src/HOL/Auth/Kerberos_BAN.ML
author paulson
Tue, 08 Sep 1998 15:17:11 +0200
changeset 5434 9b4bed3f394c
parent 5421 01fc8d6a40f2
child 5479 5a5dfb0f0d7d
permissions -rw-r--r--
Got rid of not_Says_to_self and most uses of ~= in definitions and theorems
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
5053
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
     1
(*  Title:      HOL/Auth/Kerberos_BAN
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
     2
    ID:         $Id$
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
     3
    Author:     Giampaolo Bella, Cambridge University Computer Laboratory
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
     4
    Copyright   1998  University of Cambridge
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
     5
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
     6
The Kerberos protocol, BAN version.
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
     7
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
     8
From page 251 of
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
     9
  Burrows, Abadi and Needham.  A Logic of Authentication.
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
    10
  Proc. Royal Soc. 426 (1989)
5064
77bd19f782e6 simplified and tidied the proofs
paulson
parents: 5053
diff changeset
    11
5223
4cb05273f764 Removal of obsolete "open" commands from heads of .ML files
paulson
parents: 5114
diff changeset
    12
  Confidentiality (secrecy) and authentication properties rely on 
4cb05273f764 Removal of obsolete "open" commands from heads of .ML files
paulson
parents: 5114
diff changeset
    13
  temporal checks: strong guarantees in a little abstracted - but
4cb05273f764 Removal of obsolete "open" commands from heads of .ML files
paulson
parents: 5114
diff changeset
    14
  very realistic - model (see .thy).
5053
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
    15
5223
4cb05273f764 Removal of obsolete "open" commands from heads of .ML files
paulson
parents: 5114
diff changeset
    16
Tidied by lcp.
5053
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
    17
*)
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
    18
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
    19
AddEs spies_partsEs;
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
    20
AddDs [impOfSubs analz_subset_parts];
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
    21
AddDs [impOfSubs Fake_parts_insert];
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
    22
5064
77bd19f782e6 simplified and tidied the proofs
paulson
parents: 5053
diff changeset
    23
AddIffs [SesKeyLife_LB, AutLife_LB];
5053
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
    24
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
    25
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
    26
(*A "possibility property": there are traces that reach the end.*)
5434
9b4bed3f394c Got rid of not_Says_to_self and most uses of ~= in definitions and theorems
paulson
parents: 5421
diff changeset
    27
Goal "EX Timestamp K. EX evs: kerberos_ban.    \
5114
c729d4c299c1 Deleted leading parameters thanks to new Goal command
paulson
parents: 5076
diff changeset
    28
\            Says B A (Crypt K (Number Timestamp)) \
c729d4c299c1 Deleted leading parameters thanks to new Goal command
paulson
parents: 5076
diff changeset
    29
\                 : set evs";
5352
paulson
parents: 5223
diff changeset
    30
by (cut_facts_tac [SesKeyLife_LB] 1);
5053
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
    31
by (REPEAT (resolve_tac [exI,bexI] 1));
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
    32
by (rtac (kerberos_ban.Nil RS kerberos_ban.Kb1 RS kerberos_ban.Kb2 RS 
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
    33
          kerberos_ban.Kb3 RS kerberos_ban.Kb4) 2);
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
    34
by possibility_tac;
5352
paulson
parents: 5223
diff changeset
    35
by (ALLGOALS Asm_simp_tac);
paulson
parents: 5223
diff changeset
    36
by (ALLGOALS trans_tac);
5053
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
    37
result();
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
    38
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
    39
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
    40
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
    41
(**** Inductive proofs about kerberos_ban ****)
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
    42
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
    43
(*Forwarding Lemma for reasoning about the encrypted portion of message Kb3*)
5114
c729d4c299c1 Deleted leading parameters thanks to new Goal command
paulson
parents: 5076
diff changeset
    44
Goal "Says S A (Crypt KA {|Timestamp, B, K, X|}) : set evs \
c729d4c299c1 Deleted leading parameters thanks to new Goal command
paulson
parents: 5076
diff changeset
    45
\             ==> X : parts (spies evs)";
5053
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
    46
by (Blast_tac 1);
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
    47
qed "Kb3_msg_in_parts_spies";
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
    48
                              
5114
c729d4c299c1 Deleted leading parameters thanks to new Goal command
paulson
parents: 5076
diff changeset
    49
Goal "Says Server A (Crypt (shrK A) {|Timestamp, B, K, X|}) : set evs \
c729d4c299c1 Deleted leading parameters thanks to new Goal command
paulson
parents: 5076
diff changeset
    50
