src/HOL/Auth/Public.thy
changeset 21588 cd0dc678a205
parent 21404 eb85850d3eb7
child 21619 dea0914773f7
--- a/src/HOL/Auth/Public.thy	Wed Nov 29 15:44:46 2006 +0100
+++ b/src/HOL/Auth/Public.thy	Wed Nov 29 15:44:51 2006 +0100
@@ -415,8 +415,8 @@
 
 method_setup analz_freshK = {*
     Method.ctxt_args (fn ctxt =>
-     (Method.METHOD
-      (fn facts => EVERY [REPEAT_FIRST (resolve_tac [allI, ballI, impI]),
+     (Method.SIMPLE_METHOD
+      (EVERY [REPEAT_FIRST (resolve_tac [allI, ballI, impI]),
                           REPEAT_FIRST (rtac analz_image_freshK_lemma),
                           ALLGOALS (asm_simp_tac (Simplifier.context ctxt analz_image_freshK_ss))]))) *}
     "for proving the Session Key Compromise theorem"
@@ -449,8 +449,7 @@
 
 method_setup possibility = {*
     Method.ctxt_args (fn ctxt =>
-        Method.METHOD (fn facts =>
-            gen_possibility_tac (local_simpset_of ctxt))) *}
+        Method.SIMPLE_METHOD (gen_possibility_tac (local_simpset_of ctxt))) *}
     "for proving possibility theorems"
 
 end