doc-src/IsarImplementation/Thy/proof.thy
changeset 20547 796ae7fa1049
parent 20542 a54ca4e90874
child 20797 c1f0bc7e7d80
equal deleted inserted replaced
20546:8923deb735ad 20547:796ae7fa1049
   288   \begin{mldecls}
   288   \begin{mldecls}
   289   @{index_ML SUBPROOF:
   289   @{index_ML SUBPROOF:
   290   "({context: Proof.context, schematics: ctyp list * cterm list,
   290   "({context: Proof.context, schematics: ctyp list * cterm list,
   291     params: cterm list, asms: cterm list, concl: cterm,
   291     params: cterm list, asms: cterm list, concl: cterm,
   292     prems: thm list} -> tactic) -> Proof.context -> int -> tactic"} \\
   292     prems: thm list} -> tactic) -> Proof.context -> int -> tactic"} \\
       
   293   \end{mldecls}
       
   294   \begin{mldecls}
   293   @{index_ML Goal.prove: "Proof.context -> string list -> term list -> term ->
   295   @{index_ML Goal.prove: "Proof.context -> string list -> term list -> term ->
   294   ({prems: thm list, context: Proof.context} -> tactic) -> thm"} \\
   296   ({prems: thm list, context: Proof.context} -> tactic) -> thm"} \\
   295   @{index_ML Goal.prove_multi: "Proof.context -> string list -> term list -> term list ->
   297   @{index_ML Goal.prove_multi: "Proof.context -> string list -> term list -> term list ->
   296   ({prems: thm list, context: Proof.context} -> tactic) -> thm list"} \\
   298   ({prems: thm list, context: Proof.context} -> tactic) -> thm list"} \\
       
   299   \end{mldecls}
       
   300   \begin{mldecls}
   297   @{index_ML Obtain.result: "(Proof.context -> tactic) ->
   301   @{index_ML Obtain.result: "(Proof.context -> tactic) ->
   298   thm list -> Proof.context -> (cterm list * thm list) * Proof.context"} \\
   302   thm list -> Proof.context -> (cterm list * thm list) * Proof.context"} \\
   299   \end{mldecls}
   303   \end{mldecls}
   300 
   304 
   301   \begin{description}
   305   \begin{description}