src/HOL/Auth/Shared.thy
changeset 60754 02924903a6fd
parent 59498 50b60f501b05
child 61830 4f5ab843cf5b
equal deleted inserted replaced
60753:80ca4a065a48 60754:02924903a6fd
   236 
   236 
   237 method_setup analz_freshK = {*
   237 method_setup analz_freshK = {*
   238     Scan.succeed (fn ctxt =>
   238     Scan.succeed (fn ctxt =>
   239      (SIMPLE_METHOD
   239      (SIMPLE_METHOD
   240       (EVERY [REPEAT_FIRST (resolve_tac ctxt [allI, ballI, impI]),
   240       (EVERY [REPEAT_FIRST (resolve_tac ctxt [allI, ballI, impI]),
   241           REPEAT_FIRST (rtac @{thm analz_image_freshK_lemma}),
   241           REPEAT_FIRST (resolve_tac ctxt @{thms analz_image_freshK_lemma}),
   242           ALLGOALS (asm_simp_tac (put_simpset Shared.analz_image_freshK_ss ctxt))]))) *}
   242           ALLGOALS (asm_simp_tac (put_simpset Shared.analz_image_freshK_ss ctxt))]))) *}
   243     "for proving the Session Key Compromise theorem"
   243     "for proving the Session Key Compromise theorem"
   244 
   244 
   245 method_setup possibility = {*
   245 method_setup possibility = {*
   246     Scan.succeed (fn ctxt => SIMPLE_METHOD (Shared.possibility_tac ctxt)) *}
   246     Scan.succeed (fn ctxt => SIMPLE_METHOD (Shared.possibility_tac ctxt)) *}