# HG changeset patch # User cu # Date 1507631507 -3600 # Node ID f754a10875c7f04ff82aaa74da24d1fb46cfd8fe # Parent 424bdcd01016b740c408ab85210b40ec6289cda3 updated for Isabelle 2017 diff -r 424bdcd01016 -r f754a10875c7 thys/Spec.thy --- a/thys/Spec.thy Tue Oct 10 10:40:44 2017 +0100 +++ b/thys/Spec.thy Tue Oct 10 11:31:47 2017 +0100 @@ -376,7 +376,7 @@ fix s::"char list" assume "\s'. length s' < length s \ finite (LV (STAR r) s')" then have IH: "\s' \ SSuffixes s. finite (LV (STAR r) s')" - by (auto simp add: strict_suffix_def) + by (force simp add: strict_suffix_def suffix_def) define f where "f \ \(v, vs). Stars (v # vs)" define S1 where "S1 \ \s' \ Prefixes s. LV r s'" define S2 where "S2 \ \s2 \ SSuffixes s. Stars -` (LV (STAR r) s2)" @@ -404,7 +404,8 @@ apply(rule conjI) apply(rule_tac x="flats list" in exI) apply(simp) - apply(blast) + apply(blast) + apply(simp add: suffix_def) using Prf.intros(6) by blast ultimately show "finite (LV (STAR r) s)" by (simp add: finite_subset) diff -r 424bdcd01016 -r f754a10875c7 thys/SpecExt.thy --- 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 "\s'. length s' < length s \ finite (LV (STAR r) s')" then have IH: "\s' \ 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 \ \(v, vs). Stars (v # vs)" define S1 where "S1 \ \s' \ Prefixes s. LV r s'" define S2 where "S2 \ \s2 \ 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