src/HOL/Library/Efficient_Nat.thy
changeset 48431 6efff142bb54
parent 48073 1b609a7837ef
child 48568 084cd758a8ab
--- a/src/HOL/Library/Efficient_Nat.thy	Mon Jul 23 09:26:55 2012 +0200
+++ b/src/HOL/Library/Efficient_Nat.thy	Mon Jul 23 09:28:03 2012 +0200
@@ -162,7 +162,7 @@
 text {* For Haskell and Scala, things are slightly different again. *}
 
 code_const int and nat
-  (Haskell "toInteger" and "fromInteger")
+  (Haskell "Prelude.toInteger" and "Prelude.fromInteger")
   (Scala "!_.as'_BigInt" and "Nat")
 
 text {* Alternativ implementation for @{const of_nat} *}
@@ -189,14 +189,14 @@
 code_const Code_Numeral.of_nat
   (SML "IntInf.toInt")
   (OCaml "_")
-  (Haskell "!(fromInteger/ ./ toInteger)")
+  (Haskell "!(Prelude.fromInteger/ ./ Prelude.toInteger)")
   (Scala "!Natural(_.as'_BigInt)")
   (Eval "_")
 
 code_const Code_Numeral.nat_of
   (SML "IntInf.fromInt")
   (OCaml "_")
-  (Haskell "!(fromInteger/ ./ toInteger)")
+  (Haskell "!(Prelude.fromInteger/ ./ Prelude.toInteger)")
   (Scala "!Nat(_.as'_BigInt)")
   (Eval "_")