doc-src/IsarImplementation/Thy/proof.thy
changeset 21827 0b1d07f79c1e
parent 20797 c1f0bc7e7d80
child 22568 ed7aa5a350ef
equal deleted inserted replaced
21826:b90d927e0a4b 21827:0b1d07f79c1e
   316   it.  The latter may depend on the local assumptions being presented
   316   it.  The latter may depend on the local assumptions being presented
   317   as facts.  The result is in HHF normal form.
   317   as facts.  The result is in HHF normal form.
   318 
   318 
   319   \item @{ML Goal.prove_multi} is simular to @{ML Goal.prove}, but
   319   \item @{ML Goal.prove_multi} is simular to @{ML Goal.prove}, but
   320   states several conclusions simultaneously.  The goal is encoded by
   320   states several conclusions simultaneously.  The goal is encoded by
   321   means of Pure conjunction; @{ML Tactic.conjunction_tac} will turn
   321   means of Pure conjunction; @{ML Goal.conjunction_tac} will turn this
   322   this into a collection of individual subgoals.
   322   into a collection of individual subgoals.
   323 
   323 
   324   \item @{ML Obtain.result}~@{text "tac thms ctxt"} eliminates the
   324   \item @{ML Obtain.result}~@{text "tac thms ctxt"} eliminates the
   325   given facts using a tactic, which results in additional fixed
   325   given facts using a tactic, which results in additional fixed
   326   variables and assumptions in the context.  Final results need to be
   326   variables and assumptions in the context.  Final results need to be
   327   exported explicitly.
   327   exported explicitly.