src/HOL/Auth/NS_Shared.thy
changeset 1976 1cff1f4fdb8a
parent 1965 789c12ea0b30
child 1997 6efba890341e
--- a/src/HOL/Auth/NS_Shared.thy	Wed Sep 11 18:00:53 1996 +0200
+++ b/src/HOL/Auth/NS_Shared.thy	Wed Sep 11 18:40:55 1996 +0200
@@ -21,12 +21,12 @@
          (*The enemy 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: ns_shared;  B ~= Enemy;  X: synth (analz (sees Enemy evs))
-          |] ==> Says Enemy B X # evs : ns_shared"
+    Fake "[| evs: ns_shared;  B ~= Enemy;  X: synth (analz (sees Enemy evs)) |]
+          ==> Says Enemy B X # evs : ns_shared"
 
          (*Alice initiates a protocol run, requesting to talk to any B*)
-    NS1  "[| evs: ns_shared;  A ~= Server
-          |] ==> Says A Server {|Agent A, Agent B, Nonce (newN evs)|} # evs
+    NS1  "[| evs: ns_shared;  A ~= Server |]
+          ==> Says A Server {|Agent A, Agent B, Nonce (newN evs)|} # evs
                  : ns_shared"
 
          (*Server's response to Alice's message.
@@ -34,8 +34,8 @@
 	   Server doesn't know who the true sender is, hence the A' in
                the sender field.*)
     NS2  "[| evs: ns_shared;  A ~= B;  A ~= Server;
-             Says A' Server {|Agent A, Agent B, Nonce NA|} : set_of_list evs
-          |] ==> Says Server A 
+             Says A' Server {|Agent A, Agent B, Nonce NA|} : set_of_list evs |]
+          ==> Says Server A 
                   (Crypt {|Nonce NA, Agent B, Key (newK evs),   
                            (Crypt {|Key (newK evs), Agent A|} (shrK B))|}
                    (shrK A)) # evs : ns_shared"
@@ -47,14 +47,14 @@
              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"
+             Says A Server {|Agent A, Agent B, Nonce NA|} : set_of_list evs |]
+          ==> Says A B X # evs : ns_shared"
 
          (*Bob's nonce exchange.  He does not know who the message came
            from, but responds to A because she is mentioned inside.*)
     NS4  "[| evs: ns_shared;  A ~= B;  
-             Says A' B (Crypt {|Key K, Agent A|} (shrK B)) : set_of_list evs
-          |] ==> Says B A (Crypt (Nonce (newN evs)) K) # evs : ns_shared"
+             Says A' B (Crypt {|Key K, Agent A|} (shrK B)) : set_of_list evs |]
+          ==> Says B A (Crypt (Nonce (newN evs)) K) # evs : ns_shared"
 
          (*Alice responds with the Nonce, if she has seen the key before.
            We do NOT use N-1 or similar as the Enemy cannot spoof such things.
@@ -64,7 +64,7 @@
     NS5  "[| evs: ns_shared;  A ~= B;  
              Says B' A (Crypt (Nonce N) K) : set_of_list evs;
              Says S  A (Crypt {|Nonce NA, Agent B, Key K, X|} (shrK A))
-               : set_of_list evs
-          |] ==> Says A B (Crypt {|Nonce N, Nonce N|} K) # evs : ns_shared"
+               : set_of_list evs |]
+          ==> Says A B (Crypt {|Nonce N, Nonce N|} K) # evs : ns_shared"
 
 end