| changeset 12489 | c92e38c3cbaa |
| parent 12473 | f41e477576b9 |
| child 12699 | deae80045527 |
--- a/doc-src/TutorialI/CTL/CTL.thy Thu Dec 13 16:48:07 2001 +0100 +++ b/doc-src/TutorialI/CTL/CTL.thy Thu Dec 13 16:48:34 2001 +0100 @@ -203,7 +203,8 @@ both the path property and the fact that @{term Q} holds: *}; -apply(subgoal_tac "\<exists>p. s = p (0::nat) \<and> (\<forall>i. (p i, p(i+1)) \<in> M \<and> Q(p i))"); +apply(subgoal_tac + "\<exists>p. s = p 0 \<and> (\<forall>i::nat. (p i, p(i+1)) \<in> M \<and> Q(p i))"); txt{*\noindent From this proposition the original goal follows easily: