src/HOL/Auth/Message.ML
author paulson
Fri, 13 Dec 1996 10:17:35 +0100
changeset 2373 490ffa16952e
parent 2327 00ac25b2791d
child 2415 46de4b035f00
permissions -rw-r--r--
Addition of the Hash constructor Strengthening spy_analz_tac
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
     1
(*  Title:      HOL/Auth/Message
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
     2
    ID:         $Id$
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
     3
    Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
     4
    Copyright   1996  University of Cambridge
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
     5
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
     6
Datatypes of agents and messages;
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
     7
Inductive relations "parts", "analz" and "synth"
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
     8
*)
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
     9
2327
00ac25b2791d Moved much common material to Message.ML
paulson
parents: 2284
diff changeset
    10
val prems = goal HOL.thy "[| P ==> Q(True); ~P ==> Q(False) |] ==> Q(P)";
00ac25b2791d Moved much common material to Message.ML
paulson
parents: 2284
diff changeset
    11
by (case_tac "P" 1);
00ac25b2791d Moved much common material to Message.ML
paulson
parents: 2284
diff changeset
    12
by (ALLGOALS (asm_simp_tac (!simpset addsimps prems)));
00ac25b2791d Moved much common material to Message.ML
paulson
parents: 2284
diff changeset
    13
val expand_case = result();
00ac25b2791d Moved much common material to Message.ML
paulson
parents: 2284
diff changeset
    14
00ac25b2791d Moved much common material to Message.ML
paulson
parents: 2284
diff changeset
    15
fun expand_case_tac P i =
00ac25b2791d Moved much common material to Message.ML
paulson
parents: 2284
diff changeset
    16
    res_inst_tac [("P",P)] expand_case i THEN
00ac25b2791d Moved much common material to Message.ML
paulson
parents: 2284
diff changeset
    17
    Simp_tac (i+1) THEN 
00ac25b2791d Moved much common material to Message.ML
paulson
parents: 2284
diff changeset
    18
    Simp_tac i;
00ac25b2791d Moved much common material to Message.ML
paulson
parents: 2284
diff changeset
    19
00ac25b2791d Moved much common material to Message.ML
paulson
parents: 2284
diff changeset
    20
00ac25b2791d Moved much common material to Message.ML
paulson
parents: 2284
diff changeset
    21
00ac25b2791d Moved much common material to Message.ML
paulson
parents: 2284
diff changeset
    22
(*GOALS.ML??*)
00ac25b2791d Moved much common material to Message.ML
paulson
parents: 2284
diff changeset
    23
fun prlim n = (goals_limit:=n; pr());
00ac25b2791d Moved much common material to Message.ML
paulson
parents: 2284
diff changeset
    24
00ac25b2791d Moved much common material to Message.ML
paulson
parents: 2284
diff changeset
    25
(*FUN.ML??  WE NEED A NOTION OF INVERSE IMAGE, OR GRAPH!!*)
00ac25b2791d Moved much common material to Message.ML
paulson
parents: 2284
diff changeset
    26
goal Set.thy "!!f. B <= range f = (B = f`` {x. f x: B})";
00ac25b2791d Moved much common material to Message.ML
paulson
parents: 2284
diff changeset
    27
by (fast_tac (!claset addEs [equalityE]) 1);
00ac25b2791d Moved much common material to Message.ML
paulson
parents: 2284
diff changeset
    28
val subset_range_iff = result();
00ac25b2791d Moved much common material to Message.ML
paulson
parents: 2284
diff changeset
    29
00ac25b2791d Moved much common material to Message.ML
paulson
parents: 2284
diff changeset
    30
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
    31
open Message;
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
    32
2373
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
    33
AddIffs (msg.inject);
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
    34
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
    35
(** Inverse of keys **)
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
    36
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
    37
goal thy "!!K K'. (invKey K = invKey K') = (K=K')";
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
    38
by (Step_tac 1);
2032
1bbf1bdcaf56 Introduction of "lost" argument
paulson
parents: 2028
diff changeset
    39
by (rtac box_equals 1);
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
    40
by (REPEAT (rtac invKey 2));
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
    41
by (Asm_simp_tac 1);
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
    42
qed "invKey_eq";
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
    43
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
    44
Addsimps [invKey, invKey_eq];
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
    45
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
    46
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
    47
(**** keysFor operator ****)
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
    48
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
    49
goalw thy [keysFor_def] "keysFor {} = {}";
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
    50
by (Fast_tac 1);
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
    51
qed "keysFor_empty";
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
    52
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
    53
goalw thy [keysFor_def] "keysFor (H Un H') = keysFor H Un keysFor H'";
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
    54
by (Fast_tac 1);
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
    55
qed "keysFor_Un";
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
    56
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
    57
goalw thy [keysFor_def] "keysFor (UN i. H i) = (UN i. keysFor (H i))";
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
    58
by (Fast_tac 1);
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
    59
qed "keysFor_UN";
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
    60
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
    61
(*Monotonicity*)
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
    62
goalw thy [keysFor_def] "!!G H. G<=H ==> keysFor(G) <= keysFor(H)";
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
    63
by (Fast_tac 1);
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
    64
qed "keysFor_mono";
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
    65
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
    66
goalw thy [keysFor_def] "keysFor (insert (Agent A) H) = keysFor H";
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
    67
by (fast_tac (!claset addss (!simpset)) 1);
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
    68
qed "keysFor_insert_Agent";
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
    69
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
    70
goalw thy [keysFor_def] "keysFor (insert (Nonce N) H) = keysFor H";
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
    71
by (fast_tac (!claset addss (!simpset)) 1);
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
    72
qed "keysFor_insert_Nonce";
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
    73
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
    74
goalw thy [keysFor_def] "keysFor (insert (Key K) H) = keysFor H";
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
    75
by (fast_tac (!claset addss (!simpset)) 1);
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
    76
qed "keysFor_insert_Key";
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
    77
2373
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
    78
goalw thy [keysFor_def] "keysFor (insert (Hash X) H) = keysFor H";
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
    79
by (fast_tac (!claset addss (!simpset)) 1);
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
    80
qed "keysFor_insert_Hash";
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
    81
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
    82
goalw thy [keysFor_def] "keysFor (insert {|X,Y|} H) = keysFor H";
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
    83
by (fast_tac (!claset addss (!simpset)) 1);
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
    84
qed "keysFor_insert_MPair";
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
    85
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
    86
goalw thy [keysFor_def]
2284
80ebd1a213fd Swapped arguments of Crypt (for clarity and because it is conventional)
paulson
parents: 2170
diff changeset
    87
    "keysFor (insert (Crypt K X) H) = insert (invKey K) (keysFor H)";
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
    88
by (Auto_tac());
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
    89
qed "keysFor_insert_Crypt";
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
    90
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
    91
Addsimps [keysFor_empty, keysFor_Un, keysFor_UN, 
2373
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
    92
          keysFor_insert_Agent, keysFor_insert_Nonce, keysFor_insert_Key, 
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
    93
	  keysFor_insert_Hash, keysFor_insert_MPair, keysFor_insert_Crypt];
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
    94
2284
80ebd1a213fd Swapped arguments of Crypt (for clarity and because it is conventional)
paulson
parents: 2170
diff changeset
    95
goalw thy [keysFor_def] "!!H. Crypt K X : H ==> invKey K : keysFor H";
2068
0d05468dc80c New theorem Crypt_imp_invKey_keysFor
paulson
parents: 2061
diff changeset
    96
by (Fast_tac 1);
0d05468dc80c New theorem Crypt_imp_invKey_keysFor
paulson
parents: 2061
diff changeset
    97
qed "Crypt_imp_invKey_keysFor";
0d05468dc80c New theorem Crypt_imp_invKey_keysFor
paulson
parents: 2061
diff changeset
    98
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
    99
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   100
(**** Inductive relation "parts" ****)
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   101
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   102
val major::prems = 
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   103
goal thy "[| {|X,Y|} : parts H;       \
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   104
\            [| X : parts H; Y : parts H |] ==> P  \
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   105
\         |] ==> P";
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   106
by (cut_facts_tac [major] 1);
2032
1bbf1bdcaf56 Introduction of "lost" argument
paulson
parents: 2028
diff changeset
   107
by (resolve_tac prems 1);
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   108
by (REPEAT (eresolve_tac [asm_rl, parts.Fst, parts.Snd] 1));
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   109
qed "MPair_parts";
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   110
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   111
AddIs  [parts.Inj];
1929
f0839bab4b00 Working version of NS, messages 1-3, WITH INTERLEAVING
paulson
parents: 1913
diff changeset
   112
f0839bab4b00 Working version of NS, messages 1-3, WITH INTERLEAVING
paulson
parents: 1913
diff changeset
   113
val partsEs = [MPair_parts, make_elim parts.Body];
f0839bab4b00 Working version of NS, messages 1-3, WITH INTERLEAVING
paulson
parents: 1913
diff changeset
   114
