src/HOL/Library/Efficient_Nat.thy
changeset 24630 351a308ab58d
parent 24423 ae9cd0e92423
child 24715 f96d86cdbe5a
--- a/src/HOL/Library/Efficient_Nat.thy	Tue Sep 18 11:06:22 2007 +0200
+++ b/src/HOL/Library/Efficient_Nat.thy	Tue Sep 18 16:08:00 2007 +0200
@@ -164,14 +164,14 @@
 *}
 
 code_type nat
-  (SML "IntInf.int")
+  (SML "int")
   (OCaml "Big'_int.big'_int")
   (Haskell "Integer")
 
 types_code
   nat ("int")
 attach (term_of) {*
-val term_of_nat = HOLogic.mk_number HOLogic.natT o IntInf.fromInt;
+val term_of_nat = HOLogic.mk_number HOLogic.natT;
 *}
 attach (test) {*
 fun gen_nat i = random_range 0 i;
@@ -224,7 +224,7 @@
     val simplify_less = Simplifier.rewrite 
       (HOL_basic_ss addsimps (@{thms less_numeral_code} @ @{thms less_eq_numeral_code}));
     fun mk_rew (t, ty) =
-      if ty = HOLogic.natT andalso IntInf.<= (0, HOLogic.dest_numeral t) then
+      if ty = HOLogic.natT andalso 0 <= HOLogic.dest_numeral t then
         Thm.capply @{cterm "(op \<le>) Numeral.Pls"} (Thm.cterm_of thy t)
         |> simplify_less
         |> (fn thm => @{thm nat_of_int_of_number_of_aux} OF [thm])