src/HOL/Library/Code_Char.thy
changeset 28346 b8390cd56b8f
parent 28244 f433e544a855
child 29944 74d83bd18977
     1.1 --- a/src/HOL/Library/Code_Char.thy	Wed Sep 24 19:39:25 2008 +0200
     1.2 +++ b/src/HOL/Library/Code_Char.thy	Thu Sep 25 09:28:03 2008 +0200
     1.3 @@ -28,7 +28,7 @@
     1.4  code_reserved OCaml
     1.5    char
     1.6  
     1.7 -code_const "op = \<Colon> char \<Rightarrow> char \<Rightarrow> bool"
     1.8 +code_const "eq_class.eq \<Colon> char \<Rightarrow> char \<Rightarrow> bool"
     1.9    (SML "!((_ : char) = _)")
    1.10    (OCaml "!((_ : char) = _)")
    1.11    (Haskell infixl 4 "==")