src/HOL/Library/Code_Integer.thy
changeset 49446 6efff142bb54
parent 49088 1b609a7837ef
     1.1 --- a/src/HOL/Library/Code_Integer.thy	Mon Jul 23 09:26:55 2012 +0200
     1.2 +++ b/src/HOL/Library/Code_Integer.thy	Mon Jul 23 09:28:03 2012 +0200
     1.3 @@ -151,7 +151,7 @@
     1.4  code_const Code_Numeral.int_of
     1.5    (SML "IntInf.fromInt")
     1.6    (OCaml "_")
     1.7 -  (Haskell "toInteger")
     1.8 +  (Haskell "Prelude.toInteger")
     1.9    (Scala "!_.as'_BigInt")
    1.10    (Eval "_")
    1.11