src/HOL/Auth/OtwayRees_AN.thy
changeset 11185 1b737b4c2108
parent 6333 b1dec44d0018
child 11230 756c5034f08b
--- a/src/HOL/Auth/OtwayRees_AN.thy	Tue Feb 27 12:28:42 2001 +0100
+++ b/src/HOL/Auth/OtwayRees_AN.thy	Tue Feb 27 16:13:23 2001 +0100
@@ -28,50 +28,50 @@
          (*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: otway;  X: synth (analz (knows Spy evs)) |]
-          ==> Says Spy B X  # evs : otway"
+    Fake "[| evs \\<in> otway;  X \\<in> synth (analz (knows Spy evs)) |]
+          ==> Says Spy B X  # evs \\<in> otway"
 
          (*A message that has been sent can be received by the
            intended recipient.*)
-    Reception "[| evsr: otway;  Says A B X : set evsr |]
-               ==> Gets B X # evsr : otway"
+    Reception "[| evsr \\<in> otway;  Says A B X \\<in>set evsr |]
+               ==> Gets B X # evsr \\<in> otway"
 
          (*Alice initiates a protocol run*)
-    OR1  "[| evs1: otway |]
-          ==> Says A B {|Agent A, Agent B, Nonce NA|} # evs1 : otway"
+    OR1  "[| evs1 \\<in> otway |]
+          ==> Says A B {|Agent A, Agent B, Nonce NA|} # evs1 \\<in> otway"
 
          (*Bob's response to Alice's message.*)
-    OR2  "[| evs2: otway;  
-             Gets B {|Agent A, Agent B, Nonce NA|} : set evs2 |]
+    OR2  "[| evs2 \\<in> otway;  
+             Gets B {|Agent A, Agent B, Nonce NA|} \\<in>set evs2 |]
           ==> Says B Server {|Agent A, Agent B, Nonce NA, Nonce NB|}
-                 # evs2 : otway"
+                 # evs2 \\<in> otway"
 
          (*The Server receives Bob's message.  Then he sends a new
            session key to Bob with a packet for forwarding to Alice.*)
-    OR3  "[| evs3: otway;  Key KAB ~: used evs3;
+    OR3  "[| evs3 \\<in> otway;  Key KAB \\<notin> used evs3;
              Gets Server {|Agent A, Agent B, Nonce NA, Nonce NB|}
-               : set evs3 |]
+               \\<in>set evs3 |]
           ==> Says Server B 
                {|Crypt (shrK A) {|Nonce NA, Agent A, Agent B, Key KAB|},
                  Crypt (shrK B) {|Nonce NB, Agent A, Agent B, Key KAB|}|}
-              # evs3 : otway"
+              # evs3 \\<in> otway"
 
          (*Bob receives the Server's (?) message and compares the Nonces with
 	   those in the message he previously sent the Server.
            Need B ~= Server because we allow messages to self.*)
-    OR4  "[| evs4: otway;  B ~= Server; 
-             Says B Server {|Agent A, Agent B, Nonce NA, Nonce NB|} : set evs4;
+    OR4  "[| evs4 \\<in> otway;  B ~= Server; 
+             Says B Server {|Agent A, Agent B, Nonce NA, Nonce NB|} \\<in>set evs4;
              Gets B {|X, Crypt(shrK B){|Nonce NB,Agent A,Agent B,Key K|}|}
-               : set evs4 |]
-          ==> Says B A X # evs4 : otway"
+               \\<in>set evs4 |]
+          ==> Says B A X # evs4 \\<in> otway"
 
          (*This message models possible leaks of session keys.  The nonces
            identify the protocol run.  B is not assumed to know shrK A.*)
-    Oops "[| evso: otway;  
+    Oops "[| evso \\<in> otway;  
              Says Server B 
                       {|Crypt (shrK A) {|Nonce NA, Agent A, Agent B, Key K|}, 
                         Crypt (shrK B) {|Nonce NB, Agent A, Agent B, Key K|}|}
-               : set evso |]
-          ==> Notes Spy {|Nonce NA, Nonce NB, Key K|} # evso : otway"
+               \\<in>set evso |]
+          ==> Notes Spy {|Nonce NA, Nonce NB, Key K|} # evso \\<in> otway"
 
 end