doc-src/IsarImplementation/Thy/Proof.thy
changeset 40126 916cb4a28ffd
parent 39864 f3b4fde34cd1
child 40153 b6fe3b189725
--- a/doc-src/IsarImplementation/Thy/Proof.thy	Mon Oct 25 11:39:52 2010 +0200
+++ b/doc-src/IsarImplementation/Thy/Proof.thy	Mon Oct 25 16:14:40 2010 +0200
@@ -180,13 +180,12 @@
   val t2 = Syntax.read_term ctxt2 "x";  (*x::nat is enforced*)
 *}
 
-text {* In the above example, the starting context had been derived
-  from the toplevel theory, which means that fixed variables are
-  internalized literally: @{verbatim "x"} is mapped again to
-  @{verbatim "x"}, and attempting to fix it again in the subsequent
-  context is an error.  Alternatively, fixed parameters can be renamed
-  explicitly as follows:
-*}
+text {* In the above example, the starting context is derived from the
+  toplevel theory, which means that fixed variables are internalized
+  literally: @{verbatim "x"} is mapped again to @{verbatim "x"}, and
+  attempting to fix it again in the subsequent context is an error.
+  Alternatively, fixed parameters can be renamed explicitly as
+  follows: *}
 
 ML {*
   val ctxt0 = @{context};