src/HOL/Library/Code_Integer.thy
changeset 38185 844977c7abeb
parent 34931 970e1466028d
child 38195 9728342bcd56
     1.1 --- a/src/HOL/Library/Code_Integer.thy	Fri Jul 23 10:25:00 2010 +0200
     1.2 +++ b/src/HOL/Library/Code_Integer.thy	Fri Jul 23 10:58:13 2010 +0200
     1.3 @@ -112,7 +112,7 @@
     1.4  code_const Code_Numeral.int_of
     1.5    (SML "IntInf.fromInt")
     1.6    (OCaml "_")
     1.7 -  (Haskell "toEnum")
     1.8 +  (Haskell "_")
     1.9    (Scala "!BigInt((_))")
    1.10  
    1.11  text {* Evaluation *}