src/Doc/IsarImplementation/Logic.thy
changeset 52788 da1fdbfebd39
parent 52630 fe411c1dc180
child 53015 a1119cf551e8
--- a/src/Doc/IsarImplementation/Logic.thy	Tue Jul 30 12:07:14 2013 +0200
+++ b/src/Doc/IsarImplementation/Logic.thy	Tue Jul 30 15:09:25 2013 +0200
@@ -718,8 +718,8 @@
   \item Type @{ML_type thm} represents proven propositions.  This is
   an abstract datatype that guarantees that its values have been
   constructed by basic principles of the @{ML_struct Thm} module.
-  Every @{ML_type thm} value contains a sliding back-reference to the
-  enclosing theory, cf.\ \secref{sec:context-theory}.
+  Every @{ML_type thm} value refers its background theory,
+  cf.\ \secref{sec:context-theory}.
 
   \item @{ML Thm.transfer}~@{text "thy thm"} transfers the given
   theorem to a \emph{larger} theory, see also \secref{sec:context}.