src/HOL/Library/Code_Integer.thy
changeset 39499 0b61951d2682
parent 39086 97775f3e8722
child 47978 2a1953f0d20d
     1.1 --- a/src/HOL/Library/Code_Integer.thy	Fri Sep 10 09:56:28 2010 +0200
     1.2 +++ b/src/HOL/Library/Code_Integer.thy	Fri Sep 10 10:21:25 2010 +0200
     1.3 @@ -99,7 +99,7 @@
     1.4  code_const "HOL.equal \<Colon> int \<Rightarrow> int \<Rightarrow> bool"
     1.5    (SML "!((_ : IntInf.int) = _)")
     1.6    (OCaml "Big'_int.eq'_big'_int")
     1.7 -  (Haskell infixl 4 "==")
     1.8 +  (Haskell infix 4 "==")
     1.9    (Scala infixl 5 "==")
    1.10    (Eval infixl 6 "=")
    1.11