src/HOL/SET_Protocol/Merchant_Registration.thy
author wenzelm
Sat, 18 Jan 2025 13:20:47 +0100
changeset 81913 5b9aca9b073b
parent 69597 ff784d5a5bfb
permissions -rw-r--r--
tuned names;
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
33028
9aa8bfb1649d modernized session SET_Protocol;
wenzelm
parents: 32960
diff changeset
     1
(*  Title:      HOL/SET_Protocol/Merchant_Registration.thy
32960
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 24123
diff changeset
     2
    Author:     Giampaolo Bella
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 24123
diff changeset
     3
    Author:     Fabio Massacci
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 24123
diff changeset
     4
    Author:     Lawrence C Paulson
14199
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
     5
*)
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
     6
63167
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 61984
diff changeset
     7
section\<open>The SET Merchant Registration Protocol\<close>
14199
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
     8
33028
9aa8bfb1649d modernized session SET_Protocol;
wenzelm
parents: 32960
diff changeset
     9
theory Merchant_Registration
9aa8bfb1649d modernized session SET_Protocol;
wenzelm
parents: 32960
diff changeset
    10
imports Public_SET
9aa8bfb1649d modernized session SET_Protocol;
wenzelm
parents: 32960
diff changeset
    11
begin
14199
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
    12
63167
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 61984
diff changeset
    13
text\<open>Copmpared with Cardholder Reigstration, \<open>KeyCryptKey\<close> is not
14199
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
    14
  needed: no session key encrypts another.  Instead we
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
    15
  prove the "key compromise" theorems for sets KK that contain no private
69597
ff784d5a5bfb isabelle update -u control_cartouches;
wenzelm
parents: 67613
diff changeset
    16
  encryption keys (\<^term>\<open>priEK C\<close>).\<close>
14199
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
    17
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
    18
23755
1c4672d130b1 Adapted to new inductive definition package.
berghofe
parents: 16417
diff changeset
    19
inductive_set
1c4672d130b1 Adapted to new inductive definition package.
berghofe
parents: 16417
diff changeset
    20
  set_mr :: "event list set"
1c4672d130b1 Adapted to new inductive definition package.
berghofe
parents: 16417
diff changeset
    21
where
14199
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
    22
67443
3abf6a722518 standardized towards new-style formal comments: isabelle update_comments;
wenzelm
parents: 63167
diff changeset
    23
  Nil:    \<comment> \<open>Initial trace is empty\<close>
32960
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 24123
diff changeset
    24
           "[] \<in> set_mr"
14199
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
    25
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
    26
67443
3abf6a722518 standardized towards new-style formal comments: isabelle update_comments;
wenzelm
parents: 63167
diff changeset
    27
| Fake:    \<comment> \<open>The spy MAY say anything he CAN say.\<close>
32960
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 24123
diff changeset
    28
           "[| evsf \<in> set_mr; X \<in> synth (analz (knows Spy evsf)) |]
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 24123
diff changeset
    29
            ==> Says Spy B X  # evsf \<in> set_mr"
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 24123
diff changeset
    30
        
14199
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
    31
67443
3abf6a722518 standardized towards new-style formal comments: isabelle update_comments;
wenzelm
parents: 63167
diff changeset
    32
| Reception: \<comment> \<open>If A sends a message X to B, then B might receive it\<close>
32960
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 24123
diff changeset
    33
             "[| evsr \<in> set_mr; Says A B X \<in> set evsr |]
14199
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
    34
              ==> Gets B X  # evsr \<in> set_mr"
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
    35
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
    36
67443
3abf6a722518 standardized towards new-style formal comments: isabelle update_comments;
wenzelm
parents: 63167
diff changeset
    37
| SET_MR1: \<comment> \<open>RegFormReq: M requires a registration form to a CA\<close>
32960
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 24123
diff changeset
    38
           "[| evs1 \<in> set_mr; M = Merchant k; Nonce NM1 \<notin> used evs1 |]
61984
cdea44c775fa more symbols;
wenzelm
parents: 58889
diff changeset
    39
            ==> Says M (CA i) \<lbrace>Agent M, Nonce NM1\<rbrace> # evs1 \<in> set_mr"
14199
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
    40
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
    41
67443
3abf6a722518 standardized towards new-style formal comments: isabelle update_comments;
wenzelm
parents: 63167
diff changeset
    42
| SET_MR2: \<comment> \<open>RegFormRes: CA replies with the registration form and the 
63167
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 61984
diff changeset
    43
               certificates for her keys\<close>
14199
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
    44
  "[| evs2 \<in> set_mr; Nonce NCA \<notin> used evs2;
61984
cdea44c775fa more symbols;
wenzelm
parents: 58889
diff changeset
    45
      Gets (CA i) \<lbrace>Agent M, Nonce NM1\<rbrace> \<in> set evs2 |]