f0839bab4b00 Working version of NS, messages 1-3, WITH INTERLEAVING
paulson
parents: 1913
diff changeset
   115
AddSEs partsEs;
f0839bab4b00 Working version of NS, messages 1-3, WITH INTERLEAVING
paulson
parents: 1913
diff changeset
   116
(*NB These two rules are UNSAFE in the formal sense, as they discard the
f0839bab4b00 Working version of NS, messages 1-3, WITH INTERLEAVING
paulson
parents: 1913
diff changeset
   117
     compound message.  They work well on THIS FILE, perhaps because its
f0839bab4b00 Working version of NS, messages 1-3, WITH INTERLEAVING
paulson
parents: 1913
diff changeset
   118
     proofs concern only atomic messages.*)
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   119
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   120
goal thy "H <= parts(H)";
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   121
by (Fast_tac 1);
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   122
qed "parts_increasing";
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   123
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   124
(*Monotonicity*)
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   125
goalw thy parts.defs "!!G H. G<=H ==> parts(G) <= parts(H)";
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   126
by (rtac lfp_mono 1);
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   127
by (REPEAT (ares_tac basic_monos 1));
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   128
qed "parts_mono";
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   129
2373
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   130
val parts_insertI = impOfSubs (subset_insertI RS parts_mono);
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   131
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   132
goal thy "parts{} = {}";
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   133
by (Step_tac 1);
2032
1bbf1bdcaf56 Introduction of "lost" argument
paulson
parents: 2028
diff changeset
   134
by (etac parts.induct 1);
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   135
by (ALLGOALS Fast_tac);
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   136
qed "parts_empty";
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   137
Addsimps [parts_empty];
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   138
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   139
goal thy "!!X. X: parts{} ==> P";
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   140
by (Asm_full_simp_tac 1);
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   141
qed "parts_emptyE";
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   142
AddSEs [parts_emptyE];
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   143
1893
fa58f4a06f21 Works up to main theorem, then XXX...X
paulson
parents: 1885
diff changeset
   144
(*WARNING: loops if H = {Y}, therefore must not be repeated!*)
fa58f4a06f21 Works up to main theorem, then XXX...X
paulson
parents: 1885
diff changeset
   145
goal thy "!!H. X: parts H ==> EX Y:H. X: parts {Y}";
2032
1bbf1bdcaf56 Introduction of "lost" argument
paulson
parents: 2028
diff changeset
   146
by (etac parts.induct 1);
1893
fa58f4a06f21 Works up to main theorem, then XXX...X
paulson
parents: 1885
diff changeset
   147
by (ALLGOALS Fast_tac);
fa58f4a06f21 Works up to main theorem, then XXX...X
paulson
parents: 1885
diff changeset
   148
qed "parts_singleton";
fa58f4a06f21 Works up to main theorem, then XXX...X
paulson
parents: 1885
diff changeset
   149
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   150
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   151
(** Unions **)
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   152
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   153
goal thy "parts(G) Un parts(H) <= parts(G Un H)";
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   154
by (REPEAT (ares_tac [Un_least, parts_mono, Un_upper1, Un_upper2] 1));
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   155
val parts_Un_subset1 = result();
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   156
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   157
goal thy "parts(G Un H) <= parts(G) Un parts(H)";
2032
1bbf1bdcaf56 Introduction of "lost" argument
paulson
parents: 2028
diff changeset
   158
by (rtac subsetI 1);
1bbf1bdcaf56 Introduction of "lost" argument
paulson
parents: 2028
diff changeset
   159
by (etac parts.induct 1);
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   160
by (ALLGOALS Fast_tac);
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   161
val parts_Un_subset2 = result();
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   162
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   163
goal thy "parts(G Un H) = parts(G) Un parts(H)";
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   164
by (REPEAT (ares_tac [equalityI, parts_Un_subset1, parts_Un_subset2] 1));
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   165
qed "parts_Un";
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   166
2011
d9af64c26be6 New laws for messages
paulson
parents: 1998
diff changeset
   167
goal thy "parts (insert X H) = parts {X} Un parts H";
1852
289ce6cb5c84 Added Msg 3; works up to Says_Server_imp_Key_newK
paulson
parents: 1839
diff changeset
   168
by (stac (read_instantiate [("A","H")] insert_is_Un) 1);
2011
d9af64c26be6 New laws for messages
paulson
parents: 1998
diff changeset
   169
by (simp_tac (HOL_ss addsimps [parts_Un]) 1);
d9af64c26be6 New laws for messages
paulson
parents: 1998
diff changeset
   170
qed "parts_insert";
d9af64c26be6 New laws for messages
paulson
parents: 1998
diff changeset
   171
d9af64c26be6 New laws for messages
paulson
parents: 1998
diff changeset
   172
(*TWO inserts to avoid looping.  This rewrite is better than nothing.
d9af64c26be6 New laws for messages
paulson
parents: 1998
diff changeset
   173
  Not suitable for Addsimps: its behaviour can be strange.*)
d9af64c26be6 New laws for messages
paulson
parents: 1998
diff changeset
   174
goal thy "parts (insert X (insert Y H)) = parts {X} Un parts {Y} Un parts H";
d9af64c26be6 New laws for messages
paulson
parents: 1998
diff changeset
   175
by (simp_tac (!simpset addsimps [Un_assoc]) 1);
d9af64c26be6 New laws for messages
paulson
parents: 1998
diff changeset
   176
by (simp_tac (!simpset addsimps [parts_insert RS sym]) 1);
1852
289ce6cb5c84 Added Msg 3; works up to Says_Server_imp_Key_newK
paulson
parents: 1839
diff changeset
   177
qed "parts_insert2";
289ce6cb5c84 Added Msg 3; works up to Says_Server_imp_Key_newK
paulson
parents: 1839
diff changeset
   178
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   179
goal thy "(UN x:A. parts(H x)) <= parts(UN x:A. H x)";
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   180
by (REPEAT (ares_tac [UN_least, parts_mono, UN_upper] 1));
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   181
val parts_UN_subset1 = result();
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   182
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   183
goal thy "parts(UN x:A. H x) <= (UN x:A. parts(H x))";
2032
1bbf1bdcaf56 Introduction of "lost" argument
paulson
parents: 2028
diff changeset
   184
by (rtac subsetI 1);
1bbf1bdcaf56 Introduction of "lost" argument
paulson
parents: 2028
diff changeset
   185
by (etac parts.induct 1);
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   186
by (ALLGOALS Fast_tac);
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   187
val parts_UN_subset2 = result();
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   188
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   189
goal thy "parts(UN x:A. H x) = (UN x:A. parts(H x))";
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   190
by (REPEAT (ares_tac [equalityI, parts_UN_subset1, parts_UN_subset2] 1));
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   191
qed "parts_UN";
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   192
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   193
goal thy "parts(UN x. H x) = (UN x. parts(H x))";
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   194
by (simp_tac (!simpset addsimps [UNION1_def, parts_UN]) 1);
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   195
qed "parts_UN1";
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   196
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   197
(*Added to simplify arguments to parts, analz and synth*)
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   198
Addsimps [parts_Un, parts_UN, parts_UN1];
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   199
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   200
goal thy "insert X (parts H) <= parts(insert X H)";
1852
289ce6cb5c84 Added Msg 3; works up to Says_Server_imp_Key_newK
paulson
parents: 1839
diff changeset
   201
by (fast_tac (!claset addEs [impOfSubs parts_mono]) 1);
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   202
qed "parts_insert_subset";
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   203
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   204
(** Idempotence and transitivity **)
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   205
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   206
goal thy "!!H. X: parts (parts H) ==> X: parts H";
2032
1bbf1bdcaf56 Introduction of "lost" argument
paulson
parents: 2028
diff changeset
   207
by (etac parts.induct 1);
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   208
by (ALLGOALS Fast_tac);
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   209
qed "parts_partsE";
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   210
AddSEs [parts_partsE];
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   211
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   212
goal thy "parts (parts H) = parts H";
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   213
by (Fast_tac 1);
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   214
qed "parts_idem";
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   215
Addsimps [parts_idem];
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   216
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   217
goal thy "!!H. [| X: parts G;  G <= parts H |] ==> X: parts H";
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   218
by (dtac parts_mono 1);
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   219
by (Fast_tac 1);
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   220
qed "parts_trans";
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   221
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   222
(*Cut*)
2373
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   223
goal thy "!!H. [| Y: parts (insert X G);  X: parts H |] \
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   224
\              ==> Y: parts (G Un H)";
2032
1bbf1bdcaf56 Introduction of "lost" argument
paulson
parents: 2028
diff changeset
   225
