equal
deleted
inserted
replaced
381 THEN |
381 THEN |
382 REPEAT_FIRST (resolve_tac ctxt [refl, conjI])) |
382 REPEAT_FIRST (resolve_tac ctxt [refl, conjI])) |
383 |
383 |
384 val analz_image_freshK_ss = |
384 val analz_image_freshK_ss = |
385 simpset_of |
385 simpset_of |
386 (\<^context> delsimps [image_insert, image_Un] |
386 (\<^context> delsimps @{thms image_insert image_Un} |
387 delsimps [@{thm imp_disjL}] (*reduces blow-up*) |
387 delsimps @{thms imp_disjL} (*reduces blow-up*) |
388 addsimps @{thms analz_image_freshK_simps}) |
388 addsimps @{thms analz_image_freshK_simps}) |
389 end |
389 end |
390 \<close> |
390 \<close> |
391 |
391 |
392 |
392 |
398 (*Specialized methods*) |
398 (*Specialized methods*) |
399 |
399 |
400 method_setup analz_freshK = \<open> |
400 method_setup analz_freshK = \<open> |
401 Scan.succeed (fn ctxt => |
401 Scan.succeed (fn ctxt => |
402 (SIMPLE_METHOD |
402 (SIMPLE_METHOD |
403 (EVERY [REPEAT_FIRST (resolve_tac ctxt [allI, ballI, impI]), |
403 (EVERY [REPEAT_FIRST (resolve_tac ctxt @{thms allI ballI impI}), |
404 REPEAT_FIRST (resolve_tac ctxt @{thms analz_image_freshK_lemma}), |
404 REPEAT_FIRST (resolve_tac ctxt @{thms analz_image_freshK_lemma}), |
405 ALLGOALS (asm_simp_tac (put_simpset Smartcard.analz_image_freshK_ss ctxt))])))\<close> |
405 ALLGOALS (asm_simp_tac (put_simpset Smartcard.analz_image_freshK_ss ctxt))])))\<close> |
406 "for proving the Session Key Compromise theorem" |
406 "for proving the Session Key Compromise theorem" |
407 |
407 |
408 method_setup possibility = \<open> |
408 method_setup possibility = \<open> |