load Product_Type before Nat; dropped junk
authorhaftmann
Wed, 28 Oct 2009 17:44:03 +0100
changeset 33275 b497b2574bf6
parent 33274 b6ff7db522b5
child 33284 b5347c65bcab
child 33296 a3924d1069e5
child 33563 4c983a9d4207
load Product_Type before Nat; dropped junk
src/HOL/Product_Type.thy
--- a/src/HOL/Product_Type.thy	Wed Oct 28 17:44:03 2009 +0100
+++ b/src/HOL/Product_Type.thy	Wed Oct 28 17:44:03 2009 +0100
@@ -6,7 +6,7 @@
 header {* Cartesian products *}
 
 theory Product_Type
-imports Inductive Nat
+imports Inductive
 uses
   ("Tools/split_rule.ML")
   ("Tools/inductive_set.ML")
@@ -94,8 +94,6 @@
 
 text {* code generator setup *}
 
-instance unit :: eq ..
-
 lemma [code]:
   "eq_class.eq (u\<Colon>unit) v \<longleftrightarrow> True" unfolding eq unit_eq [of u] unit_eq [of v] by rule+
 
@@ -932,8 +930,6 @@
 
 subsubsection {* Code generator setup *}
 
-instance * :: (eq, eq) eq ..
-
 lemma [code]:
   "eq_class.eq (x1\<Colon>'a\<Colon>eq, y1\<Colon>'b\<Colon>eq) (x2, y2) \<longleftrightarrow> x1 = x2 \<and> y1 = y2" by (simp add: eq)