src/HOL/Auth/WooLam.thy
author paulson
Tue, 01 Jul 1997 10:37:42 +0200
changeset 3470 8160cc3f6d40
parent 3465 e85c24717cad
child 3481 256f38c01b98
permissions -rw-r--r--
Added a comment

(*  Title:      HOL/Auth/WooLam
    ID:         $Id$
    Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
    Copyright   1996  University of Cambridge

Inductive relation "woolam" for the Woo-Lam protocol.

Simplified version from page 11 of
  Abadi and Needham.  Prudent Engineering Practice for Cryptographic Protocols.
  IEEE Trans. S.E. 22(1), 1996, pages 6-15.

Note: this differs from the Woo-Lam protocol discussed by Lowe in his paper
  Some New Attacks upon Security Protocols.
  Computer Security Foundations Workshop, 1996.
*)

WooLam = Shared + 

consts  lost    :: agent set        (*No need for it to be a variable*)
	woolam  :: event list set
inductive woolam
  intrs 
         (*Initial trace is empty*)
    Nil  "[]: woolam"

         (*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: woolam;  B ~= Spy;  
             X: synth (analz (sees lost Spy evs)) |]
          ==> Says Spy B X  # evs : woolam"

         (*Alice initiates a protocol run*)
    WL1  "[| evs: woolam;  A ~= B |]
          ==> Says A B (Agent A) # evs : woolam"

         (*Bob responds to Alice's message with a challenge.*)
    WL2  "[| evs: woolam;  A ~= B;  
             Says A' B (Agent A) : set evs |]
          ==> Says B A (Nonce NB) # evs : woolam"

         (*Alice responds to Bob's challenge by encrypting NB with her key.
           B is *not* properly determined -- Alice essentially broadcasts
           her reply.*)
    WL3  "[| evs: woolam;  A ~= B;
             Says A  B (Agent A)  : set evs;
             Says B' A (Nonce NB) : set evs |]
          ==> Says A B (Crypt (shrK A) (Nonce NB)) # evs : woolam"

         (*Bob forwards Alice's response to the Server.  NOTE: usually
           the messages are shown in chronological order, for clarity.
           But here, exchanging the two events would cause the lemma
           WL4_analz_sees_Spy to pick up the wrong assumption!*)
    WL4  "[| evs: woolam;  B ~= Server;  
             Says A'  B X         : set evs;
             Says A'' B (Agent A) : set evs |]
          ==> Says B Server {|Agent A, Agent B, X|} # evs : woolam"

         (*Server decrypts Alice's response for Bob.*)
    WL5  "[| evs: woolam;  B ~= Server;
             Says B' Server {|Agent A, Agent B, Crypt (shrK A) (Nonce NB)|}
               : set evs |]
          ==> Says Server B (Crypt (shrK B) {|Agent A, Nonce NB|})
                 # evs : woolam"

end