doc-src/IsarImplementation/Thy/integration.thy
changeset 21401 faddc6504177
parent 21168 0f869edd6cc1
child 22090 bc8aee017f8a
equal deleted inserted replaced
21400:4788fc8e66ea 21401:faddc6504177
   282 
   282 
   283   \begin{mldecls}
   283   \begin{mldecls}
   284   @{index_ML Isar.main: "unit -> unit"} \\
   284   @{index_ML Isar.main: "unit -> unit"} \\
   285   @{index_ML Isar.loop: "unit -> unit"} \\
   285   @{index_ML Isar.loop: "unit -> unit"} \\
   286   @{index_ML Isar.state: "unit -> Toplevel.state"} \\
   286   @{index_ML Isar.state: "unit -> Toplevel.state"} \\
       
   287   @{index_ML Isar.exn: "unit -> (exn * string) option"} \\
   287   @{index_ML Isar.context: "unit -> Proof.context"} \\
   288   @{index_ML Isar.context: "unit -> Proof.context"} \\
   288   @{index_ML Isar.exn: "unit -> (exn * string) option"} \\
   289   @{index_ML Isar.goal: "unit -> thm list * thm"} \\
   289   \end{mldecls}
   290   \end{mldecls}
   290 
   291 
   291   \begin{description}
   292   \begin{description}
   292 
   293 
   293   \item @{ML "Isar.main ()"} invokes the Isar toplevel from {\ML},
   294   \item @{ML "Isar.main ()"} invokes the Isar toplevel from {\ML},
   301   after having dropped out of the Isar toplevel loop.
   302   after having dropped out of the Isar toplevel loop.
   302 
   303 
   303   \item @{ML "Isar.context ()"} produces the proof context from @{ML
   304   \item @{ML "Isar.context ()"} produces the proof context from @{ML
   304   "Isar.state ()"}, analogous to @{ML Context.proof_of}
   305   "Isar.state ()"}, analogous to @{ML Context.proof_of}
   305   (\secref{sec:generic-context}).
   306   (\secref{sec:generic-context}).
       
   307 
       
   308   \item @{ML "Isar.goal ()"} picks the goal configuration from @{ML
       
   309   "Isar.state ()"}, consisting on the current facts and the goal
       
   310   represented as a theorem according to \secref{sec:tactical-goals}.
   306 
   311 
   307   \end{description}
   312   \end{description}
   308 *}
   313 *}
   309 
   314 
   310 
   315