diff -r eab03e9cee8a -r 05f5fdb8d093 src/Doc/Tutorial/CTL/CTL.thy --- a/src/Doc/Tutorial/CTL/CTL.thy Wed Feb 12 08:35:57 2014 +0100 +++ b/src/Doc/Tutorial/CTL/CTL.thy Wed Feb 12 08:35:57 2014 +0100 @@ -258,9 +258,9 @@ @{thm[source]infinity_lemma}. Aficionados of minimal proofs might like to know that we could have given the witness without having to define a new function: the term -@{term[display]"nat_rec s (\n t. SOME u. (t,u)\M \ Q u)"} +@{term[display]"rec_nat s (\n t. SOME u. (t,u)\M \ Q u)"} is extensionally equal to @{term"path s Q"}, -where @{term nat_rec} is the predefined primitive recursor on @{typ nat}. +where @{term rec_nat} is the predefined primitive recursor on @{typ nat}. *}; (*<*) lemma @@ -270,7 +270,7 @@ "\ p. s = p 0 \ (\ i. (p i,p(Suc i))\M \ Q(p i))"); apply(simp add: Paths_def); apply(blast); -apply(rule_tac x = "nat_rec s (\n t. SOME u. (t,u)\M \ Q u)" in exI); +apply(rule_tac x = "rec_nat s (\n t. SOME u. (t,u)\M \ Q u)" in exI); apply(simp); apply(intro strip); apply(induct_tac i);