hope it works
authorChengsong
Mon, 19 Aug 2019 16:22:58 +0100
changeset 341 abf178a5db58
parent 340 6c71db65bdec
child 342 f0e876ed43fa
hope it works
thys/BitCoded.thy
--- a/thys/BitCoded.thy	Mon Aug 19 13:33:53 2019 +0100
+++ b/thys/BitCoded.thy	Mon Aug 19 16:22:58 2019 +0100
@@ -1,5 +1,5 @@
 
-theory BitCoded
+theory BitCodedCT
   imports "Lexer" 
 begin
 
@@ -2756,7 +2756,7 @@
   shows " \<exists> a aa list. y = a#aa#list"
   by (metis Nil_is_map_conv arexp.simps(13) assms bsimp_AALTs.elims flts1 good.simps(5) good1 k0a)
 
-
+(*SAD*)
 (*this does not hold actually
 lemma bsimp_equiv0:
   shows "bsimp(bsimp r) = bsimp(bsimp (AALTs []  [r]))"
@@ -2881,7 +2881,7 @@
   shows"map f [a,b] = [f a, f b]"
   apply simp
   done
-
+(*SAD*)
 (* bsimp (bder c (bsimp_AALTs x51 (flts [bsimp a1, bsimp a2]))) =
        bsimp (AALT x51 (bder c (bsimp a1)) (bder c (bsimp a2)))*)
 (*This equality does not hold*)