cdea44c775fa more symbols;
wenzelm
parents: 58889
diff changeset
    46
   ==> Says (CA i) M \<lbrace>sign (priSK (CA i)) \<lbrace>Agent M, Nonce NM1, Nonce NCA\<rbrace>,
32960
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 24123
diff changeset
    47
                       cert (CA i) (pubEK (CA i)) onlyEnc (priSK RCA),
61984
cdea44c775fa more symbols;
wenzelm
parents: 58889
diff changeset
    48
                       cert (CA i) (pubSK (CA i)) onlySig (priSK RCA) \<rbrace>
32960
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 24123
diff changeset
    49
         # evs2 \<in> set_mr"
14199
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
    50
23755
1c4672d130b1 Adapted to new inductive definition package.
berghofe
parents: 16417
diff changeset
    51
| SET_MR3:
67443
3abf6a722518 standardized towards new-style formal comments: isabelle update_comments;
wenzelm
parents: 63167
diff changeset
    52
         \<comment> \<open>CertReq: M submits the key pair to be certified.  The Notes
14199
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
    53
             event allows KM1 to be lost if M is compromised. Piero remarks
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
    54
             that the agent mentioned inside the signature is not verified to
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
    55
             correspond to M.  As in CR, each Merchant has fixed key pairs.  M
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
    56
             is only optionally required to send NCA back, so M doesn't do so
63167
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 61984
diff changeset
    57
             in the model\<close>
14199
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
    58
  "[| evs3 \<in> set_mr; M = Merchant k; Nonce NM2 \<notin> used evs3;
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
    59
      Key KM1 \<notin> used evs3;  KM1 \<in> symKeys;
61984
cdea44c775fa more symbols;
wenzelm
parents: 58889
diff changeset
    60
      Gets M \<lbrace>sign (invKey SKi) \<lbrace>Agent X, Nonce NM1, Nonce NCA\<rbrace>,
32960
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 24123
diff changeset
    61
               cert (CA i) EKi onlyEnc (priSK RCA),
61984
cdea44c775fa more symbols;
wenzelm
parents: 58889
diff changeset
    62
               cert (CA i) SKi onlySig (priSK RCA) \<rbrace>
32960
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 24123
diff changeset
    63
        \<in> set evs3;
61984
cdea44c775fa more symbols;
wenzelm
parents: 58889
diff changeset
    64
      Says M (CA i) \<lbrace>Agent M, Nonce NM1\<rbrace> \<in> set evs3 |]
14199
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
    65
   ==> Says M (CA i)
61984
cdea44c775fa more symbols;
wenzelm
parents: 58889
diff changeset
    66
            \<lbrace>Crypt KM1 (sign (priSK M) \<lbrace>Agent M, Nonce NM2,
cdea44c775fa more symbols;
wenzelm
parents: 58889
diff changeset
    67
                                          Key (pubSK M), Key (pubEK M)\<rbrace>),
cdea44c775fa more symbols;
wenzelm
parents: 58889
diff changeset
    68
              Crypt EKi (Key KM1)\<rbrace>
cdea44c775fa more symbols;
wenzelm
parents: 58889
diff changeset
    69
         # Notes M \<lbrace>Key KM1, Agent (CA i)\<rbrace>
32960
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 24123
diff changeset
    70
         # evs3 \<in> set_mr"
14199
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
    71
23755
1c4672d130b1 Adapted to new inductive definition package.
berghofe
parents: 16417
diff changeset
    72
| SET_MR4:
67443
3abf6a722518 standardized towards new-style formal comments: isabelle update_comments;
wenzelm
parents: 63167
diff changeset
    73
         \<comment> \<open>CertRes: CA issues the certificates for merSK and merEK,
14199
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
    74
             while checking never to have certified the m even
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
    75
             separately. NOTE: In Cardholder Registration the
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
    76
             corresponding rule (6) doesn't use the "sign" primitive. "The
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
    77
             CertRes shall be signed but not encrypted if the EE is a Merchant
63167
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 61984
diff changeset
    78
             or Payment Gateway."-- Programmer's Guide, page 191.\<close>
14199
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
    79
    "[| evs4 \<in> set_mr; M = Merchant k;
32960
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 24123
diff changeset
    80
        merSK \<notin> symKeys;  merEK \<notin> symKeys;
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 24123
diff changeset
    81
        Notes (CA i) (Key merSK) \<notin> set evs4;
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 24123
diff changeset
    82
        Notes (CA i) (Key merEK) \<notin> set evs4;
61984
cdea44c775fa more symbols;
wenzelm
parents: 58889
diff changeset
    83
        Gets (CA i) \<lbrace>Crypt KM1 (sign (invKey merSK)
cdea44c775fa more symbols;
wenzelm
parents: 58889
diff changeset
    84
                                 \<lbrace>Agent M, Nonce NM2, Key merSK, Key merEK\<rbrace>),
