18886
|
1 |
(* ID: $Id$
|
|
2 |
Author: Giampaolo Bella, Catania University
|
|
3 |
*)
|
|
4 |
|
|
5 |
header{*Bella's version of the Otway-Rees protocol*}
|
|
6 |
|
|
7 |
|
|
8 |
theory OtwayReesBella imports Public begin
|
|
9 |
|
|
10 |
text{*Bella's modifications to a version of the Otway-Rees protocol taken from
|
|
11 |
the BAN paper only concern message 7. The updated protocol makes the goal of
|
|
12 |
key distribution of the session key available to A. Investigating the
|
|
13 |
principle of Goal Availability undermines the BAN claim about the original
|
|
14 |
protocol, that "this protocol does not make use of Kab as an encryption key,
|
|
15 |
so neither principal can know whether the key is known to the other". The
|
|
16 |
updated protocol makes no use of the session key to encrypt but informs A that
|
|
17 |
B knows it.*}
|
|
18 |
|
23746
|
19 |
inductive_set orb :: "event list set"
|
|
20 |
where
|
18886
|
21 |
|
|
22 |
Nil: "[]\<in> orb"
|
|
23 |
|
23746
|
24 |
| Fake: "\<lbrakk>evsa\<in> orb; X\<in> synth (analz (knows Spy evsa))\<rbrakk>
|
18886
|
25 |
\<Longrightarrow> Says Spy B X # evsa \<in> orb"
|
|
26 |
|
23746
|
27 |
| Reception: "\<lbrakk>evsr\<in> orb; Says A B X \<in> set evsr\<rbrakk>
|
18886
|
28 |
\<Longrightarrow> Gets B X # evsr \<in> orb"
|
|
29 |
|
23746
|
30 |
| OR1: "\<lbrakk>evs1\<in> orb; Nonce NA \<notin> used evs1\<rbrakk>
|
18886
|
31 |
\<Longrightarrow> Says A B \<lbrace>Nonce M, Agent A, Agent B,
|
|
32 |
Crypt (shrK A) \<lbrace>Nonce NA, Nonce M, Agent A, Agent B\<rbrace>\<rbrace>
|
|
33 |
# evs1 \<in> orb"
|
|
34 |
|
23746
|
35 |
| OR2: "\<lbrakk>evs2\<in> orb; Nonce NB \<notin> used evs2;
|
18886
|
36 |
Gets B \<lbrace>Nonce M, Agent A, Agent B, X\<rbrace> \<in> set evs2\<rbrakk>
|
|
37 |
\<Longrightarrow> Says B Server
|
|
38 |
\<lbrace>Nonce M, Agent A, Agent B, X,
|
|
39 |
Crypt (shrK B) \<lbrace>Nonce NB, Nonce M, Nonce M, Agent A, Agent B\<rbrace>\<rbrace>
|
|
40 |
# evs2 \<in> orb"
|
|
41 |
|
23746
|
42 |
| OR3: "\<lbrakk>evs3\<in> orb; Key KAB \<notin> used evs3;
|
18886
|
43 |
Gets Server
|
|
44 |
\<lbrace>Nonce M, Agent A, Agent B,
|
|
45 |
Crypt (shrK A) \<lbrace>Nonce NA, Nonce M, Agent A, Agent B\<rbrace>,
|
|
46 |
Crypt (shrK B) \<lbrace>Nonce NB, Nonce M, Nonce M, Agent A, Agent B\<rbrace>\<rbrace>
|
|
47 |
\<in> set evs3\<rbrakk>
|
|
48 |
\<Longrightarrow> Says Server B \<lbrace>Nonce M,
|
|
49 |
Crypt (shrK B) \<lbrace>Crypt (shrK A) \<lbrace>Nonce NA, Key KAB\<rbrace>,
|
|
50 |
Nonce NB, Key KAB\<rbrace>\<rbrace>
|
|
51 |
# evs3 \<in> orb"
|
|
52 |
|
|
53 |
(*B can only check that the message he is bouncing is a ciphertext*)
|
|
54 |
(*Sending M back is omitted*)
|
23746
|
55 |
| OR4: "\<lbrakk>evs4\<in> orb; B \<noteq> Server; \<forall> p q. X \<noteq> \<lbrace>p, q\<rbrace>;
|
18886
|
56 |
Says B Server \<lbrace>Nonce M, Agent A, Agent B, X',
|
|
57 |
Crypt (shrK B) \<lbrace>Nonce NB, Nonce M, Nonce M, Agent A, Agent B\<rbrace>\<rbrace>
|
|
58 |
\<in> set evs4;
|
|
59 |
Gets B \<lbrace>Nonce M, Crypt (shrK B) \<lbrace>X, Nonce NB, Key KAB\<rbrace>\<rbrace>
|
|
60 |
\<in> set evs4\<rbrakk>
|
|
61 |
\<Longrightarrow> Says B A \<lbrace>Nonce M, X\<rbrace> # evs4 \<in> orb"
|
|
62 |
|
|
63 |
|
23746
|
64 |
| Oops: "\<lbrakk>evso\<in> orb;
|
18886
|
65 |
Says Server B \<lbrace>Nonce M,
|
|
66 |
Crypt (shrK B) \<lbrace>Crypt (shrK A) \<lbrace>Nonce NA, Key KAB\<rbrace>,
|
|
67 |
Nonce NB, Key KAB\<rbrace>\<rbrace>
|
|
68 |
\<in> set evso\<rbrakk>
|
|
69 |
\<Longrightarrow> Notes Spy \<lbrace>Agent A, Agent B, Nonce NA, Nonce NB, Key KAB\<rbrace> # evso
|
|
70 |
\<in> orb"
|
|
71 |
|
|
72 |
|
|
73 |
|
|
74 |
declare knows_Spy_partsEs [elim]
|
|
75 |
declare analz_into_parts [dest]
|
|
76 |
declare Fake_parts_insert_in_Un [dest]
|
|
77 |
|
|
78 |
|
|
79 |
text{*Fragile proof, with backtracking in the possibility call.*}
|
|
80 |
lemma possibility_thm: "\<lbrakk>A \<noteq> Server; B \<noteq> Server; Key K \<notin> used[]\<rbrakk>
|
|
81 |
\<Longrightarrow> \<exists> evs \<in> orb.
|
|
82 |
Says B A \<lbrace>Nonce M, Crypt (shrK A) \<lbrace>Nonce Na, Key K\<rbrace>\<rbrace> \<in> set evs"
|
|
83 |
apply (intro exI bexI)
|
|
84 |
apply (rule_tac [2] orb.Nil
|
|
85 |
[THEN orb.OR1, THEN orb.Reception,
|
|
86 |
THEN orb.OR2, THEN orb.Reception,
|
|
87 |
THEN orb.OR3, THEN orb.Reception, THEN orb.OR4])
|
|
88 |
apply (possibility, simp add: used_Cons)
|
|
89 |
done
|
|
90 |
|
|
91 |
|
|
92 |
lemma Gets_imp_Says :
|
|
93 |
"\<lbrakk>Gets B X \<in> set evs; evs \<in> orb\<rbrakk> \<Longrightarrow> \<exists>A. Says A B X \<in> set evs"
|
|
94 |
apply (erule rev_mp)
|
|
95 |
apply (erule orb.induct)
|
|
96 |
apply auto
|
|
97 |
done
|
|
98 |
|
|
99 |
lemma Gets_imp_knows_Spy:
|
|
100 |
"\<lbrakk>Gets B X \<in> set evs; evs \<in> orb\<rbrakk> \<Longrightarrow> X \<in> knows Spy evs"
|
|
101 |
by (blast dest!: Gets_imp_Says Says_imp_knows_Spy)
|
|
102 |
|
|
103 |
declare Gets_imp_knows_Spy [THEN parts.Inj, dest]
|
|
104 |
|
|
105 |
lemma Gets_imp_knows:
|
|
106 |
"\<lbrakk>Gets B X \<in> set evs; evs \<in> orb\<rbrakk> \<Longrightarrow> X \<in> knows B evs"
|
|
107 |
apply (case_tac "B = Spy")
|
|
108 |
apply (blast dest!: Gets_imp_knows_Spy)
|
|
109 |
apply (blast dest!: Gets_imp_knows_agents)
|
|
110 |
done
|
|
111 |
|
|
112 |
|
|
113 |
lemma OR2_analz_knows_Spy:
|
|
114 |
"\<lbrakk>Gets B \<lbrace>Nonce M, Agent A, Agent B, X\<rbrace> \<in> set evs; evs \<in> orb\<rbrakk>
|
|
115 |
\<Longrightarrow> X \<in> analz (knows Spy evs)"
|
|
116 |
by (blast dest!: Gets_imp_knows_Spy [THEN analz.Inj])
|
|
117 |
|
|
118 |
lemma OR4_parts_knows_Spy:
|
|
119 |
"\<lbrakk>Gets B \<lbrace>Nonce M, Crypt (shrK B) \<lbrace>X, Nonce Nb, Key Kab\<rbrace>\<rbrace> \<in> set evs;
|
|
120 |
evs \<in> orb\<rbrakk> \<Longrightarrow> X \<in> parts (knows Spy evs)"
|
|
121 |
by blast
|
|
122 |
|
|
123 |
lemma Oops_parts_knows_Spy:
|
|
124 |
"Says Server B \<lbrace>Nonce M, Crypt K' \<lbrace>X, Nonce Nb, K\<rbrace>\<rbrace> \<in> set evs
|
|
125 |
\<Longrightarrow> K \<in> parts (knows Spy evs)"
|
|
126 |
by blast
|
|
127 |
|
|
128 |
lemmas OR2_parts_knows_Spy =
|
|
129 |
OR2_analz_knows_Spy [THEN analz_into_parts, standard]
|
|
130 |
|
|
131 |
ML
|
|
132 |
{*
|
|
133 |
val Oops_parts_knows_Spy = thm "Oops_parts_knows_Spy"
|
|
134 |
val OR4_parts_knows_Spy = thm "OR4_parts_knows_Spy"
|
|
135 |
val OR2_parts_knows_Spy = thm "OR2_parts_knows_Spy"
|
|
136 |
|
|
137 |
fun parts_explicit_tac i =
|
|
138 |
forward_tac [Oops_parts_knows_Spy] (i+7) THEN
|
|
139 |
forward_tac [OR4_parts_knows_Spy] (i+6) THEN
|
|
140 |
forward_tac [OR2_parts_knows_Spy] (i+4)
|
|
141 |
*}
|
|
142 |
|
|
143 |
method_setup parts_explicit = {*
|
21588
|
144 |
Method.no_args (Method.SIMPLE_METHOD' parts_explicit_tac) *}
|
18886
|
145 |
"to explicitly state that some message components belong to parts knows Spy"
|
|
146 |
|
|
147 |
|
|
148 |
lemma Spy_see_shrK [simp]:
|
|
149 |
"evs \<in> orb \<Longrightarrow> (Key (shrK A) \<in> parts (knows Spy evs)) = (A \<in> bad)"
|
|
150 |
by (erule orb.induct, parts_explicit, simp_all, blast+)
|
|
151 |
|
|
152 |
lemma Spy_analz_shrK [simp]:
|
|
153 |
"evs \<in> orb \<Longrightarrow> (Key (shrK A) \<in> analz (knows Spy evs)) = (A \<in> bad)"
|
|
154 |
by auto
|
|
155 |
|
|
156 |
lemma Spy_see_shrK_D [dest!]:
|
|
157 |
"[|Key (shrK A) \<in> parts (knows Spy evs); evs \<in> orb|] ==> A \<in> bad"
|
|
158 |
by (blast dest: Spy_see_shrK)
|
|
159 |
|
|
160 |
lemma new_keys_not_used [simp]:
|
|
161 |
"\<lbrakk>Key K \<notin> used evs; K \<in> symKeys; evs \<in> orb\<rbrakk> \<Longrightarrow> K \<notin> keysFor (parts (knows Spy evs))"
|
|
162 |
apply (erule rev_mp)
|
|
163 |
apply (erule orb.induct, parts_explicit, simp_all)
|
|
164 |
apply (force dest!: keysFor_parts_insert)
|
|
165 |
apply (blast+)
|
|
166 |
done
|
|
167 |
|
|
168 |
|
|
169 |
|
|
170 |
subsection{* Proofs involving analz *}
|
|
171 |
|
|
172 |
text{*Describes the form of K and NA when the Server sends this message. Also
|
|
173 |
for Oops case.*}
|
|
174 |
lemma Says_Server_message_form:
|
|
175 |
"\<lbrakk>Says Server B \<lbrace>Nonce M, Crypt (shrK B) \<lbrace>X, Nonce Nb, Key K\<rbrace>\<rbrace> \<in> set evs;
|
|
176 |
evs \<in> orb\<rbrakk>
|
|
177 |
\<Longrightarrow> K \<notin> range shrK & (\<exists> A Na. X=(Crypt (shrK A) \<lbrace>Nonce Na, Key K\<rbrace>))"
|
|
178 |
by (erule rev_mp, erule orb.induct, simp_all)
|
|
179 |
|
|
180 |
lemma Says_Server_imp_Gets:
|
|
181 |
"\<lbrakk>Says Server B \<lbrace>Nonce M, Crypt (shrK B) \<lbrace>Crypt (shrK A) \<lbrace>Nonce Na, Key K\<rbrace>,
|
|
182 |
Nonce Nb, Key K\<rbrace>\<rbrace> \<in> set evs;
|
|
183 |
evs \<in> orb\<rbrakk>
|
|
184 |
\<Longrightarrow> Gets Server \<lbrace>Nonce M, Agent A, Agent B,
|
|
185 |
Crypt (shrK A) \<lbrace>Nonce Na, Nonce M, Agent A, Agent B\<rbrace>,
|
|
186 |
Crypt (shrK B) \<lbrace>Nonce Nb, Nonce M, Nonce M, Agent A, Agent B\<rbrace>\<rbrace>
|
|
187 |
\<in> set evs"
|
|
188 |
by (erule rev_mp, erule orb.induct, simp_all)
|
|
189 |
|
|
190 |
|
|
191 |
lemma A_trusts_OR1:
|
|
192 |
"\<lbrakk>Crypt (shrK A) \<lbrace>Nonce Na, Nonce M, Agent A, Agent B\<rbrace> \<in> parts (knows Spy evs);
|
|
193 |
A \<notin> bad; evs \<in> orb\<rbrakk>
|
|
194 |
\<Longrightarrow> Says A B \<lbrace>Nonce M, Agent A, Agent B, Crypt (shrK A) \<lbrace>Nonce Na, Nonce M, Agent A, Agent B\<rbrace>\<rbrace> \<in> set evs"
|
|
195 |
apply (erule rev_mp, erule orb.induct, parts_explicit, simp_all)
|
|
196 |
apply (blast)
|
|
197 |
done
|
|
198 |
|
|
199 |
|
|
200 |
lemma B_trusts_OR2:
|
|
201 |
"\<lbrakk>Crypt (shrK B) \<lbrace>Nonce Nb, Nonce M, Nonce M, Agent A, Agent B\<rbrace>
|
|
202 |
\<in> parts (knows Spy evs); B \<notin> bad; evs \<in> orb\<rbrakk>
|
|
203 |
\<Longrightarrow> (\<exists> X. Says B Server \<lbrace>Nonce M, Agent A, Agent B, X,
|
|
204 |
Crypt (shrK B) \<lbrace>Nonce Nb, Nonce M, Nonce M, Agent A, Agent B\<rbrace>\<rbrace>
|
|
205 |
\<in> set evs)"
|
|
206 |
apply (erule rev_mp, erule orb.induct, parts_explicit, simp_all)
|
|
207 |
apply (blast+)
|
|
208 |
done
|
|
209 |
|
|
210 |
|
|
211 |
lemma B_trusts_OR3:
|
|
212 |
"\<lbrakk>Crypt (shrK B) \<lbrace>X, Nonce Nb, Key K\<rbrace> \<in> parts (knows Spy evs);
|
|
213 |
B \<notin> bad; evs \<in> orb\<rbrakk>
|
|
214 |
\<Longrightarrow> \<exists> M. Says Server B \<lbrace>Nonce M, Crypt (shrK B) \<lbrace>X, Nonce Nb, Key K\<rbrace>\<rbrace>
|
|
215 |
\<in> set evs"
|
|
216 |
apply (erule rev_mp, erule orb.induct, parts_explicit, simp_all)
|
|
217 |
apply (blast+)
|
|
218 |
done
|
|
219 |
|
|
220 |
lemma Gets_Server_message_form:
|
|
221 |
"\<lbrakk>Gets B \<lbrace>Nonce M, Crypt (shrK B) \<lbrace>X, Nonce Nb, Key K\<rbrace>\<rbrace> \<in> set evs;
|
|
222 |
evs \<in> orb\<rbrakk>
|
|
223 |
\<Longrightarrow> (K \<notin> range shrK & (\<exists> A Na. X = (Crypt (shrK A) \<lbrace>Nonce Na, Key K\<rbrace>)))
|
|
224 |
| X \<in> analz (knows Spy evs)"
|
|
225 |
apply (case_tac "B \<in> bad")
|
|
226 |
apply (drule Gets_imp_knows_Spy [THEN analz.Inj, THEN analz.Snd,
|
|
227 |
THEN analz.Decrypt, THEN analz.Fst])
|
|
228 |
prefer 3 apply blast
|
|
229 |
prefer 3 apply (blast dest!: Gets_imp_knows_Spy [THEN parts.Inj, THEN
|
|
230 |
parts.Snd, THEN B_trusts_OR3]
|
|
231 |
Says_Server_message_form)
|
|
232 |
apply simp_all
|
|
233 |
done
|
|
234 |
|
|
235 |
lemma unique_Na: "\<lbrakk>Says A B \<lbrace>Nonce M, Agent A, Agent B, Crypt (shrK A) \<lbrace>Nonce Na, Nonce M, Agent A, Agent B\<rbrace>\<rbrace> \<in> set evs;
|
|
236 |
Says A B' \<lbrace>Nonce M', Agent A, Agent B', Crypt (shrK A) \<lbrace>Nonce Na, Nonce M', Agent A, Agent B'\<rbrace>\<rbrace> \<in> set evs;
|
|
237 |
A \<notin> bad; evs \<in> orb\<rbrakk> \<Longrightarrow> B=B' & M=M'"
|
|
238 |
by (erule rev_mp, erule rev_mp, erule orb.induct, simp_all, blast+)
|
|
239 |
|
|
240 |
lemma unique_Nb: "\<lbrakk>Says B Server \<lbrace>Nonce M, Agent A, Agent B, X, Crypt (shrK B) \<lbrace>Nonce Nb, Nonce M, Nonce M, Agent A, Agent B\<rbrace>\<rbrace> \<in> set evs;
|
|
241 |
Says B Server \<lbrace>Nonce M', Agent A', Agent B, X', Crypt (shrK B) \<lbrace>Nonce Nb,Nonce M', Nonce M', Agent A', Agent B\<rbrace>\<rbrace> \<in> set evs;
|
|
242 |
B \<notin> bad; evs \<in> orb\<rbrakk> \<Longrightarrow> M=M' & A=A' & X=X'"
|
|
243 |
by (erule rev_mp, erule rev_mp, erule orb.induct, simp_all, blast+)
|
|
244 |
|
|
245 |
lemma analz_image_freshCryptK_lemma:
|
|
246 |
"(Crypt K X \<in> analz (Key`nE \<union> H)) \<longrightarrow> (Crypt K X \<in> analz H) \<Longrightarrow>
|
|
247 |
(Crypt K X \<in> analz (Key`nE \<union> H)) = (Crypt K X \<in> analz H)";
|
|
248 |
by (blast intro: analz_mono [THEN [2] rev_subsetD])
|
|
249 |
|
|
250 |
ML
|
|
251 |
{*
|
|
252 |
val analz_image_freshCryptK_lemma = thm "analz_image_freshCryptK_lemma";
|
|
253 |
val analz_image_freshK_simps = thms "analz_image_freshK_simps";
|
|
254 |
|
|
255 |
val analz_image_freshK_ss =
|
|
256 |
simpset() delsimps [image_insert, image_Un]
|
|
257 |
delsimps [imp_disjL] (*reduces blow-up*)
|
|
258 |
addsimps thms "analz_image_freshK_simps"
|
|
259 |
*}
|
|
260 |
|
|
261 |
method_setup analz_freshCryptK = {*
|
20048
|
262 |
Method.ctxt_args (fn ctxt =>
|
21588
|
263 |
(Method.SIMPLE_METHOD
|
|
264 |
(EVERY [REPEAT_FIRST (resolve_tac [allI, ballI, impI]),
|
18886
|
265 |
REPEAT_FIRST (rtac analz_image_freshCryptK_lemma),
|
20048
|
266 |
ALLGOALS (asm_simp_tac (Simplifier.context ctxt analz_image_freshK_ss))]))) *}
|
18886
|
267 |
"for proving useful rewrite rule"
|
|
268 |
|
|
269 |
|
|
270 |
method_setup disentangle = {*
|
|
271 |
Method.no_args
|
21588
|
272 |
(Method.SIMPLE_METHOD
|
|
273 |
(REPEAT_FIRST (eresolve_tac [asm_rl, conjE, disjE]
|
18886
|
274 |
ORELSE' hyp_subst_tac))) *}
|
|
275 |
"for eliminating conjunctions, disjunctions and the like"
|
|
276 |
|
|
277 |
|
|
278 |
|
|
279 |
lemma analz_image_freshCryptK [rule_format]:
|
|
280 |
"evs \<in> orb \<Longrightarrow>
|
|
281 |
Key K \<notin> analz (knows Spy evs) \<longrightarrow>
|
|
282 |
(\<forall> KK. KK \<subseteq> - (range shrK) \<longrightarrow>
|
|
283 |
(Crypt K X \<in> analz (Key`KK \<union> (knows Spy evs))) =
|
|
284 |
(Crypt K X \<in> analz (knows Spy evs)))"
|
|
285 |
apply (erule orb.induct)
|
|
286 |
apply (analz_mono_contra)
|
|
287 |
apply (frule_tac [7] Gets_Server_message_form)
|
|
288 |
apply (frule_tac [9] Says_Server_message_form)
|
|
289 |
apply disentangle
|
|
290 |
apply (drule_tac [5] Gets_imp_knows_Spy [THEN analz.Inj, THEN analz.Snd, THEN analz.Snd, THEN analz.Snd])
|
|
291 |
prefer 8 apply clarify
|
|
292 |
apply (analz_freshCryptK, spy_analz, fastsimp)
|
|
293 |
done
|
|
294 |
|
|
295 |
|
|
296 |
|
|
297 |
lemma analz_insert_freshCryptK:
|
|
298 |
"\<lbrakk>evs \<in> orb; Key K \<notin> analz (knows Spy evs);
|
|
299 |
Seskey \<notin> range shrK\<rbrakk> \<Longrightarrow>
|
|
300 |
(Crypt K X \<in> analz (insert (Key Seskey) (knows Spy evs))) =
|
|
301 |
(Crypt K X \<in> analz (knows Spy evs))"
|
|
302 |
by (simp only: analz_image_freshCryptK analz_image_freshK_simps)
|
|
303 |
|
|
304 |
|
|
305 |
lemma analz_hard:
|
|
306 |
"\<lbrakk>Says A B \<lbrace>Nonce M, Agent A, Agent B,
|
|
307 |
Crypt (shrK A) \<lbrace>Nonce Na, Nonce M, Agent A, Agent B\<rbrace>\<rbrace> \<in>set evs;
|
|
308 |
Crypt (shrK A) \<lbrace>Nonce Na, Key K\<rbrace> \<in> analz (knows Spy evs);
|
|
309 |
A \<notin> bad; B \<notin> bad; evs \<in> orb\<rbrakk>
|
|
310 |
\<Longrightarrow> Says B A \<lbrace>Nonce M, Crypt (shrK A) \<lbrace>Nonce Na, Key K\<rbrace>\<rbrace> \<in> set evs"
|
|
311 |
apply (erule rev_mp)
|
|
312 |
apply (erule rev_mp)
|
|
313 |
apply (erule orb.induct)
|
|
314 |
apply (frule_tac [7] Gets_Server_message_form)
|
|
315 |
apply (frule_tac [9] Says_Server_message_form)
|
|
316 |
apply disentangle
|
|
317 |
txt{*letting the simplifier solve OR2*}
|
|
318 |
apply (drule_tac [5] Gets_imp_knows_Spy [THEN analz.Inj, THEN analz.Snd, THEN analz.Snd, THEN analz.Snd])
|
|
319 |
apply (simp_all (no_asm_simp) add: analz_insert_eq pushes split_ifs)
|
|
320 |
apply (spy_analz)
|
|
321 |
txt{*OR1*}
|
|
322 |
apply blast
|
|
323 |
txt{*Oops*}
|
|
324 |
prefer 4 apply (blast dest: analz_insert_freshCryptK)
|
|
325 |
txt{*OR4 - ii*}
|
|
326 |
prefer 3 apply (blast)
|
|
327 |
txt{*OR3*}
|
|
328 |
(*adding Gets_imp_ and Says_imp_ for efficiency*)
|
|
329 |
apply (blast dest:
|
|
330 |
A_trusts_OR1 unique_Na Key_not_used analz_insert_freshCryptK)
|
|
331 |
txt{*OR4 - i *}
|
|
332 |
apply clarify
|
|
333 |
apply (simp add: pushes split_ifs)
|
|
334 |
apply (case_tac "Aaa\<in>bad")
|
|
335 |
apply (blast dest: analz_insert_freshCryptK)
|
|
336 |
apply clarify
|
|
337 |
apply simp
|
|
338 |
apply (case_tac "Ba\<in>bad")
|
|
339 |
apply (frule Gets_imp_knows_Spy [THEN analz.Inj, THEN analz.Snd, THEN analz.Decrypt, THEN analz.Fst] , assumption)
|
|
340 |
apply (simp (no_asm_simp))
|
|
341 |
apply clarify
|
|
342 |
apply (frule Gets_imp_knows_Spy
|
|
343 |
[THEN parts.Inj, THEN parts.Snd, THEN B_trusts_OR3],
|
|
344 |
assumption, assumption, assumption, erule exE)
|
|
345 |
apply (frule Says_Server_imp_Gets
|
|
346 |
[THEN Gets_imp_knows_Spy, THEN parts.Inj, THEN parts.Snd,
|
|
347 |
THEN parts.Snd, THEN parts.Snd, THEN parts.Fst, THEN A_trusts_OR1],
|
|
348 |
assumption, assumption, assumption, assumption)
|
|
349 |
apply (blast dest: Says_Server_imp_Gets B_trusts_OR2 unique_Na unique_Nb)
|
|
350 |
done
|
|
351 |
|
|
352 |
|
|
353 |
lemma Gets_Server_message_form':
|
|
354 |
"\<lbrakk>Gets B \<lbrace>Nonce M, Crypt (shrK B) \<lbrace>X, Nonce Nb, Key K\<rbrace>\<rbrace> \<in> set evs;
|
|
355 |
B \<notin> bad; evs \<in> orb\<rbrakk>
|
|
356 |
\<Longrightarrow> K \<notin> range shrK & (\<exists> A Na. X = (Crypt (shrK A) \<lbrace>Nonce Na, Key K\<rbrace>))"
|
|
357 |
by (blast dest!: B_trusts_OR3 Says_Server_message_form)
|
|
358 |
|
|
359 |
|
|
360 |
lemma OR4_imp_Gets:
|
|
361 |
"\<lbrakk>Says B A \<lbrace>Nonce M, Crypt (shrK A) \<lbrace>Nonce Na, Key K\<rbrace>\<rbrace> \<in> set evs;
|
|
362 |
B \<notin> bad; evs \<in> orb\<rbrakk>
|
|
363 |
\<Longrightarrow> (\<exists> Nb. Gets B \<lbrace>Nonce M, Crypt (shrK B) \<lbrace>Crypt (shrK A) \<lbrace>Nonce Na, Key K\<rbrace>,
|
|
364 |
Nonce Nb, Key K\<rbrace>\<rbrace> \<in> set evs)"
|
|
365 |
apply (erule rev_mp, erule orb.induct, parts_explicit, simp_all)
|
|
366 |
prefer 3 apply (blast dest: Gets_Server_message_form')
|
|
367 |
apply blast+
|
|
368 |
done
|
|
369 |
|
|
370 |
|
|
371 |
lemma A_keydist_to_B:
|
|
372 |
"\<lbrakk>Says A B \<lbrace>Nonce M, Agent A, Agent B,
|
|
373 |
Crypt (shrK A) \<lbrace>Nonce Na, Nonce M, Agent A, Agent B\<rbrace>\<rbrace> \<in>set evs;
|
|
374 |
Gets A \<lbrace>Nonce M, Crypt (shrK A) \<lbrace>Nonce Na, Key K\<rbrace>\<rbrace> \<in> set evs;
|
|
375 |
A \<notin> bad; B \<notin> bad; evs \<in> orb\<rbrakk>
|
|
376 |
\<Longrightarrow> Key K \<in> analz (knows B evs)"
|
|
377 |
apply (drule Gets_imp_knows_Spy [THEN analz.Inj, THEN analz.Snd], assumption)
|
|
378 |
apply (drule analz_hard, assumption, assumption, assumption, assumption)
|
|
379 |
apply (drule OR4_imp_Gets, assumption, assumption)
|
|
380 |
apply (erule exE)
|
|
381 |
(*blast doesn't do because it can't infer that Key (shrK P) \<in> (knows P evs)*)
|
|
382 |
apply (fastsimp dest!: Gets_imp_knows [THEN analz.Inj] analz.Decrypt)
|
|
383 |
done
|
|
384 |
|
|
385 |
|
|
386 |
text{*Other properties as for the original protocol*}
|
|
387 |
|
|
388 |
|
|
389 |
end
|