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