src/Pure/Isar/element.ML
changeset 32194 966e166d039d
parent 32091 30e2ffbba718
child 32199 82c4c570310a
equal deleted inserted replaced
32193:c314b4836031 32194:966e166d039d
   270 
   270 
   271 val refine_witness =
   271 val refine_witness =
   272   Proof.refine (Method.Basic (K (RAW_METHOD
   272   Proof.refine (Method.Basic (K (RAW_METHOD
   273     (K (ALLGOALS
   273     (K (ALLGOALS
   274       (CONJUNCTS (ALLGOALS
   274       (CONJUNCTS (ALLGOALS
   275         (CONJUNCTS (TRYALL (Tactic.rtac Drule.protectI)))))))), Position.none));
   275         (CONJUNCTS (TRYALL (Tactic.rtac Drule.protectI))))))))));
   276 
   276 
   277 fun gen_witness_proof proof after_qed wit_propss eq_props =
   277 fun gen_witness_proof proof after_qed wit_propss eq_props =
   278   let
   278   let
   279     val propss = (map o map) (fn prop => (mark_witness prop, [])) wit_propss
   279     val propss = (map o map) (fn prop => (mark_witness prop, [])) wit_propss
   280       @ [map (rpair []) eq_props];
   280       @ [map (rpair []) eq_props];