CookBook/Base.thy
changeset 23 1322990e4ee7
child 43 02f76f1b6e7b
--- /dev/null	Thu Jan 01 00:00:00 1970 +0000
+++ b/CookBook/Base.thy	Fri Oct 10 16:59:35 2008 +0200
@@ -0,0 +1,9 @@
+theory Base
+imports Main
+uses
+  "antiquote_setup.ML"
+  "chunks.ML"
+  "antiquote_setup_plus.ML"
+begin
+
+end