changeset 59499 | 14095f771781 |
parent 58963 | 26bf09b95dda |
child 61984 | cdea44c775fa |
--- a/src/HOL/SET_Protocol/Purchase.thy Tue Feb 10 14:48:26 2015 +0100 +++ b/src/HOL/SET_Protocol/Purchase.thy Tue Feb 10 16:46:21 2015 +0100 @@ -482,7 +482,7 @@ method_setup valid_certificate_tac = {* Args.goal_spec >> (fn quant => fn ctxt => SIMPLE_METHOD'' quant (fn i => - EVERY [ftac @{thm Gets_certificate_valid} i, + EVERY [forward_tac ctxt @{thms Gets_certificate_valid} i, assume_tac ctxt i, REPEAT (hyp_subst_tac ctxt i)])) *}