by (etac parts_trans 1);
2373
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   226
by (Auto_tac());
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   227
qed "parts_cut";
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   228
1929
f0839bab4b00 Working version of NS, messages 1-3, WITH INTERLEAVING
paulson
parents: 1913
diff changeset
   229
goal thy "!!H. X: parts H ==> parts (insert X H) = parts H";
2373
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   230
by (fast_tac (!claset addSDs [parts_cut]
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   231
                      addIs  [parts_insertI] 
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   232
                      addss (!simpset)) 1);
1929
f0839bab4b00 Working version of NS, messages 1-3, WITH INTERLEAVING
paulson
parents: 1913
diff changeset
   233
qed "parts_cut_eq";
f0839bab4b00 Working version of NS, messages 1-3, WITH INTERLEAVING
paulson
parents: 1913
diff changeset
   234
2028
738bb98d65ec Last working version prior to addition of "lost" component
paulson
parents: 2026
diff changeset
   235
Addsimps [parts_cut_eq];
738bb98d65ec Last working version prior to addition of "lost" component
paulson
parents: 2026
diff changeset
   236
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   237
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   238
(** Rewrite rules for pulling out atomic messages **)
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   239
2373
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   240
fun parts_tac i =
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   241
  EVERY [rtac ([subsetI, parts_insert_subset] MRS equalityI) i,
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   242
	 etac parts.induct i,
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   243
	 REPEAT (fast_tac (!claset addss (!simpset)) i)];
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   244
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   245
goal thy "parts (insert (Agent agt) H) = insert (Agent agt) (parts H)";
2373
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   246
by (parts_tac 1);
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   247
qed "parts_insert_Agent";
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   248
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   249
goal thy "parts (insert (Nonce N) H) = insert (Nonce N) (parts H)";
2373
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   250
by (parts_tac 1);
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   251
qed "parts_insert_Nonce";
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   252
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   253
goal thy "parts (insert (Key K) H) = insert (Key K) (parts H)";
2373
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   254
by (parts_tac 1);
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   255
qed "parts_insert_Key";
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   256
2373
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   257
goal thy "parts (insert (Hash X) H) = insert (Hash X) (parts H)";
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   258
by (parts_tac 1);
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   259
qed "parts_insert_Hash";
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   260
2284
80ebd1a213fd Swapped arguments of Crypt (for clarity and because it is conventional)
paulson
parents: 2170
diff changeset
   261
goal thy "parts (insert (Crypt K X) H) = \
80ebd1a213fd Swapped arguments of Crypt (for clarity and because it is conventional)
paulson
parents: 2170
diff changeset
   262
\         insert (Crypt K X) (parts (insert X H))";
2032
1bbf1bdcaf56 Introduction of "lost" argument
paulson
parents: 2028
diff changeset
   263
by (rtac equalityI 1);
1bbf1bdcaf56 Introduction of "lost" argument
paulson
parents: 2028
diff changeset
   264
by (rtac subsetI 1);
1bbf1bdcaf56 Introduction of "lost" argument
paulson
parents: 2028
diff changeset
   265
by (etac parts.induct 1);
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   266
by (Auto_tac());
2032
1bbf1bdcaf56 Introduction of "lost" argument
paulson
parents: 2028
diff changeset
   267
by (etac parts.induct 1);
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   268
by (ALLGOALS (best_tac (!claset addIs [parts.Body])));
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   269
qed "parts_insert_Crypt";
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   270
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   271
goal thy "parts (insert {|X,Y|} H) = \
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   272
\         insert {|X,Y|} (parts (insert X (insert Y H)))";
2032
1bbf1bdcaf56 Introduction of "lost" argument
paulson
parents: 2028
diff changeset
   273
by (rtac equalityI 1);
1bbf1bdcaf56 Introduction of "lost" argument
paulson
parents: 2028
diff changeset
   274
by (rtac subsetI 1);
1bbf1bdcaf56 Introduction of "lost" argument
paulson
parents: 2028
diff changeset
   275
by (etac parts.induct 1);
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   276
by (Auto_tac());
2032
1bbf1bdcaf56 Introduction of "lost" argument
paulson
parents: 2028
diff changeset
   277
by (etac parts.induct 1);
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   278
by (ALLGOALS (best_tac (!claset addIs [parts.Fst, parts.Snd])));
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   279
qed "parts_insert_MPair";
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   280
2373
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   281
Addsimps [parts_insert_Agent, parts_insert_Nonce, parts_insert_Key, 
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   282
          parts_insert_Hash, parts_insert_Crypt, parts_insert_MPair];
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   283
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   284
2026
0df5a96bf77e Last working version prior to introduction of "lost"
paulson
parents: 2011
diff changeset
   285
goal thy "parts (Key``N) = Key``N";
0df5a96bf77e Last working version prior to introduction of "lost"
paulson
parents: 2011
diff changeset
   286
by (Auto_tac());
2032
1bbf1bdcaf56 Introduction of "lost" argument
paulson
parents: 2028
diff changeset
   287
by (etac parts.induct 1);
2026
0df5a96bf77e Last working version prior to introduction of "lost"
paulson
parents: 2011
diff changeset
   288
by (Auto_tac());
0df5a96bf77e Last working version prior to introduction of "lost"
paulson
parents: 2011
diff changeset
   289
qed "parts_image_Key";
0df5a96bf77e Last working version prior to introduction of "lost"
paulson
parents: 2011
diff changeset
   290
0df5a96bf77e Last working version prior to introduction of "lost"
paulson
parents: 2011
diff changeset
   291
Addsimps [parts_image_Key];
0df5a96bf77e Last working version prior to introduction of "lost"
paulson
parents: 2011
diff changeset
   292
0df5a96bf77e Last working version prior to introduction of "lost"
paulson
parents: 2011
diff changeset
   293
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   294
(**** Inductive relation "analz" ****)
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   295
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   296
val major::prems = 
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   297
goal thy "[| {|X,Y|} : analz H;       \
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   298
\            [| X : analz H; Y : analz H |] ==> P  \
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   299
\         |] ==> P";
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   300
by (cut_facts_tac [major] 1);
2032
1bbf1bdcaf56 Introduction of "lost" argument
paulson
parents: 2028
diff changeset
   301
by (resolve_tac prems 1);
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   302
by (REPEAT (eresolve_tac [asm_rl, analz.Fst, analz.Snd] 1));
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   303
qed "MPair_analz";
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   304
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   305
AddIs  [analz.Inj];
2011
d9af64c26be6 New laws for messages
paulson
parents: 1998
diff changeset
   306
AddSEs [MPair_analz];      (*Perhaps it should NOT be deemed safe!*)
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   307
AddDs  [analz.Decrypt];
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   308
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   309
Addsimps [analz.Inj];
1885
a18a6dc14f76 Auth proofs work up to the XXX...
paulson
parents: 1852
diff changeset
   310
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   311
goal thy "H <= analz(H)";
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   312
by (Fast_tac 1);
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   313
qed "analz_increasing";
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   314
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   315
goal thy "analz H <= parts H";
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   316
by (rtac subsetI 1);
2032
1bbf1bdcaf56 Introduction of "lost" argument
paulson
parents: 2028
diff changeset
   317
by (etac analz.induct 1);
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   318
by (ALLGOALS Fast_tac);
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   319
qed "analz_subset_parts";
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   320
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   321
bind_thm ("not_parts_not_analz", analz_subset_parts RS contra_subsetD);
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   322
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   323
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   324
goal thy "parts (analz H) = parts H";
2032
1bbf1bdcaf56 Introduction of "lost" argument
paulson
parents: 2028
diff changeset
   325
by (rtac equalityI 1);
1bbf1bdcaf56 Introduction of "lost" argument
paulson
parents: 2028
diff changeset
   326
by (rtac (analz_subset_parts RS parts_mono RS subset_trans) 1);
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   327
by (Simp_tac 1);
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   328
by (fast_tac (!claset addDs [analz_increasing RS parts_mono RS subsetD]) 1);
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   329
qed "parts_analz";
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   330
Addsimps [parts_analz];
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   331
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   332
goal thy "analz (parts H) = parts H";
1885
a18a6dc14f76 Auth proofs work up to the XXX...
paulson
parents: 1852
diff changeset
   333
by (Auto_tac());
2032
1bbf1bdcaf56 Introduction of "lost" argument
paulson
parents: 2028
diff changeset
   334
by (etac analz.induct 1);
1885
a18a6dc14f76 Auth proofs work up to the XXX...
paulson
parents: 1852
diff changeset
   335
