doc-src/TutorialI/CTL/PDL.thy
changeset 11231 30d96882f915
parent 11207 08188224c24e
child 11458 09a6c44a48ea
--- a/doc-src/TutorialI/CTL/PDL.thy	Thu Mar 29 10:44:37 2001 +0200
+++ b/doc-src/TutorialI/CTL/PDL.thy	Thu Mar 29 12:26:37 2001 +0200
@@ -152,7 +152,7 @@
 is solved by unrolling @{term lfp} once
 *}
 
- apply(rule ssubst[OF lfp_unfold[OF mono_ef]])
+ apply(subst lfp_unfold[OF mono_ef])
 
 txt{*
 @{subgoals[display,indent=0,goals_limit=1]}
@@ -165,7 +165,7 @@
 The proof of the induction step is identical to the one for the base case:
 *}
 
-apply(rule ssubst[OF lfp_unfold[OF mono_ef]])
+apply(subst lfp_unfold[OF mono_ef])
 apply(blast)
 done
 
@@ -205,7 +205,7 @@
 lemma "(s \<Turnstile> EF f) = (s \<Turnstile> f | s \<Turnstile> Neg(AX(Neg(EF f))))";
 apply(simp only:aux);
 apply(simp);
-apply(rule ssubst[OF lfp_unfold[OF mono_ef]], fast);
+apply(subst lfp_unfold[OF mono_ef], fast);
 done
 
 end