cdea44c775fa more symbols;
wenzelm
parents: 58889
diff changeset
    85
                      Crypt (pubEK (CA i)) (Key KM1) \<rbrace>
32960
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 24123
diff changeset
    86
          \<in> set evs4 |]
61984
cdea44c775fa more symbols;
wenzelm
parents: 58889
diff changeset
    87
    ==> Says (CA i) M \<lbrace>sign (priSK(CA i)) \<lbrace>Agent M, Nonce NM2, Agent(CA i)\<rbrace>,
32960
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 24123
diff changeset
    88
                        cert  M      merSK    onlySig (priSK (CA i)),
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 24123
diff changeset
    89
                        cert  M      merEK    onlyEnc (priSK (CA i)),
61984
cdea44c775fa more symbols;
wenzelm
parents: 58889
diff changeset
    90
                        cert (CA i) (pubSK (CA i)) onlySig (priSK RCA)\<rbrace>
32960
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 24123
diff changeset
    91
          # Notes (CA i) (Key merSK)
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 24123
diff changeset
    92
          # Notes (CA i) (Key merEK)
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 24123
diff changeset
    93
          # evs4 \<in> set_mr"
14199
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
    94
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
    95
63167
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 61984
diff changeset
    96
text\<open>Note possibility proofs are missing.\<close>
14199
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
    97
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
    98
declare Says_imp_knows_Spy [THEN parts.Inj, dest]
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
    99
declare parts.Body [dest]
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   100
declare analz_into_parts [dest]
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   101
declare Fake_parts_insert_in_Un [dest]
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   102
63167
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 61984
diff changeset
   103
text\<open>General facts about message reception\<close>
14199
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   104
lemma Gets_imp_Says:
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   105
     "[| Gets B X \<in> set evs; evs \<in> set_mr |] ==> \<exists>A. Says A B X \<in> set evs"
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   106
apply (erule rev_mp)
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   107
apply (erule set_mr.induct, auto)
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   108
done
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   109
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   110
lemma Gets_imp_knows_Spy:
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   111
     "[| Gets B X \<in> set evs; evs \<in> set_mr |]  ==> X \<in> knows Spy evs"
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   112
by (blast dest!: Gets_imp_Says Says_imp_knows_Spy)
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   113
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   114
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   115
declare Gets_imp_knows_Spy [THEN parts.Inj, dest]
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   116
63167
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 61984
diff changeset
   117
subsubsection\<open>Proofs on keys\<close>
14199
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   118
63167
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 61984
diff changeset
   119
text\<open>Spy never sees an agent's private keys! (unless it's bad at start)\<close>
14199
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   120
lemma Spy_see_private_Key [simp]:
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   121
     "evs \<in> set_mr
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   122
      ==> (Key(invKey (publicKey b A)) \<in> parts(knows Spy evs)) = (A \<in> bad)"
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   123
apply (erule set_mr.induct)
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   124
apply (auto dest!: Gets_imp_knows_Spy [THEN parts.Inj])
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   125
done
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   126
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   127
lemma Spy_analz_private_Key [simp]:
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   128
     "evs \<in> set_mr ==>
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   129
     (Key(invKey (publicKey b A)) \<in> analz(knows Spy evs)) = (A \<in> bad)"
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   130
by auto
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   131
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   132
declare Spy_see_private_Key [THEN [2] rev_iffD1, dest!]
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   133
declare Spy_analz_private_Key [THEN [2] rev_iffD1, dest!]
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   134
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   135
(*This is to state that the signed keys received in step 4
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   136
  are into parts - rather than installing sign_def each time.
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   137
  Needed in Spy_see_priSK_RCA, Spy_see_priEK and in Spy_see_priSK
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   138
Goal "[|Gets C \<lbrace>Crypt KM1
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   139
                (sign K \<lbrace>Agent M, Nonce NM2, Key merSK, Key merEK\<rbrace>), X\<rbrace>
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   140
          \<in> set evs;  evs \<in> set_mr |]
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   141
    ==> Key merSK \<in> parts (knows Spy evs) \<and>
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   142
        Key merEK \<in> parts (knows Spy evs)"
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   143
by (fast_tac (claset() addss (simpset())) 1);
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   144
qed "signed_keys_in_parts";
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   145
???*)
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   146
63167
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 61984
diff changeset
   147
text\<open>Proofs on certificates -
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 61984
diff changeset
   148
  they hold, as in CR, because RCA's keys are secure\<close>
14199
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   149
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   150
lemma Crypt_valid_pubEK:
61984
cdea44c775fa more symbols;
wenzelm
parents: 58889
diff changeset
   151
     "[| Crypt (priSK RCA) \<lbrace>Agent (CA i), Key EKi, onlyEnc\<rbrace>
