src/HOL/Auth/Message.thy
changeset 11245 3d9d25a3375b
parent 11230 756c5034f08b
child 11251 a6816d47f41d
--- a/src/HOL/Auth/Message.thy	Mon Apr 09 10:12:33 2001 +0200
+++ b/src/HOL/Auth/Message.thy	Mon Apr 09 14:49:51 2001 +0200
@@ -135,6 +135,11 @@
 
 use "Message_lemmas.ML"
 
+lemma Fake_parts_insert_in_Un:
+     "[|Z \<in> parts (insert X H);  X: synth (analz H)|] 
+      ==> Z \<in>  synth (analz H) \<union> parts H";
+by (blast dest: Fake_parts_insert  [THEN subsetD, dest])
+
 method_setup spy_analz = {*
     Method.no_args (Method.METHOD (fn facts => spy_analz_tac 1)) *}
     "for proving the Fake case when analz is involved"