by (Auto_tac());
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   336
qed "analz_parts";
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   337
Addsimps [analz_parts];
1885
a18a6dc14f76 Auth proofs work up to the XXX...
paulson
parents: 1852
diff changeset
   338
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   339
(*Monotonicity; Lemma 1 of Lowe*)
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   340
goalw thy analz.defs "!!G H. G<=H ==> analz(G) <= analz(H)";
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   341
by (rtac lfp_mono 1);
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   342
by (REPEAT (ares_tac basic_monos 1));
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   343
qed "analz_mono";
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   344
2373
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   345
val analz_insertI = impOfSubs (subset_insertI RS analz_mono);
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   346
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   347
(** General equational properties **)
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   348
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   349
goal thy "analz{} = {}";
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   350
by (Step_tac 1);
2032
1bbf1bdcaf56 Introduction of "lost" argument
paulson
parents: 2028
diff changeset
   351
by (etac analz.induct 1);
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   352
by (ALLGOALS Fast_tac);
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   353
qed "analz_empty";
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   354
Addsimps [analz_empty];
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   355
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   356
(*Converse fails: we can analz more from the union than from the 
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   357
  separate parts, as a key in one might decrypt a message in the other*)
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   358
goal thy "analz(G) Un analz(H) <= analz(G Un H)";
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   359
by (REPEAT (ares_tac [Un_least, analz_mono, Un_upper1, Un_upper2] 1));
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   360
qed "analz_Un";
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   361
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   362
goal thy "insert X (analz H) <= analz(insert X H)";
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   363
by (fast_tac (!claset addEs [impOfSubs analz_mono]) 1);
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   364
qed "analz_insert";
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   365
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   366
(** Rewrite rules for pulling out atomic messages **)
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   367
2373
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   368
fun analz_tac i =
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   369
  EVERY [rtac ([subsetI, analz_insert] MRS equalityI) i,
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   370
	 etac analz.induct i,
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   371
	 REPEAT (fast_tac (!claset addss (!simpset)) i)];
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   372
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   373
goal thy "analz (insert (Agent agt) H) = insert (Agent agt) (analz H)";
2373
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   374
by (analz_tac 1);
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   375
qed "analz_insert_Agent";
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   376
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   377
goal thy "analz (insert (Nonce N) H) = insert (Nonce N) (analz H)";
2373
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   378
by (analz_tac 1);
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   379
qed "analz_insert_Nonce";
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   380
2373
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   381
goal thy "analz (insert (Hash X) H) = insert (Hash X) (analz H)";
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   382
by (analz_tac 1);
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   383
qed "analz_insert_Hash";
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   384
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   385
(*Can only pull out Keys if they are not needed to decrypt the rest*)
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   386
goalw thy [keysFor_def]
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   387
    "!!K. K ~: keysFor (analz H) ==>  \
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   388
\         analz (insert (Key K) H) = insert (Key K) (analz H)";
2373
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   389
by (analz_tac 1);
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   390
qed "analz_insert_Key";
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   391
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   392
goal thy "analz (insert {|X,Y|} H) = \
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   393
\         insert {|X,Y|} (analz (insert X (insert Y H)))";
2032
1bbf1bdcaf56 Introduction of "lost" argument
paulson
parents: 2028
diff changeset
   394
by (rtac equalityI 1);
1bbf1bdcaf56 Introduction of "lost" argument
paulson
parents: 2028
diff changeset
   395
by (rtac subsetI 1);
1bbf1bdcaf56 Introduction of "lost" argument
paulson
parents: 2028
diff changeset
   396
by (etac analz.induct 1);
1885
a18a6dc14f76 Auth proofs work up to the XXX...
paulson
parents: 1852
diff changeset
   397
by (Auto_tac());
2032
1bbf1bdcaf56 Introduction of "lost" argument
paulson
parents: 2028
diff changeset
   398
by (etac analz.induct 1);
2102
41a667d2c3fa Replaced excluded_middle_tac by case_tac
paulson
parents: 2068
diff changeset
   399
by (ALLGOALS
41a667d2c3fa Replaced excluded_middle_tac by case_tac
paulson
parents: 2068
diff changeset
   400
    (deepen_tac (!claset addIs [analz.Fst, analz.Snd, analz.Decrypt]) 0));
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   401
qed "analz_insert_MPair";
1885
a18a6dc14f76 Auth proofs work up to the XXX...
paulson
parents: 1852
diff changeset
   402
a18a6dc14f76 Auth proofs work up to the XXX...
paulson
parents: 1852
diff changeset
   403
(*Can pull out enCrypted message if the Key is not known*)
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   404
goal thy "!!H. Key (invKey K) ~: analz H ==>  \
2284
80ebd1a213fd Swapped arguments of Crypt (for clarity and because it is conventional)
paulson
parents: 2170
diff changeset
   405
\              analz (insert (Crypt K X) H) = \
80ebd1a213fd Swapped arguments of Crypt (for clarity and because it is conventional)
paulson
parents: 2170
diff changeset
   406
\              insert (Crypt K X) (analz H)";
2373
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   407
by (analz_tac 1);
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   408
qed "analz_insert_Crypt";
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   409
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   410
goal thy "!!H. Key (invKey K) : analz H ==>  \
2284
80ebd1a213fd Swapped arguments of Crypt (for clarity and because it is conventional)
paulson
parents: 2170
diff changeset
   411
\              analz (insert (Crypt K X) H) <= \
80ebd1a213fd Swapped arguments of Crypt (for clarity and because it is conventional)
paulson
parents: 2170
diff changeset
   412
\              insert (Crypt K X) (analz (insert X H))";
2032
1bbf1bdcaf56 Introduction of "lost" argument
paulson
parents: 2028
diff changeset
   413
by (rtac subsetI 1);
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   414
by (eres_inst_tac [("za","x")] analz.induct 1);
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   415
by (ALLGOALS (fast_tac (!claset addss (!simpset))));
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   416
val lemma1 = result();
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   417
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   418
goal thy "!!H. Key (invKey K) : analz H ==>  \
2284
80ebd1a213fd Swapped arguments of Crypt (for clarity and because it is conventional)
paulson
parents: 2170
diff changeset
   419
\              insert (Crypt K X) (analz (insert X H)) <= \
80ebd1a213fd Swapped arguments of Crypt (for clarity and because it is conventional)
paulson
parents: 2170
diff changeset
   420
\              analz (insert (Crypt K X) H)";
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   421
by (Auto_tac());
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   422
by (eres_inst_tac [("za","x")] analz.induct 1);
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   423
by (Auto_tac());
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   424
by (best_tac (!claset addIs [subset_insertI RS analz_mono RS subsetD,
2032
1bbf1bdcaf56 Introduction of "lost" argument
paulson
parents: 2028
diff changeset
   425
                             analz.Decrypt]) 1);
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   426
val lemma2 = result();
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   427
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   428
goal thy "!!H. Key (invKey K) : analz H ==>  \
2284
80ebd1a213fd Swapped arguments of Crypt (for clarity and because it is conventional)
paulson
parents: 2170
diff changeset
   429
\              analz (insert (Crypt K X) H) = \
80ebd1a213fd Swapped arguments of Crypt (for clarity and because it is conventional)
paulson
parents: 2170
diff changeset
   430
\              insert (Crypt K X) (analz (insert X H))";
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   431
by (REPEAT (ares_tac [equalityI, lemma1, lemma2] 1));
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   432
qed "analz_insert_Decrypt";
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   433
1885
a18a6dc14f76 Auth proofs work up to the XXX...
paulson
parents: 1852
diff changeset
   434
(*Case analysis: either the message is secure, or it is not!
1946
b59a3d686436 New theorems for Fake case
paulson
parents: 1929
diff changeset
   435
  Effective, but can cause subgoals to blow up!
1885
a18a6dc14f76 Auth proofs work up to the XXX...
paulson
parents: 1852
diff changeset
   436
  Use with expand_if;  apparently split_tac does not cope with patterns
2284
80ebd1a213fd Swapped arguments of Crypt (for clarity and because it is conventional)
paulson
parents: 2170
diff changeset
   437
  such as "analz (insert (Crypt K X) H)" *)
80ebd1a213fd Swapped arguments of Crypt (for clarity and because it is conventional)
paulson
parents: 2170
diff changeset
   438
goal thy "analz (insert (Crypt K X) H) =                \
2154
913b4fc7670a New, purely illustrative result Crypt_synth_analz
paulson
parents: 2102
diff changeset
   439
\         (if (Key (invKey K) : analz H)                \
2284
80ebd1a213fd Swapped arguments of Crypt (for clarity and because it is conventional)
paulson
parents: 2170
diff changeset
   440
\          then insert (Crypt K X) (analz (insert X H)) \
80ebd1a213fd Swapped arguments of Crypt (for clarity and because it is conventional)
paulson
parents: 2170
diff changeset
   441
\          else insert (Crypt K X) (analz H))";
2102
41a667d2c3fa Replaced excluded_middle_tac by case_tac
paulson
parents: 2068
diff changeset
   442
