src/HOL/Datatype.thy
changeset 21454 a1937c51ed88
parent 21407 af60523da908
child 21669 c68717c16013
--- a/src/HOL/Datatype.thy	Wed Nov 22 10:20:11 2006 +0100
+++ b/src/HOL/Datatype.thy	Wed Nov 22 10:20:12 2006 +0100
@@ -799,7 +799,7 @@
 code_instance option :: eq
   (Haskell -)
 
-code_const "Code_Generator.eq \<Colon> 'a\<Colon>eq option \<Rightarrow> 'a option \<Rightarrow> bool"
+code_const "op = \<Colon> 'a\<Colon>eq option \<Rightarrow> 'a option \<Rightarrow> bool"
   (Haskell infixl 4 "==")
 
 code_reserved SML