src/HOL/Auth/WooLam.thy
changeset 67613 ce654b0e6d69
parent 61956 38b73f7940af
child 76287 cdc14f94c754
--- a/src/HOL/Auth/WooLam.thy	Tue Feb 13 14:24:50 2018 +0100
+++ b/src/HOL/Auth/WooLam.thy	Thu Feb 15 12:11:00 2018 +0100
@@ -142,7 +142,7 @@
   But A may have sent the nonce to some other agent and it could have reached
   the Server via the Spy.*)
 lemma B_trusts_WL5:
-     "[| Says S B (Crypt (shrK B) \<lbrace>Agent A, Nonce NB\<rbrace>): set evs;
+     "[| Says S B (Crypt (shrK B) \<lbrace>Agent A, Nonce NB\<rbrace>) \<in> set evs;
          A \<notin> bad;  B \<notin> bad;  evs \<in> woolam  |]
       ==> \<exists>B. Says A B (Crypt (shrK A) (Nonce NB)) \<in> set evs"
 by (blast dest!: NB_Crypt_imp_Server_msg)
@@ -157,9 +157,9 @@
 
 (**CANNOT be proved because A doesn't know where challenges come from...*)
 lemma "[| A \<notin> bad;  B \<noteq> Spy;  evs \<in> woolam |]
-  ==> Crypt (shrK A) (Nonce NB) \<in> parts (spies evs) &
+  ==> Crypt (shrK A) (Nonce NB) \<in> parts (spies evs) \<and>
       Says B A (Nonce NB) \<in> set evs
-      --> Says A B (Crypt (shrK A) (Nonce NB)) \<in> set evs"
+      \<longrightarrow> Says A B (Crypt (shrK A) (Nonce NB)) \<in> set evs"
 apply (erule rev_mp, erule woolam.induct, force, simp_all, blast, auto)
 oops