src/HOL/Auth/NS_Shared.thy
changeset 1997 6efba890341e
parent 1976 1cff1f4fdb8a
child 2032 1bbf1bdcaf56
--- a/src/HOL/Auth/NS_Shared.thy	Fri Sep 13 13:20:22 1996 +0200
+++ b/src/HOL/Auth/NS_Shared.thy	Fri Sep 13 13:22:08 1996 +0200
@@ -41,12 +41,10 @@
                    (shrK A)) # evs : ns_shared"
 
           (*We can't assume S=Server.  Agent A "remembers" her nonce.
-            May assume WLOG that she is NOT the Enemy: the Fake rule
-            covers this case.  Can inductively show A ~= Server*)
+            Can inductively show A ~= Server*)
     NS3  "[| evs: ns_shared;  A ~= B;
              Says S A (Crypt {|Nonce NA, Agent B, Key K, X|} (shrK A)) 
                : set_of_list evs;
-             A = Friend i;
              Says A Server {|Agent A, Agent B, Nonce NA|} : set_of_list evs |]
           ==> Says A B X # evs : ns_shared"