diff -r 3ed58bbcf4bd -r 332347b9b942 doc-src/TutorialI/Misc/natsum.thy --- a/doc-src/TutorialI/Misc/natsum.thy Mon Jul 16 13:14:19 2001 +0200 +++ b/doc-src/TutorialI/Misc/natsum.thy Tue Jul 17 13:46:21 2001 +0200 @@ -24,13 +24,13 @@ } The usual arithmetic operations \ttindexboldpos{+}{$HOL2arithfun}, \ttindexboldpos{-}{$HOL2arithfun}, \ttindexboldpos{\mystar}{$HOL2arithfun}, -\isaindexbold{div}, \isaindexbold{mod}, \isaindexbold{min} and -\isaindexbold{max} are predefined, as are the relations +\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"} if @{prop"m"}), the relations @{text"="}, @{text"\"} 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. +known as the class of (quantifier free) \textbf{linear arithmetic} formulae. For example, *} @@ -97,8 +97,8 @@ \begin{warn} The running time of @{text arith} is exponential in the number of occurrences - of \ttindexboldpos{-}{$HOL2arithfun}, \isaindexbold{min} and - \isaindexbold{max} because they are first eliminated by case distinctions. + of \ttindexboldpos{-}{$HOL2arithfun}, \cdx{min} and + \cdx{max} because they are first eliminated by case distinctions. \isa{arith} is incomplete even for the restricted class of linear arithmetic formulae. If divisibility plays a