src/HOL/Auth/OtwayRees_AN.thy
changeset 32366 b269b56b6a14
parent 23746 a455e69c31cc
child 32960 69916a850301
--- a/src/HOL/Auth/OtwayRees_AN.thy	Mon Aug 10 17:00:41 2009 +0200
+++ b/src/HOL/Auth/OtwayRees_AN.thy	Thu Aug 13 17:19:10 2009 +0100
@@ -246,7 +246,7 @@
          Notes Spy {|NA, NB, Key K|} \<notin> set evs;
          A \<notin> bad;  B \<notin> bad;  evs \<in> otway |]
       ==> Key K \<notin> analz (knows Spy evs)"
-by (blast dest: Says_Server_message_form secrecy_lemma)
+  by (metis secrecy_lemma)
 
 
 text{*A's guarantee.  The Oops premise quantifies over NB because A cannot know
@@ -256,7 +256,7 @@
          \<forall>NB. Notes Spy {|NA, NB, Key K|} \<notin> set evs;
          A \<notin> bad;  B \<notin> bad;  A \<noteq> B;  evs \<in> otway |]
       ==> Key K \<notin> analz (knows Spy evs)"
-by (blast dest!: A_trusts_OR4 Spy_not_see_encrypted_key)
+  by (metis A_trusts_OR4 secrecy_lemma)