diff -r a99747ccba87 -r 9a9cc62932d9 doc-src/TutorialI/Misc/natsum.thy --- a/doc-src/TutorialI/Misc/natsum.thy Thu Jun 12 14:20:25 2008 +0200 +++ b/doc-src/TutorialI/Misc/natsum.thy Thu Jun 12 14:20:52 2008 +0200 @@ -103,13 +103,13 @@ succeeds because @{term"k*k"} can be treated as atomic. In contrast, *} -lemma "n*n = n \ n=0 \ n=1" +lemma "n*n = n+1 \ n=0" (*<*)oops(*>*) text{*\noindent -is not proved even by @{text arith} because the proof relies +is not proved by @{text arith} because the proof relies on properties of multiplication. Only multiplication by numerals (which is -the same as iterated addition) is allowed. +the same as iterated addition) is taken into account. \begin{warn} The running time of @{text arith} is exponential in the number of occurrences of \ttindexboldpos{-}{$HOL2arithfun}, \cdx{min} and