CookBook/Package/Simple_Inductive_Package.thy
changeset 32 5bb2d29553c2
child 159 64fa844064fa
--- /dev/null	Thu Jan 01 00:00:00 1970 +0000
+++ b/CookBook/Package/Simple_Inductive_Package.thy	Fri Oct 10 17:13:21 2008 +0200
@@ -0,0 +1,8 @@
+theory Simple_Inductive_Package
+imports Main
+uses ("simple_inductive_package.ML")
+begin
+
+use_chunks "simple_inductive_package.ML"
+
+end