diff -r 885a40edcdba -r 0c3891c3528f doc-src/TutorialI/Misc/natsum.thy --- a/doc-src/TutorialI/Misc/natsum.thy Thu Dec 02 12:28:09 2004 +0100 +++ b/doc-src/TutorialI/Misc/natsum.thy Thu Dec 02 14:47:07 2004 +0100 @@ -23,20 +23,20 @@ text{*\newcommand{\mystar}{*% } \index{arithmetic operations!for \protect\isa{nat}}% -The arithmetic operations \ttindexboldpos{+}{$HOL2arithfun}, -\ttindexboldpos{-}{$HOL2arithfun}, \ttindexboldpos{\mystar}{$HOL2arithfun}, +The arithmetic operations \isadxboldpos{+}{$HOL2arithfun}, +\isadxboldpos{-}{$HOL2arithfun}, \isadxboldpos{\mystar}{$HOL2arithfun}, \sdx{div}, \sdx{mod}, \cdx{min} and \cdx{max} are predefined, as are the relations -\indexboldpos{\isasymle}{$HOL2arithrel} and -\ttindexboldpos{<}{$HOL2arithrel}. As usual, @{prop"m-n = (0::nat)"} if +\isadxboldpos{\isasymle}{$HOL2arithrel} and +\isadxboldpos{<}{$HOL2arithrel}. As usual, @{prop"m-n = (0::nat)"} if @{prop"m}{$HOL2arithrel} and + \isadxboldpos{\isasymge}{$HOL2arithrel} are merely syntax: @{text"x > y"} + stands for @{prop"y < x"} and similary for @{text"\"} and + @{text"\"}. +\end{warn} +\begin{warn} Constant @{text"1::nat"} is defined to equal @{term"Suc 0"}. This definition (see \S\ref{sec:ConstDefinitions}) is unfolded automatically by some tactics (like @{text auto}, @{text simp} and @{text arith}) but not by