\        ==> K : parts (spies evs)";
5053
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
    51
by (Blast_tac 1);
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
    52
qed "Oops_parts_spies";
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
    53
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
    54
(*For proving the easier theorems about X ~: parts (spies evs).*)
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
    55
fun parts_induct_tac i = 
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
    56
    etac kerberos_ban.induct i  THEN 
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
    57
    forward_tac [Oops_parts_spies] (i+6)  THEN
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
    58
    forward_tac [Kb3_msg_in_parts_spies] (i+4)     THEN
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
    59
    prove_simple_subgoals_tac i;
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
    60
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
    61
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
    62
(*Spy never sees another agent's shared key! (unless it's bad at start)*)
5114
c729d4c299c1 Deleted leading parameters thanks to new Goal command
paulson
parents: 5076
diff changeset
    63
Goal "evs : kerberos_ban ==> (Key (shrK A) : parts (spies evs)) = (A : bad)";
5053
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
    64
by (parts_induct_tac 1);
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
    65
by (ALLGOALS Blast_tac);
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
    66
qed "Spy_see_shrK";
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
    67
Addsimps [Spy_see_shrK];
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
    68
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
    69
5114
c729d4c299c1 Deleted leading parameters thanks to new Goal command
paulson
parents: 5076
diff changeset
    70
Goal "evs : kerberos_ban ==> (Key (shrK A) : analz (spies evs)) = (A : bad)";
5053
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
    71
by Auto_tac;
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
    72
qed "Spy_analz_shrK";
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
    73
Addsimps [Spy_analz_shrK];
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
    74
5114
c729d4c299c1 Deleted leading parameters thanks to new Goal command
paulson
parents: 5076
diff changeset
    75
Goal  "[| Key (shrK A) : parts (spies evs);       \
c729d4c299c1 Deleted leading parameters thanks to new Goal command
paulson
parents: 5076
diff changeset
    76
\               evs : kerberos_ban |] ==> A:bad";
5053
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
    77
by (blast_tac (claset() addDs [Spy_see_shrK]) 1);
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
    78
qed "Spy_see_shrK_D";
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
    79
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
    80
bind_thm ("Spy_analz_shrK_D", analz_subset_parts RS subsetD RS Spy_see_shrK_D);
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
    81
AddSDs [Spy_see_shrK_D, Spy_analz_shrK_D];
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
    82
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
    83
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
    84
(*Nobody can have used non-existent keys!*)
5114
c729d4c299c1 Deleted leading parameters thanks to new Goal command
paulson
parents: 5076
diff changeset
    85
Goal "evs : kerberos_ban ==>      \
c729d4c299c1 Deleted leading parameters thanks to new Goal command
paulson
parents: 5076
diff changeset
    86
\      Key K ~: used evs --> K ~: keysFor (parts (spies evs))";
5053
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
    87
by (parts_induct_tac 1);
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
    88
(*Fake*)
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
    89
by (blast_tac (claset() addSDs [keysFor_parts_insert]) 1);
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
    90
(*Kb2, Kb3, Kb4*)
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
    91
by (ALLGOALS Blast_tac);
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
    92
qed_spec_mp "new_keys_not_used";
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
    93
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
    94
bind_thm ("new_keys_not_analzd",
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
    95
          [analz_subset_parts RS keysFor_mono,
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
    96
           new_keys_not_used] MRS contra_subsetD);
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
    97
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
    98
Addsimps [new_keys_not_used, new_keys_not_analzd];
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
    99
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   100
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   101
(** Lemmas concerning the form of items passed in messages **)
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   102
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   103
(*Describes the form of K, X and K' when the Server sends this message.*)
5114
c729d4c299c1 Deleted leading parameters thanks to new Goal command
paulson
parents: 5076
diff changeset
   104
Goal "[| Says Server A (Crypt K' {|Number Ts, Agent B, Key K, X|})  \
c729d4c299c1 Deleted leading parameters thanks to new Goal command
paulson
parents: 5076
diff changeset
   105
\        : set evs; evs : kerberos_ban |]                           \
c729d4c299c1 Deleted leading parameters thanks to new Goal command
paulson
parents: 5076
diff changeset
   106
\     ==> K ~: range shrK &                                         \
c729d4c299c1 Deleted leading parameters thanks to new Goal command
paulson
parents: 5076
diff changeset
   107