14199
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   152
           \<in> parts (knows Spy evs);
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   153
         evs \<in> set_mr |] ==> EKi = pubEK (CA i)"
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   154
apply (erule rev_mp)
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   155
apply (erule set_mr.induct, auto)
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   156
done
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   157
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   158
lemma certificate_valid_pubEK:
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   159
    "[| cert (CA i) EKi onlyEnc (priSK RCA) \<in> parts (knows Spy evs);
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   160
        evs \<in> set_mr |]
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   161
     ==> EKi = pubEK (CA i)"
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   162
apply (unfold cert_def signCert_def)
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   163
apply (blast dest!: Crypt_valid_pubEK)
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   164
done
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   165
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   166
lemma Crypt_valid_pubSK:
61984
cdea44c775fa more symbols;
wenzelm
parents: 58889
diff changeset
   167
     "[| Crypt (priSK RCA) \<lbrace>Agent (CA i), Key SKi, onlySig\<rbrace>
14199
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   168
           \<in> parts (knows Spy evs);
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   169
         evs \<in> set_mr |] ==> SKi = pubSK (CA i)"
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   170
apply (erule rev_mp)
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   171
apply (erule set_mr.induct, auto)
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   172
done
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   173
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   174
lemma certificate_valid_pubSK:
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   175
    "[| cert (CA i) SKi onlySig (priSK RCA) \<in> parts (knows Spy evs);
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   176
        evs \<in> set_mr |] ==> SKi = pubSK (CA i)"
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   177
apply (unfold cert_def signCert_def)
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   178
apply (blast dest!: Crypt_valid_pubSK)
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   179
done
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   180
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   181
lemma Gets_certificate_valid:
61984
cdea44c775fa more symbols;
wenzelm
parents: 58889
diff changeset
   182
     "[| Gets A \<lbrace> X, cert (CA i) EKi onlyEnc (priSK RCA),
cdea44c775fa more symbols;
wenzelm
parents: 58889
diff changeset
   183
                      cert (CA i) SKi onlySig (priSK RCA)\<rbrace> \<in> set evs;
14199
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   184
         evs \<in> set_mr |]
67613
ce654b0e6d69 more symbols;
wenzelm
parents: 67443
diff changeset
   185
      ==> EKi = pubEK (CA i) \<and> SKi = pubSK (CA i)"
14199
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   186
by (blast dest: certificate_valid_pubEK certificate_valid_pubSK)
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   187
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   188
63167
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 61984
diff changeset
   189
text\<open>Nobody can have used non-existent keys!\<close>
14199
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   190
lemma new_keys_not_used [rule_format,simp]:
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   191
     "evs \<in> set_mr
67613
ce654b0e6d69 more symbols;
wenzelm
parents: 67443
diff changeset
   192
      ==> Key K \<notin> used evs \<longrightarrow> K \<in> symKeys \<longrightarrow>
14199
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   193
          K \<notin> keysFor (parts (knows Spy evs))"
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   194
apply (erule set_mr.induct, simp_all)
67443
3abf6a722518 standardized towards new-style formal comments: isabelle update_comments;
wenzelm
parents: 63167
diff changeset
   195
apply (force dest!: usedI keysFor_parts_insert)  \<comment> \<open>Fake\<close>
3abf6a722518 standardized towards new-style formal comments: isabelle update_comments;
wenzelm
parents: 63167
diff changeset
   196
apply force  \<comment> \<open>Message 2\<close>
3abf6a722518 standardized towards new-style formal comments: isabelle update_comments;
wenzelm
parents: 63167
diff changeset
   197
apply (blast dest: Gets_certificate_valid)  \<comment> \<open>Message 3\<close>
3abf6a722518 standardized towards new-style formal comments: isabelle update_comments;
wenzelm
parents: 63167
diff changeset
   198
apply force  \<comment> \<open>Message 4\<close>
14199
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   199
done
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   200
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   201
63167
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 61984
diff changeset
   202
subsubsection\<open>New Versions: As Above, but Generalized with the Kk Argument\<close>
14199
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   203
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   204
lemma gen_new_keys_not_used [rule_format]:
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   205
     "evs \<in> set_mr
67613
ce654b0e6d69 more symbols;
wenzelm
parents: 67443
diff changeset
   206
      ==> Key K \<notin> used evs \<longrightarrow> K \<in> symKeys \<longrightarrow>
ce654b0e6d69 more symbols;
wenzelm
parents: 67443
diff changeset
   207
          K \<notin> keysFor (parts (Key`KK \<union> knows Spy evs))"
14199
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   208
by auto
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   209
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   210
lemma gen_new_keys_not_analzd:
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   211
     "[|Key K \<notin> used evs; K \<in> symKeys; evs \<in> set_mr |]
67613
ce654b0e6d69 more symbols;
wenzelm
parents: 67443
diff changeset
   212
      ==> K \<notin> keysFor (analz (Key`KK \<union> knows Spy evs))"
