src/HOL/ex/BinEx.thy
changeset 15965 f422f8283491
parent 15013 34264f5e4691
child 16417 9bc16273c2d4
--- a/src/HOL/ex/BinEx.thy	Mon May 16 09:35:05 2005 +0200
+++ b/src/HOL/ex/BinEx.thy	Mon May 16 10:29:15 2005 +0200
@@ -186,6 +186,10 @@
 lemma "(1234567::int) \<le> 1234567"
   by simp
 
+text{*No integer overflow!*}
+lemma "1234567 * (1234567::int) < 1234567*1234567*1234567"
+  by simp
+
 
 text {* \medskip Quotient and Remainder *}
 
@@ -205,7 +209,7 @@
 
 text {*
   A negative dividend\footnote{The definition agrees with mathematical
-  convention but not with the hardware of most computers}
+  convention and with ML, but not with the hardware of most computers}
 *}
 
 lemma "(-10::int) div 3 = -4"