\         X = (Crypt (shrK B) {|Number Ts, Agent A, Key K|}) &      \
c729d4c299c1 Deleted leading parameters thanks to new Goal command
paulson
parents: 5076
diff changeset
   108
\         K' = shrK A";
5053
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   109
by (etac rev_mp 1);
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   110
by (etac kerberos_ban.induct 1);
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   111
by Auto_tac;
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   112
qed "Says_Server_message_form";
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   113
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   114
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   115
(*If the encrypted message appears then it originated with the Server
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   116
  PROVIDED that A is NOT compromised!
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   117
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   118
  This shows implicitly the FRESHNESS OF THE SESSION KEY to A
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   119
*)
5114
c729d4c299c1 Deleted leading parameters thanks to new Goal command
paulson
parents: 5076
diff changeset
   120
Goal "[| Crypt (shrK A) {|Number Ts, Agent B, Key K, X|} \
c729d4c299c1 Deleted leading parameters thanks to new Goal command
paulson
parents: 5076
diff changeset
   121
\          : parts (spies evs);                          \
c729d4c299c1 Deleted leading parameters thanks to new Goal command
paulson
parents: 5076
diff changeset
   122
\        A ~: bad;  evs : kerberos_ban |]                \
c729d4c299c1 Deleted leading parameters thanks to new Goal command
paulson
parents: 5076
diff changeset
   123
\      ==> Says Server A (Crypt (shrK A) {|Number Ts, Agent B, Key K, X|}) \
c729d4c299c1 Deleted leading parameters thanks to new Goal command
paulson
parents: 5076
diff changeset
   124
\            : set evs";
5053
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   125
by (etac rev_mp 1);
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   126
by (parts_induct_tac 1);
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   127
by (Blast_tac 1);
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   128
qed "A_trusts_K_by_Kb2";
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   129
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   130
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   131
(*If the TICKET appears then it originated with the Server*)
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   132
(*FRESHNESS OF THE SESSION KEY to B*)
5114
c729d4c299c1 Deleted leading parameters thanks to new Goal command
paulson
parents: 5076
diff changeset
   133
Goal "[| Crypt (shrK B) {|Number Ts, Agent A, Key K|} : parts (spies evs); \
c729d4c299c1 Deleted leading parameters thanks to new Goal command
paulson
parents: 5076
diff changeset
   134
\        B ~: bad;  evs : kerberos_ban |]                        \
c729d4c299c1 Deleted leading parameters thanks to new Goal command
paulson
parents: 5076
diff changeset
   135
\      ==> Says Server A                                         \
c729d4c299c1 Deleted leading parameters thanks to new Goal command
paulson
parents: 5076
diff changeset
   136
\           (Crypt (shrK A) {|Number Ts, Agent B, Key K,                   \
c729d4c299c1 Deleted leading parameters thanks to new Goal command
paulson
parents: 5076
diff changeset
   137
\                         Crypt (shrK B) {|Number Ts, Agent A, Key K|}|})  \
c729d4c299c1 Deleted leading parameters thanks to new Goal command
paulson
parents: 5076
diff changeset
   138
\          : set evs";
5053
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   139
by (etac rev_mp 1);
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   140
by (parts_induct_tac 1);
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   141
by (Blast_tac 1);
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   142
qed "B_trusts_K_by_Kb3";
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   143
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   144
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   145
(*EITHER describes the form of X when the following message is sent, 
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   146
  OR     reduces it to the Fake case.
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   147
  Use Says_Server_message_form if applicable.*)
5114
c729d4c299c1 Deleted leading parameters thanks to new Goal command
paulson
parents: 5076
diff changeset
   148
Goal "[| Says S A (Crypt (shrK A) {|Number Ts, Agent B, Key K, X|})     \
c729d4c299c1 Deleted leading parameters thanks to new Goal command
paulson
parents: 5076
diff changeset
   149
\           : set evs;                                                  \
c729d4c299c1 Deleted leading parameters thanks to new Goal command
paulson
parents: 5076
diff changeset
   150
\        evs : kerberos_ban |]                                          \
c729d4c299c1 Deleted leading parameters thanks to new Goal command
paulson
parents: 5076
diff changeset
   151
\==> (K ~: range shrK & X = (Crypt (shrK B) {|Number Ts, Agent A, Key K|}))\
c729d4c299c1 Deleted leading parameters thanks to new Goal command
paulson
parents: 5076
diff changeset
   152
