doc-src/IsarImplementation/Thy/integration.thy
changeset 18590 f6a553aa3d81
parent 18563 1df7022eac6f
child 20025 95aeaa3ef35d
equal deleted inserted replaced
18589:c27c9fa9e83d 18590:f6a553aa3d81
   134   Toplevel.transition -> Toplevel.transition"} \\
   134   Toplevel.transition -> Toplevel.transition"} \\
   135   @{index_ML Toplevel.theory: "(theory -> theory) ->
   135   @{index_ML Toplevel.theory: "(theory -> theory) ->
   136   Toplevel.transition -> Toplevel.transition"} \\
   136   Toplevel.transition -> Toplevel.transition"} \\
   137   @{index_ML Toplevel.theory_to_proof: "(theory -> Proof.state) ->
   137   @{index_ML Toplevel.theory_to_proof: "(theory -> Proof.state) ->
   138   Toplevel.transition -> Toplevel.transition"} \\
   138   Toplevel.transition -> Toplevel.transition"} \\
   139   @{index_ML Toplevel.theory_theory_to_proof: "(theory -> Proof.state) ->
       
   140   Toplevel.transition -> Toplevel.transition"} \\
       
   141   @{index_ML Toplevel.proof: "(Proof.state -> Proof.state) ->
   139   @{index_ML Toplevel.proof: "(Proof.state -> Proof.state) ->
   142   Toplevel.transition -> Toplevel.transition"} \\
   140   Toplevel.transition -> Toplevel.transition"} \\
   143   @{index_ML Toplevel.proofs: "(Proof.state -> Proof.state Seq.seq) ->
   141   @{index_ML Toplevel.proofs: "(Proof.state -> Proof.state Seq.seq) ->
   144   Toplevel.transition -> Toplevel.transition"} \\
   142   Toplevel.transition -> Toplevel.transition"} \\
   145   @{index_ML Toplevel.proof_to_theory: "(Proof.state -> theory) ->
   143   @{index_ML Toplevel.proof_to_theory: "(Proof.state -> theory) ->
   158   \item @{ML Toplevel.keep} adjoins a diagnostic function.
   156   \item @{ML Toplevel.keep} adjoins a diagnostic function.
   159 
   157 
   160   \item @{ML Toplevel.theory} adjoins a theory transformer.
   158   \item @{ML Toplevel.theory} adjoins a theory transformer.
   161 
   159 
   162   \item @{ML Toplevel.theory_to_proof} adjoins a global goal function,
   160   \item @{ML Toplevel.theory_to_proof} adjoins a global goal function,
   163   which turns a theory into a proof state.  The theory must not be
   161   which turns a theory into a proof state.  The theory may be changed
   164   changed here!  The generic Isar goal setup includes an argument that
   162   before entering the proof; the generic Isar goal setup includes an
   165   specifies how to apply the proven result to the theory, when the
   163   argument that specifies how to apply the proven result to the
   166   proof is finished.
   164   theory, when the proof is finished.
   167 
       
   168   \item @{ML Toplevel.theory_theory_to_proof} is like @{ML
       
   169   Toplevel.theory_to_proof}, but allows the initial theory to be
       
   170   changed before entering proof state.
       
   171 
   165 
   172   \item @{ML Toplevel.proof} adjoins a deterministic proof command,
   166   \item @{ML Toplevel.proof} adjoins a deterministic proof command,
   173   with a singleton result state.
   167   with a singleton result state.
   174 
   168 
   175   \item @{ML Toplevel.proofs} adjoins a general proof command, with
   169   \item @{ML Toplevel.proofs} adjoins a general proof command, with