diff -r 05c4c6a99b3f -r bd4d37edfee4 src/Doc/Implementation/Logic.thy --- a/src/Doc/Implementation/Logic.thy Sun Oct 20 16:16:23 2019 +0200 +++ b/src/Doc/Implementation/Logic.thy Sun Oct 20 20:38:22 2019 +0200 @@ -1189,7 +1189,7 @@ @{index_ML Proofterm.reconstruct_proof: "theory -> term -> proof -> proof"} \\ @{index_ML Proofterm.expand_proof: "theory -> - (string * term option) list -> proof -> proof"} \\ + (Proofterm.thm_header -> string option) -> proof -> proof"} \\ @{index_ML Proof_Checker.thm_of_proof: "theory -> proof -> thm"} \\ @{index_ML Proof_Syntax.read_proof: "theory -> bool -> bool -> string -> proof"} \\ @{index_ML Proof_Syntax.pretty_proof: "Proof.context -> proof -> Pretty.T"} \\ @@ -1228,10 +1228,11 @@ for proofs that are constructed manually, but not for those produced automatically by the inference kernel. - \<^descr> \<^ML>\Proofterm.expand_proof\~\thy [thm\<^sub>1, \, thm\<^sub>n] prf\ expands and - reconstructs the proofs of all specified theorems, with the given (full) - proof. Theorems that are not unique specified via their name may be - disambiguated by giving their proposition. + \<^descr> \<^ML>\Proofterm.expand_proof\~\thy expand prf\ reconstructs and expands + the proofs of nested theorems according to the given \expand\ function: a + result of @{ML \SOME ""\} means full expansion, @{ML \SOME\}~\name\ means to + keep the theorem node but replace its internal name, @{ML NONE} means no + change. \<^descr> \<^ML>\Proof_Checker.thm_of_proof\~\thy prf\ turns the given (full) proof into a theorem, by replaying it using only primitive rules of the inference