doc-src/TutorialI/CTL/PDL.thy
changeset 12631 7648ac4a6b95
parent 11458 09a6c44a48ea
child 12815 1f073030b97a
--- a/doc-src/TutorialI/CTL/PDL.thy	Fri Jan 04 19:23:28 2002 +0100
+++ b/doc-src/TutorialI/CTL/PDL.thy	Fri Jan 04 19:24:43 2002 +0100
@@ -38,7 +38,7 @@
 "s \<Turnstile> Neg f   = (\<not>(s \<Turnstile> f))"
 "s \<Turnstile> And f g = (s \<Turnstile> f \<and> s \<Turnstile> g)"
 "s \<Turnstile> AX f    = (\<forall>t. (s,t) \<in> M \<longrightarrow> t \<Turnstile> f)"
-"s \<Turnstile> EF f    = (\<exists>t. (s,t) \<in> M\<^sup>* \<and> t \<Turnstile> f)";
+"s \<Turnstile> EF f    = (\<exists>t. (s,t) \<in> M\<^sup>* \<and> t \<Turnstile> f)"
 
 text{*\noindent
 The first three equations should be self-explanatory. The temporal formula
@@ -51,7 +51,7 @@
 states where the formula is true.  It too is defined by recursion over the syntax:
 *}
 
-consts mc :: "formula \<Rightarrow> state set";
+consts mc :: "formula \<Rightarrow> state set"
 primrec
 "mc(Atom a)  = {s. a \<in> L s}"
 "mc(Neg f)   = -mc f"
@@ -92,8 +92,8 @@
 includes the other; the inclusion is shown pointwise:
 *}
 
-apply(rule equalityI);
- apply(rule subsetI);
+apply(rule equalityI)
+ apply(rule subsetI)
  apply(simp)(*<*)apply(rename_tac s)(*>*)
 
 txt{*\noindent
@@ -118,7 +118,7 @@
 \isa{M\isactrlsup {\isacharasterisk}}.
 *}
 
- apply(blast intro: rtrancl_trans);
+ apply(blast intro: rtrancl_trans)
 
 txt{*
 We now return to the second set inclusion subgoal, which is again proved
@@ -172,10 +172,10 @@
 @{text auto} augmented with the lemma as a simplification rule.
 *}
 
-theorem "mc f = {s. s \<Turnstile> f}";
-apply(induct_tac f);
-apply(auto simp add:EF_lemma);
-done;
+theorem "mc f = {s. s \<Turnstile> f}"
+apply(induct_tac f)
+apply(auto simp add:EF_lemma)
+done
 
 text{*
 \begin{exercise}
@@ -193,19 +193,19 @@
 \index{PDL|)}
 *}
 (*<*)
-theorem main: "mc f = {s. s \<Turnstile> f}";
-apply(induct_tac f);
-apply(auto simp add:EF_lemma);
-done;
+theorem main: "mc f = {s. s \<Turnstile> f}"
+apply(induct_tac f)
+apply(auto simp add: EF_lemma)
+done
 
-lemma aux: "s \<Turnstile> f = (s : mc f)";
-apply(simp add:main);
-done;
+lemma aux: "s \<Turnstile> f = (s : mc f)"
+apply(simp add: main)
+done
 
-lemma "(s \<Turnstile> EF f) = (s \<Turnstile> f | s \<Turnstile> Neg(AX(Neg(EF f))))";
-apply(simp only:aux);
-apply(simp);
-apply(subst lfp_unfold[OF mono_ef], fast);
+lemma "(s \<Turnstile> EF f) = (s \<Turnstile> f | s \<Turnstile> Neg(AX(Neg(EF f))))"
+apply(simp only: aux)
+apply(simp)
+apply(subst lfp_unfold[OF mono_ef], fast)
 done
 
 end