src/HOL/SET-Protocol/Cardholder_Registration.thy
changeset 16417 9bc16273c2d4
parent 14218 db95d1c2f51b
child 23755 1c4672d130b1
equal deleted inserted replaced
16416:6061ae1f90f2 16417:9bc16273c2d4
     4                 Piero Tramontano
     4                 Piero Tramontano
     5 *)
     5 *)
     6 
     6 
     7 header{*The SET Cardholder Registration Protocol*}
     7 header{*The SET Cardholder Registration Protocol*}
     8 
     8 
     9 theory Cardholder_Registration = PublicSET:
     9 theory Cardholder_Registration imports PublicSET begin
    10 
    10 
    11 text{*Note: nonces seem to consist of 20 bytes.  That includes both freshness
    11 text{*Note: nonces seem to consist of 20 bytes.  That includes both freshness
    12 challenges (Chall-EE, etc.) and important secrets (CardSecret, PANsecret)
    12 challenges (Chall-EE, etc.) and important secrets (CardSecret, PANsecret)
    13 *}
    13 *}
    14 
    14