\         | X : analz (spies evs)";
5053
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   153
by (case_tac "A : bad" 1);
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   154
by (fast_tac (claset() addSDs [Says_imp_spies RS analz.Inj]
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   155
                      addss (simpset())) 1);
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   156
by (forward_tac [Says_imp_spies RS parts.Inj] 1);
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   157
by (blast_tac (claset() addSDs [A_trusts_K_by_Kb2, 
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   158
				Says_Server_message_form]) 1);
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   159
qed "Says_S_message_form";
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   160
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   161
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   162
(*For proofs involving analz.*)
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   163
val analz_spies_tac = 
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   164
    forward_tac [Says_Server_message_form] 7 THEN
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   165
    forward_tac [Says_S_message_form] 5 THEN 
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   166
    REPEAT_FIRST (eresolve_tac [asm_rl, conjE, disjE] ORELSE' hyp_subst_tac);
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   167
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   168
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   169
(****
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   170
 The following is to prove theorems of the form
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   171
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   172
  Key K : analz (insert (Key KAB) (spies evs)) ==>
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   173
  Key K : analz (spies evs)
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   174
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   175
 A more general formula must be proved inductively.
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   176
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   177
****)
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   178
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   179
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   180
(** Session keys are not used to encrypt other session keys **)
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   181
5114
c729d4c299c1 Deleted leading parameters thanks to new Goal command
paulson
parents: 5076
diff changeset
   182
Goal "evs : kerberos_ban ==>                          \
5053
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   183
\  ALL K KK. KK <= Compl (range shrK) -->                \
5114
c729d4c299c1 Deleted leading parameters thanks to new Goal command
paulson
parents: 5076
diff changeset
   184
\         (Key K : analz (Key``KK Un (spies evs))) =  \
c729d4c299c1 Deleted leading parameters thanks to new Goal command
paulson
parents: 5076
diff changeset
   185
\         (K : KK | Key K : analz (spies evs))";
5053
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   186
by (etac kerberos_ban.induct 1);
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   187
by analz_spies_tac;
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   188
by (REPEAT_FIRST (resolve_tac [allI, impI]));
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   189
by (REPEAT_FIRST (rtac analz_image_freshK_lemma));
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   190
(*Takes 5 secs*)
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   191
by (ALLGOALS (asm_simp_tac analz_image_freshK_ss));
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   192
(*Fake*) 
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   193
by (spy_analz_tac 1);
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   194
qed_spec_mp "analz_image_freshK";
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   195
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   196
5114
c729d4c299c1 Deleted leading parameters thanks to new Goal command
paulson
parents: 5076
diff changeset
   197
Goal "[| evs : kerberos_ban;  KAB ~: range shrK |] ==>     \
c729d4c299c1 Deleted leading parameters thanks to new Goal command
paulson
parents: 5076
diff changeset
   198
\     Key K : analz (insert (Key KAB) (spies evs)) =       \
c729d4c299c1 Deleted leading parameters thanks to new Goal command
paulson
parents: 5076
diff changeset
   199
\     (K = KAB | Key K : analz (spies evs))";
5053
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   200
by (asm_simp_tac (analz_image_freshK_ss addsimps [analz_image_freshK]) 1);
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   201
qed "analz_insert_freshK";
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   202
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   203
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   204
(** The session key K uniquely identifies the message **)
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   205
5114
c729d4c299c1 Deleted leading parameters thanks to new Goal command
paulson
parents: 5076
diff changeset
   206
Goal "evs : kerberos_ban ==>                                         \
c729d4c299c1 Deleted leading parameters thanks to new Goal command
paulson
parents: 5076
diff changeset
   207
\   EX A' Ts' B' X'. ALL A Ts B X.                                   \
c729d4c299c1 Deleted leading parameters thanks to new Goal command
paulson
parents: 5076
diff changeset
   208
\    Says Server A (Crypt (shrK A) {|Number Ts, Agent B, Key K, X|}) \
c729d4c299c1 Deleted leading parameters thanks to new Goal command
paulson
parents: 5076
diff changeset
   209
\          : set evs \
c729d4c299c1 Deleted leading parameters thanks to new Goal command
paulson
parents: 5076
diff changeset
   210
\    -->         A=A' & Ts=Ts' & B=B' & X=X'";
5053
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   211
by (etac kerberos_ban.induct 1);
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   212
by (ALLGOALS (asm_simp_tac (simpset() addsimps [all_conj_distrib])));
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   213
by Safe_tac;
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   214
(*Kb2: it can't be a new key*)
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   215
by (expand_case_tac "K = ?y" 1);
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   216
by (REPEAT (ares_tac [refl,exI,impI,conjI] 2));
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   217
by (blast_tac (claset() delrules [conjI]) 1);
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   218
val lemma = result();
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   219
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   220
(*In messages of this form, the session key uniquely identifies the rest*)
5114
c729d4c299c1 Deleted leading parameters thanks to new Goal command
paulson
parents: 5076
diff changeset
   221
Goal "[| Says Server A                                    \
c729d4c299c1 Deleted leading parameters thanks to new Goal command
paulson
parents: 5076
diff changeset
   222
\          (Crypt (shrK A) {|Number Ts, Agent B, Key K, X|}) : set evs; \ 
c729d4c299c1 Deleted leading parameters thanks to new Goal command
paulson
parents: 5076
diff changeset
   223
\        Says Server A'                                   \
c729d4c299c1 Deleted leading parameters thanks to new Goal command
paulson
parents: 5076
diff changeset
   224
\         (Crypt (shrK A') {|Number Ts', Agent B', Key K, X'|}) : set evs;\
c729d4c299c1 Deleted leading parameters thanks to new Goal command
paulson
parents: 5076
diff changeset
   225
\        evs : kerberos_ban |] ==> A=A' & Ts=Ts' & B=B' & X = X'";
5053
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   226
by (prove_unique_tac lemma 1);
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   227
qed "unique_session_keys";
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   228
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   229
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   230
(** Lemma: the session key sent in msg Kb2 would be EXPIRED
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   231
    if the spy could see it!
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   232
**)
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   233
5114
c729d4c299c1 Deleted leading parameters thanks to new Goal command
paulson
parents: 5076
diff changeset
   234
Goal "[| A ~: bad;  B ~: bad;  evs : kerberos_ban |]           \
c729d4c299c1 Deleted leading parameters thanks to new Goal command
paulson
parents: 5076
diff changeset
   235
\ ==> Says Server A                                            \
c729d4c299c1 Deleted leading parameters thanks to new Goal command
paulson
parents: 5076
diff changeset
   236
\         (Crypt (shrK A) {|Number Ts, Agent B, Key K,         \
c729d4c299c1 Deleted leading parameters thanks to new Goal command
paulson
parents: 5076
diff changeset
   237
\                           Crypt (shrK B) {|Number Ts, Agent A, Key K|}|})\
c729d4c299c1 Deleted leading parameters thanks to new Goal command
paulson
parents: 5076
diff changeset
   238
\        : set evs -->                                         \
c729d4c299c1 Deleted leading parameters thanks to new Goal command
paulson
parents: 5076
diff changeset
   239
\     Key K : analz (spies evs) --> Expired Ts evs"; 
5053
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   240
by (etac kerberos_ban.induct 1);
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   241
by analz_spies_tac;
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   242
by (ALLGOALS
5064
77bd19f782e6 simplified and tidied the proofs
paulson
parents: 5053
diff changeset
   243
    (asm_simp_tac (simpset() addsimps ([analz_insert_eq, analz_insert_freshK]
77bd19f782e6 simplified and tidied the proofs
paulson
parents: 5053
diff changeset
   244
				       @ pushes))));
5053
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   245
(*Oops*)
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   246
by (blast_tac (claset() addDs [unique_session_keys] addIs [less_SucI]) 4);
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   247
(*Kb2*)
5064
77bd19f782e6 simplified and tidied the proofs
paulson
parents: 5053
diff changeset
   248
by (blast_tac (claset() addIs [parts_insertI, less_SucI]) 2);
5053
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   249
(*Fake*) 
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   250
by (spy_analz_tac 1);
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   251
(**LEVEL 6 **)
5064
77bd19f782e6 simplified and tidied the proofs
paulson
parents: 5053
diff changeset
   252
(*Kb3*)
5053
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   253
by (case_tac "Aa : bad" 1);
5064
77bd19f782e6 simplified and tidied the proofs
paulson
parents: 5053
diff changeset
   254
by (blast_tac (claset() addDs [A_trusts_K_by_Kb2, unique_session_keys]) 2);
77bd19f782e6 simplified and tidied the proofs
paulson
parents: 5053
diff changeset
   255
by (blast_tac (claset() addDs [Says_imp_spies RS analz.Inj,
77bd19f782e6 simplified and tidied the proofs
paulson
parents: 5053
diff changeset
   256
                               Crypt_Spy_analz_bad, analz.Fst, analz.Snd]
5053
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   257
                        addIs [less_SucI]) 1);
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   258
val lemma = result() RS mp RS mp RSN(1,rev_notE);
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   259
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   260
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   261
(** CONFIDENTIALITY for the SERVER:
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   262
                     Spy does not see the keys sent in msg Kb2 
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   263
                     as long as they have NOT EXPIRED
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   264
**)
5114
c729d4c299c1 Deleted leading parameters thanks to new Goal command
paulson
parents: 5076
diff changeset
   265
Goal "[| Says Server A                                           \
c729d4c299c1 Deleted leading parameters thanks to new Goal command
paulson
parents: 5076
diff changeset
   266
\         (Crypt K' {|Number T, Agent B, Key K, X|}) : set evs;  \
c729d4c299c1 Deleted leading parameters thanks to new Goal command
paulson
parents: 5076
diff changeset
   267
\        ~ Expired T evs;                                        \
c729d4c299c1 Deleted leading parameters thanks to new Goal command
paulson
parents: 5076
diff changeset
   268
\        A ~: bad;  B ~: bad;  evs : kerberos_ban                \
c729d4c299c1 Deleted leading parameters thanks to new Goal command
paulson
parents: 5076
diff changeset
   269
\     |] ==> Key K ~: analz (spies evs)";
5053
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   270
by (forward_tac [Says_Server_message_form] 1 THEN assume_tac 1);
5064
77bd19f782e6 simplified and tidied the proofs
paulson
parents: 5053
diff changeset
   271
by (Clarify_tac 1);   (*prevents PROOF FAILED*)
5053
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   272
by (blast_tac (claset() addSEs [lemma]) 1);
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   273
qed "Confidentiality_S";
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   274
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   275
(**** THE COUNTERPART OF CONFIDENTIALITY 
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   276
      [|...; Expired Ts evs; ...|] ==> Key K : analz (spies evs)
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   277
      WOULD HOLD ONLY IF AN OOPS OCCURRED! ---> Nothing to prove!   ****)
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   278
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   279
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   280
(** CONFIDENTIALITY for ALICE: **)
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   281
(** Also A_trusts_K_by_Kb2 RS Confidentiality_S **)
5114
c729d4c299c1 Deleted leading parameters thanks to new Goal command
paulson
parents: 5076
diff changeset
   282
Goal "[| Crypt (shrK A) {|Number T, Agent B, Key K, X|} : parts (spies evs);\
c729d4c299c1 Deleted leading parameters thanks to new Goal command
paulson
parents: 5076
diff changeset
   283
\        ~ Expired T evs;          \
c729d4c299c1 Deleted leading parameters thanks to new Goal command
paulson
parents: 5076
diff changeset
   284
\        A ~: bad;  B ~: bad;  evs : kerberos_ban                \
c729d4c299c1 Deleted leading parameters thanks to new Goal command
paulson
parents: 5076
diff changeset
   285
\     |] ==> Key K ~: analz (spies evs)";
5064
77bd19f782e6 simplified and tidied the proofs
paulson
parents: 5053
diff changeset
   286
