src/HOL/Library/ML_Int.thy
changeset 24354 0fdabe28f0e6
parent 24219 e558fe311376
child 24423 ae9cd0e92423
--- a/src/HOL/Library/ML_Int.thy	Mon Aug 20 19:51:01 2007 +0200
+++ b/src/HOL/Library/ML_Int.thy	Mon Aug 20 19:52:24 2007 +0200
@@ -109,9 +109,9 @@
   case 0 show ?case by simp
 next
   case (Suc n)
-  then have "int_of_ml_int (ml_int_of_int (int_of_nat n))
+  then have "int_of_ml_int (ml_int_of_int (int n))
     = int_of_ml_int (of_nat n)" by simp
-  then have "int_of_nat n = int_of_ml_int (of_nat n)" by simp
+  then have "int n = int_of_ml_int (of_nat n)" by simp
   then show ?case by simp
 qed
 
@@ -127,7 +127,7 @@
   "(1\<Colon>ml_int) = Numeral1"
   by simp
 
-instance ml_int :: minus
+instance ml_int :: abs
   "\<bar>k\<bar> \<equiv> if k < 0 then -k else k" ..