src/HOL/Auth/OtwayRees_AN.thy
changeset 11230 756c5034f08b
parent 11185 1b737b4c2108
child 11251 a6816d47f41d
equal deleted inserted replaced
11229:f417841385b7 11230:756c5034f08b
    56                  Crypt (shrK B) {|Nonce NB, Agent A, Agent B, Key KAB|}|}
    56                  Crypt (shrK B) {|Nonce NB, Agent A, Agent B, Key KAB|}|}
    57               # evs3 \\<in> otway"
    57               # evs3 \\<in> otway"
    58 
    58 
    59          (*Bob receives the Server's (?) message and compares the Nonces with
    59          (*Bob receives the Server's (?) message and compares the Nonces with
    60 	   those in the message he previously sent the Server.
    60 	   those in the message he previously sent the Server.
    61            Need B ~= Server because we allow messages to self.*)
    61            Need B \\<noteq> Server because we allow messages to self.*)
    62     OR4  "[| evs4 \\<in> otway;  B ~= Server; 
    62     OR4  "[| evs4 \\<in> otway;  B \\<noteq> Server; 
    63              Says B Server {|Agent A, Agent B, Nonce NA, Nonce NB|} \\<in>set evs4;
    63              Says B Server {|Agent A, Agent B, Nonce NA, Nonce NB|} \\<in>set evs4;
    64              Gets B {|X, Crypt(shrK B){|Nonce NB,Agent A,Agent B,Key K|}|}
    64              Gets B {|X, Crypt(shrK B){|Nonce NB,Agent A,Agent B,Key K|}|}
    65                \\<in>set evs4 |]
    65                \\<in>set evs4 |]
    66           ==> Says B A X # evs4 \\<in> otway"
    66           ==> Says B A X # evs4 \\<in> otway"
    67 
    67