by (blast_tac (claset() addSDs [A_trusts_K_by_Kb2, Confidentiality_S]) 1);
5053
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   287
qed "Confidentiality_A";
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   288
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   289
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   290
(** CONFIDENTIALITY for BOB: **)
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   291
(** Also B_trusts_K_by_Kb3 RS Confidentiality_S **)
5114
c729d4c299c1 Deleted leading parameters thanks to new Goal command
paulson
parents: 5076
diff changeset
   292
Goal "[| Crypt (shrK B) {|Number Tk, Agent A, Key K|} \
c729d4c299c1 Deleted leading parameters thanks to new Goal command
paulson
parents: 5076
diff changeset
   293
\         : parts (spies evs);              \
c729d4c299c1 Deleted leading parameters thanks to new Goal command
paulson
parents: 5076
diff changeset
   294
\       ~ Expired Tk evs;          \
c729d4c299c1 Deleted leading parameters thanks to new Goal command
paulson
parents: 5076
diff changeset
   295
\       A ~: bad;  B ~: bad;  evs : kerberos_ban                \
c729d4c299c1 Deleted leading parameters thanks to new Goal command
paulson
parents: 5076
diff changeset
   296
\     |] ==> Key K ~: analz (spies evs)";             
5053
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   297
by (blast_tac (claset() addSDs [B_trusts_K_by_Kb3, 
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   298
                                Confidentiality_S]) 1);
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   299
qed "Confidentiality_B";
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   300
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   301
5114
c729d4c299c1 Deleted leading parameters thanks to new Goal command
paulson
parents: 5076
diff changeset
   302
