thys/SpecExt.thy
changeset 279 f754a10875c7
parent 278 424bdcd01016
child 280 c840a99a3e05
--- a/thys/SpecExt.thy	Tue Oct 10 10:40:44 2017 +0100
+++ b/thys/SpecExt.thy	Tue Oct 10 11:31:47 2017 +0100
@@ -885,7 +885,8 @@
   fix s::"char list"
   assume "\<forall>s'. length s' < length s \<longrightarrow> finite (LV (STAR r) s')"
   then have IH: "\<forall>s' \<in> SSuffixes s. finite (LV (STAR r) s')"
-    by (auto simp add: strict_suffix_def) 
+    apply(auto simp add: strict_suffix_def suffix_def)
+    by force    
   define f where "f \<equiv> \<lambda>(v, vs). Stars (v # vs)"
   define S1 where "S1 \<equiv> \<Union>s' \<in> Prefixes s. LV r s'"
   define S2 where "S2 \<equiv> \<Union>s2 \<in> SSuffixes s. LV (STAR r) s2"
@@ -912,9 +913,8 @@
   apply(rule exI)
   apply(rule conjI)
   apply(rule_tac x="flats list" in exI)
-  apply(rule conjI)
-  apply(rule_tac x="flat a" in exI)
-  apply(simp)
+   apply(rule conjI)
+  apply(simp add: suffix_def)
   apply(blast)
   using Prf.intros(6) flat_Stars by blast  
   ultimately