src/HOL/Library/Code_Integer.thy
changeset 38053 9102e859dc0b
parent 37968 52fdcb76c0af
child 38773 f9837065b5e8
--- a/src/HOL/Library/Code_Integer.thy	Tue Jul 27 20:16:14 2010 +0200
+++ b/src/HOL/Library/Code_Integer.thy	Wed Jul 28 12:12:29 2010 +0200
@@ -19,6 +19,7 @@
   (OCaml "Big'_int.big'_int")
   (Haskell "Integer")
   (Scala "BigInt")
+  (Eval "int")
 
 code_instance int :: eq
   (Haskell -)