ProgTutorial/Base.thy
changeset 255 ef1da1abee46
parent 239 b63c72776f03
child 256 1fb8d62c88a0
--- a/ProgTutorial/Base.thy	Fri May 29 12:15:48 2009 +0200
+++ b/ProgTutorial/Base.thy	Sat May 30 11:12:46 2009 +0200
@@ -1,6 +1,7 @@
 theory Base
 imports Main
 uses
+  "outputfn.ML"
   "chunks.ML"
   "antiquote_setup.ML"
 begin
@@ -37,4 +38,5 @@
 
 *}
 
+
 end
\ No newline at end of file