by (case_tac "Key (invKey K)  : analz H " 1);
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   443
by (ALLGOALS (asm_simp_tac (!simpset addsimps [analz_insert_Crypt, 
2032
1bbf1bdcaf56 Introduction of "lost" argument
paulson
parents: 2028
diff changeset
   444
                                               analz_insert_Decrypt])));
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   445
qed "analz_Crypt_if";
1885
a18a6dc14f76 Auth proofs work up to the XXX...
paulson
parents: 1852
diff changeset
   446
2373
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   447
Addsimps [analz_insert_Agent, analz_insert_Nonce, analz_insert_Key, 
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   448
	  analz_insert_Hash, analz_insert_MPair, analz_Crypt_if];
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   449
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   450
(*This rule supposes "for the sake of argument" that we have the key.*)
2284
80ebd1a213fd Swapped arguments of Crypt (for clarity and because it is conventional)
paulson
parents: 2170
diff changeset
   451
goal thy  "analz (insert (Crypt K X) H) <=  \
80ebd1a213fd Swapped arguments of Crypt (for clarity and because it is conventional)
paulson
parents: 2170
diff changeset
   452
\          insert (Crypt K X) (analz (insert X H))";
2032
1bbf1bdcaf56 Introduction of "lost" argument
paulson
parents: 2028
diff changeset
   453
by (rtac subsetI 1);
1bbf1bdcaf56 Introduction of "lost" argument
paulson
parents: 2028
diff changeset
   454
by (etac analz.induct 1);
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   455
by (Auto_tac());
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   456
qed "analz_insert_Crypt_subset";
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   457
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   458
2026
0df5a96bf77e Last working version prior to introduction of "lost"
paulson
parents: 2011
diff changeset
   459
goal thy "analz (Key``N) = Key``N";
0df5a96bf77e Last working version prior to introduction of "lost"
paulson
parents: 2011
diff changeset
   460
by (Auto_tac());
2032
1bbf1bdcaf56 Introduction of "lost" argument
paulson
parents: 2028
diff changeset
   461
by (etac analz.induct 1);
2026
0df5a96bf77e Last working version prior to introduction of "lost"
paulson
parents: 2011
diff changeset
   462
by (Auto_tac());
0df5a96bf77e Last working version prior to introduction of "lost"
paulson
parents: 2011
diff changeset
   463
qed "analz_image_Key";
0df5a96bf77e Last working version prior to introduction of "lost"
paulson
parents: 2011
diff changeset
   464
0df5a96bf77e Last working version prior to introduction of "lost"
paulson
parents: 2011
diff changeset
   465
Addsimps [analz_image_Key];
0df5a96bf77e Last working version prior to introduction of "lost"
paulson
parents: 2011
diff changeset
   466
0df5a96bf77e Last working version prior to introduction of "lost"
paulson
parents: 2011
diff changeset
   467
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   468
(** Idempotence and transitivity **)
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   469
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   470
goal thy "!!H. X: analz (analz H) ==> X: analz H";
2032
1bbf1bdcaf56 Introduction of "lost" argument
paulson
parents: 2028
diff changeset
   471
by (etac analz.induct 1);
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   472
by (ALLGOALS Fast_tac);
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   473
qed "analz_analzE";
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   474
AddSEs [analz_analzE];
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   475
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   476
goal thy "analz (analz H) = analz H";
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   477
by (Fast_tac 1);
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   478
qed "analz_idem";
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   479
Addsimps [analz_idem];
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   480
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   481
goal thy "!!H. [| X: analz G;  G <= analz H |] ==> X: analz H";
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   482
by (dtac analz_mono 1);
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   483
by (Fast_tac 1);
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   484
qed "analz_trans";
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   485
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   486
(*Cut; Lemma 2 of Lowe*)
1998
f8230821f1e8 Reordering of premises for cut theorems, and new law MPair_synth_analz
paulson
parents: 1994
diff changeset
   487
goal thy "!!H. [| Y: analz (insert X H);  X: analz H |] ==> Y: analz H";
2032
1bbf1bdcaf56 Introduction of "lost" argument
paulson
parents: 2028
diff changeset
   488
by (etac analz_trans 1);
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   489
by (Fast_tac 1);
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   490
qed "analz_cut";
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   491
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   492
(*Cut can be proved easily by induction on
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   493
   "!!H. Y: analz (insert X H) ==> X: analz H --> Y: analz H"
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   494
*)
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   495
1885
a18a6dc14f76 Auth proofs work up to the XXX...
paulson
parents: 1852
diff changeset
   496
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   497
(** A congruence rule for "analz" **)
1885
a18a6dc14f76 Auth proofs work up to the XXX...
paulson
parents: 1852
diff changeset
   498
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   499
goal thy "!!H. [| analz G <= analz G'; analz H <= analz H' \
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   500
\              |] ==> analz (G Un H) <= analz (G' Un H')";
1885
a18a6dc14f76 Auth proofs work up to the XXX...
paulson
parents: 1852
diff changeset
   501
by (Step_tac 1);
2032
1bbf1bdcaf56 Introduction of "lost" argument
paulson
parents: 2028
diff changeset
   502
