src/HOL/Auth/Smartcard/ShoupRubinBella.thy
changeset 21588 cd0dc678a205
parent 20048 a7964311f1fb
child 23746 a455e69c31cc
equal deleted inserted replaced
21587:a3561bfe0ada 21588:cd0dc678a205
   780          REPEAT_FIRST (eresolve_tac [asm_rl, conjE] ORELSE' hyp_subst_tac)
   780          REPEAT_FIRST (eresolve_tac [asm_rl, conjE] ORELSE' hyp_subst_tac)
   781 
   781 
   782 *}
   782 *}
   783 
   783 
   784 method_setup prepare = {*
   784 method_setup prepare = {*
   785     Method.no_args (Method.METHOD (fn facts => prepare_tac)) *}
   785     Method.no_args (Method.SIMPLE_METHOD prepare_tac) *}
   786   "to launch a few simple facts that'll help the simplifier"
   786   "to launch a few simple facts that'll help the simplifier"
   787 
   787 
   788 method_setup parts_prepare = {*
   788 method_setup parts_prepare = {*
   789     Method.no_args (Method.METHOD (fn facts => parts_prepare_tac)) *}
   789     Method.no_args (Method.SIMPLE_METHOD parts_prepare_tac) *}
   790   "additional facts to reason about parts"
   790   "additional facts to reason about parts"
   791 
   791 
   792 method_setup analz_prepare = {*
   792 method_setup analz_prepare = {*
   793     Method.no_args (Method.METHOD (fn facts => analz_prepare_tac)) *}
   793     Method.no_args (Method.SIMPLE_METHOD analz_prepare_tac) *}
   794   "additional facts to reason about analz"
   794   "additional facts to reason about analz"
   795 
   795 
   796 
   796 
   797 
   797 
   798 lemma Spy_parts_keys [simp]: "evs \<in> srb \<Longrightarrow>  
   798 lemma Spy_parts_keys [simp]: "evs \<in> srb \<Longrightarrow>  
   843 val analz_image_Key_Un_Nonce= thm "analz_image_Key_Un_Nonce"
   843 val analz_image_Key_Un_Nonce= thm "analz_image_Key_Un_Nonce"
   844 *}
   844 *}
   845 
   845 
   846 method_setup sc_analz_freshK = {*
   846 method_setup sc_analz_freshK = {*
   847     Method.ctxt_args (fn ctxt =>
   847     Method.ctxt_args (fn ctxt =>
   848      (Method.METHOD
   848      (Method.SIMPLE_METHOD
   849       (fn facts => EVERY [REPEAT_FIRST (resolve_tac [allI, ballI, impI]),
   849       (EVERY [REPEAT_FIRST (resolve_tac [allI, ballI, impI]),
   850                           REPEAT_FIRST (rtac analz_image_freshK_lemma),
   850                           REPEAT_FIRST (rtac analz_image_freshK_lemma),
   851                           ALLGOALS (asm_simp_tac (Simplifier.context ctxt analz_image_freshK_ss
   851                           ALLGOALS (asm_simp_tac (Simplifier.context ctxt analz_image_freshK_ss
   852                                     addsimps [knows_Spy_Inputs_secureM_srb_Spy,
   852                                     addsimps [knows_Spy_Inputs_secureM_srb_Spy,
   853                                               knows_Spy_Outpts_secureM_srb_Spy,
   853                                               knows_Spy_Outpts_secureM_srb_Spy,
   854                                               shouprubin_assumes_securemeans, 
   854                                               shouprubin_assumes_securemeans,