ProgTutorial/Base.thy
changeset 256 1fb8d62c88a0
parent 255 ef1da1abee46
child 260 5accec94b6df
--- a/ProgTutorial/Base.thy	Sat May 30 11:12:46 2009 +0200
+++ b/ProgTutorial/Base.thy	Sat May 30 17:40:20 2009 +0200
@@ -1,7 +1,7 @@
 theory Base
 imports Main
 uses
-  "outputfn.ML"
+  "output_tutorial.ML"
   "chunks.ML"
   "antiquote_setup.ML"
 begin