CookBook/Base.thy
changeset 57 065f472c09ab
parent 43 02f76f1b6e7b
child 64 9a6e5e0c4906
--- a/CookBook/Base.thy	Tue Dec 16 08:08:44 2008 +0000
+++ b/CookBook/Base.thy	Tue Dec 16 17:37:39 2008 +0100
@@ -1,8 +1,8 @@
 theory Base
 imports Main
 uses
+  "chunks.ML"
   "antiquote_setup.ML"
-  "chunks.ML"
 begin
 
 end