14199
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   213
by (blast intro: keysFor_mono [THEN [2] rev_subsetD]
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   214
          dest: gen_new_keys_not_used)
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   215
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   216
lemma analz_Key_image_insert_eq:
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   217
     "[|Key K \<notin> used evs; K \<in> symKeys; evs \<in> set_mr |]
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   218
      ==> analz (Key ` (insert K KK) \<union> knows Spy evs) =
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   219
          insert (Key K) (analz (Key ` KK \<union> knows Spy evs))"
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   220
by (simp add: gen_new_keys_not_analzd)
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   221
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   222
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   223
lemma Crypt_parts_imp_used:
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   224
     "[|Crypt K X \<in> parts (knows Spy evs);
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   225
        K \<in> symKeys; evs \<in> set_mr |] ==> Key K \<in> used evs"
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   226
apply (rule ccontr)
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   227
apply (force dest: new_keys_not_used Crypt_imp_invKey_keysFor)
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   228
done
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   229
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   230
lemma Crypt_analz_imp_used:
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   231
     "[|Crypt K X \<in> analz (knows Spy evs);
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   232
        K \<in> symKeys; evs \<in> set_mr |] ==> Key K \<in> used evs"
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   233
by (blast intro: Crypt_parts_imp_used)
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   234
63167
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 61984
diff changeset
   235
text\<open>Rewriting rule for private encryption keys.  Analogous rewriting rules
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 61984
diff changeset
   236
for other keys aren't needed.\<close>
14199
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   237
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   238
lemma parts_image_priEK:
67613
ce654b0e6d69 more symbols;
wenzelm
parents: 67443
diff changeset
   239
     "[|Key (priEK (CA i)) \<in> parts (Key`KK \<union> (knows Spy evs));
14199
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   240
        evs \<in> set_mr|] ==> priEK (CA i) \<in> KK | CA i \<in> bad"
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   241
by auto
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   242
63167
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 61984
diff changeset
   243
text\<open>trivial proof because (priEK (CA i)) never appears even in (parts evs)\<close>
14199
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   244
lemma analz_image_priEK:
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   245
     "evs \<in> set_mr ==>
67613
ce654b0e6d69 more symbols;
wenzelm
parents: 67443
diff changeset
   246
          (Key (priEK (CA i)) \<in> analz (Key`KK \<union> (knows Spy evs))) =
14199
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   247
          (priEK (CA i) \<in> KK | CA i \<in> bad)"
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   248
by (blast dest!: parts_image_priEK intro: analz_mono [THEN [2] rev_subsetD])
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   249
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   250
63167
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 61984
diff changeset
   251
subsection\<open>Secrecy of Session Keys\<close>
14199
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   252
63167
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 61984
diff changeset
   253
text\<open>This holds because if (priEK (CA i)) appears in any traffic then it must
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 61984
diff changeset
   254
  be known to the Spy, by \<open>Spy_see_private_Key\<close>\<close>
14199
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   255
lemma merK_neq_priEK:
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   256
     "[|Key merK \<notin> analz (knows Spy evs);
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   257
        Key merK \<in> parts (knows Spy evs);
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   258
        evs \<in> set_mr|] ==> merK \<noteq> priEK C"
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   259
by blast
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   260
63167
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 61984
diff changeset
   261
text\<open>Lemma for message 4: either merK is compromised (when we don't care)
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 61984
diff changeset
   262
  or else merK hasn't been used to encrypt K.\<close>
14199
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   263
lemma msg4_priEK_disj:
61984
cdea44c775fa more symbols;
wenzelm
parents: 58889
diff changeset
   264
     "[|Gets B \<lbrace>Crypt KM1
cdea44c775fa more symbols;
wenzelm
parents: 58889
diff changeset
   265
                       (sign K \<lbrace>Agent M, Nonce NM2, Key merSK, Key merEK\<rbrace>),
cdea44c775fa more symbols;
wenzelm
parents: 58889
diff changeset
   266
                 Y\<rbrace> \<in> set evs;
14199
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   267
        evs \<in> set_mr|]
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   268
  ==> (Key merSK \<in> analz (knows Spy evs) | merSK \<notin> range(\<lambda>C. priEK C))
67613
ce654b0e6d69 more symbols;
wenzelm
parents: 67443
diff changeset
   269
   \<and>  (Key merEK \<in> analz (knows Spy evs) | merEK \<notin> range(\<lambda>C. priEK C))"
14199
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   270
apply (unfold sign_def)
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   271
apply (blast dest: merK_neq_priEK)
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   272
done
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   273
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   274
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   275
lemma Key_analz_image_Key_lemma:
67613
ce654b0e6d69 more symbols;
wenzelm
parents: 67443
diff changeset
   276
     "P \<longrightarrow> (Key K \<in> analz (Key`KK \<union> H)) \<longrightarrow> (K\<in>KK | Key K \<in> analz H)
