src/HOL/Product_Type.thy
changeset 23247 b99dce43d252
parent 22886 cdff6ef76009
child 24162 8dfd5dd65d82
--- a/src/HOL/Product_Type.thy	Tue Jun 05 12:12:25 2007 +0200
+++ b/src/HOL/Product_Type.thy	Tue Jun 05 15:16:08 2007 +0200
@@ -7,7 +7,7 @@
 header {* Cartesian products *}
 
 theory Product_Type
-imports Typedef Fun Code_Generator
+imports Typedef Fun
 uses ("Tools/split_rule.ML")
 begin