by (etac analz.induct 1);
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   503
by (ALLGOALS (best_tac (!claset addIs [analz_mono RS subsetD])));
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   504
qed "analz_subset_cong";
1885
a18a6dc14f76 Auth proofs work up to the XXX...
paulson
parents: 1852
diff changeset
   505
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   506
goal thy "!!H. [| analz G = analz G'; analz H = analz H' \
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   507
\              |] ==> analz (G Un H) = analz (G' Un H')";
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   508
by (REPEAT_FIRST (ares_tac [equalityI, analz_subset_cong]
2032
1bbf1bdcaf56 Introduction of "lost" argument
paulson
parents: 2028
diff changeset
   509
          ORELSE' etac equalityE));
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   510
qed "analz_cong";
1885
a18a6dc14f76 Auth proofs work up to the XXX...
paulson
parents: 1852
diff changeset
   511
a18a6dc14f76 Auth proofs work up to the XXX...
paulson
parents: 1852
diff changeset
   512
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   513
goal thy "!!H. analz H = analz H' ==> analz(insert X H) = analz(insert X H')";
1885
a18a6dc14f76 Auth proofs work up to the XXX...
paulson
parents: 1852
diff changeset
   514
by (asm_simp_tac (!simpset addsimps [insert_def] 
2032
1bbf1bdcaf56 Introduction of "lost" argument
paulson
parents: 2028
diff changeset
   515
                           setloop (rtac analz_cong)) 1);
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   516
qed "analz_insert_cong";
1885
a18a6dc14f76 Auth proofs work up to the XXX...
paulson
parents: 1852
diff changeset
   517
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   518
(*If there are no pairs or encryptions then analz does nothing*)
2284
80ebd1a213fd Swapped arguments of Crypt (for clarity and because it is conventional)
paulson
parents: 2170
diff changeset
   519
goal thy "!!H. [| ALL X Y. {|X,Y|} ~: H;  ALL X K. Crypt K X ~: H |] ==> \
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   520
\         analz H = H";
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   521
by (Step_tac 1);
2032
1bbf1bdcaf56 Introduction of "lost" argument
paulson
parents: 2028
diff changeset
   522
by (etac analz.induct 1);
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   523
by (ALLGOALS Fast_tac);
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   524
qed "analz_trivial";
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   525
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   526
(*Helps to prove Fake cases*)
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   527
goal thy "!!X. X: analz (UN i. analz (H i)) ==> X: analz (UN i. H i)";
2032
1bbf1bdcaf56 Introduction of "lost" argument
paulson
parents: 2028
diff changeset
   528
by (etac analz.induct 1);
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   529
by (ALLGOALS (fast_tac (!claset addEs [impOfSubs analz_mono])));
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   530
val lemma = result();
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   531
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   532
goal thy "analz (UN i. analz (H i)) = analz (UN i. H i)";
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   533
by (fast_tac (!claset addIs [lemma]
2032
1bbf1bdcaf56 Introduction of "lost" argument
paulson
parents: 2028
diff changeset
   534
                      addEs [impOfSubs analz_mono]) 1);
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   535
qed "analz_UN_analz";
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   536
Addsimps [analz_UN_analz];
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   537
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   538
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   539
(**** Inductive relation "synth" ****)
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   540
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   541
AddIs  synth.intrs;
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   542
2011
d9af64c26be6 New laws for messages
paulson
parents: 1998
diff changeset
   543
(*Can only produce a nonce or key if it is already known,
d9af64c26be6 New laws for messages
paulson
parents: 1998
diff changeset
   544
  but can synth a pair or encryption from its components...*)
d9af64c26be6 New laws for messages
paulson
parents: 1998
diff changeset
   545
val mk_cases = synth.mk_cases msg.simps;
d9af64c26be6 New laws for messages
paulson
parents: 1998
diff changeset
   546
d9af64c26be6 New laws for messages
paulson
parents: 1998
diff changeset
   547
(*NO Agent_synth, as any Agent name can be synthd*)
d9af64c26be6 New laws for messages
paulson
parents: 1998
diff changeset
   548
val Nonce_synth = mk_cases "Nonce n : synth H";
d9af64c26be6 New laws for messages
paulson
parents: 1998
diff changeset
   549
val Key_synth   = mk_cases "Key K : synth H";
2373
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   550
val Hash_synth  = mk_cases "Hash X : synth H";
2011
d9af64c26be6 New laws for messages
paulson
parents: 1998
diff changeset
   551
val MPair_synth = mk_cases "{|X,Y|} : synth H";
2284
80ebd1a213fd Swapped arguments of Crypt (for clarity and because it is conventional)
paulson
parents: 2170
diff changeset
   552
val Crypt_synth = mk_cases "Crypt K X : synth H";
2011
d9af64c26be6 New laws for messages
paulson
parents: 1998
diff changeset
   553
2373
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   554
AddSEs [Nonce_synth, Key_synth, Hash_synth, MPair_synth, Crypt_synth];
2011
d9af64c26be6 New laws for messages
paulson
parents: 1998
diff changeset
   555
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   556
goal thy "H <= synth(H)";
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   557
by (Fast_tac 1);
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   558
qed "synth_increasing";
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   559
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   560
(*Monotonicity*)
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   561
goalw thy synth.defs "!!G H. G<=H ==> synth(G) <= synth(H)";
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   562
by (rtac lfp_mono 1);
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   563
by (REPEAT (ares_tac basic_monos 1));
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   564
qed "synth_mono";
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   565
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   566
(** Unions **)
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   567
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   568
(*Converse fails: we can synth more from the union than from the 
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   569
  separate parts, building a compound message using elements of each.*)
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   570
goal thy "synth(G) Un synth(H) <= synth(G Un H)";
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   571
by (REPEAT (ares_tac [Un_least, synth_mono, Un_upper1, Un_upper2] 1));
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   572
qed "synth_Un";
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   573
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   574
goal thy "insert X (synth H) <= synth(insert X H)";
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   575
by (fast_tac (!claset addEs [impOfSubs synth_mono]) 1);
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   576
qed "synth_insert";
1885
a18a6dc14f76 Auth proofs work up to the XXX...
paulson
parents: 1852
diff changeset
   577
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   578
(** Idempotence and transitivity **)
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   579
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   580
goal thy "!!H. X: synth (synth H) ==> X: synth H";
2032
1bbf1bdcaf56 Introduction of "lost" argument
paulson
parents: 2028
diff changeset
   581
by (etac synth.induct 1);
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   582
by (ALLGOALS Fast_tac);
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   583
qed "synth_synthE";
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   584
AddSEs [synth_synthE];
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   585
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   586
goal thy "synth (synth H) = synth H";
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   587
by (Fast_tac 1);
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   588
qed "synth_idem";
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   589
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   590
goal thy "!!H. [| X: synth G;  G <= synth H |] ==> X: synth H";
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   591
by (dtac synth_mono 1);
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   592
by (Fast_tac 1);
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   593
qed "synth_trans";
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   594
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   595
(*Cut; Lemma 2 of Lowe*)
1998
f8230821f1e8 Reordering of premises for cut theorems, and new law MPair_synth_analz
paulson
parents: 1994
diff changeset
   596
goal thy "!!H. [| Y: synth (insert X H);  X: synth H |] ==> Y: synth H";
2032
1bbf1bdcaf56 Introduction of "lost" argument
paulson
parents: 2028
diff changeset
   597
by (etac synth_trans 1);
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   598
by (Fast_tac 1);
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   599
qed "synth_cut";
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   600
1946
b59a3d686436 New theorems for Fake case
paulson
parents: 1929
diff changeset
   601
goal thy "Agent A : synth H";
b59a3d686436 New theorems for Fake case
paulson
parents: 1929
diff changeset
   602
by (Fast_tac 1);
b59a3d686436 New theorems for Fake case
paulson
parents: 1929
diff changeset
   603
qed "Agent_synth";
b59a3d686436 New theorems for Fake case
paulson
parents: 1929
diff changeset
   604
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   605
goal thy "(Nonce N : synth H) = (Nonce N : H)";
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   606
by (Fast_tac 1);
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   607
qed "Nonce_synth_eq";
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   608
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   609
goal thy "(Key K : synth H) = (Key K : H)";
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   610
by (Fast_tac 1);
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   611
qed "Key_synth_eq";
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   612
2373
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   613
goal thy "!!K. Key K ~: H ==> (Crypt K X : synth H) = (Crypt K X : H)";
2011
d9af64c26be6 New laws for messages
paulson
parents: 1998
diff changeset
   614
by (Fast_tac 1);
d9af64c26be6 New laws for messages
paulson
parents: 1998
diff changeset
   615
qed "Crypt_synth_eq";
d9af64c26be6 New laws for messages
paulson
parents: 1998
diff changeset
   616
d9af64c26be6 New laws for messages
paulson
parents: 1998
diff changeset
   617
Addsimps [Agent_synth, Nonce_synth_eq, Key_synth_eq, Crypt_synth_eq];
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   618
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   619
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   620
goalw thy [keysFor_def]
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   621
    "keysFor (synth H) = keysFor H Un invKey``{K. Key K : H}";
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   622
by (Fast_tac 1);
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   623
qed "keysFor_synth";
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   624
Addsimps [keysFor_synth];
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   625
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   626
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   627
(*** Combinations of parts, analz and synth ***)
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   628
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   629
goal thy "parts (synth H) = parts H Un synth H";
2032
1bbf1bdcaf56 Introduction of "lost" argument
paulson
parents: 2028
diff changeset
   630
by (rtac equalityI 1);
1bbf1bdcaf56 Introduction of "lost" argument
paulson
parents: 2028
diff changeset
   631
by (rtac subsetI 1);
1bbf1bdcaf56 Introduction of "lost" argument
paulson
parents: 2028
diff changeset
   632
by (etac parts.induct 1);
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   633
by (ALLGOALS
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   634
    (best_tac (!claset addIs ((synth_increasing RS parts_mono RS subsetD)
2032
1bbf1bdcaf56 Introduction of "lost" argument
paulson
parents: 2028
diff changeset
   635
                             ::parts.intrs))));
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   636
qed "parts_synth";
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   637
Addsimps [parts_synth];
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   638
2373
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   639
goal thy "analz (analz G Un H) = analz (G Un H)";
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   640
by (REPEAT_FIRST (resolve_tac [equalityI, analz_subset_cong]));
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   641
by (ALLGOALS Simp_tac);
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   642
qed "analz_analz_Un";
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   643
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   644
goal thy "analz (synth G Un H) = analz (G Un H) Un synth G";
2032
1bbf1bdcaf56 Introduction of "lost" argument
paulson
parents: 2028
diff changeset
   645
by (rtac equalityI 1);
1bbf1bdcaf56 Introduction of "lost" argument
paulson
parents: 2028
diff changeset
   646
by (rtac subsetI 1);
1bbf1bdcaf56 Introduction of "lost" argument
paulson
parents: 2028
diff changeset
   647
by (etac analz.induct 1);
2373
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   648
by (deepen_tac (!claset addIs [impOfSubs analz_mono]) 0 5);
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   649
(*Strange that best_tac just can't hack this one...*)
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   650
by (ALLGOALS (deepen_tac (!claset addIs analz.intrs) 0));
2373
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   651
qed "analz_synth_Un";
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   652
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   653
goal thy "analz (synth H) = analz H Un synth H";
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   654
by (cut_inst_tac [("H","{}")] analz_synth_Un 1);
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   655
by (Full_simp_tac 1);
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   656
qed "analz_synth";
2373
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   657
Addsimps [analz_analz_Un, analz_synth_Un, analz_synth];
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   658
2032
1bbf1bdcaf56 Introduction of "lost" argument
paulson
parents: 2028
diff changeset
   659
(*Hard to prove; still needed now that there's only one Spy?*)
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   660
goal thy "analz (UN i. synth (H i)) = \
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   661
\         analz (UN i. H i) Un (UN i. synth (H i))";
2032
1bbf1bdcaf56 Introduction of "lost" argument
paulson
parents: 2028
diff changeset
   662
by (rtac equalityI 1);
1bbf1bdcaf56 Introduction of "lost" argument
paulson
parents: 2028
diff changeset
   663
by (rtac subsetI 1);
1bbf1bdcaf56 Introduction of "lost" argument
paulson
parents: 2028
diff changeset
   664
by (etac analz.induct 1);
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   665
by (best_tac
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   666
    (!claset addEs [impOfSubs synth_increasing,
2032
1bbf1bdcaf56 Introduction of "lost" argument
paulson
parents: 2028
diff changeset
   667
                    impOfSubs analz_mono]) 5);
1839
199243afac2b Proving safety properties of authentication protocols
paulson
parents:
diff changeset
   668
by (Best_tac 1);
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   669
by (deepen_tac (!claset addIs [analz.Fst]) 0 1);
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   670
by (deepen_tac (!claset addIs [analz.Snd]) 0 1);
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   671
by (deepen_tac (!claset addSEs [analz.Decrypt]
2032
1bbf1bdcaf56 Introduction of "lost" argument
paulson
parents: 2028
diff changeset
   672
                        addIs  [analz.Decrypt]) 0 1);
1913
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   673
qed "analz_UN1_synth";
2809adb15eb0 Renaming of functions, and tidying
paulson
parents: 1893
diff changeset
   674
Addsimps [analz_UN1_synth];
1929
f0839bab4b00 Working version of NS, messages 1-3, WITH INTERLEAVING
paulson
parents: 1913
diff changeset
   675
1946
b59a3d686436 New theorems for Fake case
paulson
parents: 1929
diff changeset
   676
b59a3d686436 New theorems for Fake case
paulson
parents: 1929
diff changeset
   677
(** For reasoning about the Fake rule in traces **)
b59a3d686436 New theorems for Fake case
paulson
parents: 1929
diff changeset
   678
1929
f0839bab4b00 Working version of NS, messages 1-3, WITH INTERLEAVING
paulson
parents: 1913
diff changeset
   679
goal thy "!!Y. X: G ==> parts(insert X H) <= parts G Un parts H";
2032
1bbf1bdcaf56 Introduction of "lost" argument
paulson
parents: 2028
diff changeset
   680
by (rtac ([parts_mono, parts_Un_subset2] MRS subset_trans) 1);
1929
f0839bab4b00 Working version of NS, messages 1-3, WITH INTERLEAVING
paulson
parents: 1913
diff changeset
   681
by (Fast_tac 1);
f0839bab4b00 Working version of NS, messages 1-3, WITH INTERLEAVING
paulson
parents: 1913
diff changeset
   682
qed "parts_insert_subset_Un";
f0839bab4b00 Working version of NS, messages 1-3, WITH INTERLEAVING
paulson
parents: 1913
diff changeset
   683
1946
b59a3d686436 New theorems for Fake case
paulson
parents: 1929
diff changeset
   684
(*More specifically for Fake*)
b59a3d686436 New theorems for Fake case
paulson
parents: 1929
diff changeset
   685
goal thy "!!H. X: synth (analz G) ==> \
b59a3d686436 New theorems for Fake case
paulson
parents: 1929
diff changeset
   686
\              parts (insert X H) <= synth (analz G) Un parts G Un parts H";
2032
1bbf1bdcaf56 Introduction of "lost" argument
paulson
parents: 2028
diff changeset
   687
by (dtac parts_insert_subset_Un 1);
1946
b59a3d686436 New theorems for Fake case
paulson
parents: 1929
diff changeset
   688
by (Full_simp_tac 1);
b59a3d686436 New theorems for Fake case
paulson
parents: 1929
diff changeset
   689
by (Deepen_tac 0 1);
b59a3d686436 New theorems for Fake case
paulson
parents: 1929
diff changeset
   690
qed "Fake_parts_insert";
b59a3d686436 New theorems for Fake case
paulson
parents: 1929
diff changeset
   691
2061
b14a08bf61bf New theorem Crypt_Fake_parts_insert
paulson
parents: 2032
diff changeset
   692
goal thy
2284
80ebd1a213fd Swapped arguments of Crypt (for clarity and because it is conventional)
paulson
parents: 2170
diff changeset
   693
     "!!H. [| Crypt K Y : parts (insert X H);  X: synth (analz G);  \
2061
b14a08bf61bf New theorem Crypt_Fake_parts_insert
paulson
parents: 2032
diff changeset
   694
\             Key K ~: analz G |]                                   \
2284
80ebd1a213fd Swapped arguments of Crypt (for clarity and because it is conventional)
paulson
parents: 2170
diff changeset
   695
\          ==> Crypt K Y : parts G Un parts H";
2061
b14a08bf61bf New theorem Crypt_Fake_parts_insert
paulson
parents: 2032
diff changeset
   696
by (dtac (impOfSubs Fake_parts_insert) 1);
2170
c5e460f1ebb4 Ran expandshort
paulson
parents: 2154
diff changeset
   697
by (assume_tac 1);
2061
b14a08bf61bf New theorem Crypt_Fake_parts_insert
paulson
parents: 2032
diff changeset
   698
by (fast_tac (!claset addDs [impOfSubs analz_subset_parts]
b14a08bf61bf New theorem Crypt_Fake_parts_insert
paulson
parents: 2032
diff changeset
   699
                      addss (!simpset)) 1);
b14a08bf61bf New theorem Crypt_Fake_parts_insert
paulson
parents: 2032
diff changeset
   700
qed "Crypt_Fake_parts_insert";
b14a08bf61bf New theorem Crypt_Fake_parts_insert
paulson
parents: 2032
diff changeset
   701
2373
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   702
goal thy "!!H. X: synth (analz G) ==> \
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   703
\              analz (insert X H) <= synth (analz G) Un analz (G Un H)";
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   704
by (rtac subsetI 1);
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   705
by (subgoal_tac "x : analz (synth (analz G) Un H)" 1);
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   706
by (best_tac (!claset addIs [impOfSubs (analz_mono RS synth_mono)]
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   707
                      addSEs [impOfSubs analz_mono]) 2);
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   708
by (Full_simp_tac 1);
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   709
by (Fast_tac 1);
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   710
qed "Fake_analz_insert";
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   711
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   712
(*Needed????????????????*)
1946
b59a3d686436 New theorems for Fake case
paulson
parents: 1929
diff changeset
   713
goal thy "!!H. [| X: synth (analz G); G <= H |] ==> \
b59a3d686436 New theorems for Fake case
paulson
parents: 1929
diff changeset
   714
\              analz (insert X H) <= synth (analz H) Un analz H";
2032
1bbf1bdcaf56 Introduction of "lost" argument
paulson
parents: 2028
diff changeset
   715
by (rtac subsetI 1);
1946
b59a3d686436 New theorems for Fake case
paulson
parents: 1929
diff changeset
   716
by (subgoal_tac "x : analz (synth (analz H))" 1);
b59a3d686436 New theorems for Fake case
paulson
parents: 1929
diff changeset
   717
by (best_tac (!claset addIs [impOfSubs (analz_mono RS synth_mono)]
b59a3d686436 New theorems for Fake case
paulson
parents: 1929
diff changeset
   718
                      addSEs [impOfSubs analz_mono]) 2);
b59a3d686436 New theorems for Fake case
paulson
parents: 1929
diff changeset
   719
by (Full_simp_tac 1);
b59a3d686436 New theorems for Fake case
paulson
parents: 1929
diff changeset
   720
by (Fast_tac 1);
2373
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   721
qed "Fake_analz_insert_old";
1929
f0839bab4b00 Working version of NS, messages 1-3, WITH INTERLEAVING
paulson
parents: 1913
diff changeset
   722
2011
d9af64c26be6 New laws for messages
paulson
parents: 1998
diff changeset
   723
goal thy "(X: analz H & X: parts H) = (X: analz H)";
d9af64c26be6 New laws for messages
paulson
parents: 1998
diff changeset
   724
by (fast_tac (!claset addDs [impOfSubs analz_subset_parts]) 1);
d9af64c26be6 New laws for messages
paulson
parents: 1998
diff changeset
   725
val analz_conj_parts = result();
d9af64c26be6 New laws for messages
paulson
parents: 1998
diff changeset
   726
d9af64c26be6 New laws for messages
paulson
parents: 1998
diff changeset
   727
goal thy "(X: analz H | X: parts H) = (X: parts H)";
d9af64c26be6 New laws for messages
paulson
parents: 1998
diff changeset
   728
by (fast_tac (!claset addDs [impOfSubs analz_subset_parts]) 1);
d9af64c26be6 New laws for messages
paulson
parents: 1998
diff changeset
   729
val analz_disj_parts = result();
d9af64c26be6 New laws for messages
paulson
parents: 1998
diff changeset
   730
d9af64c26be6 New laws for messages
paulson
parents: 1998
diff changeset
   731
AddIffs [analz_conj_parts, analz_disj_parts];
d9af64c26be6 New laws for messages
paulson
parents: 1998
diff changeset
   732
1998
f8230821f1e8 Reordering of premises for cut theorems, and new law MPair_synth_analz
paulson
parents: 1994
diff changeset
   733
(*Without this equation, other rules for synth and analz would yield
f8230821f1e8 Reordering of premises for cut theorems, and new law MPair_synth_analz
paulson
parents: 1994
diff changeset
   734
  redundant cases*)
f8230821f1e8 Reordering of premises for cut theorems, and new law MPair_synth_analz
paulson
parents: 1994
diff changeset
   735
goal thy "({|X,Y|} : synth (analz H)) = \
f8230821f1e8 Reordering of premises for cut theorems, and new law MPair_synth_analz
paulson
parents: 1994
diff changeset
   736
\         (X : synth (analz H) & Y : synth (analz H))";
f8230821f1e8 Reordering of premises for cut theorems, and new law MPair_synth_analz
paulson
parents: 1994
diff changeset
   737
by (Fast_tac 1);
f8230821f1e8 Reordering of premises for cut theorems, and new law MPair_synth_analz
paulson
parents: 1994
diff changeset
   738
qed "MPair_synth_analz";
f8230821f1e8 Reordering of premises for cut theorems, and new law MPair_synth_analz
paulson
parents: 1994
diff changeset
   739
f8230821f1e8 Reordering of premises for cut theorems, and new law MPair_synth_analz
paulson
parents: 1994
diff changeset
   740
AddIffs [MPair_synth_analz];
1929
f0839bab4b00 Working version of NS, messages 1-3, WITH INTERLEAVING
paulson
parents: 1913
diff changeset
   741
2154
913b4fc7670a New, purely illustrative result Crypt_synth_analz
paulson
parents: 2102
diff changeset
   742
goal thy "!!K. [| Key K : analz H;  Key (invKey K) : analz H |] \
2284
80ebd1a213fd Swapped arguments of Crypt (for clarity and because it is conventional)
paulson
parents: 2170
diff changeset
   743
\              ==> (Crypt K X : synth (analz H)) = (X : synth (analz H))";
2154
913b4fc7670a New, purely illustrative result Crypt_synth_analz
paulson
parents: 2102
diff changeset
   744
by (Fast_tac 1);
913b4fc7670a New, purely illustrative result Crypt_synth_analz
paulson
parents: 2102
diff changeset
   745
qed "Crypt_synth_analz";
913b4fc7670a New, purely illustrative result Crypt_synth_analz
paulson
parents: 2102
diff changeset
   746
1929
f0839bab4b00 Working version of NS, messages 1-3, WITH INTERLEAVING
paulson
parents: 1913
diff changeset
   747
2373
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   748
goal thy "!!K. Key K ~: analz H \
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   749
\   ==> (Hash{|Key K,X|} : synth (analz H)) = (Hash{|Key K,X|} : analz H)";
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   750
by (Fast_tac 1);
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   751
qed "Hash_synth_analz";
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   752
Addsimps [Hash_synth_analz];
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   753
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   754
1929
f0839bab4b00 Working version of NS, messages 1-3, WITH INTERLEAVING
paulson
parents: 1913
diff changeset
   755
(*We do NOT want Crypt... messages broken up in protocols!!*)
f0839bab4b00 Working version of NS, messages 1-3, WITH INTERLEAVING
paulson
parents: 1913
diff changeset
   756
Delrules partsEs;
f0839bab4b00 Working version of NS, messages 1-3, WITH INTERLEAVING
paulson
parents: 1913
diff changeset
   757
2327
00ac25b2791d Moved much common material to Message.ML
paulson
parents: 2284
diff changeset
   758
00ac25b2791d Moved much common material to Message.ML
paulson
parents: 2284
diff changeset
   759
(** Rewrites to push in Key and Crypt messages, so that other messages can
00ac25b2791d Moved much common material to Message.ML
paulson
parents: 2284
diff changeset
   760
    be pulled out using the analz_insert rules **)
00ac25b2791d Moved much common material to Message.ML
paulson
parents: 2284
diff changeset
   761
00ac25b2791d Moved much common material to Message.ML
paulson
parents: 2284
diff changeset
   762
fun insComm thy x y = read_instantiate_sg (sign_of thy) [("x",x), ("y",y)] 
00ac25b2791d Moved much common material to Message.ML
paulson
parents: 2284
diff changeset
   763
                          insert_commute;
00ac25b2791d Moved much common material to Message.ML
paulson
parents: 2284
diff changeset
   764
00ac25b2791d Moved much common material to Message.ML
paulson
parents: 2284
diff changeset
   765
val pushKeys = map (insComm thy "Key ?K") 
2373
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   766
                   ["Agent ?C", "Nonce ?N", "Hash ?X", 
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   767
		    "MPair ?X ?Y", "Crypt ?X ?K'"];
2327
00ac25b2791d Moved much common material to Message.ML
paulson
parents: 2284
diff changeset
   768
00ac25b2791d Moved much common material to Message.ML
paulson
parents: 2284
diff changeset
   769
val pushCrypts = map (insComm thy "Crypt ?X ?K") 
2373
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   770
                     ["Agent ?C", "Nonce ?N", "Hash ?X'", "MPair ?X' ?Y"];
2327
00ac25b2791d Moved much common material to Message.ML
paulson
parents: 2284
diff changeset
   771
00ac25b2791d Moved much common material to Message.ML
paulson
parents: 2284
diff changeset
   772
(*Cannot be added with Addsimps -- we don't always want to re-order messages*)
00ac25b2791d Moved much common material to Message.ML
paulson
parents: 2284
diff changeset
   773
val pushes = pushKeys@pushCrypts;
00ac25b2791d Moved much common material to Message.ML
paulson
parents: 2284
diff changeset
   774
00ac25b2791d Moved much common material to Message.ML
paulson
parents: 2284
diff changeset
   775
00ac25b2791d Moved much common material to Message.ML
paulson
parents: 2284
diff changeset
   776
(*No premature instantiation of variables.  For proving weak liveness.*)
00ac25b2791d Moved much common material to Message.ML
paulson
parents: 2284
diff changeset
   777
fun safe_solver prems =
00ac25b2791d Moved much common material to Message.ML
paulson
parents: 2284
diff changeset
   778
    match_tac (TrueI::refl::prems) ORELSE' eq_assume_tac
00ac25b2791d Moved much common material to Message.ML
paulson
parents: 2284
diff changeset
   779
    ORELSE' etac FalseE;
00ac25b2791d Moved much common material to Message.ML
paulson
parents: 2284
diff changeset
   780
2373
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   781
val Fake_insert_tac = 
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   782
    dresolve_tac [impOfSubs Fake_analz_insert,
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   783
		  impOfSubs Fake_parts_insert] THEN'
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   784
    eresolve_tac [asm_rl, synth.Inj];
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   785
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   786
(*Analysis of Fake cases and of messages that forward unknown parts.
2327
00ac25b2791d Moved much common material to Message.ML
paulson
parents: 2284
diff changeset
   787
  Abstraction over i is ESSENTIAL: it delays the dereferencing of claset
00ac25b2791d Moved much common material to Message.ML
paulson
parents: 2284
diff changeset
   788
  DEPENDS UPON "X" REFERRING TO THE FRADULENT MESSAGE *)
00ac25b2791d Moved much common material to Message.ML
paulson
parents: 2284
diff changeset
   789
fun spy_analz_tac i =
2373
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   790
  DETERM
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   791
   (SELECT_GOAL
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   792
     (EVERY 
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   793
      [  (*push in occurrences of X...*)
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   794
       (REPEAT o CHANGED)
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   795
           (res_inst_tac [("x1","X")] (insert_commute RS ssubst) 1),
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   796
       (*...allowing further simplifications*)
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   797
       simp_tac (!simpset setloop split_tac [expand_if]) 1,
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   798
       REPEAT (FIRSTGOAL (resolve_tac [allI,impI,notI,conjI])),
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   799
       DEPTH_SOLVE 
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   800
         (REPEAT (Fake_insert_tac 1) THEN Asm_full_simp_tac 1
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   801
	  THEN
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   802
	  IF_UNSOLVED (depth_tac (!claset addIs [impOfSubs analz_mono,
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   803
						 impOfSubs analz_subset_parts]) 2 1))
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   804
       ]) i);
2327
00ac25b2791d Moved much common material to Message.ML
paulson
parents: 2284
diff changeset
   805
00ac25b2791d Moved much common material to Message.ML
paulson
parents: 2284
diff changeset
   806
(*Useful in many uniqueness proofs*)
00ac25b2791d Moved much common material to Message.ML
paulson
parents: 2284
diff changeset
   807
fun ex_strip_tac i = REPEAT (swap_res_tac [exI, conjI] i) THEN 
00ac25b2791d Moved much common material to Message.ML
paulson
parents: 2284
diff changeset
   808
                     assume_tac (i+1);
00ac25b2791d Moved much common material to Message.ML
paulson
parents: 2284
diff changeset
   809
2373
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   810
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   811
(*Needed occasionally with spy_analz_tac, e.g. in analz_insert_Key_newK*)
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   812
goal Set.thy "A Un (B Un A) = B Un A";
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   813
by (Fast_tac 1);
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   814
val Un_absorb3 = result();
490ffa16952e Addition of the Hash constructor
paulson
parents: 2327
diff changeset
   815
Addsimps [Un_absorb3];