doc-src/TutorialI/Misc/natsum.thy
changeset 13181 dc393bbee6ce
parent 12699 deae80045527
child 13996 a994b92ab1ea
--- a/doc-src/TutorialI/Misc/natsum.thy	Fri May 24 16:56:25 2002 +0200
+++ b/doc-src/TutorialI/Misc/natsum.thy	Mon May 27 17:20:16 2002 +0200
@@ -75,10 +75,10 @@
 text{*\noindent
 For efficiency's sake, this built-in prover ignores quantified formulae,
 logical connectives, and all arithmetic operations apart from addition.
-In consequence, @{text auto} cannot prove this slightly more complex goal:
+In consequence, @{text auto} and @{text simp} cannot prove this slightly more complex goal:
 *}
 
-lemma "\<not> m < n \<and> m < n + (1::nat) \<Longrightarrow> m = n";
+lemma "m \<noteq> (n::nat) \<Longrightarrow> m < n \<or> n < m"
 (*<*)by(arith)(*>*)
 
 text{*\noindent