Goal "[| B ~: bad;  evs : kerberos_ban |]                        \
c729d4c299c1 Deleted leading parameters thanks to new Goal command
paulson
parents: 5076
diff changeset
   303
\     ==> Key K ~: analz (spies evs) -->                    \
c729d4c299c1 Deleted leading parameters thanks to new Goal command
paulson
parents: 5076
diff changeset
   304
\         Says Server A (Crypt (shrK A) {|Number Ts, Agent B, Key K, X|}) \
c729d4c299c1 Deleted leading parameters thanks to new Goal command
paulson
parents: 5076
diff changeset
   305
\         : set evs -->                                             \
c729d4c299c1 Deleted leading parameters thanks to new Goal command
paulson
parents: 5076
diff changeset
   306
\         Crypt K (Number Ta) : parts (spies evs) -->        \
c729d4c299c1 Deleted leading parameters thanks to new Goal command
paulson
parents: 5076
diff changeset
   307
\         Says B A (Crypt K (Number Ta)) : set evs";
5053
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   308
by (etac kerberos_ban.induct 1);
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   309
by (forward_tac [Says_S_message_form] 5 THEN assume_tac 5);     
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   310
by (dtac Kb3_msg_in_parts_spies 5);
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   311
by (forward_tac [Oops_parts_spies] 7);
5064
77bd19f782e6 simplified and tidied the proofs
paulson
parents: 5053
diff changeset
   312
