src/HOL/Library/Efficient_Nat.thy
changeset 27673 52056ddac194
parent 27609 b23c9ad0fe7d
child 28228 7ebe8dc06cbb
--- a/src/HOL/Library/Efficient_Nat.thy	Mon Jul 21 15:26:23 2008 +0200
+++ b/src/HOL/Library/Efficient_Nat.thy	Mon Jul 21 15:26:24 2008 +0200
@@ -376,12 +376,12 @@
 code_const index_of_nat
   (SML "IntInf.toInt")
   (OCaml "Big'_int.int'_of'_big'_int")
-  (Haskell "toEnum")
+  (Haskell "fromEnum")
 
 code_const nat_of_index
   (SML "IntInf.fromInt")
   (OCaml "Big'_int.big'_int'_of'_int")
-  (Haskell "fromEnum")
+  (Haskell "toEnum")
 
 text {* Using target language arithmetic operations whenever appropriate *}