--- a/CookBook/Recipes/Config.thy Wed Jan 14 16:46:07 2009 +0000
+++ b/CookBook/Recipes/Config.thy Wed Jan 14 17:47:49 2009 +0000
@@ -17,11 +17,9 @@
containing a string. These values can be declared on the ML-level with
*}
-ML {*
-val (bval, setup_bval) = Attrib.config_bool "bval" false
+ML{*val (bval, setup_bval) = Attrib.config_bool "bval" false
val (ival, setup_ival) = Attrib.config_int "ival" 0
-val (sval, setup_sval) = Attrib.config_string "sval" "some string"
-*}
+val (sval, setup_sval) = Attrib.config_string "sval" "some string" *}
text {*
where each value needs to be given a default. To enable these values, they need to
@@ -33,9 +31,7 @@
text {* or on the ML-level *}
-ML {*
-setup_sval @{theory}
-*}
+ML{*setup_sval @{theory} *}
text {*
The user can now manipulate the values from within Isabelle with the command