14199
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   277
      ==>
67613
ce654b0e6d69 more symbols;
wenzelm
parents: 67443
diff changeset
   278
      P \<longrightarrow> (Key K \<in> analz (Key`KK \<union> H)) = (K\<in>KK | Key K \<in> analz H)"
14199
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   279
by (blast intro: analz_mono [THEN [2] rev_subsetD])
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   280
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   281
lemma symKey_compromise:
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   282
     "evs \<in> set_mr ==>
67613
ce654b0e6d69 more symbols;
wenzelm
parents: 67443
diff changeset
   283
      (\<forall>SK KK. SK \<in> symKeys \<longrightarrow> (\<forall>K \<in> KK. K \<notin> range(\<lambda>C. priEK C)) \<longrightarrow>
ce654b0e6d69 more symbols;
wenzelm
parents: 67443
diff changeset
   284
               (Key SK \<in> analz (Key`KK \<union> (knows Spy evs))) =
14199
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   285
               (SK \<in> KK | Key SK \<in> analz (knows Spy evs)))"
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   286
apply (erule set_mr.induct)
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   287
apply (safe del: impI intro!: Key_analz_image_Key_lemma [THEN impI])
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   288
apply (drule_tac [7] msg4_priEK_disj)
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   289
apply (frule_tac [6] Gets_certificate_valid)
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   290
apply (safe del: impI)
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   291
apply (simp_all del: image_insert image_Un imp_disjL
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   292
         add: analz_image_keys_simps abbrev_simps analz_knows_absorb
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   293
              analz_knows_absorb2 analz_Key_image_insert_eq notin_image_iff
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   294
              Spy_analz_private_Key analz_image_priEK)
67443
3abf6a722518 standardized towards new-style formal comments: isabelle update_comments;
wenzelm
parents: 63167
diff changeset
   295
  \<comment> \<open>5 seconds on a 1.6GHz machine\<close>
3abf6a722518 standardized towards new-style formal comments: isabelle update_comments;
wenzelm
parents: 63167
diff changeset
   296
apply spy_analz  \<comment> \<open>Fake\<close>
3abf6a722518 standardized towards new-style formal comments: isabelle update_comments;
wenzelm
parents: 63167
diff changeset
   297
apply auto  \<comment> \<open>Message 3\<close>
14199
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   298
done
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   299
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   300
lemma symKey_secrecy [rule_format]:
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   301
     "[|CA i \<notin> bad; K \<in> symKeys;  evs \<in> set_mr|]
67613
ce654b0e6d69 more symbols;
wenzelm
parents: 67443
diff changeset
   302
      ==> \<forall>X m. Says (Merchant m) (CA i) X \<in> set evs \<longrightarrow>
ce654b0e6d69 more symbols;
wenzelm
parents: 67443
diff changeset
   303
                Key K \<in> parts{X} \<longrightarrow>
ce654b0e6d69 more symbols;
wenzelm
parents: 67443
diff changeset
   304
                Merchant m \<notin> bad \<longrightarrow>
14199
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   305
                Key K \<notin> analz (knows Spy evs)"
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   306
apply (erule set_mr.induct)
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   307
apply (drule_tac [7] msg4_priEK_disj)
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   308
apply (frule_tac [6] Gets_certificate_valid)
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   309
apply (safe del: impI)
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   310
apply (simp_all del: image_insert image_Un imp_disjL
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   311
         add: analz_image_keys_simps abbrev_simps analz_knows_absorb
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   312
              analz_knows_absorb2 analz_Key_image_insert_eq
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   313
              symKey_compromise notin_image_iff Spy_analz_private_Key
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   314
              analz_image_priEK)
67443
3abf6a722518 standardized towards new-style formal comments: isabelle update_comments;
wenzelm
parents: 63167
diff changeset
   315
apply spy_analz  \<comment> \<open>Fake\<close>
3abf6a722518 standardized towards new-style formal comments: isabelle update_comments;
wenzelm
parents: 63167
diff changeset
   316
apply force  \<comment> \<open>Message 1\<close>
3abf6a722518 standardized towards new-style formal comments: isabelle update_comments;
wenzelm
parents: 63167
diff changeset
   317
apply (auto intro: analz_into_parts [THEN usedI] in_parts_Says_imp_used)  \<comment> \<open>Message 3\<close>
14199
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   318
done
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   319
63167
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 61984
diff changeset
   320
subsection\<open>Unicity\<close>
14199
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   321
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   322
lemma msg4_Says_imp_Notes:
61984
cdea44c775fa more symbols;
wenzelm
parents: 58889
diff changeset
   323
 "[|Says (CA i) M \<lbrace>sign (priSK (CA i)) \<lbrace>Agent M, Nonce NM2, Agent (CA i)\<rbrace>,
