src/HOL/Datatype.thy
changeset 21046 fe1db2f991a7
parent 20847 7e8c724339e0
child 21060 bc1fa6f47ced
--- a/src/HOL/Datatype.thy	Mon Oct 16 14:07:21 2006 +0200
+++ b/src/HOL/Datatype.thy	Mon Oct 16 14:07:31 2006 +0200
@@ -804,7 +804,7 @@
 code_instance option :: eq
   (Haskell -)
 
-code_const "OperationalEquality.eq \<Colon> 'a\<Colon>eq option \<Rightarrow> 'a option \<Rightarrow> bool"
+code_const "Code_Generator.eq \<Colon> 'a\<Colon>eq option \<Rightarrow> 'a option \<Rightarrow> bool"
   (Haskell infixl 4 "==")
 
 ML