doc-src/IsarImplementation/Thy/integration.thy
changeset 21168 0f869edd6cc1
parent 20491 98ba42f19995
child 21401 faddc6504177
equal deleted inserted replaced
21167:276dd93cfa97 21168:0f869edd6cc1
   139   Toplevel.transition -> Toplevel.transition"} \\
   139   Toplevel.transition -> Toplevel.transition"} \\
   140   @{index_ML Toplevel.proof: "(Proof.state -> Proof.state) ->
   140   @{index_ML Toplevel.proof: "(Proof.state -> Proof.state) ->
   141   Toplevel.transition -> Toplevel.transition"} \\
   141   Toplevel.transition -> Toplevel.transition"} \\
   142   @{index_ML Toplevel.proofs: "(Proof.state -> Proof.state Seq.seq) ->
   142   @{index_ML Toplevel.proofs: "(Proof.state -> Proof.state Seq.seq) ->
   143   Toplevel.transition -> Toplevel.transition"} \\
   143   Toplevel.transition -> Toplevel.transition"} \\
   144   @{index_ML Toplevel.proof_to_theory: "(Proof.state -> theory) ->
   144   @{index_ML Toplevel.end_proof: "(bool -> Proof.state -> Proof.context) ->
   145   Toplevel.transition -> Toplevel.transition"} \\
   145   Toplevel.transition -> Toplevel.transition"} \\
   146   \end{mldecls}
   146   \end{mldecls}
   147 
   147 
   148   \begin{description}
   148   \begin{description}
   149 
   149 
   172 
   172 
   173   \item @{ML Toplevel.proofs}~@{text "tr"} adjoins a general proof
   173   \item @{ML Toplevel.proofs}~@{text "tr"} adjoins a general proof
   174   command, with zero or more result states (represented as a lazy
   174   command, with zero or more result states (represented as a lazy
   175   list).
   175   list).
   176 
   176 
   177   \item @{ML Toplevel.proof_to_theory}~@{text "tr"} adjoins a
   177   \item @{ML Toplevel.end_proof}~@{text "tr"} adjoins a concluding
   178   concluding proof command, that returns the resulting theory, after
   178   proof command, that returns the resulting theory, after storing the
   179   storing the resulting facts etc.
   179   resulting facts in the context etc.
   180 
   180 
   181   \end{description}
   181   \end{description}
   182 *}
   182 *}
   183 
   183 
   184 
   184