author | wenzelm |
Tue, 06 Aug 2002 11:22:05 +0200 | |
changeset 13462 | 56610e2ba220 |
parent 11655 | 923e4d0d36d5 |
child 13507 | febb8e5d2a9d |
permissions | -rw-r--r-- |
2090 | 1 |
(* Title: HOL/Auth/OtwayRees |
2 |
ID: $Id$ |
|
3 |
Author: Lawrence C Paulson, Cambridge University Computer Laboratory |
|
4 |
Copyright 1996 University of Cambridge |
|
5 |
||
6 |
Inductive relation "otway" for the Otway-Rees protocol. |
|
7 |
||
11251 | 8 |
Abadi-Needham simplified version: minimal encryption, explicit messages |
2090 | 9 |
|
2516
4d68fbe6378b
Now with Andy Gordon's treatment of freshness to replace newN/K
paulson
parents:
2451
diff
changeset
|
10 |
Note that the formalization does not even assume that nonces are fresh. |
4d68fbe6378b
Now with Andy Gordon's treatment of freshness to replace newN/K
paulson
parents:
2451
diff
changeset
|
11 |
This is because the protocol does not rely on uniqueness of nonces for |
4d68fbe6378b
Now with Andy Gordon's treatment of freshness to replace newN/K
paulson
parents:
2451
diff
changeset
|
12 |
security, only for freshness, and the proof script does not prove freshness |
4d68fbe6378b
Now with Andy Gordon's treatment of freshness to replace newN/K
paulson
parents:
2451
diff
changeset
|
13 |
properties. |
4d68fbe6378b
Now with Andy Gordon's treatment of freshness to replace newN/K
paulson
parents:
2451
diff
changeset
|
14 |
|
2090 | 15 |
From page 11 of |
16 |
Abadi and Needham. Prudent Engineering Practice for Cryptographic Protocols. |
|
17 |
IEEE Trans. SE 22 (1), 1996 |
|
18 |
*) |
|
19 |
||
11251 | 20 |
theory OtwayRees_AN = Shared: |
2090 | 21 |
|
11251 | 22 |
consts otway :: "event list set" |
3519
ab0a9fbed4c0
Changing "lost" from a parameter of protocol definitions to a constant.
paulson
parents:
3466
diff
changeset
|
23 |
inductive "otway" |
11251 | 24 |
intros |
2090 | 25 |
(*Initial trace is empty*) |
11251 | 26 |
Nil: "[] \<in> otway" |
2090 | 27 |
|
28 |
(*The spy MAY say anything he CAN say. We do not expect him to |
|
29 |
invent new nonces here, but he can also use NS1. Common to |
|
30 |
all similar protocols.*) |
|
11251 | 31 |
Fake: "[| evsf \<in> otway; X \<in> synth (analz (knows Spy evsf)) |] |
32 |
==> Says Spy B X # evsf \<in> otway" |
|
2090 | 33 |
|
6308
76f3865a2b1d
Added Bella's "Gets" model for Otway_Rees. Also affects some other theories.
paulson
parents:
5434
diff
changeset
|
34 |
(*A message that has been sent can be received by the |
76f3865a2b1d
Added Bella's "Gets" model for Otway_Rees. Also affects some other theories.
paulson
parents:
5434
diff
changeset
|
35 |
intended recipient.*) |
11251 | 36 |
Reception: "[| evsr \<in> otway; Says A B X \<in>set evsr |] |
37 |
==> Gets B X # evsr \<in> otway" |
|
6308
76f3865a2b1d
Added Bella's "Gets" model for Otway_Rees. Also affects some other theories.
paulson
parents:
5434
diff
changeset
|
38 |
|
2090 | 39 |
(*Alice initiates a protocol run*) |
11251 | 40 |
OR1: "evs1 \<in> otway |
41 |
==> Says A B {|Agent A, Agent B, Nonce NA|} # evs1 \<in> otway" |
|
2090 | 42 |
|
6333 | 43 |
(*Bob's response to Alice's message.*) |
11251 | 44 |
OR2: "[| evs2 \<in> otway; |
45 |
Gets B {|Agent A, Agent B, Nonce NA|} \<in>set evs2 |] |
|
2516
4d68fbe6378b
Now with Andy Gordon's treatment of freshness to replace newN/K
paulson
parents:
2451
diff
changeset
|
46 |
==> Says B Server {|Agent A, Agent B, Nonce NA, Nonce NB|} |
11251 | 47 |
# evs2 \<in> otway" |
2090 | 48 |
|
49 |
(*The Server receives Bob's message. Then he sends a new |
|
50 |
session key to Bob with a packet for forwarding to Alice.*) |
|
11251 | 51 |
OR3: "[| evs3 \<in> otway; Key KAB \<notin> used evs3; |
6308
76f3865a2b1d
Added Bella's "Gets" model for Otway_Rees. Also affects some other theories.
paulson
parents:
5434
diff
changeset
|
52 |
Gets Server {|Agent A, Agent B, Nonce NA, Nonce NB|} |
11251 | 53 |
\<in>set evs3 |] |
54 |
==> Says Server B |
|
2516
4d68fbe6378b
Now with Andy Gordon's treatment of freshness to replace newN/K
paulson
parents:
2451
diff
changeset
|
55 |
{|Crypt (shrK A) {|Nonce NA, Agent A, Agent B, Key KAB|}, |
4d68fbe6378b
Now with Andy Gordon's treatment of freshness to replace newN/K
paulson
parents:
2451
diff
changeset
|
56 |
Crypt (shrK B) {|Nonce NB, Agent A, Agent B, Key KAB|}|} |
11251 | 57 |
# evs3 \<in> otway" |
2090 | 58 |
|
59 |
(*Bob receives the Server's (?) message and compares the Nonces with |
|
5434
9b4bed3f394c
Got rid of not_Says_to_self and most uses of ~= in definitions and theorems
paulson
parents:
5359
diff
changeset
|
60 |
those in the message he previously sent the Server. |
11251 | 61 |
Need B \<noteq> Server because we allow messages to self.*) |
62 |
OR4: "[| evs4 \<in> otway; B \<noteq> Server; |
|
63 |
Says B Server {|Agent A, Agent B, Nonce NA, Nonce NB|} \<in>set evs4; |
|
6308
76f3865a2b1d
Added Bella's "Gets" model for Otway_Rees. Also affects some other theories.
paulson
parents:
5434
diff
changeset
|
64 |
Gets B {|X, Crypt(shrK B){|Nonce NB,Agent A,Agent B,Key K|}|} |
11251 | 65 |
\<in>set evs4 |] |
66 |
==> Says B A X # evs4 \<in> otway" |
|
2090 | 67 |
|
2131 | 68 |
(*This message models possible leaks of session keys. The nonces |
69 |
identify the protocol run. B is not assumed to know shrK A.*) |
|
11251 | 70 |
Oops: "[| evso \<in> otway; |
71 |
Says Server B |
|
72 |
{|Crypt (shrK A) {|Nonce NA, Agent A, Agent B, Key K|}, |
|
2284
80ebd1a213fd
Swapped arguments of Crypt (for clarity and because it is conventional)
paulson
parents:
2131
diff
changeset
|
73 |
Crypt (shrK B) {|Nonce NB, Agent A, Agent B, Key K|}|} |
11251 | 74 |
\<in>set evso |] |
75 |
==> Notes Spy {|Nonce NA, Nonce NB, Key K|} # evso \<in> otway" |
|
76 |
||
77 |
||
78 |
declare Says_imp_knows_Spy [THEN analz.Inj, dest] |
|
79 |
declare parts.Body [dest] |
|
80 |
declare analz_into_parts [dest] |
|
81 |
declare Fake_parts_insert_in_Un [dest] |
|
82 |
||
83 |
||
84 |
(*A "possibility property": there are traces that reach the end*) |
|
85 |
lemma "B \<noteq> Server |
|
86 |
==> \<exists>K. \<exists>evs \<in> otway. |
|
87 |
Says B A (Crypt (shrK A) {|Nonce NA, Agent A, Agent B, Key K|}) |
|
88 |
\<in> set evs" |
|
89 |
apply (intro exI bexI) |
|
90 |
apply (rule_tac [2] otway.Nil |
|
91 |
[THEN otway.OR1, THEN otway.Reception, |
|
92 |
THEN otway.OR2, THEN otway.Reception, |
|
93 |
THEN otway.OR3, THEN otway.Reception, THEN otway.OR4]) |
|
94 |
apply possibility |
|
95 |
done |
|
96 |
||
97 |
lemma Gets_imp_Says [dest!]: |
|
98 |
"[| Gets B X \<in> set evs; evs \<in> otway |] ==> \<exists>A. Says A B X \<in> set evs" |
|
99 |
by (erule rev_mp, erule otway.induct, auto) |
|
100 |
||
101 |
||
102 |
(**** Inductive proofs about otway ****) |
|
103 |
||
104 |
(** For reasoning about the encrypted portion of messages **) |
|
105 |
||
106 |
lemma OR4_analz_knows_Spy: |
|
107 |
"[| Gets B {|X, Crypt(shrK B) X'|} \<in> set evs; evs \<in> otway |] |
|
108 |
==> X \<in> analz (knows Spy evs)" |
|
109 |
by blast |
|
110 |
||
111 |
||
112 |
(** Theorems of the form X \<notin> parts (knows Spy evs) imply that NOBODY |
|
113 |
sends messages containing X! **) |
|
114 |
||
115 |
(*Spy never sees a good agent's shared key!*) |
|
116 |
lemma Spy_see_shrK [simp]: |
|
117 |
"evs \<in> otway ==> (Key (shrK A) \<in> parts (knows Spy evs)) = (A \<in> bad)" |
|
118 |
apply (erule otway.induct, simp_all) |
|
119 |
apply blast+ |
|
120 |
done |
|
121 |
||
122 |
lemma Spy_analz_shrK [simp]: |
|
123 |
"evs \<in> otway ==> (Key (shrK A) \<in> analz (knows Spy evs)) = (A \<in> bad)" |
|
124 |
by auto |
|
125 |
||
126 |
lemma Spy_see_shrK_D [dest!]: |
|
127 |
"[|Key (shrK A) \<in> parts (knows Spy evs); evs \<in> otway|] ==> A \<in> bad" |
|
128 |
by (blast dest: Spy_see_shrK) |
|
129 |
||
130 |
||
131 |
(*** Proofs involving analz ***) |
|
132 |
||
133 |
(*Describes the form of K and NA when the Server sends this message.*) |
|
134 |
lemma Says_Server_message_form: |
|
135 |
"[| Says Server B |
|
136 |
{|Crypt (shrK A) {|NA, Agent A, Agent B, Key K|}, |
|
137 |
Crypt (shrK B) {|NB, Agent A, Agent B, Key K|}|} |
|
138 |
\<in> set evs; |
|
139 |
evs \<in> otway |] |
|
140 |
==> K \<notin> range shrK & (\<exists>i. NA = Nonce i) & (\<exists>j. NB = Nonce j)" |
|
141 |
apply (erule rev_mp) |
|
142 |
apply (erule otway.induct) |
|
143 |
apply simp_all |
|
144 |
apply blast |
|
145 |
done |
|
146 |
||
147 |
||
148 |
||
149 |
(**** |
|
150 |
The following is to prove theorems of the form |
|
151 |
||
152 |
Key K \<in> analz (insert (Key KAB) (knows Spy evs)) ==> |
|
153 |
Key K \<in> analz (knows Spy evs) |
|
154 |
||
155 |
A more general formula must be proved inductively. |
|
156 |
****) |
|
157 |
||
158 |
||
159 |
(** Session keys are not used to encrypt other session keys **) |
|
160 |
||
161 |
(*The equality makes the induction hypothesis easier to apply*) |
|
162 |
lemma analz_image_freshK [rule_format]: |
|
163 |
"evs \<in> otway ==> |
|
164 |
\<forall>K KK. KK <= -(range shrK) --> |
|
165 |
(Key K \<in> analz (Key`KK Un (knows Spy evs))) = |
|
166 |
(K \<in> KK | Key K \<in> analz (knows Spy evs))" |
|
167 |
apply (erule otway.induct, force) |
|
168 |
apply (frule_tac [7] Says_Server_message_form) |
|
169 |
apply (drule_tac [6] OR4_analz_knows_Spy) |
|
170 |
apply analz_freshK |
|
171 |
apply spy_analz |
|
172 |
done |
|
173 |
||
174 |
lemma analz_insert_freshK: |
|
175 |
"[| evs \<in> otway; KAB \<notin> range shrK |] ==> |
|
11655 | 176 |
(Key K \<in> analz (insert (Key KAB) (knows Spy evs))) = |
11251 | 177 |
(K = KAB | Key K \<in> analz (knows Spy evs))" |
178 |
by (simp only: analz_image_freshK analz_image_freshK_simps) |
|
179 |
||
180 |
||
181 |
(*** The Key K uniquely identifies the Server's message. **) |
|
182 |
||
183 |
lemma unique_session_keys: |
|
184 |
"[| Says Server B |
|
185 |
{|Crypt (shrK A) {|NA, Agent A, Agent B, K|}, |
|
186 |
Crypt (shrK B) {|NB, Agent A, Agent B, K|}|} |
|
187 |
\<in> set evs; |
|
188 |
Says Server B' |
|
189 |
{|Crypt (shrK A') {|NA', Agent A', Agent B', K|}, |
|
190 |
Crypt (shrK B') {|NB', Agent A', Agent B', K|}|} |
|
191 |
\<in> set evs; |
|
192 |
evs \<in> otway |] |
|
193 |
==> A=A' & B=B' & NA=NA' & NB=NB'" |
|
194 |
apply (erule rev_mp, erule rev_mp, erule otway.induct) |
|
195 |
apply simp_all |
|
196 |
(*Remaining cases: OR3 and OR4*) |
|
197 |
apply blast+ |
|
198 |
done |
|
199 |
||
200 |
||
201 |
(**** Authenticity properties relating to NA ****) |
|
202 |
||
203 |
(*If the encrypted message appears then it originated with the Server!*) |
|
204 |
lemma NA_Crypt_imp_Server_msg [rule_format]: |
|
205 |
"[| A \<notin> bad; A \<noteq> B; evs \<in> otway |] |
|
206 |
==> Crypt (shrK A) {|NA, Agent A, Agent B, Key K|} \<in> parts (knows Spy evs) |
|
207 |
--> (\<exists>NB. Says Server B |
|
208 |
{|Crypt (shrK A) {|NA, Agent A, Agent B, Key K|}, |
|
209 |
Crypt (shrK B) {|NB, Agent A, Agent B, Key K|}|} |
|
210 |
\<in> set evs)" |
|
211 |
apply (erule otway.induct, force) |
|
212 |
apply (simp_all add: ex_disj_distrib) |
|
213 |
(*Fake, OR3*) |
|
214 |
apply blast+; |
|
215 |
done |
|
216 |
||
217 |
||
218 |
(*Corollary: if A receives B's OR4 message then it originated with the Server. |
|
219 |
Freshness may be inferred from nonce NA.*) |
|
220 |
lemma A_trusts_OR4: |
|
221 |
"[| Says B' A (Crypt (shrK A) {|NA, Agent A, Agent B, Key K|}) \<in> set evs; |
|
222 |
A \<notin> bad; A \<noteq> B; evs \<in> otway |] |
|
223 |
==> \<exists>NB. Says Server B |
|
224 |
{|Crypt (shrK A) {|NA, Agent A, Agent B, Key K|}, |
|
225 |
Crypt (shrK B) {|NB, Agent A, Agent B, Key K|}|} |
|
226 |
\<in> set evs" |
|
227 |
by (blast intro!: NA_Crypt_imp_Server_msg) |
|
228 |
||
229 |
||
230 |
(** Crucial secrecy property: Spy does not see the keys sent in msg OR3 |
|
231 |
Does not in itself guarantee security: an attack could violate |
|
232 |
the premises, e.g. by having A=Spy **) |
|
233 |
||
234 |
lemma secrecy_lemma: |
|
235 |
"[| A \<notin> bad; B \<notin> bad; evs \<in> otway |] |
|
236 |
==> Says Server B |
|
237 |
{|Crypt (shrK A) {|NA, Agent A, Agent B, Key K|}, |
|
238 |
Crypt (shrK B) {|NB, Agent A, Agent B, Key K|}|} |
|
239 |
\<in> set evs --> |
|
240 |
Notes Spy {|NA, NB, Key K|} \<notin> set evs --> |
|
241 |
Key K \<notin> analz (knows Spy evs)" |
|
242 |
apply (erule otway.induct, force) |
|
243 |
apply (frule_tac [7] Says_Server_message_form) |
|
244 |
apply (drule_tac [6] OR4_analz_knows_Spy) |
|
245 |
apply (simp_all add: analz_insert_eq analz_insert_freshK pushes) |
|
246 |
apply spy_analz (*Fake*) |
|
247 |
(*OR3, OR4, Oops*) |
|
248 |
apply (blast dest: unique_session_keys)+ |
|
249 |
done |
|
250 |
||
251 |
||
252 |
lemma Spy_not_see_encrypted_key: |
|
253 |
"[| Says Server B |
|
254 |
{|Crypt (shrK A) {|NA, Agent A, Agent B, Key K|}, |
|
255 |
Crypt (shrK B) {|NB, Agent A, Agent B, Key K|}|} |
|
256 |
\<in> set evs; |
|
257 |
Notes Spy {|NA, NB, Key K|} \<notin> set evs; |
|
258 |
A \<notin> bad; B \<notin> bad; evs \<in> otway |] |
|
259 |
==> Key K \<notin> analz (knows Spy evs)" |
|
260 |
by (blast dest: Says_Server_message_form secrecy_lemma) |
|
261 |
||
262 |
||
263 |
(*A's guarantee. The Oops premise quantifies over NB because A cannot know |
|
264 |
what it is.*) |
|
265 |
lemma A_gets_good_key: |
|
266 |
"[| Says B' A (Crypt (shrK A) {|NA, Agent A, Agent B, Key K|}) \<in> set evs; |
|
267 |
\<forall>NB. Notes Spy {|NA, NB, Key K|} \<notin> set evs; |
|
268 |
A \<notin> bad; B \<notin> bad; A \<noteq> B; evs \<in> otway |] |
|
269 |
==> Key K \<notin> analz (knows Spy evs)" |
|
270 |
by (blast dest!: A_trusts_OR4 Spy_not_see_encrypted_key) |
|
271 |
||
272 |
||
273 |
||
274 |
(**** Authenticity properties relating to NB ****) |
|
275 |
||
276 |
(*If the encrypted message appears then it originated with the Server!*) |
|
277 |
||
278 |
lemma NB_Crypt_imp_Server_msg [rule_format]: |
|
279 |
"[| B \<notin> bad; A \<noteq> B; evs \<in> otway |] |
|
280 |
==> Crypt (shrK B) {|NB, Agent A, Agent B, Key K|} \<in> parts (knows Spy evs) |
|
281 |
--> (\<exists>NA. Says Server B |
|
282 |
{|Crypt (shrK A) {|NA, Agent A, Agent B, Key K|}, |
|
283 |
Crypt (shrK B) {|NB, Agent A, Agent B, Key K|}|} |
|
284 |
\<in> set evs)" |
|
285 |
apply (erule otway.induct, force, simp_all add: ex_disj_distrib) |
|
286 |
(*Fake, OR3*) |
|
287 |
apply blast+; |
|
288 |
done |
|
289 |
||
290 |
||
291 |
||
292 |
(*Guarantee for B: if it gets a well-formed certificate then the Server |
|
293 |
has sent the correct message in round 3.*) |
|
294 |
lemma B_trusts_OR3: |
|
295 |
"[| Says S B {|X, Crypt (shrK B) {|NB, Agent A, Agent B, Key K|}|} |
|
296 |
\<in> set evs; |
|
297 |
B \<notin> bad; A \<noteq> B; evs \<in> otway |] |
|
298 |
==> \<exists>NA. Says Server B |
|
299 |
{|Crypt (shrK A) {|NA, Agent A, Agent B, Key K|}, |
|
300 |
Crypt (shrK B) {|NB, Agent A, Agent B, Key K|}|} |
|
301 |
\<in> set evs" |
|
302 |
by (blast intro!: NB_Crypt_imp_Server_msg) |
|
303 |
||
304 |
||
305 |
(*The obvious combination of B_trusts_OR3 with Spy_not_see_encrypted_key*) |
|
306 |
lemma B_gets_good_key: |
|
307 |
"[| Gets B {|X, Crypt (shrK B) {|NB, Agent A, Agent B, Key K|}|} |
|
308 |
\<in> set evs; |
|
309 |
\<forall>NA. Notes Spy {|NA, NB, Key K|} \<notin> set evs; |
|
310 |
A \<notin> bad; B \<notin> bad; A \<noteq> B; evs \<in> otway |] |
|
311 |
==> Key K \<notin> analz (knows Spy evs)" |
|
312 |
by (blast dest: B_trusts_OR3 Spy_not_see_encrypted_key) |
|
2090 | 313 |
|
314 |
end |