doc-src/TutorialI/Misc/natsum.thy
changeset 10971 6852682eaf16
parent 10788 ea48dd8b0232
child 10978 5eebea8f359f
--- a/doc-src/TutorialI/Misc/natsum.thy	Wed Jan 24 11:59:15 2001 +0100
+++ b/doc-src/TutorialI/Misc/natsum.thy	Wed Jan 24 12:29:10 2001 +0100
@@ -69,7 +69,8 @@
 For more complex goals, there is the special method \isaindexbold{arith}
 (which attacks the first subgoal). It proves arithmetic goals involving the
 usual logical connectives (@{text"\<not>"}, @{text"\<and>"}, @{text"\<or>"},
-@{text"\<longrightarrow>"}), the relations @{text"\<le>"} and @{text"<"}, and the operations
+@{text"\<longrightarrow>"}), the relations @{text"="}, @{text"\<le>"} and @{text"<"},
+and the operations
 @{text"+"}, @{text"-"}, @{term min} and @{term max}. Technically, this is
 known as the class of (quantifier free) \bfindex{linear arithmetic} formulae.
 For example,