doc-src/IsarImplementation/Thy/document/integration.tex
changeset 26617 e99719e70925
parent 26464 aedaf65f7a57
child 26854 9b4aec46ad78
equal deleted inserted replaced
26616:b5fd3ad271ec 26617:e99719e70925
   333   \indexml{Isar.main}\verb|Isar.main: unit -> unit| \\
   333   \indexml{Isar.main}\verb|Isar.main: unit -> unit| \\
   334   \indexml{Isar.loop}\verb|Isar.loop: unit -> unit| \\
   334   \indexml{Isar.loop}\verb|Isar.loop: unit -> unit| \\
   335   \indexml{Isar.state}\verb|Isar.state: unit -> Toplevel.state| \\
   335   \indexml{Isar.state}\verb|Isar.state: unit -> Toplevel.state| \\
   336   \indexml{Isar.exn}\verb|Isar.exn: unit -> (exn * string) option| \\
   336   \indexml{Isar.exn}\verb|Isar.exn: unit -> (exn * string) option| \\
   337   \indexml{Isar.context}\verb|Isar.context: unit -> Proof.context| \\
   337   \indexml{Isar.context}\verb|Isar.context: unit -> Proof.context| \\
   338   \indexml{Isar.goal}\verb|Isar.goal: unit -> thm list * thm| \\
   338   \indexml{Isar.goal}\verb|Isar.goal: unit -> thm| \\
   339   \end{mldecls}
   339   \end{mldecls}
   340 
   340 
   341   \begin{description}
   341   \begin{description}
   342 
   342 
   343   \item \verb|Isar.main ()| invokes the Isar toplevel from {\ML},
   343   \item \verb|Isar.main ()| invokes the Isar toplevel from {\ML},
   351   after having dropped out of the Isar toplevel loop.
   351   after having dropped out of the Isar toplevel loop.
   352 
   352 
   353   \item \verb|Isar.context ()| produces the proof context from \verb|Isar.state ()|, analogous to \verb|Context.proof_of|
   353   \item \verb|Isar.context ()| produces the proof context from \verb|Isar.state ()|, analogous to \verb|Context.proof_of|
   354   (\secref{sec:generic-context}).
   354   (\secref{sec:generic-context}).
   355 
   355 
   356   \item \verb|Isar.goal ()| picks the goal configuration from \verb|Isar.state ()|, consisting on the current facts and the goal
   356   \item \verb|Isar.goal ()| picks the tactical goal from \verb|Isar.state ()|, represented as a theorem according to
   357   represented as a theorem according to \secref{sec:tactical-goals}.
   357   \secref{sec:tactical-goals}.
   358 
   358 
   359   \end{description}%
   359   \end{description}%
   360 \end{isamarkuptext}%
   360 \end{isamarkuptext}%
   361 \isamarkuptrue%
   361 \isamarkuptrue%
   362 %
   362 %