src/HOL/SET_Protocol/Purchase.thy
changeset 58963 26bf09b95dda
parent 58889 5b7a9633cfa8
child 59499 14095f771781
--- a/src/HOL/SET_Protocol/Purchase.thy	Sun Nov 09 20:49:28 2014 +0100
+++ b/src/HOL/SET_Protocol/Purchase.thy	Mon Nov 10 21:49:48 2014 +0100
@@ -483,7 +483,7 @@
   Args.goal_spec >> (fn quant =>
     fn ctxt => SIMPLE_METHOD'' quant (fn i =>
       EVERY [ftac @{thm Gets_certificate_valid} i,
-             assume_tac i, REPEAT (hyp_subst_tac ctxt i)]))
+             assume_tac ctxt i, REPEAT (hyp_subst_tac ctxt i)]))
 *}