doc-src/TutorialI/Recdef/Induction.thy
changeset 11428 332347b9b942
parent 11159 07b13770c4d6
child 11458 09a6c44a48ea
--- a/doc-src/TutorialI/Recdef/Induction.thy	Mon Jul 16 13:14:19 2001 +0200
+++ b/doc-src/TutorialI/Recdef/Induction.thy	Tue Jul 17 13:46:21 2001 +0200
@@ -48,7 +48,7 @@
 In general, the format of invoking recursion induction is
 \begin{quote}
 \isacommand{apply}@{text"(induct_tac"} $x@1 \dots x@n$ @{text"rule:"} $f$@{text".induct)"}
-\end{quote}\index{*induct_tac}%
+\end{quote}\index{*induct_tac (method)}%
 where $x@1~\dots~x@n$ is a list of free variables in the subgoal and $f$ the
 name of a function that takes an $n$-tuple. Usually the subgoal will
 contain the term $f(x@1,\dots,x@n)$ but this need not be the case. The