by (REPEAT (FIRSTGOAL analz_mono_contra_tac));
5053
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   313
by (ALLGOALS (asm_simp_tac (simpset() addsimps [all_conj_distrib])));
5064
77bd19f782e6 simplified and tidied the proofs
paulson
parents: 5053
diff changeset
   314
(**LEVEL 6**)
5053
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   315
by (Blast_tac 1);
5064
77bd19f782e6 simplified and tidied the proofs
paulson
parents: 5053
diff changeset
   316
by (Clarify_tac 1);
5053
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   317
(*
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   318
Subgoal 1: contradiction from the assumptions  
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   319
Key K ~: used evs2  and Crypt K (Number Ta) : parts (spies evs2)
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   320
*)
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   321
by (dtac Crypt_imp_invKey_keysFor 1);
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   322
by (Asm_full_simp_tac 1);
5064
77bd19f782e6 simplified and tidied the proofs
paulson
parents: 5053
diff changeset
   323
(* the two tactics above detect the contradiction*)
5053
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   324
by (case_tac "Ba : bad" 1);  (*splits up the subgoal by the stated case*)
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   325
by (blast_tac (claset() addDs [Says_imp_spies RS parts.Inj RS parts.Fst RS 
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   326
                              B_trusts_K_by_Kb3, 
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   327
			      unique_session_keys]) 2);
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   328
by (blast_tac (claset() addDs [Says_imp_spies RS analz.Inj RS analz.Fst RS 
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   329
			      Crypt_Spy_analz_bad]) 1);
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   330
val lemma_B = result();
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   331
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   332
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   333
(*AUTHENTICATION OF B TO A*)
5114
c729d4c299c1 Deleted leading parameters thanks to new Goal command
paulson
parents: 5076
diff changeset
   334
Goal "[| Crypt K (Number Ta) : parts (spies evs);           \
c729d4c299c1 Deleted leading parameters thanks to new Goal command
paulson
parents: 5076
diff changeset
   335
\        Crypt (shrK A) {|Number Ts, Agent B, Key K, X|}    \
c729d4c299c1 Deleted leading parameters thanks to new Goal command
paulson
parents: 5076
diff changeset
   336
\        : parts (spies evs);                               \
c729d4c299c1 Deleted leading parameters thanks to new Goal command
paulson
parents: 5076
diff changeset
   337
\        ~ Expired Ts evs;                                  \
c729d4c299c1 Deleted leading parameters thanks to new Goal command
paulson
parents: 5076
diff changeset
   338
\        A ~: bad;  B ~: bad;  evs : kerberos_ban |]        \
c729d4c299c1 Deleted leading parameters thanks to new Goal command
paulson
parents: 5076
diff changeset
   339
\     ==> Says B A (Crypt K (Number Ta)) : set evs";
5053
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   340
by (blast_tac (claset() addSDs [A_trusts_K_by_Kb2]
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   341
                        addSIs [lemma_B RS mp RS mp RS mp]
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   342
                        addSEs [Confidentiality_S RSN (2,rev_notE)]) 1);
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   343
qed "Authentication_B";
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   344
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   345
5114
c729d4c299c1 Deleted leading parameters thanks to new Goal command
paulson
parents: 5076
diff changeset
   346
