src/HOL/Typedef.thy
changeset 22846 fb79144af9a3
parent 20426 9ffea7a8b31c
child 23247 b99dce43d252
--- a/src/HOL/Typedef.thy	Sun May 06 21:50:17 2007 +0200
+++ b/src/HOL/Typedef.thy	Mon May 07 00:49:59 2007 +0200
@@ -90,8 +90,7 @@
 use "Tools/typedef_codegen.ML"
 
 setup {*
-  TypedefPackage.setup
-  #> TypecopyPackage.setup
+  TypecopyPackage.setup
   #> TypedefCodegen.setup
 *}