changeset 39272 | 0b61951d2682 |
parent 38857 | 97775f3e8722 |
child 47108 | 2a1953f0d20d |
--- a/src/HOL/Library/Code_Integer.thy Fri Sep 10 09:56:28 2010 +0200 +++ b/src/HOL/Library/Code_Integer.thy Fri Sep 10 10:21:25 2010 +0200 @@ -99,7 +99,7 @@ code_const "HOL.equal \<Colon> int \<Rightarrow> int \<Rightarrow> bool" (SML "!((_ : IntInf.int) = _)") (OCaml "Big'_int.eq'_big'_int") - (Haskell infixl 4 "==") + (Haskell infix 4 "==") (Scala infixl 5 "==") (Eval infixl 6 "=")