doc-src/IsarImplementation/Thy/integration.thy
changeset 22090 bc8aee017f8a
parent 21401 faddc6504177
child 22095 07875394618e
--- a/doc-src/IsarImplementation/Thy/integration.thy	Fri Jan 19 13:09:37 2007 +0100
+++ b/doc-src/IsarImplementation/Thy/integration.thy	Fri Jan 19 13:16:37 2007 +0100
@@ -240,18 +240,12 @@
 
 text %mlref {*
   \begin{mldecls}
-  @{index_ML context: "theory -> unit"} \\
   @{index_ML the_context: "unit -> theory"} \\
   @{index_ML "Context.>> ": "(theory -> theory) -> unit"} \\
   \end{mldecls}
 
   \begin{description}
 
-  \item @{ML context}~@{text thy} sets the {\ML} theory context to
-  @{text thy}.  This is usually performed automatically by the system,
-  when dropping out of the interactive Isar toplevel into {\ML}, or
-  when Isar invokes {\ML} to process code from a string or a file.
-
   \item @{ML "the_context ()"} refers to the theory context of the
   {\ML} toplevel --- at compile time!  {\ML} code needs to take care
   to refer to @{ML "the_context ()"} correctly.  Recall that