doc-src/IsarImplementation/Thy/Prelim.thy
changeset 40126 916cb4a28ffd
parent 39876 1ff9bce085bd
child 40153 b6fe3b189725
--- a/doc-src/IsarImplementation/Thy/Prelim.thy	Mon Oct 25 11:39:52 2010 +0200
+++ b/doc-src/IsarImplementation/Thy/Prelim.thy	Mon Oct 25 16:14:40 2010 +0200
@@ -640,7 +640,7 @@
 setup my_flag_setup
 
 text {* Now the user can refer to @{attribute my_flag} in
-  declarations, while we can retrieve the current value from the
+  declarations, while ML tools can retrieve the current value from the
   context via @{ML Config.get}.  *}
 
 ML_val {* @{assert} (Config.get @{context} my_flag = false) *}
@@ -897,7 +897,7 @@
   @{assert} (list2 = ["x", "xa", "a", "aa", "'a", "'aa"]);
 *}
 
-text {* \medskip The same works reletively to the formal context as
+text {* \medskip The same works relatively to the formal context as
   follows. *}
 
 locale ex = fixes a b c :: 'a
@@ -1210,13 +1210,13 @@
 *}
 
 text %mlex {* The following example yields the source position of some
-  concrete binding inlined into the text.
+  concrete binding inlined into the text:
 *}
 
 ML {* Binding.pos_of @{binding here} *}
 
 text {* \medskip That position can be also printed in a message as
-  follows. *}
+  follows: *}
 
 ML_command {*
   writeln
@@ -1225,6 +1225,7 @@
 
 text {* This illustrates a key virtue of formalized bindings as
   opposed to raw specifications of base names: the system can use this
-  additional information for advanced feedback given to the user. *}
+  additional information for feedback given to the user (error
+  messages etc.). *}
 
 end