changeset 35689 | c3bef0c972d7 |
parent 35625 | 9c818cab0dd0 |
child 36176 | 3fe7e97ccca8 |
--- a/src/HOL/Library/Efficient_Nat.thy Wed Mar 10 15:29:22 2010 +0100 +++ b/src/HOL/Library/Efficient_Nat.thy Wed Mar 10 15:29:22 2010 +0100 @@ -400,7 +400,7 @@ (SML "IntInf.max/ (/0,/ _)") (OCaml "Big'_int.max'_big'_int/ Big'_int.zero'_big'_int") -text {* For Haskell ans Scala, things are slightly different again. *} +text {* For Haskell and Scala, things are slightly different again. *} code_const int and nat (Haskell "toInteger" and "fromInteger")