32960
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 24123
diff changeset
   324
                    cert  M      merSK    onlySig (priSK (CA i)),
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 24123
diff changeset
   325
                    cert  M      merEK    onlyEnc (priSK (CA i)),
61984
cdea44c775fa more symbols;
wenzelm
parents: 58889
diff changeset
   326
                    cert (CA i) (pubSK (CA i)) onlySig (priSK RCA)\<rbrace> \<in> set evs;
14199
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   327
    evs \<in> set_mr |]
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   328
  ==> Notes (CA i) (Key merSK) \<in> set evs
67613
ce654b0e6d69 more symbols;
wenzelm
parents: 67443
diff changeset
   329
   \<and>  Notes (CA i) (Key merEK) \<in> set evs"
14199
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   330
apply (erule rev_mp)
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   331
apply (erule set_mr.induct)
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   332
apply (simp_all (no_asm_simp))
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   333
done
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   334
63167
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 61984
diff changeset
   335
text\<open>Unicity of merSK wrt a given CA:
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 61984
diff changeset
   336
  merSK uniquely identifies the other components, including merEK\<close>
14199
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   337
lemma merSK_unicity:
61984
cdea44c775fa more symbols;
wenzelm
parents: 58889
diff changeset
   338
 "[|Says (CA i) M \<lbrace>sign (priSK(CA i)) \<lbrace>Agent M, Nonce NM2, Agent (CA i)\<rbrace>,
32960
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 24123
diff changeset
   339
                    cert  M      merSK    onlySig (priSK (CA i)),
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 24123
diff changeset
   340
                    cert  M      merEK    onlyEnc (priSK (CA i)),
61984
cdea44c775fa more symbols;
wenzelm
parents: 58889
diff changeset
   341
                    cert (CA i) (pubSK (CA i)) onlySig (priSK RCA)\<rbrace> \<in> set evs;
cdea44c775fa more symbols;
wenzelm
parents: 58889
diff changeset
   342
    Says (CA i) M' \<lbrace>sign (priSK(CA i)) \<lbrace>Agent M', Nonce NM2', Agent (CA i)\<rbrace>,
32960
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 24123
diff changeset
   343
                    cert  M'      merSK    onlySig (priSK (CA i)),
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 24123
diff changeset
   344
                    cert  M'      merEK'    onlyEnc (priSK (CA i)),
61984
cdea44c775fa more symbols;
wenzelm
parents: 58889
diff changeset
   345
                    cert (CA i) (pubSK(CA i)) onlySig (priSK RCA)\<rbrace> \<in> set evs;
67613
ce654b0e6d69 more symbols;
wenzelm
parents: 67443
diff changeset
   346
    evs \<in> set_mr |] ==> M=M' \<and> NM2=NM2' \<and> merEK=merEK'"
14199
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   347
apply (erule rev_mp)
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   348
apply (erule rev_mp)
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   349
apply (erule set_mr.induct)
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   350
apply (simp_all (no_asm_simp))
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   351
apply (blast dest!: msg4_Says_imp_Notes)
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   352
done
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   353
63167
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 61984
diff changeset
   354
text\<open>Unicity of merEK wrt a given CA:
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 61984
diff changeset
   355
  merEK uniquely identifies the other components, including merSK\<close>
14199
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   356
lemma merEK_unicity:
61984
cdea44c775fa more symbols;
wenzelm
parents: 58889
diff changeset
   357
 "[|Says (CA i) M \<lbrace>sign (priSK(CA i)) \<lbrace>Agent M, Nonce NM2, Agent (CA i)\<rbrace>,
32960
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 24123
diff changeset
   358
                    cert  M      merSK    onlySig (priSK (CA i)),
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 24123
diff changeset
   359
                    cert  M      merEK    onlyEnc (priSK (CA i)),
61984
cdea44c775fa more symbols;
wenzelm
parents: 58889
diff changeset
   360
                    cert (CA i) (pubSK (CA i)) onlySig (priSK RCA)\<rbrace> \<in> set evs;
cdea44c775fa more symbols;
wenzelm
parents: 58889
diff changeset
   361
    Says (CA i) M' \<lbrace>sign (priSK(CA i)) \<lbrace>Agent M', Nonce NM2', Agent (CA i)\<rbrace>,
32960
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 24123
diff changeset
   362
                     cert  M'      merSK'    onlySig (priSK (CA i)),
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 24123
diff changeset
   363
                     cert  M'      merEK    onlyEnc (priSK (CA i)),
61984
cdea44c775fa more symbols;
wenzelm
parents: 58889
diff changeset
   364
                     cert (CA i) (pubSK(CA i)) onlySig (priSK RCA)\<rbrace> \<in> set evs;
14199
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   365
    evs \<in> set_mr |] 