Goal "[| A ~: bad; B ~: bad; evs : kerberos_ban |]      ==>         \ 
c729d4c299c1 Deleted leading parameters thanks to new Goal command
paulson
parents: 5076
diff changeset
   347
\        Key K ~: analz (spies evs) -->         \
c729d4c299c1 Deleted leading parameters thanks to new Goal command
paulson
parents: 5076
diff changeset
   348
\        Says Server A (Crypt (shrK A) {|Number Ts, Agent B, Key K, X|})  \
c729d4c299c1 Deleted leading parameters thanks to new Goal command
paulson
parents: 5076
diff changeset
   349
\        : set evs -->  \
c729d4c299c1 Deleted leading parameters thanks to new Goal command
paulson
parents: 5076
diff changeset
   350
\         Crypt K {|Agent A, Number Ta|} : parts (spies evs) -->\
c729d4c299c1 Deleted leading parameters thanks to new Goal command
paulson
parents: 5076
diff changeset
   351
\        Says A B {|X, Crypt K {|Agent A, Number Ta|}|}  \
c729d4c299c1 Deleted leading parameters thanks to new Goal command
paulson
parents: 5076
diff changeset
   352
\            : set evs";
5053
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   353
by (etac kerberos_ban.induct 1);
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   354
by (forward_tac [Says_S_message_form] 5 THEN assume_tac 5);     
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   355
by (forward_tac [Kb3_msg_in_parts_spies] 5);
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   356
by (forward_tac [Oops_parts_spies] 7);
5064
77bd19f782e6 simplified and tidied the proofs
paulson
parents: 5053
diff changeset
   357
by (REPEAT (FIRSTGOAL analz_mono_contra_tac));
5053
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   358
by (ALLGOALS (asm_simp_tac (simpset() addsimps [all_conj_distrib])));
5064
77bd19f782e6 simplified and tidied the proofs
paulson
parents: 5053
diff changeset
   359
(**LEVEL 6**)
5053
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   360
by (Blast_tac 1);
5064
77bd19f782e6 simplified and tidied the proofs
paulson
parents: 5053
diff changeset
   361
by (Clarify_tac 1);
5053
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   362
by (dtac Crypt_imp_invKey_keysFor 1);
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   363
by (Asm_full_simp_tac 1);
5064
77bd19f782e6 simplified and tidied the proofs
paulson
parents: 5053
diff changeset
   364
by (blast_tac (claset() addDs [A_trusts_K_by_Kb2, unique_session_keys]) 1);
5053
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   365
val lemma_A = result();
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   366
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   367
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   368
(*AUTHENTICATION OF A TO B*)
5114
c729d4c299c1 Deleted leading parameters thanks to new Goal command
paulson
parents: 5076
diff changeset
   369
Goal "[| Crypt K {|Agent A, Number Ta|} : parts (spies evs);  \
c729d4c299c1 Deleted leading parameters thanks to new Goal command
paulson
parents: 5076
diff changeset
   370
\        Crypt (shrK B) {|Number Ts, Agent A, Key K|}         \
c729d4c299c1 Deleted leading parameters thanks to new Goal command
paulson
parents: 5076
diff changeset
   371
\        : parts (spies evs);                                 \
c729d4c299c1 Deleted leading parameters thanks to new Goal command
paulson
parents: 5076
diff changeset
   372
\        ~ Expired Ts evs;                                    \
c729d4c299c1 Deleted leading parameters thanks to new Goal command
paulson
parents: 5076
diff changeset
   373
\        A ~: bad;  B ~: bad;  evs : kerberos_ban |]          \
c729d4c299c1 Deleted leading parameters thanks to new Goal command
paulson
parents: 5076
diff changeset
   374
\     ==> Says A B {|Crypt (shrK B) {|Number Ts, Agent A, Key K|}, \    
c729d4c299c1 Deleted leading parameters thanks to new Goal command
paulson
parents: 5076
diff changeset
   375
\                    Crypt K {|Agent A, Number Ta|}|} : set evs";
5053
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   376
by (blast_tac (claset() addSDs [B_trusts_K_by_Kb3]
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   377
                        addSIs [lemma_A RS mp RS mp RS mp]
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   378
                        addSEs [Confidentiality_S RSN (2,rev_notE)]) 1);
75d20f367e94 New example Kerberos_BAN by G Bella
paulson
parents:
diff changeset
   379
qed "Authentication_A";