src/HOL/List.thy
changeset 28346 b8390cd56b8f
parent 28262 aa7ca36d67fd
child 28370 37f56e6e702d
--- a/src/HOL/List.thy	Wed Sep 24 19:39:25 2008 +0200
+++ b/src/HOL/List.thy	Thu Sep 25 09:28:03 2008 +0200
@@ -3625,7 +3625,7 @@
 code_instance list :: eq
   (Haskell -)
 
-code_const "op = \<Colon> 'a\<Colon>eq list \<Rightarrow> 'a list \<Rightarrow> bool"
+code_const "eq_class.eq \<Colon> 'a\<Colon>eq list \<Rightarrow> 'a list \<Rightarrow> bool"
   (Haskell infixl 4 "==")
 
 setup {*