doc-src/TutorialI/CTL/PDL.thy
changeset 12815 1f073030b97a
parent 12631 7648ac4a6b95
child 17914 99ead7a7eb42
--- a/doc-src/TutorialI/CTL/PDL.thy	Fri Jan 18 17:46:17 2002 +0100
+++ b/doc-src/TutorialI/CTL/PDL.thy	Fri Jan 18 18:30:19 2002 +0100
@@ -174,7 +174,7 @@
 
 theorem "mc f = {s. s \<Turnstile> f}"
 apply(induct_tac f)
-apply(auto simp add:EF_lemma)
+apply(auto simp add: EF_lemma)
 done
 
 text{*