src/Doc/IsarImplementation/Prelim.thy
changeset 51686 532e0ac5a66d
parent 48992 0518bf89c777
child 52421 6d93140a206c
--- a/src/Doc/IsarImplementation/Prelim.thy	Wed Apr 10 15:30:19 2013 +0200
+++ b/src/Doc/IsarImplementation/Prelim.thy	Wed Apr 10 17:02:47 2013 +0200
@@ -226,10 +226,13 @@
 text %mlantiq {*
   \begin{matharray}{rcl}
   @{ML_antiquotation_def "theory"} & : & @{text ML_antiquotation} \\
+  @{ML_antiquotation_def "theory_context"} & : & @{text ML_antiquotation} \\
   \end{matharray}
 
   @{rail "
   @@{ML_antiquotation theory} nameref?
+  ;
+  @@{ML_antiquotation theory_context} nameref
   "}
 
   \begin{description}
@@ -241,6 +244,10 @@
   theory @{text "A"} of the background theory of the current context
   --- as abstract value.
 
+  \item @{text "@{theory_context A}"} is similar to @{text "@{theory
+  A}"}, but presents the result as initial @{ML_type Proof.context}
+  (see also @{ML Proof_Context.init_global}).
+
   \end{description}
 *}