src/HOL/Auth/Message.thy
changeset 11245 3d9d25a3375b
parent 11230 756c5034f08b
child 11251 a6816d47f41d
equal deleted inserted replaced
11244:ca1de97d67c8 11245:3d9d25a3375b
   133 inductive_cases MPair_synth [elim!]: "{|X,Y|} \<in> synth H"
   133 inductive_cases MPair_synth [elim!]: "{|X,Y|} \<in> synth H"
   134 inductive_cases Crypt_synth [elim!]: "Crypt K X \<in> synth H"
   134 inductive_cases Crypt_synth [elim!]: "Crypt K X \<in> synth H"
   135 
   135 
   136 use "Message_lemmas.ML"
   136 use "Message_lemmas.ML"
   137 
   137 
       
   138 lemma Fake_parts_insert_in_Un:
       
   139      "[|Z \<in> parts (insert X H);  X: synth (analz H)|] 
       
   140       ==> Z \<in>  synth (analz H) \<union> parts H";
       
   141 by (blast dest: Fake_parts_insert  [THEN subsetD, dest])
       
   142 
   138 method_setup spy_analz = {*
   143 method_setup spy_analz = {*
   139     Method.no_args (Method.METHOD (fn facts => spy_analz_tac 1)) *}
   144     Method.no_args (Method.METHOD (fn facts => spy_analz_tac 1)) *}
   140     "for proving the Fake case when analz is involved"
   145     "for proving the Fake case when analz is involved"
   141 
   146 
   142 end
   147 end