changeset 30211 | 556d1810cdad |
parent 29603 | b660ee46f2f6 |
child 30219 | 9224f88c1651 |
--- a/src/Pure/Isar/element.ML Tue Mar 03 14:07:23 2009 +0100 +++ b/src/Pure/Isar/element.ML Tue Mar 03 14:07:43 2009 +0100 @@ -296,7 +296,7 @@ gen_witness_proof (fn after_qed' => fn propss => Proof.map_context (K goal_ctxt) #> Proof.local_goal (ProofDisplay.print_results int) (K I) ProofContext.bind_propp_i - cmd NONE after_qed' (map (pair (Binding.empty, [])) propss)) + cmd NONE after_qed' (map (pair Thm.empty_binding) propss)) (fn wits => fn _ => after_qed wits) wit_propss []; end;