src/Doc/IsarImplementation/Proof.thy
changeset 54883 dd04a8b654fc
parent 53015 a1119cf551e8
equal deleted inserted replaced
54882:61276a7fc369 54883:dd04a8b654fc
   277 *}
   277 *}
   278 
   278 
   279 text %mlref {*
   279 text %mlref {*
   280   \begin{mldecls}
   280   \begin{mldecls}
   281   @{index_ML_type Assumption.export} \\
   281   @{index_ML_type Assumption.export} \\
   282   @{index_ML Assumption.assume: "cterm -> thm"} \\
   282   @{index_ML Assumption.assume: "Proof.context -> cterm -> thm"} \\
   283   @{index_ML Assumption.add_assms:
   283   @{index_ML Assumption.add_assms:
   284     "Assumption.export ->
   284     "Assumption.export ->
   285   cterm list -> Proof.context -> thm list * Proof.context"} \\
   285   cterm list -> Proof.context -> thm list * Proof.context"} \\
   286   @{index_ML Assumption.add_assumes: "
   286   @{index_ML Assumption.add_assumes: "
   287   cterm list -> Proof.context -> thm list * Proof.context"} \\
   287   cterm list -> Proof.context -> thm list * Proof.context"} \\
   294   rules, which is any function of type @{ML_type "bool -> cterm list
   294   rules, which is any function of type @{ML_type "bool -> cterm list
   295   -> thm -> thm"}, where the @{ML_type "bool"} indicates goal mode,
   295   -> thm -> thm"}, where the @{ML_type "bool"} indicates goal mode,
   296   and the @{ML_type "cterm list"} the collection of assumptions to be
   296   and the @{ML_type "cterm list"} the collection of assumptions to be
   297   discharged simultaneously.
   297   discharged simultaneously.
   298 
   298 
   299   \item @{ML Assumption.assume}~@{text "A"} turns proposition @{text
   299   \item @{ML Assumption.assume}~@{text "ctxt A"} turns proposition @{text
   300   "A"} into a primitive assumption @{text "A \<turnstile> A'"}, where the
   300   "A"} into a primitive assumption @{text "A \<turnstile> A'"}, where the
   301   conclusion @{text "A'"} is in HHF normal form.
   301   conclusion @{text "A'"} is in HHF normal form.
   302 
   302 
   303   \item @{ML Assumption.add_assms}~@{text "r As"} augments the context
   303   \item @{ML Assumption.add_assms}~@{text "r As"} augments the context
   304   by assumptions @{text "As"} with export rule @{text "r"}.  The
   304   by assumptions @{text "As"} with export rule @{text "r"}.  The