author | paulson |
Fri, 03 Mar 2000 18:26:19 +0100 | |
changeset 8334 | 7896bcbd8641 |
parent 8128 | 3a5864b465e2 |
child 9190 | b86ff604729f |
permissions | -rw-r--r-- |
8044 | 1 |
(* Title: HOL/UNITY/ELT |
2 |
ID: $Id$ |
|
3 |
Author: Lawrence C Paulson, Cambridge University Computer Laboratory |
|
4 |
Copyright 1999 University of Cambridge |
|
5 |
||
6 |
leadsTo strengthened with a specification of the allowable sets transient parts |
|
7 |
*) |
|
8 |
||
8128 | 9 |
(*** givenBy ***) |
10 |
||
11 |
Goalw [givenBy_def] "givenBy id = UNIV"; |
|
12 |
by Auto_tac; |
|
13 |
qed "givenBy_id"; |
|
14 |
Addsimps [givenBy_id]; |
|
15 |
||
16 |
Goalw [givenBy_def] "(givenBy v) = {A. ALL x:A. ALL y. v x = v y --> y: A}"; |
|
17 |
by Safe_tac; |
|
18 |
by (res_inst_tac [("x", "v `` ?u")] image_eqI 2); |
|
19 |
by Auto_tac; |
|
20 |
qed "givenBy_eq_all"; |
|
21 |
||
22 |
Goal "givenBy v = {A. EX P. A = {s. P(v s)}}"; |
|
23 |
by (simp_tac (simpset() addsimps [givenBy_eq_all]) 1); |
|
24 |
by Safe_tac; |
|
25 |
by (res_inst_tac [("x", "%n. EX s. v s = n & s : ?A")] exI 1); |
|
26 |
by (Blast_tac 1); |
|
27 |
by Auto_tac; |
|
28 |
qed "givenBy_eq_Collect"; |
|
29 |
||
30 |
val prems = |
|
31 |
Goal "(!!x y. [| x:A; v x = v y |] ==> y: A) ==> A: givenBy v"; |
|
32 |
by (stac givenBy_eq_all 1); |
|
33 |
by (blast_tac (claset() addIs prems) 1); |
|
34 |
qed "givenByI"; |
|
35 |
||
36 |
Goalw [givenBy_def] "[| A: givenBy v; x:A; v x = v y |] ==> y: A"; |
|
37 |
by Auto_tac; |
|
38 |
qed "givenByD"; |
|
39 |
||
40 |
Goal "{} : givenBy v"; |
|
41 |
by (blast_tac (claset() addSIs [givenByI]) 1); |
|
42 |
qed "empty_mem_givenBy"; |
|
43 |
||
44 |
AddIffs [empty_mem_givenBy]; |
|
45 |
||
46 |
Goal "A: givenBy v ==> EX P. A = {s. P(v s)}"; |
|
47 |
by (res_inst_tac [("x", "%n. EX s. v s = n & s : A")] exI 1); |
|
48 |
by (full_simp_tac (simpset() addsimps [givenBy_eq_all]) 1); |
|
49 |
by (Blast_tac 1); |
|
50 |
qed "givenBy_imp_eq_Collect"; |
|
51 |
||
52 |
Goalw [givenBy_def] "{s. P(v s)} : givenBy v"; |
|
53 |
by (Best_tac 1); |
|
54 |
qed "Collect_mem_givenBy"; |
|
55 |
||
56 |
Goal "givenBy v = {A. EX P. A = {s. P(v s)}}"; |
|
57 |
by (blast_tac (claset() addIs [Collect_mem_givenBy, |
|
58 |
givenBy_imp_eq_Collect]) 1); |
|
59 |
qed "givenBy_eq_eq_Collect"; |
|
60 |
||
61 |
(*preserving v preserves properties given by v*) |
|
62 |
Goal "[| F : preserves v; D : givenBy v |] ==> F : stable D"; |
|
63 |
by (force_tac (claset(), |
|
64 |
simpset() addsimps [impOfSubs preserves_subset_stable, |
|
65 |
givenBy_eq_Collect]) 1); |
|
66 |
qed "preserves_givenBy_imp_stable"; |
|
67 |
||
68 |
Goal "givenBy (w o v) <= givenBy v"; |
|
69 |
by (simp_tac (simpset() addsimps [givenBy_eq_Collect]) 1); |
|
70 |
by (Deepen_tac 0 1); |
|
71 |
qed "givenBy_o_subset"; |
|
72 |
||
73 |
Goal "[| A : givenBy v; B : givenBy v |] ==> A-B : givenBy v"; |
|
74 |
by (full_simp_tac (simpset() addsimps [givenBy_eq_Collect]) 1); |
|
75 |
by Safe_tac; |
|
76 |
by (res_inst_tac [("x", "%z. ?R z & ~ ?Q z")] exI 1); |
|
77 |
by (deepen_tac (set_cs addSIs [equalityI]) 0 1); |
|
78 |
qed "givenBy_DiffI"; |
|
79 |
||
80 |
||
8044 | 81 |
(** Standard leadsTo rules **) |
82 |
||
8072
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
83 |
Goalw [leadsETo_def] |
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
84 |
"[| F: A ensures B; A-B: insert {} CC |] ==> F : A leadsTo[CC] B"; |
8044 | 85 |
by (blast_tac (claset() addIs [elt.Basis]) 1); |
86 |
qed "leadsETo_Basis"; |
|
87 |
||
88 |
Goalw [leadsETo_def] |
|
89 |
"[| F : A leadsTo[CC] B; F : B leadsTo[CC] C |] ==> F : A leadsTo[CC] C"; |
|
90 |
by (blast_tac (claset() addIs [elt.Trans]) 1); |
|
91 |
qed "leadsETo_Trans"; |
|
92 |
||
8122
b43ad07660b9
working version, with Alloc now working on the same state space as the whole
paulson
parents:
8110
diff
changeset
|
93 |
|
8044 | 94 |
(*Useful with cancellation, disjunction*) |
95 |
Goal "F : A leadsTo[CC] (A' Un A') ==> F : A leadsTo[CC] A'"; |
|
96 |
by (asm_full_simp_tac (simpset() addsimps Un_ac) 1); |
|
97 |
qed "leadsETo_Un_duplicate"; |
|
98 |
||
99 |
Goal "F : A leadsTo[CC] (A' Un C Un C) ==> F : A leadsTo[CC] (A' Un C)"; |
|
100 |
by (asm_full_simp_tac (simpset() addsimps Un_ac) 1); |
|
101 |
qed "leadsETo_Un_duplicate2"; |
|
102 |
||
103 |
(*The Union introduction rule as we should have liked to state it*) |
|
104 |
val prems = Goalw [leadsETo_def] |
|
105 |
"(!!A. A : S ==> F : A leadsTo[CC] B) ==> F : (Union S) leadsTo[CC] B"; |
|
106 |
by (blast_tac (claset() addIs [elt.Union] addDs prems) 1); |
|
107 |
qed "leadsETo_Union"; |
|
108 |
||
109 |
val prems = Goal |
|
110 |
"(!!i. i : I ==> F : (A i) leadsTo[CC] B) \ |
|
111 |
\ ==> F : (UN i:I. A i) leadsTo[CC] B"; |
|
112 |
by (stac (Union_image_eq RS sym) 1); |
|
113 |
by (blast_tac (claset() addIs leadsETo_Union::prems) 1); |
|
114 |
qed "leadsETo_UN"; |
|
115 |
||
116 |
(*The INDUCTION rule as we should have liked to state it*) |
|
117 |
val major::prems = Goalw [leadsETo_def] |
|
118 |
"[| F : za leadsTo[CC] zb; \ |
|
8072
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
119 |
\ !!A B. [| F : A ensures B; A-B : insert {} CC |] ==> P A B; \ |
8044 | 120 |
\ !!A B C. [| F : A leadsTo[CC] B; P A B; F : B leadsTo[CC] C; P B C |] \ |
121 |
\ ==> P A C; \ |
|
122 |
\ !!B S. ALL A:S. F : A leadsTo[CC] B & P A B ==> P (Union S) B \ |
|
123 |
\ |] ==> P za zb"; |
|
124 |
by (rtac (major RS CollectD RS elt.induct) 1); |
|
125 |
by (REPEAT (blast_tac (claset() addIs prems) 1)); |
|
126 |
qed "leadsETo_induct"; |
|
127 |
||
128 |
||
129 |
(** New facts involving leadsETo **) |
|
130 |
||
131 |
Goal "CC' <= CC ==> (A leadsTo[CC'] B) <= (A leadsTo[CC] B)"; |
|
132 |
by Safe_tac; |
|
133 |
by (etac leadsETo_induct 1); |
|
134 |
by (blast_tac (claset() addIs [leadsETo_Union]) 3); |
|
135 |
by (blast_tac (claset() addIs [leadsETo_Trans]) 2); |
|
136 |
by (blast_tac (claset() addIs [leadsETo_Basis]) 1); |
|
137 |
qed "leadsETo_mono"; |
|
138 |
||
8122
b43ad07660b9
working version, with Alloc now working on the same state space as the whole
paulson
parents:
8110
diff
changeset
|
139 |
Goal "[| F : A leadsTo[CC] B; F : B leadsTo[DD] C |] \ |
b43ad07660b9
working version, with Alloc now working on the same state space as the whole
paulson
parents:
8110
diff
changeset
|
140 |
\ ==> F : A leadsTo[CC Un DD] C"; |
b43ad07660b9
working version, with Alloc now working on the same state space as the whole
paulson
parents:
8110
diff
changeset
|
141 |
by (blast_tac (claset() addIs [impOfSubs leadsETo_mono, leadsETo_Trans]) 1); |
b43ad07660b9
working version, with Alloc now working on the same state space as the whole
paulson
parents:
8110
diff
changeset
|
142 |
qed "leadsETo_Trans_Un"; |
b43ad07660b9
working version, with Alloc now working on the same state space as the whole
paulson
parents:
8110
diff
changeset
|
143 |
|
8044 | 144 |
val prems = Goalw [leadsETo_def] |
145 |
"(!!A. A : S ==> F : (A Int C) leadsTo[CC] B) ==> F : (Union S Int C) leadsTo[CC] B"; |
|
146 |
by (simp_tac (HOL_ss addsimps [Int_Union_Union]) 1); |
|
147 |
by (blast_tac (claset() addIs [elt.Union] addDs prems) 1); |
|
148 |
qed "leadsETo_Union_Int"; |
|
149 |
||
150 |
(*Binary union introduction rule*) |
|
151 |
Goal "[| F : A leadsTo[CC] C; F : B leadsTo[CC] C |] ==> F : (A Un B) leadsTo[CC] C"; |
|
152 |
by (stac Un_eq_Union 1); |
|
153 |
by (blast_tac (claset() addIs [leadsETo_Union]) 1); |
|
154 |
qed "leadsETo_Un"; |
|
155 |
||
156 |
val prems = |
|
157 |
Goal "(!!x. x : A ==> F : {x} leadsTo[CC] B) ==> F : A leadsTo[CC] B"; |
|
158 |
by (stac (UN_singleton RS sym) 1 THEN rtac leadsETo_UN 1); |
|
159 |
by (blast_tac (claset() addIs prems) 1); |
|
160 |
qed "single_leadsETo_I"; |
|
161 |
||
162 |
||
8072
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
163 |
Goal "A<=B ==> F : A leadsTo[CC] B"; |
8044 | 164 |
by (asm_simp_tac (simpset() addsimps [subset_imp_ensures RS leadsETo_Basis, |
165 |
Diff_eq_empty_iff RS iffD2]) 1); |
|
166 |
qed "subset_imp_leadsETo"; |
|
167 |
||
168 |
bind_thm ("empty_leadsETo", empty_subsetI RS subset_imp_leadsETo); |
|
169 |
Addsimps [empty_leadsETo]; |
|
170 |
||
171 |
||
8122
b43ad07660b9
working version, with Alloc now working on the same state space as the whole
paulson
parents:
8110
diff
changeset
|
172 |
|
8072
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
173 |
(** Weakening laws **) |
8044 | 174 |
|
8072
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
175 |
Goal "[| F : A leadsTo[CC] A'; A'<=B' |] ==> F : A leadsTo[CC] B'"; |
8044 | 176 |
by (blast_tac (claset() addIs [subset_imp_leadsETo, leadsETo_Trans]) 1); |
177 |
qed "leadsETo_weaken_R"; |
|
178 |
||
8072
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
179 |
Goal "[| F : A leadsTo[CC] A'; B<=A |] ==> F : B leadsTo[CC] A'"; |
8044 | 180 |
by (blast_tac (claset() addIs [leadsETo_Trans, subset_imp_leadsETo]) 1); |
181 |
qed_spec_mp "leadsETo_weaken_L"; |
|
182 |
||
183 |
(*Distributes over binary unions*) |
|
8072
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
184 |
Goal "F : (A Un B) leadsTo[CC] C = \ |
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
185 |
\ (F : A leadsTo[CC] C & F : B leadsTo[CC] C)"; |
8044 | 186 |
by (blast_tac (claset() addIs [leadsETo_Un, leadsETo_weaken_L]) 1); |
187 |
qed "leadsETo_Un_distrib"; |
|
188 |
||
8072
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
189 |
Goal "F : (UN i:I. A i) leadsTo[CC] B = \ |
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
190 |
\ (ALL i : I. F : (A i) leadsTo[CC] B)"; |
8044 | 191 |
by (blast_tac (claset() addIs [leadsETo_UN, leadsETo_weaken_L]) 1); |
192 |
qed "leadsETo_UN_distrib"; |
|
193 |
||
8072
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
194 |
Goal "F : (Union S) leadsTo[CC] B = (ALL A : S. F : A leadsTo[CC] B)"; |
8044 | 195 |
by (blast_tac (claset() addIs [leadsETo_Union, leadsETo_weaken_L]) 1); |
196 |
qed "leadsETo_Union_distrib"; |
|
197 |
||
8072
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
198 |
Goal "[| F : A leadsTo[CC'] A'; B<=A; A'<=B'; CC' <= CC |] \ |
8044 | 199 |
\ ==> F : B leadsTo[CC] B'"; |
200 |
by (dtac (impOfSubs leadsETo_mono) 1); |
|
201 |
by (assume_tac 1); |
|
8110 | 202 |
by (blast_tac (claset() delrules [subsetCE] |
203 |
addIs [leadsETo_weaken_R, leadsETo_weaken_L, |
|
8044 | 204 |
leadsETo_Trans]) 1); |
205 |
qed "leadsETo_weaken"; |
|
206 |
||
207 |
Goal "[| F : A leadsTo[CC] A'; CC <= givenBy v |] \ |
|
208 |
\ ==> F : A leadsTo[givenBy v] A'"; |
|
209 |
by (blast_tac (claset() addIs [empty_mem_givenBy, leadsETo_weaken]) 1); |
|
210 |
qed "leadsETo_givenBy"; |
|
211 |
||
212 |
||
213 |
(*Set difference*) |
|
8072
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
214 |
Goal "[| F : (A-B) leadsTo[CC] C; F : B leadsTo[CC] C |] \ |
8044 | 215 |
\ ==> F : A leadsTo[CC] C"; |
216 |
by (blast_tac (claset() addIs [leadsETo_Un, leadsETo_weaken]) 1); |
|
217 |
qed "leadsETo_Diff"; |
|
218 |
||
219 |
||
220 |
(*Binary union version*) |
|
8072
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
221 |
Goal "[| F : A leadsTo[CC] A'; F : B leadsTo[CC] B' |] \ |
8044 | 222 |
\ ==> F : (A Un B) leadsTo[CC] (A' Un B')"; |
223 |
by (blast_tac (claset() addIs [leadsETo_Un, |
|
224 |
leadsETo_weaken_R]) 1); |
|
225 |
qed "leadsETo_Un_Un"; |
|
226 |
||
227 |
||
228 |
(** The cancellation law **) |
|
229 |
||
8072
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
230 |
Goal "[| F : A leadsTo[CC] (A' Un B); F : B leadsTo[CC] B' |] \ |
8044 | 231 |
\ ==> F : A leadsTo[CC] (A' Un B')"; |
232 |
by (blast_tac (claset() addIs [leadsETo_Un_Un, |
|
233 |
subset_imp_leadsETo, leadsETo_Trans]) 1); |
|
234 |
qed "leadsETo_cancel2"; |
|
235 |
||
8072
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
236 |
Goal "[| F : A leadsTo[CC] (B Un A'); F : B leadsTo[CC] B' |] \ |
8044 | 237 |
\ ==> F : A leadsTo[CC] (B' Un A')"; |
238 |
by (asm_full_simp_tac (simpset() addsimps [Un_commute]) 1); |
|
239 |
by (blast_tac (claset() addSIs [leadsETo_cancel2]) 1); |
|
240 |
qed "leadsETo_cancel1"; |
|
241 |
||
8072
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
242 |
Goal "[| F : A leadsTo[CC] (B Un A'); F : (B-A') leadsTo[CC] B' |] \ |
8044 | 243 |
\ ==> F : A leadsTo[CC] (B' Un A')"; |
244 |
by (rtac leadsETo_cancel1 1); |
|
245 |
by (assume_tac 2); |
|
246 |
by (ALLGOALS Asm_simp_tac); |
|
247 |
qed "leadsETo_cancel_Diff1"; |
|
248 |
||
249 |
||
250 |
(** The impossibility law **) |
|
251 |
||
252 |
Goal "F : A leadsTo[CC] B ==> B={} --> A={}"; |
|
253 |
by (etac leadsETo_induct 1); |
|
254 |
by (ALLGOALS Asm_simp_tac); |
|
255 |
by (rewrite_goals_tac [ensures_def, constrains_def, transient_def]); |
|
256 |
by (Blast_tac 1); |
|
257 |
val lemma = result() RS mp; |
|
258 |
||
259 |
Goal "F : A leadsTo[CC] {} ==> A={}"; |
|
260 |
by (blast_tac (claset() addSIs [lemma]) 1); |
|
261 |
qed "leadsETo_empty"; |
|
262 |
||
263 |
||
264 |
(** PSP: Progress-Safety-Progress **) |
|
265 |
||
266 |
(*Special case of PSP: Misra's "stable conjunction"*) |
|
267 |
Goalw [stable_def] |
|
268 |
"[| F : A leadsTo[CC] A'; F : stable B; ALL C:CC. C Int B : CC |] \ |
|
269 |
\ ==> F : (A Int B) leadsTo[CC] (A' Int B)"; |
|
270 |
by (etac leadsETo_induct 1); |
|
271 |
by (blast_tac (claset() addIs [leadsETo_Union_Int]) 3); |
|
272 |
by (blast_tac (claset() addIs [leadsETo_Trans]) 2); |
|
273 |
by (rtac leadsETo_Basis 1); |
|
8072
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
274 |
by (force_tac (claset(), |
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
275 |
simpset() addsimps [Diff_Int_distrib2 RS sym]) 2); |
8044 | 276 |
by (asm_full_simp_tac |
277 |
(simpset() addsimps [ensures_def, |
|
278 |
Diff_Int_distrib2 RS sym, Int_Un_distrib2 RS sym]) 1); |
|
279 |
by (blast_tac (claset() addIs [transient_strengthen, constrains_Int]) 1); |
|
280 |
qed "e_psp_stable"; |
|
281 |
||
282 |
Goal "[| F : A leadsTo[CC] A'; F : stable B; ALL C:CC. C Int B : CC |] \ |
|
283 |
\ ==> F : (B Int A) leadsTo[CC] (B Int A')"; |
|
284 |
by (asm_simp_tac (simpset() addsimps e_psp_stable::Int_ac) 1); |
|
285 |
qed "e_psp_stable2"; |
|
286 |
||
287 |
Goal "[| F : A leadsTo[CC] A'; F : B co B'; \ |
|
8072
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
288 |
\ ALL C:CC. C Int B Int B' : CC |] \ |
8044 | 289 |
\ ==> F : (A Int B') leadsTo[CC] ((A' Int B) Un (B' - B))"; |
290 |
by (etac leadsETo_induct 1); |
|
291 |
by (blast_tac (claset() addIs [leadsETo_Union_Int]) 3); |
|
292 |
(*Transitivity case has a delicate argument involving "cancellation"*) |
|
293 |
by (rtac leadsETo_Un_duplicate2 2); |
|
294 |
by (etac leadsETo_cancel_Diff1 2); |
|
295 |
by (asm_full_simp_tac (simpset() addsimps [Int_Diff, Diff_triv]) 2); |
|
296 |
by (blast_tac (claset() addIs [leadsETo_weaken_L] |
|
297 |
addDs [constrains_imp_subset]) 2); |
|
298 |
(*Basis case*) |
|
299 |
by (rtac leadsETo_Basis 1); |
|
300 |
by (blast_tac (claset() addIs [psp_ensures]) 1); |
|
301 |
by (subgoal_tac "A Int B' - (Ba Int B Un (B' - B)) = (A - Ba) Int B Int B'" 1); |
|
302 |
by Auto_tac; |
|
303 |
qed "e_psp"; |
|
304 |
||
305 |
Goal "[| F : A leadsTo[CC] A'; F : B co B'; \ |
|
8072
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
306 |
\ ALL C:CC. C Int B Int B' : CC |] \ |
8044 | 307 |
\ ==> F : (B' Int A) leadsTo[CC] ((B Int A') Un (B' - B))"; |
308 |
by (asm_full_simp_tac (simpset() addsimps e_psp::Int_ac) 1); |
|
309 |
qed "e_psp2"; |
|
310 |
||
311 |
||
312 |
(*** Special properties involving the parameter [CC] ***) |
|
313 |
||
314 |
(*??IS THIS NEEDED?? or is it just an example of what's provable??*) |
|
8055
bb15396278fb
abolition of localTo: instead "guarantees" has local vars as extra argument
paulson
parents:
8044
diff
changeset
|
315 |
Goal "[| F: (A leadsTo[givenBy v] B); G : preserves v; \ |
8044 | 316 |
\ F Join G : stable C |] \ |
317 |
\ ==> F Join G : ((C Int A) leadsTo[(%D. C Int D) `` givenBy v] B)"; |
|
318 |
by (etac leadsETo_induct 1); |
|
319 |
by (stac Int_Union 3); |
|
320 |
by (blast_tac (claset() addIs [leadsETo_UN]) 3); |
|
321 |
by (blast_tac (claset() addIs [e_psp_stable2 RS leadsETo_weaken_L, |
|
322 |
leadsETo_Trans]) 2); |
|
323 |
by (rtac leadsETo_Basis 1); |
|
324 |
by (auto_tac (claset(), |
|
8072
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
325 |
simpset() addsimps [Diff_eq_empty_iff RS iffD2, |
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
326 |
Int_Diff, ensures_def, |
8055
bb15396278fb
abolition of localTo: instead "guarantees" has local vars as extra argument
paulson
parents:
8044
diff
changeset
|
327 |
givenBy_eq_Collect, Join_stable, |
8044 | 328 |
Join_constrains, Join_transient])); |
329 |
by (blast_tac (claset() addIs [transient_strengthen]) 3); |
|
8055
bb15396278fb
abolition of localTo: instead "guarantees" has local vars as extra argument
paulson
parents:
8044
diff
changeset
|
330 |
by (ALLGOALS (dres_inst_tac [("P1","P")] (impOfSubs preserves_subset_stable))); |
bb15396278fb
abolition of localTo: instead "guarantees" has local vars as extra argument
paulson
parents:
8044
diff
changeset
|
331 |
by (rewtac stable_def); |
bb15396278fb
abolition of localTo: instead "guarantees" has local vars as extra argument
paulson
parents:
8044
diff
changeset
|
332 |
by (blast_tac (claset() addSEs [equalityE] |
8044 | 333 |
addIs [constrains_Int RS constrains_weaken]) 2); |
8055
bb15396278fb
abolition of localTo: instead "guarantees" has local vars as extra argument
paulson
parents:
8044
diff
changeset
|
334 |
by (blast_tac (claset() addSEs [equalityE] |
bb15396278fb
abolition of localTo: instead "guarantees" has local vars as extra argument
paulson
parents:
8044
diff
changeset
|
335 |
addIs [constrains_Int RS constrains_weaken]) 1); |
bb15396278fb
abolition of localTo: instead "guarantees" has local vars as extra argument
paulson
parents:
8044
diff
changeset
|
336 |
qed "gen_leadsETo_imp_Join_leadsETo"; |
8044 | 337 |
|
338 |
(*useful??*) |
|
339 |
Goal "[| F Join G : (A leadsTo[CC] B); ALL C:CC. G : stable C |] \ |
|
340 |
\ ==> F: (A leadsTo[CC] B)"; |
|
341 |
by (etac leadsETo_induct 1); |
|
342 |
by (blast_tac (claset() addIs [leadsETo_Union]) 3); |
|
343 |
by (blast_tac (claset() addIs [leadsETo_Trans]) 2); |
|
344 |
by (rtac leadsETo_Basis 1); |
|
345 |
by (case_tac "A <= B" 1); |
|
346 |
by (etac subset_imp_ensures 1); |
|
347 |
by (auto_tac (claset() addIs [constrains_weaken], |
|
8072
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
348 |
simpset() addsimps [stable_def, ensures_def, |
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
349 |
Join_constrains, Join_transient])); |
8044 | 350 |
by (REPEAT (thin_tac "?F : ?A co ?B" 1)); |
351 |
by (etac transientE 1); |
|
352 |
by (rewtac constrains_def); |
|
353 |
by (blast_tac (claset() addSDs [bspec]) 1); |
|
354 |
qed "Join_leadsETo_stable_imp_leadsETo"; |
|
355 |
||
8067 | 356 |
(**** Relationship with traditional "leadsTo", strong & weak ****) |
357 |
||
358 |
(** strong **) |
|
359 |
||
360 |
Goal "(A leadsTo[CC] B) <= (A leadsTo B)"; |
|
361 |
by Safe_tac; |
|
362 |
by (etac leadsETo_induct 1); |
|
363 |
by (blast_tac (claset() addIs [leadsTo_Union]) 3); |
|
364 |
by (blast_tac (claset() addIs [leadsTo_Trans]) 2); |
|
365 |
by (blast_tac (claset() addIs [leadsTo_Basis]) 1); |
|
366 |
qed "leadsETo_subset_leadsTo"; |
|
367 |
||
368 |
Goal "(A leadsTo[UNIV] B) = (A leadsTo B)"; |
|
369 |
by Safe_tac; |
|
370 |
by (etac (impOfSubs leadsETo_subset_leadsTo) 1); |
|
371 |
(*right-to-left case*) |
|
372 |
by (etac leadsTo_induct 1); |
|
373 |
by (blast_tac (claset() addIs [leadsETo_Union]) 3); |
|
374 |
by (blast_tac (claset() addIs [leadsETo_Trans]) 2); |
|
375 |
by (blast_tac (claset() addIs [leadsETo_Basis]) 1); |
|
376 |
qed "leadsETo_UNIV_eq_leadsTo"; |
|
377 |
||
8072
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
378 |
(**** weak ****) |
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
379 |
|
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
380 |
Goalw [LeadsETo_def] |
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
381 |
"A LeadsTo[CC] B = \ |
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
382 |
\ {F. F : (reachable F Int A) leadsTo[(%C. reachable F Int C) `` CC] \ |
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
383 |
\ (reachable F Int B)}"; |
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
384 |
by (blast_tac (claset() addDs [e_psp_stable2] addIs [leadsETo_weaken]) 1); |
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
385 |
qed "LeadsETo_eq_leadsETo"; |
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
386 |
|
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
387 |
(*** Introduction rules: Basis, Trans, Union ***) |
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
388 |
|
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
389 |
Goal "[| F : A LeadsTo[CC] B; F : B LeadsTo[CC] C |] \ |
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
390 |
\ ==> F : A LeadsTo[CC] C"; |
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
391 |
by (asm_full_simp_tac (simpset() addsimps [LeadsETo_eq_leadsETo]) 1); |
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
392 |
by (blast_tac (claset() addIs [leadsETo_Trans]) 1); |
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
393 |
qed "LeadsETo_Trans"; |
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
394 |
|
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
395 |
val prems = Goalw [LeadsETo_def] |
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
396 |
"(!!A. A : S ==> F : A LeadsTo[CC] B) ==> F : (Union S) LeadsTo[CC] B"; |
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
397 |
by (Simp_tac 1); |
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
398 |
by (stac Int_Union 1); |
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
399 |
by (blast_tac (claset() addIs [leadsETo_UN] addDs prems) 1); |
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
400 |
qed "LeadsETo_Union"; |
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
401 |
|
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
402 |
val prems = |
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
403 |
Goal "(!!i. i : I ==> F : (A i) LeadsTo[CC] B) \ |
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
404 |
\ ==> F : (UN i:I. A i) LeadsTo[CC] B"; |
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
405 |
by (simp_tac (HOL_ss addsimps [Union_image_eq RS sym]) 1); |
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
406 |
by (blast_tac (claset() addIs (LeadsETo_Union::prems)) 1); |
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
407 |
qed "LeadsETo_UN"; |
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
408 |
|
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
409 |
(*Binary union introduction rule*) |
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
410 |
Goal "[| F : A LeadsTo[CC] C; F : B LeadsTo[CC] C |] \ |
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
411 |
\ ==> F : (A Un B) LeadsTo[CC] C"; |
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
412 |
by (stac Un_eq_Union 1); |
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
413 |
by (blast_tac (claset() addIs [LeadsETo_Union]) 1); |
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
414 |
qed "LeadsETo_Un"; |
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
415 |
|
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
416 |
(*Lets us look at the starting state*) |
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
417 |
val prems = |
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
418 |
Goal "(!!s. s : A ==> F : {s} LeadsTo[CC] B) ==> F : A LeadsTo[CC] B"; |
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
419 |
by (stac (UN_singleton RS sym) 1 THEN rtac LeadsETo_UN 1); |
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
420 |
by (blast_tac (claset() addIs prems) 1); |
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
421 |
qed "single_LeadsETo_I"; |
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
422 |
|
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
423 |
Goal "A <= B ==> F : A LeadsTo[CC] B"; |
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
424 |
by (simp_tac (simpset() addsimps [LeadsETo_def]) 1); |
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
425 |
by (blast_tac (claset() addIs [subset_imp_leadsETo]) 1); |
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
426 |
qed "subset_imp_LeadsETo"; |
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
427 |
|
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
428 |
bind_thm ("empty_LeadsETo", empty_subsetI RS subset_imp_LeadsETo); |
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
429 |
|
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
430 |
Goal "[| F : A LeadsTo[CC] A'; A' <= B' |] ==> F : A LeadsTo[CC] B'"; |
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
431 |
by (full_simp_tac (simpset() addsimps [LeadsETo_def]) 1); |
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
432 |
by (blast_tac (claset() addIs [leadsETo_weaken_R]) 1); |
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
433 |
qed_spec_mp "LeadsETo_weaken_R"; |
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
434 |
|
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
435 |
Goal "[| F : A LeadsTo[CC] A'; B <= A |] ==> F : B LeadsTo[CC] A'"; |
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
436 |
by (full_simp_tac (simpset() addsimps [LeadsETo_def]) 1); |
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
437 |
by (blast_tac (claset() addIs [leadsETo_weaken_L]) 1); |
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
438 |
qed_spec_mp "LeadsETo_weaken_L"; |
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
439 |
|
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
440 |
Goal "[| F : A LeadsTo[CC'] A'; \ |
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
441 |
\ B <= A; A' <= B'; CC' <= CC |] \ |
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
442 |
\ ==> F : B LeadsTo[CC] B'"; |
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
443 |
by (full_simp_tac (simpset() addsimps [LeadsETo_def]) 1); |
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
444 |
by (blast_tac (claset() addIs [leadsETo_weaken]) 1); |
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
445 |
qed "LeadsETo_weaken"; |
8067 | 446 |
|
447 |
Goalw [LeadsETo_def, LeadsTo_def] "(A LeadsTo[CC] B) <= (A LeadsTo B)"; |
|
448 |
by (blast_tac (claset() addIs [impOfSubs leadsETo_subset_leadsTo]) 1); |
|
449 |
qed "LeadsETo_subset_LeadsTo"; |
|
450 |
||
451 |
(*Postcondition can be strengthened to (reachable F Int B) *) |
|
452 |
Goal "F : A ensures B ==> F : (reachable F Int A) ensures B"; |
|
453 |
by (rtac (stable_ensures_Int RS ensures_weaken_R) 1); |
|
8069
19b9f92ca503
working with weak LeadsTo in guarantees precondition\!
paulson
parents:
8067
diff
changeset
|
454 |
by Auto_tac; |
8067 | 455 |
qed "reachable_ensures"; |
456 |
||
457 |
Goal "F : A leadsTo B ==> F : (reachable F Int A) leadsTo[Pow(reachable F)] B"; |
|
458 |
by (etac leadsTo_induct 1); |
|
459 |
by (stac Int_Union 3); |
|
460 |
by (blast_tac (claset() addIs [leadsETo_UN]) 3); |
|
461 |
by (blast_tac (claset() addDs [e_psp_stable2] |
|
8069
19b9f92ca503
working with weak LeadsTo in guarantees precondition\!
paulson
parents:
8067
diff
changeset
|
462 |
addIs [leadsETo_Trans, leadsETo_weaken_L]) 2); |
8067 | 463 |
by (blast_tac (claset() addIs [reachable_ensures, leadsETo_Basis]) 1); |
464 |
val lemma = result(); |
|
465 |
||
466 |
Goal "(A LeadsTo[UNIV] B) = (A LeadsTo B)"; |
|
467 |
by Safe_tac; |
|
468 |
by (etac (impOfSubs LeadsETo_subset_LeadsTo) 1); |
|
469 |
(*right-to-left case*) |
|
470 |
by (rewrite_goals_tac [LeadsETo_def, LeadsTo_def]); |
|
471 |
by (fast_tac (claset() addEs [lemma RS leadsETo_weaken]) 1); |
|
472 |
qed "LeadsETo_UNIV_eq_LeadsTo"; |
|
473 |
||
8044 | 474 |
|
475 |
(**** EXTEND/PROJECT PROPERTIES ****) |
|
476 |
||
477 |
Open_locale "Extend"; |
|
478 |
||
8334
7896bcbd8641
Added Tanja's Detects and Reachability theories. Also
paulson
parents:
8128
diff
changeset
|
479 |
(*givenBy laws that need to be in the locale*) |
7896bcbd8641
Added Tanja's Detects and Reachability theories. Also
paulson
parents:
8128
diff
changeset
|
480 |
|
7896bcbd8641
Added Tanja's Detects and Reachability theories. Also
paulson
parents:
8128
diff
changeset
|
481 |
Goal "givenBy (v o f) = extend_set h `` (givenBy v)"; |
7896bcbd8641
Added Tanja's Detects and Reachability theories. Also
paulson
parents:
8128
diff
changeset
|
482 |
by (simp_tac (simpset() addsimps [givenBy_eq_Collect]) 1); |
7896bcbd8641
Added Tanja's Detects and Reachability theories. Also
paulson
parents:
8128
diff
changeset
|
483 |
by (Deepen_tac 0 1); |
7896bcbd8641
Added Tanja's Detects and Reachability theories. Also
paulson
parents:
8128
diff
changeset
|
484 |
qed "givenBy_o_eq_extend_set"; |
7896bcbd8641
Added Tanja's Detects and Reachability theories. Also
paulson
parents:
8128
diff
changeset
|
485 |
|
7896bcbd8641
Added Tanja's Detects and Reachability theories. Also
paulson
parents:
8128
diff
changeset
|
486 |
Goal "givenBy f = range (extend_set h)"; |
7896bcbd8641
Added Tanja's Detects and Reachability theories. Also
paulson
parents:
8128
diff
changeset
|
487 |
by (simp_tac (simpset() addsimps [givenBy_eq_Collect]) 1); |
7896bcbd8641
Added Tanja's Detects and Reachability theories. Also
paulson
parents:
8128
diff
changeset
|
488 |
by (Deepen_tac 0 1); |
7896bcbd8641
Added Tanja's Detects and Reachability theories. Also
paulson
parents:
8128
diff
changeset
|
489 |
qed "givenBy_eq_extend_set"; |
7896bcbd8641
Added Tanja's Detects and Reachability theories. Also
paulson
parents:
8128
diff
changeset
|
490 |
|
7896bcbd8641
Added Tanja's Detects and Reachability theories. Also
paulson
parents:
8128
diff
changeset
|
491 |
Goal "D : givenBy v ==> extend_set h D : givenBy (v o f)"; |
7896bcbd8641
Added Tanja's Detects and Reachability theories. Also
paulson
parents:
8128
diff
changeset
|
492 |
by (full_simp_tac (simpset() addsimps [givenBy_eq_all]) 1); |
7896bcbd8641
Added Tanja's Detects and Reachability theories. Also
paulson
parents:
8128
diff
changeset
|
493 |
by (Blast_tac 1); |
7896bcbd8641
Added Tanja's Detects and Reachability theories. Also
paulson
parents:
8128
diff
changeset
|
494 |
qed "extend_set_givenBy_I"; |
7896bcbd8641
Added Tanja's Detects and Reachability theories. Also
paulson
parents:
8128
diff
changeset
|
495 |
|
8044 | 496 |
Goal "F : A leadsTo[CC] B \ |
497 |
\ ==> extend h F : (extend_set h A) leadsTo[extend_set h `` CC] \ |
|
498 |
\ (extend_set h B)"; |
|
499 |
by (etac leadsETo_induct 1); |
|
500 |
by (asm_simp_tac (simpset() addsimps [leadsETo_UN, extend_set_Union]) 3); |
|
501 |
by (blast_tac (claset() addIs [leadsETo_Trans]) 2); |
|
8072
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
502 |
by (force_tac (claset() addIs [leadsETo_Basis, subset_imp_ensures], |
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
503 |
simpset() addsimps [extend_ensures, |
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
504 |
extend_set_Diff_distrib RS sym]) 1); |
8044 | 505 |
qed "leadsETo_imp_extend_leadsETo"; |
506 |
||
8055
bb15396278fb
abolition of localTo: instead "guarantees" has local vars as extra argument
paulson
parents:
8044
diff
changeset
|
507 |
|
bb15396278fb
abolition of localTo: instead "guarantees" has local vars as extra argument
paulson
parents:
8044
diff
changeset
|
508 |
|
bb15396278fb
abolition of localTo: instead "guarantees" has local vars as extra argument
paulson
parents:
8044
diff
changeset
|
509 |
(*NOT USED, but analogous to preserves_project_transient_empty in Project.ML*) |
bb15396278fb
abolition of localTo: instead "guarantees" has local vars as extra argument
paulson
parents:
8044
diff
changeset
|
510 |
Goal "[| G : preserves (v o f); project h C G : transient D; \ |
bb15396278fb
abolition of localTo: instead "guarantees" has local vars as extra argument
paulson
parents:
8044
diff
changeset
|
511 |
\ D : givenBy v |] ==> D={}"; |
bb15396278fb
abolition of localTo: instead "guarantees" has local vars as extra argument
paulson
parents:
8044
diff
changeset
|
512 |
by (rtac stable_transient_empty 1); |
8044 | 513 |
by (assume_tac 2); |
8055
bb15396278fb
abolition of localTo: instead "guarantees" has local vars as extra argument
paulson
parents:
8044
diff
changeset
|
514 |
(*If addIs then PROOF FAILED at depth 2*) |
bb15396278fb
abolition of localTo: instead "guarantees" has local vars as extra argument
paulson
parents:
8044
diff
changeset
|
515 |
by (blast_tac (claset() addSIs [preserves_givenBy_imp_stable, |
bb15396278fb
abolition of localTo: instead "guarantees" has local vars as extra argument
paulson
parents:
8044
diff
changeset
|
516 |
project_preserves_I]) 1); |
bb15396278fb
abolition of localTo: instead "guarantees" has local vars as extra argument
paulson
parents:
8044
diff
changeset
|
517 |
result(); |
bb15396278fb
abolition of localTo: instead "guarantees" has local vars as extra argument
paulson
parents:
8044
diff
changeset
|
518 |
|
8044 | 519 |
|
520 |
(*This version's stronger in the "ensures" precondition |
|
521 |
BUT there's no ensures_weaken_L*) |
|
8055
bb15396278fb
abolition of localTo: instead "guarantees" has local vars as extra argument
paulson
parents:
8044
diff
changeset
|
522 |
Goal "[| project h C G ~: transient (project_set h C Int (A-B)) | \ |
bb15396278fb
abolition of localTo: instead "guarantees" has local vars as extra argument
paulson
parents:
8044
diff
changeset
|
523 |
\ project_set h C Int (A - B) = {}; \ |
8044 | 524 |
\ extend h F Join G : stable C; \ |
525 |
\ F Join project h C G : (project_set h C Int A) ensures B |] \ |
|
526 |
\ ==> extend h F Join G : (C Int extend_set h A) ensures (extend_set h B)"; |
|
527 |
by (stac (Int_extend_set_lemma RS sym) 1); |
|
528 |
by (rtac Join_project_ensures 1); |
|
529 |
by (auto_tac (claset(), simpset() addsimps [Int_Diff])); |
|
530 |
qed "Join_project_ensures_strong"; |
|
531 |
||
8334
7896bcbd8641
Added Tanja's Detects and Reachability theories. Also
paulson
parents:
8128
diff
changeset
|
532 |
(*Generalizes preserves_project_transient_empty*) |
7896bcbd8641
Added Tanja's Detects and Reachability theories. Also
paulson
parents:
8128
diff
changeset
|
533 |
Goal "[| G : preserves (v o f); \ |
7896bcbd8641
Added Tanja's Detects and Reachability theories. Also
paulson
parents:
8128
diff
changeset
|
534 |
\ project h C G : transient (C' Int D); \ |
7896bcbd8641
Added Tanja's Detects and Reachability theories. Also
paulson
parents:
8128
diff
changeset
|
535 |
\ project h C G : stable C'; D : givenBy v |] \ |
7896bcbd8641
Added Tanja's Detects and Reachability theories. Also
paulson
parents:
8128
diff
changeset
|
536 |
\ ==> C' Int D = {}"; |
7896bcbd8641
Added Tanja's Detects and Reachability theories. Also
paulson
parents:
8128
diff
changeset
|
537 |
by (rtac stable_transient_empty 1); |
7896bcbd8641
Added Tanja's Detects and Reachability theories. Also
paulson
parents:
8128
diff
changeset
|
538 |
by (assume_tac 2); |
7896bcbd8641
Added Tanja's Detects and Reachability theories. Also
paulson
parents:
8128
diff
changeset
|
539 |
(*If addIs then PROOF FAILED at depth 3*) |
7896bcbd8641
Added Tanja's Detects and Reachability theories. Also
paulson
parents:
8128
diff
changeset
|
540 |
by (blast_tac (claset() addSIs [stable_Int, preserves_givenBy_imp_stable, |
7896bcbd8641
Added Tanja's Detects and Reachability theories. Also
paulson
parents:
8128
diff
changeset
|
541 |
project_preserves_I]) 1); |
7896bcbd8641
Added Tanja's Detects and Reachability theories. Also
paulson
parents:
8128
diff
changeset
|
542 |
qed "preserves_o_project_transient_empty"; |
7896bcbd8641
Added Tanja's Detects and Reachability theories. Also
paulson
parents:
8128
diff
changeset
|
543 |
|
8044 | 544 |
Goal "[| extend h F Join G : stable C; \ |
8055
bb15396278fb
abolition of localTo: instead "guarantees" has local vars as extra argument
paulson
parents:
8044
diff
changeset
|
545 |
\ F Join project h C G : (project_set h C Int A) leadsTo[(%D. project_set h C Int D)``givenBy v] B; \ |
bb15396278fb
abolition of localTo: instead "guarantees" has local vars as extra argument
paulson
parents:
8044
diff
changeset
|
546 |
\ G : preserves (v o f) |] \ |
8044 | 547 |
\ ==> extend h F Join G : \ |
548 |
\ (C Int extend_set h (project_set h C Int A)) \ |
|
549 |
\ leadsTo[(%D. C Int extend_set h D)``givenBy v] (extend_set h B)"; |
|
550 |
by (etac leadsETo_induct 1); |
|
551 |
by (asm_simp_tac (simpset() delsimps UN_simps |
|
552 |
addsimps [Int_UN_distrib, leadsETo_UN, extend_set_Union]) 3); |
|
553 |
by (blast_tac (claset() addIs [e_psp_stable2 RS leadsETo_weaken_L, |
|
554 |
leadsETo_Trans]) 2); |
|
8110 | 555 |
by Auto_tac; |
8072
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
556 |
by (force_tac (claset() addIs [leadsETo_Basis, subset_imp_ensures], |
5b95377d7538
removing the "{} : CC" requirement for leadsTo[CC]
paulson
parents:
8069
diff
changeset
|
557 |
simpset()) 1); |
8044 | 558 |
by (rtac leadsETo_Basis 1); |
559 |
by (asm_simp_tac (simpset() addsimps [Int_Diff, Int_extend_set_lemma, |
|
560 |
extend_set_Diff_distrib RS sym]) 2); |
|
561 |
by (rtac Join_project_ensures_strong 1); |
|
8055
bb15396278fb
abolition of localTo: instead "guarantees" has local vars as extra argument
paulson
parents:
8044
diff
changeset
|
562 |
by (auto_tac (claset() addDs [preserves_o_project_transient_empty] |
bb15396278fb
abolition of localTo: instead "guarantees" has local vars as extra argument
paulson
parents:
8044
diff
changeset
|
563 |
addIs [project_stable_project_set], |
8044 | 564 |
simpset() addsimps [Int_left_absorb, Join_stable])); |
565 |
by (asm_simp_tac |
|
566 |
(simpset() addsimps [stable_ensures_Int RS ensures_weaken_R, |
|
567 |
Int_lower2, project_stable_project_set, |
|
568 |
Join_stable, extend_stable_project_set]) 1); |
|
569 |
val lemma = result(); |
|
570 |
||
571 |
Goal "[| extend h F Join G : stable C; \ |
|
8055
bb15396278fb
abolition of localTo: instead "guarantees" has local vars as extra argument
paulson
parents:
8044
diff
changeset
|
572 |
\ F Join project h C G : \ |
bb15396278fb
abolition of localTo: instead "guarantees" has local vars as extra argument
paulson
parents:
8044
diff
changeset
|
573 |
\ (project_set h C Int A) \ |
bb15396278fb
abolition of localTo: instead "guarantees" has local vars as extra argument
paulson
parents:
8044
diff
changeset
|
574 |
\ leadsTo[(%D. project_set h C Int D)``givenBy v] B; \ |
bb15396278fb
abolition of localTo: instead "guarantees" has local vars as extra argument
paulson
parents:
8044
diff
changeset
|
575 |
\ G : preserves (v o f) |] \ |
8044 | 576 |
\ ==> extend h F Join G : (C Int extend_set h A) \ |
577 |
\ leadsTo[(%D. C Int extend_set h D)``givenBy v] (extend_set h B)"; |
|
578 |
by (rtac (lemma RS leadsETo_weaken) 1); |
|
8069
19b9f92ca503
working with weak LeadsTo in guarantees precondition\!
paulson
parents:
8067
diff
changeset
|
579 |
by (auto_tac (claset(), |
19b9f92ca503
working with weak LeadsTo in guarantees precondition\!
paulson
parents:
8067
diff
changeset
|
580 |
simpset() addsimps [split_extended_all])); |
19b9f92ca503
working with weak LeadsTo in guarantees precondition\!
paulson
parents:
8067
diff
changeset
|
581 |
qed "project_leadsETo_D_lemma"; |
8044 | 582 |
|
8055
bb15396278fb
abolition of localTo: instead "guarantees" has local vars as extra argument
paulson
parents:
8044
diff
changeset
|
583 |
Goal "[| F Join project h UNIV G : A leadsTo[givenBy v] B; \ |
bb15396278fb
abolition of localTo: instead "guarantees" has local vars as extra argument
paulson
parents:
8044
diff
changeset
|
584 |
\ G : preserves (v o f) |] \ |
8044 | 585 |
\ ==> extend h F Join G : (extend_set h A) \ |
586 |
\ leadsTo[givenBy (v o f)] (extend_set h B)"; |
|
8069
19b9f92ca503
working with weak LeadsTo in guarantees precondition\!
paulson
parents:
8067
diff
changeset
|
587 |
by (rtac (make_elim project_leadsETo_D_lemma) 1); |
8055
bb15396278fb
abolition of localTo: instead "guarantees" has local vars as extra argument
paulson
parents:
8044
diff
changeset
|
588 |
by (stac stable_UNIV 1); |
8044 | 589 |
by Auto_tac; |
590 |
by (etac leadsETo_givenBy 1); |
|
8069
19b9f92ca503
working with weak LeadsTo in guarantees precondition\!
paulson
parents:
8067
diff
changeset
|
591 |
by (rtac (givenBy_o_eq_extend_set RS equalityD2) 1); |
8044 | 592 |
qed "project_leadsETo_D"; |
593 |
||
594 |
Goal "[| F Join project h (reachable (extend h F Join G)) G \ |
|
8055
bb15396278fb
abolition of localTo: instead "guarantees" has local vars as extra argument
paulson
parents:
8044
diff
changeset
|
595 |
\ : A LeadsTo[givenBy v] B; \ |
bb15396278fb
abolition of localTo: instead "guarantees" has local vars as extra argument
paulson
parents:
8044
diff
changeset
|
596 |
\ G : preserves (v o f) |] \ |
8044 | 597 |
\ ==> extend h F Join G : \ |
598 |
\ (extend_set h A) LeadsTo[givenBy (v o f)] (extend_set h B)"; |
|
599 |
by (rtac (make_elim (subset_refl RS stable_reachable RS |
|
8069
19b9f92ca503
working with weak LeadsTo in guarantees precondition\!
paulson
parents:
8067
diff
changeset
|
600 |
project_leadsETo_D_lemma)) 1); |
8044 | 601 |
by (auto_tac (claset(), |
8055
bb15396278fb
abolition of localTo: instead "guarantees" has local vars as extra argument
paulson
parents:
8044
diff
changeset
|
602 |
simpset() addsimps [LeadsETo_def])); |
8044 | 603 |
by (asm_full_simp_tac |
604 |
(simpset() addsimps [project_set_reachable_extend_eq RS sym]) 1); |
|
605 |
by (etac (impOfSubs leadsETo_mono) 1); |
|
606 |
by (blast_tac (claset() addIs [extend_set_givenBy_I]) 1); |
|
607 |
qed "project_LeadsETo_D"; |
|
608 |
||
609 |
Goalw [extending_def] |
|
8055
bb15396278fb
abolition of localTo: instead "guarantees" has local vars as extra argument
paulson
parents:
8044
diff
changeset
|
610 |
"extending (v o f) (%G. UNIV) h F \ |
8044 | 611 |
\ (extend_set h A leadsTo[givenBy (v o f)] extend_set h B) \ |
612 |
\ (A leadsTo[givenBy v] B)"; |
|
8055
bb15396278fb
abolition of localTo: instead "guarantees" has local vars as extra argument
paulson
parents:
8044
diff
changeset
|
613 |
by (auto_tac (claset(), simpset() addsimps [project_leadsETo_D])); |
8044 | 614 |
qed "extending_leadsETo"; |
615 |
||
616 |
||
617 |
Goalw [extending_def] |
|
8055
bb15396278fb
abolition of localTo: instead "guarantees" has local vars as extra argument
paulson
parents:
8044
diff
changeset
|
618 |
"extending (v o f) (%G. reachable (extend h F Join G)) h F \ |
8044 | 619 |
\ (extend_set h A LeadsTo[givenBy (v o f)] extend_set h B) \ |
620 |
\ (A LeadsTo[givenBy v] B)"; |
|
8055
bb15396278fb
abolition of localTo: instead "guarantees" has local vars as extra argument
paulson
parents:
8044
diff
changeset
|
621 |
by (blast_tac (claset() addIs [project_LeadsETo_D]) 1); |
8044 | 622 |
qed "extending_LeadsETo"; |
623 |
||
624 |
||
8069
19b9f92ca503
working with weak LeadsTo in guarantees precondition\!
paulson
parents:
8067
diff
changeset
|
625 |
(*** leadsETo in the precondition ***) |
19b9f92ca503
working with weak LeadsTo in guarantees precondition\!
paulson
parents:
8067
diff
changeset
|
626 |
|
19b9f92ca503
working with weak LeadsTo in guarantees precondition\!
paulson
parents:
8067
diff
changeset
|
627 |
(*Lemma for the Trans case*) |
19b9f92ca503
working with weak LeadsTo in guarantees precondition\!
paulson
parents:
8067
diff
changeset
|
628 |
Goal "[| extend h F Join G : stable C; \ |
19b9f92ca503
working with weak LeadsTo in guarantees precondition\!
paulson
parents:
8067
diff
changeset
|
629 |
\ F Join project h C G \ |
19b9f92ca503
working with weak LeadsTo in guarantees precondition\!
paulson
parents:
8067
diff
changeset
|
630 |
\ : project_set h C Int project_set h A leadsTo project_set h B |] \ |
19b9f92ca503
working with weak LeadsTo in guarantees precondition\!
paulson
parents:
8067
diff
changeset
|
631 |
\ ==> F Join project h C G \ |
19b9f92ca503
working with weak LeadsTo in guarantees precondition\!
paulson
parents:
8067
diff
changeset
|
632 |
\ : project_set h C Int project_set h A leadsTo \ |
19b9f92ca503
working with weak LeadsTo in guarantees precondition\!
paulson
parents:
8067
diff
changeset
|
633 |
\ project_set h C Int project_set h B"; |
19b9f92ca503
working with weak LeadsTo in guarantees precondition\!
paulson
parents:
8067
diff
changeset
|
634 |
by (rtac (psp_stable2 RS leadsTo_weaken_L) 1); |
19b9f92ca503
working with weak LeadsTo in guarantees precondition\!
paulson
parents:
8067
diff
changeset
|
635 |
by (auto_tac (claset(), |
19b9f92ca503
working with weak LeadsTo in guarantees precondition\!
paulson
parents:
8067
diff
changeset
|
636 |
simpset() addsimps [project_stable_project_set, Join_stable, |
19b9f92ca503
working with weak LeadsTo in guarantees precondition\!
paulson
parents:
8067
diff
changeset
|
637 |
extend_stable_project_set])); |
19b9f92ca503
working with weak LeadsTo in guarantees precondition\!
paulson
parents:
8067
diff
changeset
|
638 |
val lemma = result(); |
19b9f92ca503
working with weak LeadsTo in guarantees precondition\!
paulson
parents:
8067
diff
changeset
|
639 |
|
19b9f92ca503
working with weak LeadsTo in guarantees precondition\!
paulson
parents:
8067
diff
changeset
|
640 |
Goal "[| extend h F Join G : stable C; \ |
19b9f92ca503
working with weak LeadsTo in guarantees precondition\!
paulson
parents:
8067
diff
changeset
|
641 |
\ extend h F Join G : \ |
19b9f92ca503
working with weak LeadsTo in guarantees precondition\!
paulson
parents:
8067
diff
changeset
|
642 |
\ (C Int A) leadsTo[(%D. C Int D)``givenBy f] B |] \ |
19b9f92ca503
working with weak LeadsTo in guarantees precondition\!
paulson
parents:
8067
diff
changeset
|
643 |
\ ==> F Join project h C G \ |
19b9f92ca503
working with weak LeadsTo in guarantees precondition\!
paulson
parents:
8067
diff
changeset
|
644 |
\ : (project_set h C Int project_set h (C Int A)) leadsTo (project_set h B)"; |
19b9f92ca503
working with weak LeadsTo in guarantees precondition\!
paulson
parents:
8067
diff
changeset
|
645 |
by (etac leadsETo_induct 1); |
19b9f92ca503
working with weak LeadsTo in guarantees precondition\!
paulson
parents:
8067
diff
changeset
|
646 |
by (asm_simp_tac (HOL_ss addsimps [Int_UN_distrib, project_set_Union]) 3); |
19b9f92ca503
working with weak LeadsTo in guarantees precondition\!
paulson
parents:
8067
diff
changeset
|
647 |
by (blast_tac (claset() addIs [leadsTo_UN]) 3); |
19b9f92ca503
working with weak LeadsTo in guarantees precondition\!
paulson
parents:
8067
diff
changeset
|
648 |
by (blast_tac (claset() addIs [leadsTo_Trans, lemma]) 2); |
19b9f92ca503
working with weak LeadsTo in guarantees precondition\!
paulson
parents:
8067
diff
changeset
|
649 |
by (asm_full_simp_tac |
19b9f92ca503
working with weak LeadsTo in guarantees precondition\!
paulson
parents:
8067
diff
changeset
|
650 |
(simpset() addsimps [givenBy_eq_extend_set, Join_stable]) 1); |
19b9f92ca503
working with weak LeadsTo in guarantees precondition\!
paulson
parents:
8067
diff
changeset
|
651 |
by (rtac leadsTo_Basis 1); |
19b9f92ca503
working with weak LeadsTo in guarantees precondition\!
paulson
parents:
8067
diff
changeset
|
652 |
by (blast_tac (claset() addIs [leadsTo_Basis, |
19b9f92ca503
working with weak LeadsTo in guarantees precondition\!
paulson
parents:
8067
diff
changeset
|
653 |
ensures_extend_set_imp_project_ensures]) 1); |
19b9f92ca503
working with weak LeadsTo in guarantees precondition\!
paulson
parents:
8067
diff
changeset
|
654 |
|
19b9f92ca503
working with weak LeadsTo in guarantees precondition\!
paulson
parents:
8067
diff
changeset
|
655 |
qed "project_leadsETo_I_lemma"; |
19b9f92ca503
working with weak LeadsTo in guarantees precondition\!
paulson
parents:
8067
diff
changeset
|
656 |
|
19b9f92ca503
working with weak LeadsTo in guarantees precondition\!
paulson
parents:
8067
diff
changeset
|
657 |
Goal "extend h F Join G : (extend_set h A) leadsTo[givenBy f] (extend_set h B)\ |
19b9f92ca503
working with weak LeadsTo in guarantees precondition\!
paulson
parents:
8067
diff
changeset
|
658 |
\ ==> F Join project h UNIV G : A leadsTo B"; |
19b9f92ca503
working with weak LeadsTo in guarantees precondition\!
paulson
parents:
8067
diff
changeset
|
659 |
by (rtac (project_leadsETo_I_lemma RS leadsTo_weaken) 1); |
19b9f92ca503
working with weak LeadsTo in guarantees precondition\!
paulson
parents:
8067
diff
changeset
|
660 |
by Auto_tac; |
19b9f92ca503
working with weak LeadsTo in guarantees precondition\!
paulson
parents:
8067
diff
changeset
|
661 |
qed "project_leadsETo_I"; |
19b9f92ca503
working with weak LeadsTo in guarantees precondition\!
paulson
parents:
8067
diff
changeset
|
662 |
|
19b9f92ca503
working with weak LeadsTo in guarantees precondition\!
paulson
parents:
8067
diff
changeset
|
663 |
Goal "extend h F Join G : (extend_set h A) LeadsTo[givenBy f] (extend_set h B)\ |
19b9f92ca503
working with weak LeadsTo in guarantees precondition\!
paulson
parents:
8067
diff
changeset
|
664 |
\ ==> F Join project h (reachable (extend h F Join G)) G \ |
19b9f92ca503
working with weak LeadsTo in guarantees precondition\!
paulson
parents:
8067
diff
changeset
|
665 |
\ : A LeadsTo B"; |
19b9f92ca503
working with weak LeadsTo in guarantees precondition\!
paulson
parents:
8067
diff
changeset
|
666 |
by (full_simp_tac (simpset() addsimps [LeadsTo_def, LeadsETo_def]) 1); |
19b9f92ca503
working with weak LeadsTo in guarantees precondition\!
paulson
parents:
8067
diff
changeset
|
667 |
by (rtac (project_leadsETo_I_lemma RS leadsTo_weaken) 1); |
19b9f92ca503
working with weak LeadsTo in guarantees precondition\!
paulson
parents:
8067
diff
changeset
|
668 |
by (auto_tac (claset(), |
19b9f92ca503
working with weak LeadsTo in guarantees precondition\!
paulson
parents:
8067
diff
changeset
|
669 |
simpset() addsimps [project_set_reachable_extend_eq RS sym])); |
19b9f92ca503
working with weak LeadsTo in guarantees precondition\!
paulson
parents:
8067
diff
changeset
|
670 |
qed "project_LeadsETo_I"; |
19b9f92ca503
working with weak LeadsTo in guarantees precondition\!
paulson
parents:
8067
diff
changeset
|
671 |
|
19b9f92ca503
working with weak LeadsTo in guarantees precondition\!
paulson
parents:
8067
diff
changeset
|
672 |
Goalw [projecting_def] |
19b9f92ca503
working with weak LeadsTo in guarantees precondition\!
paulson
parents:
8067
diff
changeset
|
673 |
"projecting (%G. UNIV) h F \ |
19b9f92ca503
working with weak LeadsTo in guarantees precondition\!
paulson
parents:
8067
diff
changeset
|
674 |
\ (extend_set h A leadsTo[givenBy f] extend_set h B) \ |
19b9f92ca503
working with weak LeadsTo in guarantees precondition\!
paulson
parents:
8067
diff
changeset
|
675 |
\ (A leadsTo B)"; |
19b9f92ca503
working with weak LeadsTo in guarantees precondition\!
paulson
parents:
8067
diff
changeset
|
676 |
by (force_tac (claset() addDs [project_leadsETo_I], simpset()) 1); |
19b9f92ca503
working with weak LeadsTo in guarantees precondition\!
paulson
parents:
8067
diff
changeset
|
677 |
qed "projecting_leadsTo"; |
19b9f92ca503
working with weak LeadsTo in guarantees precondition\!
paulson
parents:
8067
diff
changeset
|
678 |
|
19b9f92ca503
working with weak LeadsTo in guarantees precondition\!
paulson
parents:
8067
diff
changeset
|
679 |
Goalw [projecting_def] |
19b9f92ca503
working with weak LeadsTo in guarantees precondition\!
paulson
parents:
8067
diff
changeset
|
680 |
"projecting (%G. reachable (extend h F Join G)) h F \ |
19b9f92ca503
working with weak LeadsTo in guarantees precondition\!
paulson
parents:
8067
diff
changeset
|
681 |
\ (extend_set h A LeadsTo[givenBy f] extend_set h B) \ |
19b9f92ca503
working with weak LeadsTo in guarantees precondition\!
paulson
parents:
8067
diff
changeset
|
682 |
\ (A LeadsTo B)"; |
19b9f92ca503
working with weak LeadsTo in guarantees precondition\!
paulson
parents:
8067
diff
changeset
|
683 |
by (force_tac (claset() addDs [project_LeadsETo_I], simpset()) 1); |
19b9f92ca503
working with weak LeadsTo in guarantees precondition\!
paulson
parents:
8067
diff
changeset
|
684 |
qed "projecting_LeadsTo"; |
19b9f92ca503
working with weak LeadsTo in guarantees precondition\!
paulson
parents:
8067
diff
changeset
|
685 |
|
8044 | 686 |
Close_locale "Extend"; |
687 |
||
688 |