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