src/HOL/Product_Type.thy
changeset 33959 2afc55e8ed27
parent 33638 548a34929e98
child 34886 873c31d9f10d
--- a/src/HOL/Product_Type.thy	Wed Nov 25 09:14:28 2009 +0100
+++ b/src/HOL/Product_Type.thy	Wed Nov 25 11:16:57 2009 +0100
@@ -6,12 +6,10 @@
 header {* Cartesian products *}
 
 theory Product_Type
-imports Inductive
+imports Typedef Inductive Fun
 uses
   ("Tools/split_rule.ML")
   ("Tools/inductive_set.ML")
-  ("Tools/inductive_realizer.ML")
-  ("Tools/Datatype/datatype_realizer.ML")
 begin
 
 subsection {* @{typ bool} is a datatype *}
@@ -1195,16 +1193,7 @@
 val unit_eq = thm "unit_eq";
 *}
 
-
-subsection {* Further inductive packages *}
-
-use "Tools/inductive_realizer.ML"
-setup InductiveRealizer.setup
-
 use "Tools/inductive_set.ML"
 setup Inductive_Set.setup
 
-use "Tools/Datatype/datatype_realizer.ML"
-setup DatatypeRealizer.setup
-
 end