src/Pure/Isar/element.ML
changeset 61841 4d3527b94f2a
parent 61814 1ca1142e1711
child 62094 7d47cf67516d
--- a/src/Pure/Isar/element.ML	Sat Dec 12 15:37:42 2015 +0100
+++ b/src/Pure/Isar/element.ML	Sun Dec 13 21:56:15 2015 +0100
@@ -272,7 +272,7 @@
 local
 
 val refine_witness =
-  Proof.refine (Method.Basic (fn ctxt => EMPTY_CASES o
+  Proof.refine_singleton (Method.Basic (fn ctxt => Method.CONTEXT_TACTIC o
     K (ALLGOALS (CONJUNCTS (ALLGOALS (CONJUNCTS (TRYALL (resolve_tac ctxt [Drule.protectI]))))))));
 
 fun gen_witness_proof proof after_qed wit_propss eq_props =
@@ -283,7 +283,7 @@
     fun after_qed' thmss =
       let val (wits, eqs) = split_last ((map o map) Thm.close_derivation thmss);
       in after_qed ((map2 o map2) (curry Witness) wit_propss wits) eqs end;
-  in proof after_qed' propss #> refine_witness #> Seq.hd end;
+  in proof after_qed' propss #> refine_witness end;
 
 fun proof_local cmd goal_ctxt int after_qed propp =
   let