ProgTutorial/Base.thy
changeset 462 1d1e795bc3ad
parent 459 4532577b61e0
child 471 f65b9f14d5de
--- a/ProgTutorial/Base.thy	Thu Apr 07 00:25:26 2011 +0100
+++ b/ProgTutorial/Base.thy	Tue May 17 18:11:21 2011 +0100
@@ -15,10 +15,9 @@
 (* they also write the code into a separate file  *)
 
 ML {*
-val (filename, setup_filename) = Attrib.config_string "filename" (K "File_Code.ML")
+val filename = Attrib.setup_config_string @{binding "filename"} (K "File_Code.ML")
 *}
 
-setup {* setup_filename *}
 
 ML {*
 fun write_file txt thy =