doc-src/TutorialI/Fun/fun0.thy
changeset 27167 a99747ccba87
parent 27015 f8537d69f514
--- a/doc-src/TutorialI/Fun/fun0.thy	Thu Jun 12 14:20:07 2008 +0200
+++ b/doc-src/TutorialI/Fun/fun0.thy	Thu Jun 12 14:20:25 2008 +0200
@@ -239,7 +239,7 @@
 \isacommand{apply}@{text"(induct_tac"} $x@1 \dots x@n$ @{text"rule:"} $f$@{text".induct)"}
 \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$ arguments. Usually the subgoal will
+name of a function that takes $n$ arguments. Usually the subgoal will
 contain the term $f x@1 \dots x@n$ but this need not be the case. The
 induction rules do not mention $f$ at all. Here is @{thm[source]sep.induct}:
 \begin{isabelle}