doc-src/TutorialI/Misc/natsum.thy
changeset 12699 deae80045527
parent 12329 8743e8305611
child 13181 dc393bbee6ce
equal deleted inserted replaced
12698:b87b41ade3b2 12699:deae80045527
   112   of \ttindexboldpos{-}{$HOL2arithfun}, \cdx{min} and
   112   of \ttindexboldpos{-}{$HOL2arithfun}, \cdx{min} and
   113   \cdx{max} because they are first eliminated by case distinctions.
   113   \cdx{max} because they are first eliminated by case distinctions.
   114 
   114 
   115   Even for linear arithmetic formulae, \isa{arith} is incomplete. If divisibility plays a
   115   Even for linear arithmetic formulae, \isa{arith} is incomplete. If divisibility plays a
   116   role, it may fail to prove a valid formula, for example
   116   role, it may fail to prove a valid formula, for example
   117   @{prop"m+m \<noteq> n+n+1"}. Fortunately, such examples are rare.
   117   @{text"m+m \<noteq> n+n+(1::nat)"}. Fortunately, such examples are rare.
   118 \end{warn}
   118 \end{warn}
   119 *}
   119 *}
   120 
   120 
   121 (*<*)
   121 (*<*)
   122 end
   122 end