src/HOL/Inductive.thy
changeset 7700 38b6d2643630
parent 7357 d0e16da40ea2
child 7710 bf8cb3fc5d64
--- a/src/HOL/Inductive.thy	Mon Oct 04 21:43:05 1999 +0200
+++ b/src/HOL/Inductive.thy	Mon Oct 04 21:43:45 1999 +0200
@@ -1,7 +1,19 @@
+(*  Title:      HOL/Inductive.thy
+    ID:         $Id$
+*)
 
 theory Inductive = Gfp + Prod + Sum
-files "Tools/inductive_package.ML":
+files
+  "Tools/inductive_package.ML"
+  "Tools/datatype_aux.ML"
+  "Tools/datatype_prop.ML"
+  "Tools/datatype_rep_proofs.ML"
+  "Tools/datatype_abs_proofs.ML"
+  "Tools/datatype_package.ML"
+  "Tools/primrec_package.ML":
 
 setup InductivePackage.setup
+setup DatatypePackage.setup
+
 
 end