doc-src/TutorialI/Inductive/Even.thy
changeset 12328 7c4ec77a8715
parent 11705 ac8ca15c556c
child 16417 9bc16273c2d4
--- a/doc-src/TutorialI/Inductive/Even.thy	Thu Nov 29 13:33:45 2001 +0100
+++ b/doc-src/TutorialI/Inductive/Even.thy	Thu Nov 29 14:12:42 2001 +0100
@@ -21,7 +21,7 @@
 
 Our first lemma states that numbers of the form $2\times k$ are even. *}
 lemma two_times_even[intro!]: "2*k \<in> even"
-apply (induct "k")
+apply (induct_tac k)
 txt{*
 The first step is induction on the natural number \isa{k}, which leaves
 two subgoals: