src/HOL/Auth/Yahalom2.thy
changeset 6335 7e4bffaa2a3e
parent 5434 9b4bed3f394c
child 11185 1b737b4c2108
--- a/src/HOL/Auth/Yahalom2.thy	Wed Mar 10 10:42:40 1999 +0100
+++ b/src/HOL/Auth/Yahalom2.thy	Wed Mar 10 10:42:57 1999 +0100
@@ -24,17 +24,21 @@
          (*The spy MAY say anything he CAN say.  We do not expect him to
            invent new nonces here, but he can also use NS1.  Common to
            all similar protocols.*)
-    Fake "[| evs: yahalom;  X: synth (analz (spies evs)) |]
+    Fake "[| evs: yahalom;  X: synth (analz (knows Spy evs)) |]
           ==> Says Spy B X  # evs : yahalom"
 
+         (*A message that has been sent can be received by the
+           intended recipient.*)
+    Reception "[| evsr: yahalom;  Says A B X : set evsr |]
+               ==> Gets B X # evsr : yahalom"
+
          (*Alice initiates a protocol run*)
     YM1  "[| evs1: yahalom;  Nonce NA ~: used evs1 |]
           ==> Says A B {|Agent A, Nonce NA|} # evs1 : yahalom"
 
-         (*Bob's response to Alice's message.  Bob doesn't know who 
-	   the sender is, hence the A' in the sender field.*)
+         (*Bob's response to Alice's message.*)
     YM2  "[| evs2: yahalom;  Nonce NB ~: used evs2;
-             Says A' B {|Agent A, Nonce NA|} : set evs2 |]
+             Gets B {|Agent A, Nonce NA|} : set evs2 |]
           ==> Says B Server 
                   {|Agent B, Nonce NB, Crypt (shrK B) {|Agent A, Nonce NA|}|}
                 # evs2 : yahalom"
@@ -43,8 +47,8 @@
            new session key to Alice, with a certificate for forwarding to Bob.
            Both agents are quoted in the 2nd certificate to prevent attacks!*)
     YM3  "[| evs3: yahalom;  Key KAB ~: used evs3;
-             Says B' Server {|Agent B, Nonce NB,
-			      Crypt (shrK B) {|Agent A, Nonce NA|}|}
+             Gets Server {|Agent B, Nonce NB,
+			   Crypt (shrK B) {|Agent A, Nonce NA|}|}
                : set evs3 |]
           ==> Says Server A
                {|Nonce NB, 
@@ -55,8 +59,8 @@
          (*Alice receives the Server's (?) message, checks her Nonce, and
            uses the new session key to send Bob his Nonce.*)
     YM4  "[| evs4: yahalom;  
-             Says S A {|Nonce NB, Crypt (shrK A) {|Agent B, Key K, Nonce NA|},
-                        X|}  : set evs4;
+             Gets A {|Nonce NB, Crypt (shrK A) {|Agent B, Key K, Nonce NA|},
+                      X|}  : set evs4;
              Says A B {|Agent A, Nonce NA|} : set evs4 |]
           ==> Says A B {|X, Crypt K (Nonce NB)|} # evs4 : yahalom"