src/HOL/Sum_Type.thy
changeset 25534 d0b74fdd6067
parent 22838 466599ecf610
child 27104 791607529f6d
--- a/src/HOL/Sum_Type.thy	Wed Dec 05 14:15:39 2007 +0100
+++ b/src/HOL/Sum_Type.thy	Wed Dec 05 14:15:45 2007 +0100
@@ -215,26 +215,6 @@
 by blast
 
 
-subsection {* Code generator setup *}
-
-instance "+" :: (eq, eq) eq ..
-
-lemma [code func]:
-  "(Inl x \<Colon> 'a\<Colon>eq + 'b\<Colon>eq) = Inl y \<longleftrightarrow> x = y"
-  unfolding Inl_eq ..
-
-lemma [code func]:
-  "(Inr x \<Colon> 'a\<Colon>eq + 'b\<Colon>eq) = Inr y \<longleftrightarrow> x = y"
-  unfolding Inr_eq ..
-
-lemma [code func]:
-  "Inl (x\<Colon>'a\<Colon>eq) = Inr (y\<Colon>'b\<Colon>eq) \<longleftrightarrow> False"
-  using Inl_not_Inr by auto
-
-lemma [code func]:
-  "Inr (x\<Colon>'b\<Colon>eq) = Inl (y\<Colon>'a\<Colon>eq) \<longleftrightarrow> False"
-  using Inr_not_Inl by auto
-
 ML
 {*
 val Inl_RepI = thm "Inl_RepI";