src/HOL/Auth/Guard/Analz.thy
changeset 17689 a04b5b43625e
parent 16417 9bc16273c2d4
child 23746 a455e69c31cc
--- a/src/HOL/Auth/Guard/Analz.thy	Wed Sep 28 11:14:26 2005 +0200
+++ b/src/HOL/Auth/Guard/Analz.thy	Wed Sep 28 11:15:33 2005 +0200
@@ -237,11 +237,6 @@
 X:analz (kparts {Z} Un kparts H)"
 by (rule analz_sub, auto)
 
-lemma Key_analz_kparts_insert: "Key K:analz (kparts {Z} Un H)
-==> Key K:analz (insert Z H)"
-apply (subgoal_tac "Key K:analz ({Z} Un H)", simp)
-by (rule_tac in_analz_subset_cong, auto dest: analz_kparts_analz)
-
 lemma Nonce_kparts_synth [rule_format]: "Y:synth (analz G)
 ==> Nonce n:kparts {Y} --> Nonce n:analz G"
 by (erule synth.induct, auto)