# HG changeset patch # User wenzelm # Date 1684608973 -7200 # Node ID 90b64ffc48a35170a90913aab2d6d1afd5825321 # Parent 5edd5b12017d5c5c0c6791f98afc82cf98482a61 more documentation; diff -r 5edd5b12017d -r 90b64ffc48a3 src/Doc/Implementation/Proof.thy --- a/src/Doc/Implementation/Proof.thy Sat May 20 17:42:01 2023 +0200 +++ b/src/Doc/Implementation/Proof.thy Sat May 20 20:56:13 2023 +0200 @@ -271,6 +271,7 @@ @{define_ML Assumption.add_assumes: " cterm list -> Proof.context -> thm list * Proof.context"} \\ @{define_ML Assumption.export: "Proof.context -> Proof.context -> thm -> thm"} \\ + @{define_ML Assumption.export_goal: "Proof.context -> Proof.context -> thm -> thm"} \\ @{define_ML Assumption.export_term: "Proof.context -> Proof.context -> term -> term"} \\ \end{mldecls} @@ -292,9 +293,10 @@ \<^descr> \<^ML>\Assumption.export\~\inner outer thm\ exports result \thm\ from the \inner\ context back into the \outer\ one; \<^ML>\Assumption.export_goal\ - does the same in a goal context. The result is in HHF normal form. Note that - \<^ML>\Proof_Context.export\ combines \<^ML>\Variable.export\ and - \<^ML>\Assumption.export\ in the canonical way. + does the same in a goal context (\<^theory_text>\fix/assume/show\ in Isabelle/Isar). The + result is always in HHF normal form. Note that \<^ML>\Proof_Context.export\ + combines \<^ML>\Variable.export\ and \<^ML>\Assumption.export\ in the + canonical way. \<^descr> \<^ML>\Assumption.export_term\~\inner outer t\ exports term \t\ from the \inner\ context back into the \outer\ one. This is analogous to