--- a/CookBook/Recipes/Config.thy Thu Jan 08 22:47:15 2009 +0000
+++ b/CookBook/Recipes/Config.thy Sat Jan 10 12:57:48 2009 +0000
@@ -33,7 +33,8 @@
text {* or on the ML-level *}
-ML {*setup_sval @{theory}
+ML {*
+setup_sval @{theory}
*}
text {*
@@ -43,7 +44,8 @@
declare [[bval = true, ival = 3]]
text {*
- On the ML-level these values can be retrieved using the function @{ML Config.get}:
+ from within Isabelle. On the ML-level these values can be retrieved using the
+ function @{ML Config.get}:
@{ML_response [display] "Config.get @{context} bval" "true"}
@@ -59,7 +61,7 @@
setup {* Config.put_thy sval "bar" *}
text {*
- Then retrival of this value yields now
+ The retrival of this value yields now
@{ML_response [display] "Config.get @{context} sval" "\"bar\""}