src/HOL/List.thy
changeset 20588 c847c56edf0c
parent 20503 503ac4c5ef91
child 20699 0cc77abb185a
--- a/src/HOL/List.thy	Tue Sep 19 15:21:41 2006 +0200
+++ b/src/HOL/List.thy	Tue Sep 19 15:21:42 2006 +0200
@@ -2282,7 +2282,8 @@
 
 text{* Defaults for generating efficient code for some standard functions. *}
 
-lemmas in_set_code[code unfold] = mem_iff[symmetric, THEN eq_reflection]
+lemmas in_set_code [code unfold] =
+  mem_iff [symmetric, THEN eq_reflection]
 
 lemma rev_code[code unfold]: "rev xs == itrev xs []"
 by simp
@@ -2760,6 +2761,15 @@
   (SML target_atom "(__,/ __)")
   (Haskell target_atom "(__,/ __)")
 
+code_instance list :: eq and char :: eq
+  (Haskell - and -)
+
+code_const "OperationalEquality.eq \<Colon> 'a\<Colon>eq list \<Rightarrow> 'a list \<Rightarrow> bool"
+  (Haskell infixl 4 "==")
+
+code_const "OperationalEquality.eq \<Colon> char \<Rightarrow> char \<Rightarrow> bool"
+  (Haskell infixl 4 "==")
+
 setup {*
 let