corrected fragile proof; tuned semicolons
authorhaftmann
Wed, 14 Mar 2012 15:54:27 +0100
changeset 46932 53d06963d83d
parent 46931 d2b92739038b
child 46933 3b02b0ef8d48
corrected fragile proof; tuned semicolons
doc-src/TutorialI/CTL/CTL.thy
--- a/doc-src/TutorialI/CTL/CTL.thy	Wed Mar 14 15:24:51 2012 +0100
+++ b/doc-src/TutorialI/CTL/CTL.thy	Wed Mar 14 15:54:27 2012 +0100
@@ -370,11 +370,11 @@
 
 lemma "lfp(eufix A B) \<subseteq> eusem A B"
 apply(rule lfp_lowerbound)
-apply(auto simp add: eusem_def eufix_def);
- apply(rule_tac x = "[]" in exI);
+apply(auto simp add: eusem_def eufix_def)
+ apply(rule_tac x = "[]" in exI)
  apply simp
-apply(rule_tac x = "y#xc" in exI);
-apply simp;
+apply(rule_tac x = "xa#xb" in exI)
+apply simp
 done
 
 lemma mono_eufix: "mono(eufix A B)";