src/HOL/SET-Protocol/PublicSET.thy
changeset 20048 a7964311f1fb
parent 16417 9bc16273c2d4
child 21588 cd0dc678a205
--- a/src/HOL/SET-Protocol/PublicSET.thy	Sat Jul 08 12:54:35 2006 +0200
+++ b/src/HOL/SET-Protocol/PublicSET.thy	Sat Jul 08 12:54:36 2006 +0200
@@ -360,13 +360,13 @@
                    resolve_tac [refl, conjI, Nonce_supply]))
 
 (*Tactic for possibility theorems (ML script version)*)
-fun possibility_tac state = gen_possibility_tac (simpset()) state
+fun possibility_tac state = gen_possibility_tac (simpset_of (Thm.theory_of_thm state)) state
 
 (*For harder protocols (such as SET_CR!), where we have to set up some
   nonces and keys initially*)
 fun basic_possibility_tac st = st |>
     REPEAT 
-    (ALLGOALS (asm_simp_tac (simpset() setSolver safe_solver))
+    (ALLGOALS (asm_simp_tac (simpset_of (Thm.theory_of_thm st) setSolver safe_solver))
      THEN
      REPEAT_FIRST (resolve_tac [refl, conjI]))
 *}