67613
ce654b0e6d69 more symbols;
wenzelm
parents: 67443
diff changeset
   366
  ==> M=M' \<and> NM2=NM2' \<and> merSK=merSK'"
14199
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   367
apply (erule rev_mp)
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   368
apply (erule rev_mp)
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   369
apply (erule set_mr.induct)
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   370
apply (simp_all (no_asm_simp))
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   371
apply (blast dest!: msg4_Says_imp_Notes)
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   372
done
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   373
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   374
63167
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 61984
diff changeset
   375
text\<open>-No interest on secrecy of nonces: they appear to be used
14199
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   376
    only for freshness.
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   377
   -No interest on secrecy of merSK or merEK, as in CR.
63167
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 61984
diff changeset
   378
   -There's no equivalent of the PAN\<close>
14199
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   379
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   380
63167
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 61984
diff changeset
   381
subsection\<open>Primary Goals of Merchant Registration\<close>
14199
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   382
63167
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 61984
diff changeset
   383
subsubsection\<open>The merchant's certificates really were created by the CA,
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 61984
diff changeset
   384
provided the CA is uncompromised\<close>
14199
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   385
69597
ff784d5a5bfb isabelle update -u control_cartouches;
wenzelm
parents: 67613
diff changeset
   386
text\<open>The assumption \<^term>\<open>CA i \<noteq> RCA\<close> is required: step 2 uses 
63167
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 61984
diff changeset
   387
  certificates of the same form.\<close>
14199
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   388
lemma certificate_merSK_valid_lemma [intro]:
61984
cdea44c775fa more symbols;
wenzelm
parents: 58889
diff changeset
   389
     "[|Crypt (priSK (CA i)) \<lbrace>Agent M, Key merSK, onlySig\<rbrace>
14199
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   390
          \<in> parts (knows Spy evs);
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   391
        CA i \<notin> bad;  CA i \<noteq> RCA;  evs \<in> set_mr|]
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   392
 ==> \<exists>X Y Z. Says (CA i) M
61984
cdea44c775fa more symbols;
wenzelm
parents: 58889
diff changeset
   393
                  \<lbrace>X, cert M merSK onlySig (priSK (CA i)), Y, Z\<rbrace> \<in> set evs"
14199
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   394
apply (erule rev_mp)
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   395
apply (erule set_mr.induct)
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   396
apply (simp_all (no_asm_simp))
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   397
apply auto
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   398
done
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   399
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   400
lemma certificate_merSK_valid:
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   401
     "[| cert M merSK onlySig (priSK (CA i)) \<in> parts (knows Spy evs);
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   402
         CA i \<notin> bad;  CA i \<noteq> RCA;  evs \<in> set_mr|]
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   403
 ==> \<exists>X Y Z. Says (CA i) M
61984
cdea44c775fa more symbols;
wenzelm
parents: 58889
diff changeset
   404
                  \<lbrace>X, cert M merSK onlySig (priSK (CA i)), Y, Z\<rbrace> \<in> set evs"
14199
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   405
by auto
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   406
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   407
lemma certificate_merEK_valid_lemma [intro]:
61984
cdea44c775fa more symbols;
wenzelm
parents: 58889
diff changeset
   408
     "[|Crypt (priSK (CA i)) \<lbrace>Agent M, Key merEK, onlyEnc\<rbrace>
14199
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   409
          \<in> parts (knows Spy evs);
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   410
        CA i \<notin> bad;  CA i \<noteq> RCA;  evs \<in> set_mr|]
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   411
 ==> \<exists>X Y Z. Says (CA i) M
61984
cdea44c775fa more symbols;
wenzelm
parents: 58889
diff changeset
   412
                  \<lbrace>X, Y, cert M merEK onlyEnc (priSK (CA i)), Z\<rbrace> \<in> set evs"
14199
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   413
apply (erule rev_mp)
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   414
apply (erule set_mr.induct)
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   415
apply (simp_all (no_asm_simp))
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   416
apply auto
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   417
done
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   418
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   419
lemma certificate_merEK_valid:
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   420
     "[| cert M merEK onlyEnc (priSK (CA i)) \<in> parts (knows Spy evs);
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   421
         CA i \<notin> bad;  CA i \<noteq> RCA;  evs \<in> set_mr|]
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   422
 ==> \<exists>X Y Z. Says (CA i) M
61984
cdea44c775fa more symbols;
wenzelm
parents: 58889
diff changeset
   423
                  \<lbrace>X, Y, cert M merEK onlyEnc (priSK (CA i)), Z\<rbrace> \<in> set evs"
14199
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   424
by auto
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   425
63167
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 61984
diff changeset
   426
text\<open>The two certificates - for merSK and for merEK - cannot be proved to
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 61984
diff changeset
   427
  have originated together\<close>
14199
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   428
d3b8d972a488 new session HOL-SET-Protocol
paulson
parents:
diff changeset
   429
end