src/HOL/SET_Protocol/Cardholder_Registration.thy
changeset 51798 ad3a241def73
parent 42814 5af15f1e2ef6
child 55417 01fbfb60c33e
--- a/src/HOL/SET_Protocol/Cardholder_Registration.thy	Sat Apr 27 11:37:50 2013 +0200
+++ b/src/HOL/SET_Protocol/Cardholder_Registration.thy	Sat Apr 27 20:50:20 2013 +0200
@@ -536,11 +536,11 @@
 by (blast intro: analz_mono [THEN [2] rev_subsetD])
 
 method_setup valid_certificate_tac = {*
-  Args.goal_spec >> (fn quant => K (SIMPLE_METHOD'' quant
+  Args.goal_spec >> (fn quant => fn ctxt => SIMPLE_METHOD'' quant
     (fn i =>
       EVERY [ftac @{thm Gets_certificate_valid} i,
              assume_tac i,
-             etac conjE i, REPEAT (hyp_subst_tac i)])))
+             etac conjE i, REPEAT (hyp_subst_tac ctxt i)]))
 *}
 
 text{*The @{text "(no_asm)"} attribute is essential, since it retains