src/HOL/Auth/NS_Shared.thy
changeset 5359 bd539b72d484
parent 4537 4e835bd9fada
child 5434 9b4bed3f394c
equal deleted inserted replaced
5358:7e046ef59fe2 5359:bd539b72d484
    69           ==> Says A B (Crypt K {|Nonce NB, Nonce NB|}) # evs5 : ns_shared"
    69           ==> Says A B (Crypt K {|Nonce NB, Nonce NB|}) # evs5 : ns_shared"
    70   
    70   
    71          (*This message models possible leaks of session keys.
    71          (*This message models possible leaks of session keys.
    72            The two Nonces identify the protocol run: the rule insists upon
    72            The two Nonces identify the protocol run: the rule insists upon
    73            the true senders in order to make them accurate.*)
    73            the true senders in order to make them accurate.*)
    74     Oops "[| evso: ns_shared;  A ~= Spy;
    74     Oops "[| evso: ns_shared;  Says B A (Crypt K (Nonce NB)) : set evso;
    75              Says B A (Crypt K (Nonce NB)) : set evso;
       
    76              Says Server A (Crypt (shrK A) {|Nonce NA, Agent B, Key K, X|})
    75              Says Server A (Crypt (shrK A) {|Nonce NA, Agent B, Key K, X|})
    77                : set evso |]
    76                : set evso |]
    78           ==> Notes Spy {|Nonce NA, Nonce NB, Key K|} # evso : ns_shared"
    77           ==> Notes Spy {|Nonce NA, Nonce NB, Key K|} # evso : ns_shared"
    79 
    78 
    80 end
    79 end