src/Pure/Isar/element.ML
changeset 60406 12cc54fac9b0
parent 60388 0c9d2a4f589d
child 60414 f25f2f2ba48c
equal deleted inserted replaced
60405:990c9fea6773 60406:12cc54fac9b0
   278       in after_qed ((map2 o map2) (curry Witness) wit_propss wits) eqs end;
   278       in after_qed ((map2 o map2) (curry Witness) wit_propss wits) eqs end;
   279   in proof after_qed' propss #> refine_witness #> Seq.hd end;
   279   in proof after_qed' propss #> refine_witness #> Seq.hd end;
   280 
   280 
   281 fun proof_local cmd goal_ctxt int after_qed' propp =
   281 fun proof_local cmd goal_ctxt int after_qed' propp =
   282   Proof.map_context (K goal_ctxt) #>
   282   Proof.map_context (K goal_ctxt) #>
   283   Proof.local_goal (K (K ())) (K I) Proof_Context.cert_propp cmd NONE
   283   Proof.internal_goal (K (K ())) (Proof_Context.get_mode goal_ctxt) cmd
   284     after_qed' (map (pair Thm.empty_binding) propp);
   284     NONE after_qed' [] (map (pair Thm.empty_binding) propp);
   285 
   285 
   286 in
   286 in
   287 
   287 
   288 fun witness_proof after_qed wit_propss =
   288 fun witness_proof after_qed wit_propss =
   289   gen_witness_proof (Proof.theorem NONE) (fn wits => fn _ => after_qed wits)
   289   gen_witness_proof (Proof.theorem NONE) (fn wits => fn _ => after_qed wits)