src/HOL/Code_Setup.thy
changeset 28687 150a8a1eae1a
parent 28562 4e74209f113e
child 28699 32b6a8f12c1c
--- a/src/HOL/Code_Setup.thy	Fri Oct 24 17:48:39 2008 +0200
+++ b/src/HOL/Code_Setup.thy	Fri Oct 24 17:48:40 2008 +0200
@@ -123,7 +123,7 @@
 text {* using built-in Haskell equality *}
 
 code_class eq
-  (Haskell "Eq" where "eq_class.eq" \<equiv> "(==)")
+  (Haskell "Eq")
 
 code_const "eq_class.eq"
   (Haskell infixl 4 "==")