src/HOL/Auth/NS_Shared.thy
changeset 2131 3106a99d30a5
parent 2069 a1c623f70407
child 2284 80ebd1a213fd
--- a/src/HOL/Auth/NS_Shared.thy	Sun Oct 27 13:47:02 1996 +0100
+++ b/src/HOL/Auth/NS_Shared.thy	Mon Oct 28 12:55:24 1996 +0100
@@ -67,10 +67,11 @@
           ==> Says A B (Crypt {|Nonce NB, Nonce NB|} K) # evs : ns_shared lost"
   
          (*This message models possible leaks of session keys.
-           The two Nonces identify the protocol run.*)
-    Revl "[| evs: ns_shared lost;  A ~= Spy;
-             Says B' A (Crypt (Nonce NB) K) : set_of_list evs;
-             Says S  A (Crypt {|Nonce NA, Agent B, Key K, X|} (shrK A))
+           The two Nonces identify the protocol run: the rule insists upon
+           the true senders in order to make them accurate.*)
+    Oops "[| evs: ns_shared lost;  A ~= Spy;
+             Says B A (Crypt (Nonce NB) K) : set_of_list evs;
+             Says Server A (Crypt {|Nonce NA, Agent B, Key K, X|} (shrK A))
                : set_of_list evs |]
           ==> Says A Spy {|Nonce NA, Nonce NB, Key K|} # evs : ns_shared lost"