author | paulson |
Fri, 16 Jun 2000 13:39:21 +0200 | |
changeset 9083 | b36787a56a1f |
parent 8948 | b797cfa3548d |
child 9190 | b86ff604729f |
permissions | -rw-r--r-- |
6297 | 1 |
(* Title: HOL/UNITY/Extend.ML |
2 |
ID: $Id$ |
|
3 |
Author: Lawrence C Paulson, Cambridge University Computer Laboratory |
|
4 |
Copyright 1999 University of Cambridge |
|
5 |
||
6 |
Extending of state sets |
|
7 |
function f (forget) maps the extended state to the original state |
|
8 |
function g (forgotten) maps the extended state to the "extending part" |
|
7482 | 9 |
*) |
7362
f08fade5ea0d
new laws; changed "guar" back to "guarantees" (sorry)
paulson
parents:
7341
diff
changeset
|
10 |
|
7482 | 11 |
(** These we prove OUTSIDE the locale. **) |
12 |
||
8948
b797cfa3548d
restructuring: LessThan.ML mostly moved to HOL/SetInterval.ML
paulson
parents:
8251
diff
changeset
|
13 |
|
b797cfa3548d
restructuring: LessThan.ML mostly moved to HOL/SetInterval.ML
paulson
parents:
8251
diff
changeset
|
14 |
(*** Restrict [MOVE to Relation.thy?] ***) |
b797cfa3548d
restructuring: LessThan.ML mostly moved to HOL/SetInterval.ML
paulson
parents:
8251
diff
changeset
|
15 |
|
b797cfa3548d
restructuring: LessThan.ML mostly moved to HOL/SetInterval.ML
paulson
parents:
8251
diff
changeset
|
16 |
Goalw [Restrict_def] "((x,y): Restrict A r) = ((x,y): r & x: A)"; |
b797cfa3548d
restructuring: LessThan.ML mostly moved to HOL/SetInterval.ML
paulson
parents:
8251
diff
changeset
|
17 |
by (Blast_tac 1); |
b797cfa3548d
restructuring: LessThan.ML mostly moved to HOL/SetInterval.ML
paulson
parents:
8251
diff
changeset
|
18 |
qed "Restrict_iff"; |
b797cfa3548d
restructuring: LessThan.ML mostly moved to HOL/SetInterval.ML
paulson
parents:
8251
diff
changeset
|
19 |
AddIffs [Restrict_iff]; |
b797cfa3548d
restructuring: LessThan.ML mostly moved to HOL/SetInterval.ML
paulson
parents:
8251
diff
changeset
|
20 |
|
b797cfa3548d
restructuring: LessThan.ML mostly moved to HOL/SetInterval.ML
paulson
parents:
8251
diff
changeset
|
21 |
Goal "Restrict UNIV = id"; |
b797cfa3548d
restructuring: LessThan.ML mostly moved to HOL/SetInterval.ML
paulson
parents:
8251
diff
changeset
|
22 |
by (rtac ext 1); |
b797cfa3548d
restructuring: LessThan.ML mostly moved to HOL/SetInterval.ML
paulson
parents:
8251
diff
changeset
|
23 |
by (auto_tac (claset(), simpset() addsimps [Restrict_def])); |
b797cfa3548d
restructuring: LessThan.ML mostly moved to HOL/SetInterval.ML
paulson
parents:
8251
diff
changeset
|
24 |
qed "Restrict_UNIV"; |
b797cfa3548d
restructuring: LessThan.ML mostly moved to HOL/SetInterval.ML
paulson
parents:
8251
diff
changeset
|
25 |
Addsimps [Restrict_UNIV]; |
b797cfa3548d
restructuring: LessThan.ML mostly moved to HOL/SetInterval.ML
paulson
parents:
8251
diff
changeset
|
26 |
|
b797cfa3548d
restructuring: LessThan.ML mostly moved to HOL/SetInterval.ML
paulson
parents:
8251
diff
changeset
|
27 |
Goal "Restrict {} r = {}"; |
b797cfa3548d
restructuring: LessThan.ML mostly moved to HOL/SetInterval.ML
paulson
parents:
8251
diff
changeset
|
28 |
by (auto_tac (claset(), simpset() addsimps [Restrict_def])); |
b797cfa3548d
restructuring: LessThan.ML mostly moved to HOL/SetInterval.ML
paulson
parents:
8251
diff
changeset
|
29 |
qed "Restrict_empty"; |
b797cfa3548d
restructuring: LessThan.ML mostly moved to HOL/SetInterval.ML
paulson
parents:
8251
diff
changeset
|
30 |
Addsimps [Restrict_empty]; |
b797cfa3548d
restructuring: LessThan.ML mostly moved to HOL/SetInterval.ML
paulson
parents:
8251
diff
changeset
|
31 |
|
b797cfa3548d
restructuring: LessThan.ML mostly moved to HOL/SetInterval.ML
paulson
parents:
8251
diff
changeset
|
32 |
Goalw [Restrict_def] "Restrict A (Restrict B r) = Restrict (A Int B) r"; |
b797cfa3548d
restructuring: LessThan.ML mostly moved to HOL/SetInterval.ML
paulson
parents:
8251
diff
changeset
|
33 |
by (Blast_tac 1); |
b797cfa3548d
restructuring: LessThan.ML mostly moved to HOL/SetInterval.ML
paulson
parents:
8251
diff
changeset
|
34 |
qed "Restrict_Int"; |
b797cfa3548d
restructuring: LessThan.ML mostly moved to HOL/SetInterval.ML
paulson
parents:
8251
diff
changeset
|
35 |
Addsimps [Restrict_Int]; |
b797cfa3548d
restructuring: LessThan.ML mostly moved to HOL/SetInterval.ML
paulson
parents:
8251
diff
changeset
|
36 |
|
b797cfa3548d
restructuring: LessThan.ML mostly moved to HOL/SetInterval.ML
paulson
parents:
8251
diff
changeset
|
37 |
Goalw [Restrict_def] "Domain r <= A ==> Restrict A r = r"; |
b797cfa3548d
restructuring: LessThan.ML mostly moved to HOL/SetInterval.ML
paulson
parents:
8251
diff
changeset
|
38 |
by Auto_tac; |
b797cfa3548d
restructuring: LessThan.ML mostly moved to HOL/SetInterval.ML
paulson
parents:
8251
diff
changeset
|
39 |
qed "Restrict_triv"; |
b797cfa3548d
restructuring: LessThan.ML mostly moved to HOL/SetInterval.ML
paulson
parents:
8251
diff
changeset
|
40 |
|
b797cfa3548d
restructuring: LessThan.ML mostly moved to HOL/SetInterval.ML
paulson
parents:
8251
diff
changeset
|
41 |
Goalw [Restrict_def] "Restrict A r <= r"; |
b797cfa3548d
restructuring: LessThan.ML mostly moved to HOL/SetInterval.ML
paulson
parents:
8251
diff
changeset
|
42 |
by Auto_tac; |
b797cfa3548d
restructuring: LessThan.ML mostly moved to HOL/SetInterval.ML
paulson
parents:
8251
diff
changeset
|
43 |
qed "Restrict_subset"; |
b797cfa3548d
restructuring: LessThan.ML mostly moved to HOL/SetInterval.ML
paulson
parents:
8251
diff
changeset
|
44 |
|
b797cfa3548d
restructuring: LessThan.ML mostly moved to HOL/SetInterval.ML
paulson
parents:
8251
diff
changeset
|
45 |
Goalw [Restrict_def] |
b797cfa3548d
restructuring: LessThan.ML mostly moved to HOL/SetInterval.ML
paulson
parents:
8251
diff
changeset
|
46 |
"[| A <= B; Restrict B r = Restrict B s |] \ |
b797cfa3548d
restructuring: LessThan.ML mostly moved to HOL/SetInterval.ML
paulson
parents:
8251
diff
changeset
|
47 |
\ ==> Restrict A r = Restrict A s"; |
b797cfa3548d
restructuring: LessThan.ML mostly moved to HOL/SetInterval.ML
paulson
parents:
8251
diff
changeset
|
48 |
by (blast_tac (claset() addSEs [equalityE]) 1); |
b797cfa3548d
restructuring: LessThan.ML mostly moved to HOL/SetInterval.ML
paulson
parents:
8251
diff
changeset
|
49 |
qed "Restrict_eq_mono"; |
b797cfa3548d
restructuring: LessThan.ML mostly moved to HOL/SetInterval.ML
paulson
parents:
8251
diff
changeset
|
50 |
|
b797cfa3548d
restructuring: LessThan.ML mostly moved to HOL/SetInterval.ML
paulson
parents:
8251
diff
changeset
|
51 |
Goalw [Restrict_def, image_def] |
b797cfa3548d
restructuring: LessThan.ML mostly moved to HOL/SetInterval.ML
paulson
parents:
8251
diff
changeset
|
52 |
"[| s : RR; Restrict A r = Restrict A s |] \ |
b797cfa3548d
restructuring: LessThan.ML mostly moved to HOL/SetInterval.ML
paulson
parents:
8251
diff
changeset
|
53 |
\ ==> Restrict A r : Restrict A `` RR"; |
b797cfa3548d
restructuring: LessThan.ML mostly moved to HOL/SetInterval.ML
paulson
parents:
8251
diff
changeset
|
54 |
by Auto_tac; |
b797cfa3548d
restructuring: LessThan.ML mostly moved to HOL/SetInterval.ML
paulson
parents:
8251
diff
changeset
|
55 |
qed "Restrict_imageI"; |
b797cfa3548d
restructuring: LessThan.ML mostly moved to HOL/SetInterval.ML
paulson
parents:
8251
diff
changeset
|
56 |
|
b797cfa3548d
restructuring: LessThan.ML mostly moved to HOL/SetInterval.ML
paulson
parents:
8251
diff
changeset
|
57 |
Goal "Domain (Restrict A r) = A Int Domain r"; |
b797cfa3548d
restructuring: LessThan.ML mostly moved to HOL/SetInterval.ML
paulson
parents:
8251
diff
changeset
|
58 |
by (Blast_tac 1); |
b797cfa3548d
restructuring: LessThan.ML mostly moved to HOL/SetInterval.ML
paulson
parents:
8251
diff
changeset
|
59 |
qed "Domain_Restrict"; |
b797cfa3548d
restructuring: LessThan.ML mostly moved to HOL/SetInterval.ML
paulson
parents:
8251
diff
changeset
|
60 |
|
b797cfa3548d
restructuring: LessThan.ML mostly moved to HOL/SetInterval.ML
paulson
parents:
8251
diff
changeset
|
61 |
Goal "(Restrict A r) ^^ B = r ^^ (A Int B)"; |
b797cfa3548d
restructuring: LessThan.ML mostly moved to HOL/SetInterval.ML
paulson
parents:
8251
diff
changeset
|
62 |
by (Blast_tac 1); |
b797cfa3548d
restructuring: LessThan.ML mostly moved to HOL/SetInterval.ML
paulson
parents:
8251
diff
changeset
|
63 |
qed "Image_Restrict"; |
b797cfa3548d
restructuring: LessThan.ML mostly moved to HOL/SetInterval.ML
paulson
parents:
8251
diff
changeset
|
64 |
|
b797cfa3548d
restructuring: LessThan.ML mostly moved to HOL/SetInterval.ML
paulson
parents:
8251
diff
changeset
|
65 |
Addsimps [Domain_Restrict, Image_Restrict]; |
b797cfa3548d
restructuring: LessThan.ML mostly moved to HOL/SetInterval.ML
paulson
parents:
8251
diff
changeset
|
66 |
|
b797cfa3548d
restructuring: LessThan.ML mostly moved to HOL/SetInterval.ML
paulson
parents:
8251
diff
changeset
|
67 |
|
8251
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
68 |
Goal "f Id = Id ==> insert Id (f``Acts F) = f `` Acts F"; |
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
69 |
by (blast_tac (claset() addIs [sym RS image_eqI]) 1); |
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
70 |
qed "insert_Id_image_Acts"; |
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
71 |
|
7482 | 72 |
(*Possibly easier than reasoning about "inv h"*) |
73 |
val [surj_h,prem] = |
|
74 |
Goalw [good_map_def] |
|
75 |
"[| surj h; !! x x' y y'. h(x,y) = h(x',y') ==> x=x' |] ==> good_map h"; |
|
76 |
by (safe_tac (claset() addSIs [surj_h])); |
|
77 |
by (rtac prem 1); |
|
78 |
by (stac (surjective_pairing RS sym) 1); |
|
79 |
by (stac (surj_h RS surj_f_inv_f) 1); |
|
80 |
by (rtac refl 1); |
|
81 |
qed "good_mapI"; |
|
82 |
||
83 |
Goalw [good_map_def] "good_map h ==> surj h"; |
|
84 |
by Auto_tac; |
|
85 |
qed "good_map_is_surj"; |
|
86 |
||
87 |
(*A convenient way of finding a closed form for inv h*) |
|
88 |
val [surj,prem] = Goalw [inv_def] |
|
89 |
"[| surj h; !! x y. g (h(x,y)) = x |] ==> fst (inv h z) = g z"; |
|
90 |
by (res_inst_tac [("y1", "z")] (surj RS surjD RS exE) 1); |
|
7499 | 91 |
by (rtac selectI2 1); |
7482 | 92 |
by (dres_inst_tac [("f", "g")] arg_cong 2); |
93 |
by (auto_tac (claset(), simpset() addsimps [prem])); |
|
94 |
qed "fst_inv_equalityI"; |
|
95 |
||
6297 | 96 |
|
97 |
Open_locale "Extend"; |
|
98 |
||
99 |
val slice_def = thm "slice_def"; |
|
100 |
||
101 |
(*** Trivial properties of f, g, h ***) |
|
102 |
||
7482 | 103 |
val good_h = rewrite_rule [good_map_def] (thm "good_h"); |
104 |
val surj_h = good_h RS conjunct1; |
|
6297 | 105 |
|
106 |
val f_def = thm "f_def"; |
|
107 |
val g_def = thm "g_def"; |
|
108 |
||
109 |
Goal "f(h(x,y)) = x"; |
|
7482 | 110 |
by (simp_tac (simpset() addsimps [f_def, good_h RS conjunct2]) 1); |
6297 | 111 |
qed "f_h_eq"; |
112 |
Addsimps [f_h_eq]; |
|
113 |
||
7482 | 114 |
Goal "h(x,y) = h(x',y') ==> x=x'"; |
115 |
by (dres_inst_tac [("f", "fst o inv h")] arg_cong 1); |
|
116 |
(*FIXME: If locales worked properly we could put just "f" above*) |
|
117 |
by (full_simp_tac (simpset() addsimps [f_def, good_h RS conjunct2]) 1); |
|
118 |
qed "h_inject1"; |
|
7878
43b03d412b82
working version with localTo[C] instead of localTo
paulson
parents:
7826
diff
changeset
|
119 |
AddDs [h_inject1]; |
6297 | 120 |
|
121 |
Goal "h(f z, g z) = z"; |
|
7482 | 122 |
by (simp_tac (simpset() addsimps [f_def, g_def, surjective_pairing RS sym, |
123 |
surj_h RS surj_f_inv_f]) 1); |
|
6297 | 124 |
qed "h_f_g_eq"; |
125 |
||
7878
43b03d412b82
working version with localTo[C] instead of localTo
paulson
parents:
7826
diff
changeset
|
126 |
|
43b03d412b82
working version with localTo[C] instead of localTo
paulson
parents:
7826
diff
changeset
|
127 |
(** A sequence of proof steps borrowed from Provers/split_paired_all.ML **) |
43b03d412b82
working version with localTo[C] instead of localTo
paulson
parents:
7826
diff
changeset
|
128 |
|
43b03d412b82
working version with localTo[C] instead of localTo
paulson
parents:
7826
diff
changeset
|
129 |
val cT = TFree ("'c", ["term"]); |
43b03d412b82
working version with localTo[C] instead of localTo
paulson
parents:
7826
diff
changeset
|
130 |
|
43b03d412b82
working version with localTo[C] instead of localTo
paulson
parents:
7826
diff
changeset
|
131 |
(* "PROP P x == PROP P (h (f x, g x))" *) |
43b03d412b82
working version with localTo[C] instead of localTo
paulson
parents:
7826
diff
changeset
|
132 |
val lemma1 = Thm.combination |
43b03d412b82
working version with localTo[C] instead of localTo
paulson
parents:
7826
diff
changeset
|
133 |
(Thm.reflexive (cterm_of (sign_of thy) (Free ("P", cT --> propT)))) |
43b03d412b82
working version with localTo[C] instead of localTo
paulson
parents:
7826
diff
changeset
|
134 |
(Drule.unvarify (h_f_g_eq RS sym RS eq_reflection)); |
43b03d412b82
working version with localTo[C] instead of localTo
paulson
parents:
7826
diff
changeset
|
135 |
|
43b03d412b82
working version with localTo[C] instead of localTo
paulson
parents:
7826
diff
changeset
|
136 |
val prems = Goalw [lemma1] "(!!u y. PROP P (h (u, y))) ==> PROP P x"; |
43b03d412b82
working version with localTo[C] instead of localTo
paulson
parents:
7826
diff
changeset
|
137 |
by (resolve_tac prems 1); |
43b03d412b82
working version with localTo[C] instead of localTo
paulson
parents:
7826
diff
changeset
|
138 |
val lemma2 = result(); |
43b03d412b82
working version with localTo[C] instead of localTo
paulson
parents:
7826
diff
changeset
|
139 |
|
43b03d412b82
working version with localTo[C] instead of localTo
paulson
parents:
7826
diff
changeset
|
140 |
val prems = Goal "(!!u y. PROP P (h (u, y))) ==> (!!z. PROP P z)"; |
43b03d412b82
working version with localTo[C] instead of localTo
paulson
parents:
7826
diff
changeset
|
141 |
by (rtac lemma2 1); |
43b03d412b82
working version with localTo[C] instead of localTo
paulson
parents:
7826
diff
changeset
|
142 |
by (resolve_tac prems 1); |
43b03d412b82
working version with localTo[C] instead of localTo
paulson
parents:
7826
diff
changeset
|
143 |
val lemma3 = result(); |
43b03d412b82
working version with localTo[C] instead of localTo
paulson
parents:
7826
diff
changeset
|
144 |
|
43b03d412b82
working version with localTo[C] instead of localTo
paulson
parents:
7826
diff
changeset
|
145 |
val prems = Goal "(!!z. PROP P z) ==> (!!u y. PROP P (h (u, y)))"; |
43b03d412b82
working version with localTo[C] instead of localTo
paulson
parents:
7826
diff
changeset
|
146 |
(*not needed for proof, but prevents generalization over h, 'c, etc.*) |
43b03d412b82
working version with localTo[C] instead of localTo
paulson
parents:
7826
diff
changeset
|
147 |
by (cut_facts_tac [surj_h] 1); |
43b03d412b82
working version with localTo[C] instead of localTo
paulson
parents:
7826
diff
changeset
|
148 |
by (resolve_tac prems 1); |
43b03d412b82
working version with localTo[C] instead of localTo
paulson
parents:
7826
diff
changeset
|
149 |
val lemma4 = result(); |
43b03d412b82
working version with localTo[C] instead of localTo
paulson
parents:
7826
diff
changeset
|
150 |
|
43b03d412b82
working version with localTo[C] instead of localTo
paulson
parents:
7826
diff
changeset
|
151 |
val split_extended_all = Thm.equal_intr lemma4 lemma3; |
43b03d412b82
working version with localTo[C] instead of localTo
paulson
parents:
7826
diff
changeset
|
152 |
|
43b03d412b82
working version with localTo[C] instead of localTo
paulson
parents:
7826
diff
changeset
|
153 |
|
6297 | 154 |
(*** extend_set: basic properties ***) |
155 |
||
8069
19b9f92ca503
working with weak LeadsTo in guarantees precondition\!
paulson
parents:
8055
diff
changeset
|
156 |
Goal "(x : project_set h C) = (EX y. h(x,y) : C)"; |
19b9f92ca503
working with weak LeadsTo in guarantees precondition\!
paulson
parents:
8055
diff
changeset
|
157 |
by (simp_tac (simpset() addsimps [project_set_def]) 1); |
19b9f92ca503
working with weak LeadsTo in guarantees precondition\!
paulson
parents:
8055
diff
changeset
|
158 |
qed "project_set_iff"; |
19b9f92ca503
working with weak LeadsTo in guarantees precondition\!
paulson
parents:
8055
diff
changeset
|
159 |
|
19b9f92ca503
working with weak LeadsTo in guarantees precondition\!
paulson
parents:
8055
diff
changeset
|
160 |
AddIffs [project_set_iff]; |
19b9f92ca503
working with weak LeadsTo in guarantees precondition\!
paulson
parents:
8055
diff
changeset
|
161 |
|
7594
8a188ef6545e
working version with co-guarantees-leadsto results
paulson
parents:
7546
diff
changeset
|
162 |
Goalw [extend_set_def] "A<=B ==> extend_set h A <= extend_set h B"; |
8a188ef6545e
working version with co-guarantees-leadsto results
paulson
parents:
7546
diff
changeset
|
163 |
by (Blast_tac 1); |
8a188ef6545e
working version with co-guarantees-leadsto results
paulson
parents:
7546
diff
changeset
|
164 |
qed "extend_set_mono"; |
8a188ef6545e
working version with co-guarantees-leadsto results
paulson
parents:
7546
diff
changeset
|
165 |
|
7826
c6a8b73b6c2a
working shapshot with "projecting" and "extending"
paulson
parents:
7689
diff
changeset
|
166 |
Goalw [extend_set_def] "z : extend_set h A = (f z : A)"; |
7341 | 167 |
by (force_tac (claset() addIs [h_f_g_eq RS sym], simpset()) 1); |
6297 | 168 |
qed "mem_extend_set_iff"; |
169 |
||
8069
19b9f92ca503
working with weak LeadsTo in guarantees precondition\!
paulson
parents:
8055
diff
changeset
|
170 |
AddIffs [mem_extend_set_iff]; |
19b9f92ca503
working with weak LeadsTo in guarantees precondition\!
paulson
parents:
8055
diff
changeset
|
171 |
|
19b9f92ca503
working with weak LeadsTo in guarantees precondition\!
paulson
parents:
8055
diff
changeset
|
172 |
Goalw [extend_set_def] "(extend_set h A <= extend_set h B) = (A <= B)"; |
7826
c6a8b73b6c2a
working shapshot with "projecting" and "extending"
paulson
parents:
7689
diff
changeset
|
173 |
by (Force_tac 1); |
c6a8b73b6c2a
working shapshot with "projecting" and "extending"
paulson
parents:
7689
diff
changeset
|
174 |
qed "extend_set_strict_mono"; |
c6a8b73b6c2a
working shapshot with "projecting" and "extending"
paulson
parents:
7689
diff
changeset
|
175 |
AddIffs [extend_set_strict_mono]; |
c6a8b73b6c2a
working shapshot with "projecting" and "extending"
paulson
parents:
7689
diff
changeset
|
176 |
|
8251
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
177 |
Goalw [extend_set_def] "extend_set h {} = {}"; |
7378 | 178 |
by Auto_tac; |
8251
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
179 |
qed "extend_set_empty"; |
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
180 |
Addsimps [extend_set_empty]; |
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
181 |
|
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
182 |
Goal "extend_set h {s. P s} = {s. P (f s)}"; |
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
183 |
by Auto_tac; |
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
184 |
qed "extend_set_eq_Collect"; |
7378 | 185 |
|
7594
8a188ef6545e
working version with co-guarantees-leadsto results
paulson
parents:
7546
diff
changeset
|
186 |
Goal "extend_set h {x} = {s. f s = x}"; |
8a188ef6545e
working version with co-guarantees-leadsto results
paulson
parents:
7546
diff
changeset
|
187 |
by Auto_tac; |
8a188ef6545e
working version with co-guarantees-leadsto results
paulson
parents:
7546
diff
changeset
|
188 |
qed "extend_set_sing"; |
8a188ef6545e
working version with co-guarantees-leadsto results
paulson
parents:
7546
diff
changeset
|
189 |
|
8251
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
190 |
Goalw [extend_set_def] "project_set h (extend_set h C) = C"; |
7341 | 191 |
by Auto_tac; |
192 |
qed "extend_set_inverse"; |
|
193 |
Addsimps [extend_set_inverse]; |
|
194 |
||
8251
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
195 |
Goalw [extend_set_def] "C <= extend_set h (project_set h C)"; |
7947 | 196 |
by (auto_tac (claset(), |
197 |
simpset() addsimps [split_extended_all])); |
|
198 |
by (Blast_tac 1); |
|
199 |
qed "extend_set_project_set"; |
|
200 |
||
6297 | 201 |
Goal "inj (extend_set h)"; |
7341 | 202 |
by (rtac inj_on_inverseI 1); |
203 |
by (rtac extend_set_inverse 1); |
|
6297 | 204 |
qed "inj_extend_set"; |
205 |
||
7689 | 206 |
Goalw [extend_set_def] "extend_set h UNIV = UNIV"; |
7878
43b03d412b82
working version with localTo[C] instead of localTo
paulson
parents:
7826
diff
changeset
|
207 |
by (auto_tac (claset(), |
43b03d412b82
working version with localTo[C] instead of localTo
paulson
parents:
7826
diff
changeset
|
208 |
simpset() addsimps [split_extended_all])); |
7689 | 209 |
qed "extend_set_UNIV_eq"; |
210 |
Addsimps [standard extend_set_UNIV_eq]; |
|
211 |
||
7482 | 212 |
(*** project_set: basic properties ***) |
213 |
||
214 |
(*project_set is simply image!*) |
|
8069
19b9f92ca503
working with weak LeadsTo in guarantees precondition\!
paulson
parents:
8055
diff
changeset
|
215 |
Goal "project_set h C = f `` C"; |
7878
43b03d412b82
working version with localTo[C] instead of localTo
paulson
parents:
7826
diff
changeset
|
216 |
by (auto_tac (claset() addIs [f_h_eq RS sym], |
43b03d412b82
working version with localTo[C] instead of localTo
paulson
parents:
7826
diff
changeset
|
217 |
simpset() addsimps [split_extended_all])); |
7482 | 218 |
qed "project_set_eq"; |
219 |
||
220 |
(*Converse appears to fail*) |
|
8069
19b9f92ca503
working with weak LeadsTo in guarantees precondition\!
paulson
parents:
8055
diff
changeset
|
221 |
Goal "!!z. z : C ==> f z : project_set h C"; |
7878
43b03d412b82
working version with localTo[C] instead of localTo
paulson
parents:
7826
diff
changeset
|
222 |
by (auto_tac (claset(), |
43b03d412b82
working version with localTo[C] instead of localTo
paulson
parents:
7826
diff
changeset
|
223 |
simpset() addsimps [split_extended_all])); |
7482 | 224 |
qed "project_set_I"; |
225 |
||
226 |
||
227 |
(*** More laws ***) |
|
228 |
||
7341 | 229 |
(*Because A and B could differ on the "other" part of the state, |
8055
bb15396278fb
abolition of localTo: instead "guarantees" has local vars as extra argument
paulson
parents:
8041
diff
changeset
|
230 |
cannot generalize to |
7341 | 231 |
project_set h (A Int B) = project_set h A Int project_set h B |
232 |
*) |
|
8069
19b9f92ca503
working with weak LeadsTo in guarantees precondition\!
paulson
parents:
8055
diff
changeset
|
233 |
Goal "project_set h ((extend_set h A) Int B) = A Int (project_set h B)"; |
7341 | 234 |
by Auto_tac; |
235 |
qed "project_set_extend_set_Int"; |
|
236 |
||
8069
19b9f92ca503
working with weak LeadsTo in guarantees precondition\!
paulson
parents:
8055
diff
changeset
|
237 |
Goal "project_set h (A Int B) <= (project_set h A) Int (project_set h B)"; |
8055
bb15396278fb
abolition of localTo: instead "guarantees" has local vars as extra argument
paulson
parents:
8041
diff
changeset
|
238 |
by Auto_tac; |
bb15396278fb
abolition of localTo: instead "guarantees" has local vars as extra argument
paulson
parents:
8041
diff
changeset
|
239 |
qed "project_set_Int_subset"; |
bb15396278fb
abolition of localTo: instead "guarantees" has local vars as extra argument
paulson
parents:
8041
diff
changeset
|
240 |
|
7341 | 241 |
Goal "extend_set h (A Un B) = extend_set h A Un extend_set h B"; |
6297 | 242 |
by Auto_tac; |
243 |
qed "extend_set_Un_distrib"; |
|
244 |
||
7341 | 245 |
Goal "extend_set h (A Int B) = extend_set h A Int extend_set h B"; |
6297 | 246 |
by Auto_tac; |
247 |
qed "extend_set_Int_distrib"; |
|
248 |
||
7341 | 249 |
Goal "extend_set h (INTER A B) = (INT x:A. extend_set h (B x))"; |
250 |
by Auto_tac; |
|
6834
44da4a2a9ef3
renamed UNION_... to UN_..., INTER_... to INT_... (to fit the convention)
paulson
parents:
6822
diff
changeset
|
251 |
qed "extend_set_INT_distrib"; |
6647 | 252 |
|
7341 | 253 |
Goal "extend_set h (A - B) = extend_set h A - extend_set h B"; |
6297 | 254 |
by Auto_tac; |
255 |
qed "extend_set_Diff_distrib"; |
|
256 |
||
7341 | 257 |
Goal "extend_set h (Union A) = (UN X:A. extend_set h X)"; |
6297 | 258 |
by (Blast_tac 1); |
259 |
qed "extend_set_Union"; |
|
260 |
||
7341 | 261 |
Goalw [extend_set_def] "(extend_set h A <= - extend_set h B) = (A <= - B)"; |
6297 | 262 |
by Auto_tac; |
263 |
qed "extend_set_subset_Compl_eq"; |
|
264 |
||
7341 | 265 |
|
6297 | 266 |
(*** extend_act ***) |
267 |
||
8216 | 268 |
(*Can't strengthen it to |
269 |
((h(s,y), h(s',y')) : extend_act h act) = ((s, s') : act & y=y') |
|
270 |
because h doesn't have to be injective in the 2nd argument*) |
|
6297 | 271 |
Goalw [extend_act_def] |
272 |
"((h(s,y), h(s',y)) : extend_act h act) = ((s, s') : act)"; |
|
273 |
by Auto_tac; |
|
274 |
qed "mem_extend_act_iff"; |
|
275 |
AddIffs [mem_extend_act_iff]; |
|
276 |
||
7878
43b03d412b82
working version with localTo[C] instead of localTo
paulson
parents:
7826
diff
changeset
|
277 |
(*Converse fails: (z,z') would include actions that changed the g-part*) |
7341 | 278 |
Goalw [extend_act_def] |
279 |
"(z, z') : extend_act h act ==> (f z, f z') : act"; |
|
280 |
by Auto_tac; |
|
281 |
qed "extend_act_D"; |
|
282 |
||
8069
19b9f92ca503
working with weak LeadsTo in guarantees precondition\!
paulson
parents:
8055
diff
changeset
|
283 |
Goalw [extend_act_def, project_act_def] |
8055
bb15396278fb
abolition of localTo: instead "guarantees" has local vars as extra argument
paulson
parents:
8041
diff
changeset
|
284 |
"project_act h (extend_act h act) = act"; |
bb15396278fb
abolition of localTo: instead "guarantees" has local vars as extra argument
paulson
parents:
8041
diff
changeset
|
285 |
by (Blast_tac 1); |
bb15396278fb
abolition of localTo: instead "guarantees" has local vars as extra argument
paulson
parents:
8041
diff
changeset
|
286 |
qed "project_act_extend_act"; |
bb15396278fb
abolition of localTo: instead "guarantees" has local vars as extra argument
paulson
parents:
8041
diff
changeset
|
287 |
|
8069
19b9f92ca503
working with weak LeadsTo in guarantees precondition\!
paulson
parents:
8055
diff
changeset
|
288 |
Goalw [extend_act_def, project_act_def] |
7878
43b03d412b82
working version with localTo[C] instead of localTo
paulson
parents:
7826
diff
changeset
|
289 |
"project_act h (Restrict C (extend_act h act)) = \ |
43b03d412b82
working version with localTo[C] instead of localTo
paulson
parents:
7826
diff
changeset
|
290 |
\ Restrict (project_set h C) act"; |
43b03d412b82
working version with localTo[C] instead of localTo
paulson
parents:
7826
diff
changeset
|
291 |
by (Blast_tac 1); |
43b03d412b82
working version with localTo[C] instead of localTo
paulson
parents:
7826
diff
changeset
|
292 |
qed "project_act_extend_act_restrict"; |
43b03d412b82
working version with localTo[C] instead of localTo
paulson
parents:
7826
diff
changeset
|
293 |
Addsimps [project_act_extend_act_restrict]; |
43b03d412b82
working version with localTo[C] instead of localTo
paulson
parents:
7826
diff
changeset
|
294 |
|
7537 | 295 |
(*Premise is still undesirably strong, since Domain act can include |
296 |
non-reachable states, but it seems necessary for this result.*) |
|
7878
43b03d412b82
working version with localTo[C] instead of localTo
paulson
parents:
7826
diff
changeset
|
297 |
Goal "Domain act <= project_set h C \ |
43b03d412b82
working version with localTo[C] instead of localTo
paulson
parents:
7826
diff
changeset
|
298 |
\ ==> project_act h (Restrict C (extend_act h act)) = act"; |
43b03d412b82
working version with localTo[C] instead of localTo
paulson
parents:
7826
diff
changeset
|
299 |
by (asm_simp_tac (simpset() addsimps [Restrict_triv]) 1); |
7341 | 300 |
qed "extend_act_inverse"; |
301 |
||
7826
c6a8b73b6c2a
working shapshot with "projecting" and "extending"
paulson
parents:
7689
diff
changeset
|
302 |
Goalw [extend_act_def, project_act_def] |
7878
43b03d412b82
working version with localTo[C] instead of localTo
paulson
parents:
7826
diff
changeset
|
303 |
"act' <= extend_act h act ==> project_act h act' <= act"; |
7826
c6a8b73b6c2a
working shapshot with "projecting" and "extending"
paulson
parents:
7689
diff
changeset
|
304 |
by (Force_tac 1); |
c6a8b73b6c2a
working shapshot with "projecting" and "extending"
paulson
parents:
7689
diff
changeset
|
305 |
qed "subset_extend_act_D"; |
c6a8b73b6c2a
working shapshot with "projecting" and "extending"
paulson
parents:
7689
diff
changeset
|
306 |
|
6297 | 307 |
Goal "inj (extend_act h)"; |
7341 | 308 |
by (rtac inj_on_inverseI 1); |
309 |
by (rtac extend_act_inverse 1); |
|
8069
19b9f92ca503
working with weak LeadsTo in guarantees precondition\!
paulson
parents:
8055
diff
changeset
|
310 |
by (Force_tac 1); |
6297 | 311 |
qed "inj_extend_act"; |
312 |
||
313 |
Goalw [extend_set_def, extend_act_def] |
|
314 |
"extend_act h act ^^ (extend_set h A) = extend_set h (act ^^ A)"; |
|
315 |
by (Force_tac 1); |
|
316 |
qed "extend_act_Image"; |
|
317 |
Addsimps [extend_act_Image]; |
|
318 |
||
7826
c6a8b73b6c2a
working shapshot with "projecting" and "extending"
paulson
parents:
7689
diff
changeset
|
319 |
Goalw [extend_act_def] "(extend_act h act' <= extend_act h act) = (act'<=act)"; |
c6a8b73b6c2a
working shapshot with "projecting" and "extending"
paulson
parents:
7689
diff
changeset
|
320 |
by Auto_tac; |
c6a8b73b6c2a
working shapshot with "projecting" and "extending"
paulson
parents:
7689
diff
changeset
|
321 |
qed "extend_act_strict_mono"; |
c6a8b73b6c2a
working shapshot with "projecting" and "extending"
paulson
parents:
7689
diff
changeset
|
322 |
|
c6a8b73b6c2a
working shapshot with "projecting" and "extending"
paulson
parents:
7689
diff
changeset
|
323 |
AddIffs [extend_act_strict_mono, inj_extend_act RS inj_eq]; |
c6a8b73b6c2a
working shapshot with "projecting" and "extending"
paulson
parents:
7689
diff
changeset
|
324 |
(*The latter theorem is (extend_act h act' = extend_act h act) = (act'=act) *) |
6297 | 325 |
|
326 |
Goalw [extend_set_def, extend_act_def] |
|
327 |
"Domain (extend_act h act) = extend_set h (Domain act)"; |
|
328 |
by (Force_tac 1); |
|
329 |
qed "Domain_extend_act"; |
|
330 |
||
7341 | 331 |
Goalw [extend_act_def] |
6297 | 332 |
"extend_act h Id = Id"; |
333 |
by (force_tac (claset() addIs [h_f_g_eq RS sym], simpset()) 1); |
|
334 |
qed "extend_act_Id"; |
|
7341 | 335 |
|
336 |
Goalw [project_act_def] |
|
7878
43b03d412b82
working version with localTo[C] instead of localTo
paulson
parents:
7826
diff
changeset
|
337 |
"!!z z'. (z, z') : act ==> (f z, f z') : project_act h act"; |
43b03d412b82
working version with localTo[C] instead of localTo
paulson
parents:
7826
diff
changeset
|
338 |
by (force_tac (claset(), |
43b03d412b82
working version with localTo[C] instead of localTo
paulson
parents:
7826
diff
changeset
|
339 |
simpset() addsimps [split_extended_all]) 1); |
7341 | 340 |
qed "project_act_I"; |
341 |
||
8251
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
342 |
Goalw [project_act_def] "project_act h Id = Id"; |
7341 | 343 |
by (Force_tac 1); |
344 |
qed "project_act_Id"; |
|
345 |
||
8069
19b9f92ca503
working with weak LeadsTo in guarantees precondition\!
paulson
parents:
8055
diff
changeset
|
346 |
Goalw [project_act_def] |
7915
c7fd7eb3b0ef
ALMOST working version: LocalTo results commented out
paulson
parents:
7880
diff
changeset
|
347 |
"Domain (project_act h act) = project_set h (Domain act)"; |
7878
43b03d412b82
working version with localTo[C] instead of localTo
paulson
parents:
7826
diff
changeset
|
348 |
by (force_tac (claset(), |
43b03d412b82
working version with localTo[C] instead of localTo
paulson
parents:
7826
diff
changeset
|
349 |
simpset() addsimps [split_extended_all]) 1); |
7482 | 350 |
qed "Domain_project_act"; |
351 |
||
8251
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
352 |
Addsimps [extend_act_Id]; |
6297 | 353 |
|
354 |
||
355 |
(**** extend ****) |
|
356 |
||
357 |
(*** Basic properties ***) |
|
358 |
||
7341 | 359 |
Goalw [extend_def] "Init (extend h F) = extend_set h (Init F)"; |
6297 | 360 |
by Auto_tac; |
361 |
qed "Init_extend"; |
|
362 |
||
7880
62fb24e28e5e
exchanged the first two args of "project" and "drop_prog"
paulson
parents:
7878
diff
changeset
|
363 |
Goalw [project_def] "Init (project h C F) = project_set h (Init F)"; |
7341 | 364 |
by Auto_tac; |
365 |
qed "Init_project"; |
|
366 |
||
6297 | 367 |
Goal "Acts (extend h F) = (extend_act h `` Acts F)"; |
8251
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
368 |
by (simp_tac (simpset() addsimps [extend_def, insert_Id_image_Acts]) 1); |
6297 | 369 |
qed "Acts_extend"; |
370 |
||
8251
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
371 |
Goal "Acts(project h C F) = insert Id (project_act h `` Restrict C `` Acts F)"; |
7546
36b26759147e
project_act no longer has a special case to allow identity actions
paulson
parents:
7538
diff
changeset
|
372 |
by (auto_tac (claset(), |
7341 | 373 |
simpset() addsimps [project_def, image_iff])); |
374 |
qed "Acts_project"; |
|
375 |
||
376 |
Addsimps [Init_extend, Init_project, Acts_extend, Acts_project]; |
|
6297 | 377 |
|
378 |
Goalw [SKIP_def] "extend h SKIP = SKIP"; |
|
379 |
by (rtac program_equalityI 1); |
|
7341 | 380 |
by Auto_tac; |
381 |
qed "extend_SKIP"; |
|
8122
b43ad07660b9
working version, with Alloc now working on the same state space as the whole
paulson
parents:
8111
diff
changeset
|
382 |
Addsimps [export extend_SKIP]; |
7341 | 383 |
|
8069
19b9f92ca503
working with weak LeadsTo in guarantees precondition\!
paulson
parents:
8055
diff
changeset
|
384 |
Goal "project_set h UNIV = UNIV"; |
7537 | 385 |
by Auto_tac; |
386 |
qed "project_set_UNIV"; |
|
7878
43b03d412b82
working version with localTo[C] instead of localTo
paulson
parents:
7826
diff
changeset
|
387 |
Addsimps [project_set_UNIV]; |
7537 | 388 |
|
8069
19b9f92ca503
working with weak LeadsTo in guarantees precondition\!
paulson
parents:
8055
diff
changeset
|
389 |
Goal "project_set h (Union A) = (UN X:A. project_set h X)"; |
19b9f92ca503
working with weak LeadsTo in guarantees precondition\!
paulson
parents:
8055
diff
changeset
|
390 |
by (Blast_tac 1); |
19b9f92ca503
working with weak LeadsTo in guarantees precondition\!
paulson
parents:
8055
diff
changeset
|
391 |
qed "project_set_Union"; |
19b9f92ca503
working with weak LeadsTo in guarantees precondition\!
paulson
parents:
8055
diff
changeset
|
392 |
|
7915
c7fd7eb3b0ef
ALMOST working version: LocalTo results commented out
paulson
parents:
7880
diff
changeset
|
393 |
Goal "project h C (extend h F) = \ |
c7fd7eb3b0ef
ALMOST working version: LocalTo results commented out
paulson
parents:
7880
diff
changeset
|
394 |
\ mk_program (Init F, Restrict (project_set h C) `` Acts F)"; |
c7fd7eb3b0ef
ALMOST working version: LocalTo results commented out
paulson
parents:
7880
diff
changeset
|
395 |
by (rtac program_equalityI 1); |
c7fd7eb3b0ef
ALMOST working version: LocalTo results commented out
paulson
parents:
7880
diff
changeset
|
396 |
by (asm_simp_tac (simpset() addsimps [image_eq_UN, |
c7fd7eb3b0ef
ALMOST working version: LocalTo results commented out
paulson
parents:
7880
diff
changeset
|
397 |
project_act_extend_act_restrict]) 2); |
c7fd7eb3b0ef
ALMOST working version: LocalTo results commented out
paulson
parents:
7880
diff
changeset
|
398 |
by (Simp_tac 1); |
c7fd7eb3b0ef
ALMOST working version: LocalTo results commented out
paulson
parents:
7880
diff
changeset
|
399 |
qed "project_extend_eq"; |
c7fd7eb3b0ef
ALMOST working version: LocalTo results commented out
paulson
parents:
7880
diff
changeset
|
400 |
|
7537 | 401 |
(*ALL act: Acts F. Domain act is MUCH TOO STRONG since Domain Id = UNIV!*) |
402 |
Goal "UNIV <= project_set h C \ |
|
7880
62fb24e28e5e
exchanged the first two args of "project" and "drop_prog"
paulson
parents:
7878
diff
changeset
|
403 |
\ ==> project h C (extend h F) = F"; |
7915
c7fd7eb3b0ef
ALMOST working version: LocalTo results commented out
paulson
parents:
7880
diff
changeset
|
404 |
by (asm_simp_tac (simpset() addsimps [project_extend_eq, image_eq_UN, |
c7fd7eb3b0ef
ALMOST working version: LocalTo results commented out
paulson
parents:
7880
diff
changeset
|
405 |
subset_UNIV RS subset_trans RS Restrict_triv]) 1); |
7341 | 406 |
qed "extend_inverse"; |
407 |
Addsimps [extend_inverse]; |
|
6297 | 408 |
|
409 |
Goal "inj (extend h)"; |
|
7341 | 410 |
by (rtac inj_on_inverseI 1); |
411 |
by (rtac extend_inverse 1); |
|
8069
19b9f92ca503
working with weak LeadsTo in guarantees precondition\!
paulson
parents:
8055
diff
changeset
|
412 |
by (Force_tac 1); |
6297 | 413 |
qed "inj_extend"; |
414 |
||
415 |
Goal "extend h (F Join G) = extend h F Join extend h G"; |
|
416 |
by (rtac program_equalityI 1); |
|
7537 | 417 |
by (simp_tac (simpset() addsimps [image_Un]) 2); |
6297 | 418 |
by (simp_tac (simpset() addsimps [extend_set_Int_distrib]) 1); |
419 |
qed "extend_Join"; |
|
420 |
Addsimps [extend_Join]; |
|
421 |
||
6647 | 422 |
Goal "extend h (JOIN I F) = (JN i:I. extend h (F i))"; |
423 |
by (rtac program_equalityI 1); |
|
7537 | 424 |
by (simp_tac (simpset() addsimps [image_UN]) 2); |
6834
44da4a2a9ef3
renamed UNION_... to UN_..., INTER_... to INT_... (to fit the convention)
paulson
parents:
6822
diff
changeset
|
425 |
by (simp_tac (simpset() addsimps [extend_set_INT_distrib]) 1); |
6647 | 426 |
qed "extend_JN"; |
427 |
Addsimps [extend_JN]; |
|
428 |
||
7689 | 429 |
(** These monotonicity results look natural but are UNUSED **) |
430 |
||
431 |
Goal "F <= G ==> extend h F <= extend h G"; |
|
432 |
by (full_simp_tac (simpset() addsimps [component_eq_subset]) 1); |
|
433 |
by Auto_tac; |
|
434 |
qed "extend_mono"; |
|
435 |
||
7880
62fb24e28e5e
exchanged the first two args of "project" and "drop_prog"
paulson
parents:
7878
diff
changeset
|
436 |
Goal "F <= G ==> project h C F <= project h C G"; |
8069
19b9f92ca503
working with weak LeadsTo in guarantees precondition\!
paulson
parents:
8055
diff
changeset
|
437 |
by (full_simp_tac (simpset() addsimps [component_eq_subset]) 1); |
7689 | 438 |
by Auto_tac; |
439 |
qed "project_mono"; |
|
440 |
||
441 |
||
6536 | 442 |
(*** Safety: co, stable ***) |
6297 | 443 |
|
6536 | 444 |
Goal "(extend h F : (extend_set h A) co (extend_set h B)) = \ |
445 |
\ (F : A co B)"; |
|
6297 | 446 |
by (simp_tac (simpset() addsimps [constrains_def]) 1); |
447 |
qed "extend_constrains"; |
|
448 |
||
449 |
Goal "(extend h F : stable (extend_set h A)) = (F : stable A)"; |
|
450 |
by (asm_simp_tac (simpset() addsimps [stable_def, extend_constrains]) 1); |
|
451 |
qed "extend_stable"; |
|
452 |
||
453 |
Goal "(extend h F : invariant (extend_set h A)) = (F : invariant A)"; |
|
454 |
by (asm_simp_tac (simpset() addsimps [invariant_def, extend_stable]) 1); |
|
455 |
qed "extend_invariant"; |
|
456 |
||
7826
c6a8b73b6c2a
working shapshot with "projecting" and "extending"
paulson
parents:
7689
diff
changeset
|
457 |
(*Converse fails: A and B may differ in their extra variables*) |
c6a8b73b6c2a
working shapshot with "projecting" and "extending"
paulson
parents:
7689
diff
changeset
|
458 |
Goal "extend h F : A co B ==> F : (project_set h A) co (project_set h B)"; |
8069
19b9f92ca503
working with weak LeadsTo in guarantees precondition\!
paulson
parents:
8055
diff
changeset
|
459 |
by (auto_tac (claset(), simpset() addsimps [constrains_def])); |
7826
c6a8b73b6c2a
working shapshot with "projecting" and "extending"
paulson
parents:
7689
diff
changeset
|
460 |
by (Force_tac 1); |
c6a8b73b6c2a
working shapshot with "projecting" and "extending"
paulson
parents:
7689
diff
changeset
|
461 |
qed "extend_constrains_project_set"; |
c6a8b73b6c2a
working shapshot with "projecting" and "extending"
paulson
parents:
7689
diff
changeset
|
462 |
|
8041 | 463 |
Goal "extend h F : stable A ==> F : stable (project_set h A)"; |
464 |
by (asm_full_simp_tac |
|
465 |
(simpset() addsimps [stable_def, extend_constrains_project_set]) 1); |
|
466 |
qed "extend_stable_project_set"; |
|
467 |
||
7341 | 468 |
|
469 |
(*** Weak safety primitives: Co, Stable ***) |
|
6297 | 470 |
|
471 |
Goal "p : reachable (extend h F) ==> f p : reachable F"; |
|
472 |
by (etac reachable.induct 1); |
|
473 |
by (auto_tac |
|
474 |
(claset() addIs reachable.intrs, |
|
7341 | 475 |
simpset() addsimps [extend_act_def, image_iff])); |
6297 | 476 |
qed "reachable_extend_f"; |
477 |
||
478 |
Goal "h(s,y) : reachable (extend h F) ==> s : reachable F"; |
|
479 |
by (force_tac (claset() addSDs [reachable_extend_f], simpset()) 1); |
|
480 |
qed "h_reachable_extend"; |
|
481 |
||
482 |
Goalw [extend_set_def] |
|
483 |
"reachable (extend h F) = extend_set h (reachable F)"; |
|
484 |
by (rtac equalityI 1); |
|
485 |
by (force_tac (claset() addIs [h_f_g_eq RS sym] |
|
486 |
addSDs [reachable_extend_f], |
|
487 |
simpset()) 1); |
|
488 |
by (Clarify_tac 1); |
|
489 |
by (etac reachable.induct 1); |
|
490 |
by (ALLGOALS (force_tac (claset() addIs reachable.intrs, |
|
491 |
simpset()))); |
|
492 |
qed "reachable_extend_eq"; |
|
493 |
||
6536 | 494 |
Goal "(extend h F : (extend_set h A) Co (extend_set h B)) = \ |
495 |
\ (F : A Co B)"; |
|
6297 | 496 |
by (simp_tac |
497 |
(simpset() addsimps [Constrains_def, reachable_extend_eq, |
|
498 |
extend_constrains, extend_set_Int_distrib RS sym]) 1); |
|
499 |
qed "extend_Constrains"; |
|
500 |
||
501 |
Goal "(extend h F : Stable (extend_set h A)) = (F : Stable A)"; |
|
502 |
by (simp_tac (simpset() addsimps [Stable_def, extend_Constrains]) 1); |
|
503 |
qed "extend_Stable"; |
|
504 |
||
6647 | 505 |
Goal "(extend h F : Always (extend_set h A)) = (F : Always A)"; |
506 |
by (asm_simp_tac (simpset() addsimps [Always_def, extend_Stable]) 1); |
|
507 |
qed "extend_Always"; |
|
508 |
||
6297 | 509 |
|
8251
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
510 |
(** Safety and "project" **) |
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
511 |
|
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
512 |
(** projection: monotonicity for safety **) |
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
513 |
|
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
514 |
Goal "D <= C ==> \ |
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
515 |
\ project_act h (Restrict D act) <= project_act h (Restrict C act)"; |
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
516 |
by (auto_tac (claset(), simpset() addsimps [project_act_def])); |
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
517 |
qed "project_act_mono"; |
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
518 |
|
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
519 |
Goal "[| D <= C; project h C F : A co B |] ==> project h D F : A co B"; |
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
520 |
by (auto_tac (claset(), simpset() addsimps [constrains_def])); |
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
521 |
by (dtac project_act_mono 1); |
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
522 |
by (Blast_tac 1); |
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
523 |
qed "project_constrains_mono"; |
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
524 |
|
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
525 |
Goal "[| D <= C; project h C F : stable A |] ==> project h D F : stable A"; |
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
526 |
by (asm_full_simp_tac |
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
527 |
(simpset() addsimps [stable_def, project_constrains_mono]) 1); |
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
528 |
qed "project_stable_mono"; |
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
529 |
|
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
530 |
Goalw [constrains_def] |
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
531 |
"(project h C F : A co B) = \ |
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
532 |
\ (F : (C Int extend_set h A) co (extend_set h B) & A <= B)"; |
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
533 |
by (auto_tac (claset() addSIs [project_act_I], simpset() addsimps [ball_Un])); |
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
534 |
by (force_tac (claset() addSIs [project_act_I] addSDs [subsetD], simpset()) 1); |
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
535 |
(*the <== direction*) |
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
536 |
by (rewtac project_act_def); |
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
537 |
by (force_tac (claset() addSDs [subsetD], simpset()) 1); |
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
538 |
qed "project_constrains"; |
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
539 |
|
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
540 |
Goalw [stable_def] |
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
541 |
"(project h UNIV F : stable A) = (F : stable (extend_set h A))"; |
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
542 |
by (simp_tac (simpset() addsimps [project_constrains]) 1); |
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
543 |
qed "project_stable"; |
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
544 |
|
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
545 |
Goal "F : stable (extend_set h A) ==> project h C F : stable A"; |
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
546 |
by (dtac (project_stable RS iffD2) 1); |
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
547 |
by (blast_tac (claset() addIs [project_stable_mono]) 1); |
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
548 |
qed "project_stable_I"; |
8122
b43ad07660b9
working version, with Alloc now working on the same state space as the whole
paulson
parents:
8111
diff
changeset
|
549 |
|
b43ad07660b9
working version, with Alloc now working on the same state space as the whole
paulson
parents:
8111
diff
changeset
|
550 |
Goal "A Int extend_set h ((project_set h A) Int B) = A Int extend_set h B"; |
b43ad07660b9
working version, with Alloc now working on the same state space as the whole
paulson
parents:
8111
diff
changeset
|
551 |
by (auto_tac (claset(), simpset() addsimps [split_extended_all])); |
b43ad07660b9
working version, with Alloc now working on the same state space as the whole
paulson
parents:
8111
diff
changeset
|
552 |
qed "Int_extend_set_lemma"; |
b43ad07660b9
working version, with Alloc now working on the same state space as the whole
paulson
parents:
8111
diff
changeset
|
553 |
|
b43ad07660b9
working version, with Alloc now working on the same state space as the whole
paulson
parents:
8111
diff
changeset
|
554 |
Goal "G : C co B ==> project h C G : project_set h C co project_set h B"; |
b43ad07660b9
working version, with Alloc now working on the same state space as the whole
paulson
parents:
8111
diff
changeset
|
555 |
by (full_simp_tac (simpset() addsimps [constrains_def, project_def, |
b43ad07660b9
working version, with Alloc now working on the same state space as the whole
paulson
parents:
8111
diff
changeset
|
556 |
project_act_def]) 1); |
b43ad07660b9
working version, with Alloc now working on the same state space as the whole
paulson
parents:
8111
diff
changeset
|
557 |
by (Blast_tac 1); |
b43ad07660b9
working version, with Alloc now working on the same state space as the whole
paulson
parents:
8111
diff
changeset
|
558 |
qed "project_constrains_project_set"; |
b43ad07660b9
working version, with Alloc now working on the same state space as the whole
paulson
parents:
8111
diff
changeset
|
559 |
|
b43ad07660b9
working version, with Alloc now working on the same state space as the whole
paulson
parents:
8111
diff
changeset
|
560 |
Goal "G : stable C ==> project h C G : stable (project_set h C)"; |
b43ad07660b9
working version, with Alloc now working on the same state space as the whole
paulson
parents:
8111
diff
changeset
|
561 |
by (asm_full_simp_tac (simpset() addsimps [stable_def, |
b43ad07660b9
working version, with Alloc now working on the same state space as the whole
paulson
parents:
8111
diff
changeset
|
562 |
project_constrains_project_set]) 1); |
b43ad07660b9
working version, with Alloc now working on the same state space as the whole
paulson
parents:
8111
diff
changeset
|
563 |
qed "project_stable_project_set"; |
b43ad07660b9
working version, with Alloc now working on the same state space as the whole
paulson
parents:
8111
diff
changeset
|
564 |
|
b43ad07660b9
working version, with Alloc now working on the same state space as the whole
paulson
parents:
8111
diff
changeset
|
565 |
|
6297 | 566 |
(*** Progress: transient, ensures ***) |
567 |
||
568 |
Goal "(extend h F : transient (extend_set h A)) = (F : transient A)"; |
|
569 |
by (auto_tac (claset(), |
|
570 |
simpset() addsimps [transient_def, extend_set_subset_Compl_eq, |
|
571 |
Domain_extend_act])); |
|
572 |
qed "extend_transient"; |
|
573 |
||
6536 | 574 |
Goal "(extend h F : (extend_set h A) ensures (extend_set h B)) = \ |
575 |
\ (F : A ensures B)"; |
|
6297 | 576 |
by (simp_tac |
577 |
(simpset() addsimps [ensures_def, extend_constrains, extend_transient, |
|
578 |
extend_set_Un_distrib RS sym, |
|
579 |
extend_set_Diff_distrib RS sym]) 1); |
|
580 |
qed "extend_ensures"; |
|
581 |
||
6536 | 582 |
Goal "F : A leadsTo B \ |
583 |
\ ==> extend h F : (extend_set h A) leadsTo (extend_set h B)"; |
|
6297 | 584 |
by (etac leadsTo_induct 1); |
585 |
by (asm_simp_tac (simpset() addsimps [leadsTo_UN, extend_set_Union]) 3); |
|
586 |
by (blast_tac (claset() addIs [leadsTo_Trans]) 2); |
|
587 |
by (asm_simp_tac (simpset() addsimps [leadsTo_Basis, extend_ensures]) 1); |
|
588 |
qed "leadsTo_imp_extend_leadsTo"; |
|
589 |
||
590 |
(*** Proving the converse takes some doing! ***) |
|
591 |
||
8111 | 592 |
Goal "(x : slice C y) = (h(x,y) : C)"; |
593 |
by (simp_tac (simpset() addsimps [slice_def]) 1); |
|
594 |
qed "slice_iff"; |
|
595 |
||
596 |
AddIffs [slice_iff]; |
|
597 |
||
598 |
Goal "slice (Union S) y = (UN x:S. slice x y)"; |
|
6297 | 599 |
by Auto_tac; |
600 |
qed "slice_Union"; |
|
601 |
||
8111 | 602 |
Goal "slice (extend_set h A) y = A"; |
6297 | 603 |
by Auto_tac; |
604 |
qed "slice_extend_set"; |
|
605 |
||
8111 | 606 |
Goal "project_set h A = (UN y. slice A y)"; |
6297 | 607 |
by Auto_tac; |
7482 | 608 |
qed "project_set_is_UN_slice"; |
6297 | 609 |
|
8111 | 610 |
Goalw [transient_def] "extend h F : transient A ==> F : transient (slice A y)"; |
6297 | 611 |
by Auto_tac; |
612 |
by (rtac bexI 1); |
|
613 |
by Auto_tac; |
|
614 |
by (force_tac (claset(), simpset() addsimps [extend_act_def]) 1); |
|
615 |
qed "extend_transient_slice"; |
|
616 |
||
8111 | 617 |
(*Converse?*) |
618 |
Goal "extend h F : A co B ==> F : (slice A y) co (slice B y)"; |
|
619 |
by (auto_tac (claset(), simpset() addsimps [constrains_def])); |
|
620 |
qed "extend_constrains_slice"; |
|
621 |
||
7482 | 622 |
Goal "extend h F : A ensures B ==> F : (slice A y) ensures (project_set h B)"; |
8111 | 623 |
by (auto_tac (claset(), |
624 |
simpset() addsimps [ensures_def, extend_constrains, |
|
625 |
extend_transient])); |
|
626 |
by (etac (extend_transient_slice RS transient_strengthen) 2); |
|
627 |
by (etac (extend_constrains_slice RS constrains_weaken) 1); |
|
628 |
by Auto_tac; |
|
6297 | 629 |
qed "extend_ensures_slice"; |
630 |
||
7482 | 631 |
Goal "ALL y. F : (slice B y) leadsTo CU ==> F : (project_set h B) leadsTo CU"; |
632 |
by (simp_tac (simpset() addsimps [project_set_is_UN_slice]) 1); |
|
6297 | 633 |
by (blast_tac (claset() addIs [leadsTo_UN]) 1); |
8111 | 634 |
qed "leadsTo_slice_project_set"; |
6297 | 635 |
|
6536 | 636 |
Goal "extend h F : AU leadsTo BU \ |
7482 | 637 |
\ ==> ALL y. F : (slice AU y) leadsTo (project_set h BU)"; |
6297 | 638 |
by (etac leadsTo_induct 1); |
8111 | 639 |
by (asm_simp_tac (simpset() addsimps [leadsTo_UN, slice_Union]) 3); |
640 |
by (blast_tac (claset() addIs [leadsTo_slice_project_set, leadsTo_Trans]) 2); |
|
6297 | 641 |
by (blast_tac (claset() addIs [extend_ensures_slice, leadsTo_Basis]) 1); |
642 |
qed_spec_mp "extend_leadsTo_slice"; |
|
643 |
||
6536 | 644 |
Goal "(extend h F : (extend_set h A) leadsTo (extend_set h B)) = \ |
645 |
\ (F : A leadsTo B)"; |
|
6297 | 646 |
by Safe_tac; |
647 |
by (etac leadsTo_imp_extend_leadsTo 2); |
|
648 |
by (dtac extend_leadsTo_slice 1); |
|
649 |
by (full_simp_tac (simpset() addsimps [slice_extend_set]) 1); |
|
8251
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
650 |
qed "extend_leadsTo"; |
6297 | 651 |
|
6536 | 652 |
Goal "(extend h F : (extend_set h A) LeadsTo (extend_set h B)) = \ |
653 |
\ (F : A LeadsTo B)"; |
|
6454 | 654 |
by (simp_tac |
655 |
(simpset() addsimps [LeadsTo_def, reachable_extend_eq, |
|
8251
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
656 |
extend_leadsTo, extend_set_Int_distrib RS sym]) 1); |
6454 | 657 |
qed "extend_LeadsTo"; |
658 |
||
6297 | 659 |
|
8251
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
660 |
(*** preserves ***) |
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
661 |
|
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
662 |
Goal "G : preserves (v o f) ==> project h C G : preserves v"; |
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
663 |
by (auto_tac (claset(), |
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
664 |
simpset() addsimps [preserves_def, project_stable_I, |
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
665 |
extend_set_eq_Collect])); |
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
666 |
qed "project_preserves_I"; |
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
667 |
|
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
668 |
(*to preserve f is to preserve the whole original state*) |
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
669 |
Goal "G : preserves f ==> project h C G : preserves id"; |
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
670 |
by (asm_simp_tac (simpset() addsimps [project_preserves_I]) 1); |
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
671 |
qed "project_preserves_id_I"; |
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
672 |
|
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
673 |
Goal "(extend h G : preserves (v o f)) = (G : preserves v)"; |
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
674 |
by (auto_tac (claset(), |
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
675 |
simpset() addsimps [preserves_def, extend_stable RS sym, |
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
676 |
extend_set_eq_Collect])); |
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
677 |
qed "extend_preserves"; |
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
678 |
|
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
679 |
Goal "inj h ==> (extend h G : preserves g)"; |
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
680 |
by (auto_tac (claset(), |
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
681 |
simpset() addsimps [preserves_def, extend_def, extend_act_def, |
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
682 |
stable_def, constrains_def, g_def])); |
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
683 |
qed "inj_extend_preserves"; |
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
684 |
|
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
685 |
|
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
686 |
(*** Guarantees ***) |
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
687 |
|
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
688 |
Goal "project h UNIV ((extend h F) Join G) = F Join (project h UNIV G)"; |
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
689 |
by (rtac program_equalityI 1); |
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
690 |
by (asm_simp_tac |
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
691 |
(simpset() addsimps [image_eq_UN, UN_Un, project_act_extend_act]) 2); |
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
692 |
by (simp_tac (simpset() addsimps [project_set_extend_set_Int]) 1); |
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
693 |
qed "project_extend_Join"; |
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
694 |
|
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
695 |
Goal "(extend h F) Join G = extend h H ==> H = F Join (project h UNIV G)"; |
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
696 |
by (dres_inst_tac [("f", "project h UNIV")] arg_cong 1); |
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
697 |
by (asm_full_simp_tac (simpset() addsimps [project_extend_Join]) 1); |
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
698 |
qed "extend_Join_eq_extend_D"; |
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
699 |
|
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
700 |
(** Strong precondition and postcondition; only useful when |
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
701 |
the old and new state sets are in bijection **) |
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
702 |
|
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
703 |
Goal "F : X guarantees[v] Y ==> \ |
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
704 |
\ extend h F : (extend h `` X) guarantees[v o f] (extend h `` Y)"; |
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
705 |
by (rtac guaranteesI 1); |
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
706 |
by Auto_tac; |
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
707 |
by (blast_tac (claset() addIs [project_preserves_I] |
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
708 |
addDs [extend_Join_eq_extend_D, guaranteesD]) 1); |
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
709 |
qed "guarantees_imp_extend_guarantees"; |
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
710 |
|
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
711 |
Goal "extend h F : (extend h `` X) guarantees[v o f] (extend h `` Y) \ |
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
712 |
\ ==> F : X guarantees[v] Y"; |
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
713 |
by (auto_tac (claset(), simpset() addsimps [guar_def])); |
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
714 |
by (dres_inst_tac [("x", "extend h G")] spec 1); |
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
715 |
by (asm_full_simp_tac |
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
716 |
(simpset() delsimps [extend_Join] |
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
717 |
addsimps [extend_Join RS sym, extend_preserves, |
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
718 |
inj_extend RS inj_image_mem_iff]) 1); |
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
719 |
qed "extend_guarantees_imp_guarantees"; |
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
720 |
|
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
721 |
Goal "(extend h F : (extend h `` X) guarantees[v o f] (extend h `` Y)) = \ |
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
722 |
\ (F : X guarantees[v] Y)"; |
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
723 |
by (blast_tac (claset() addIs [guarantees_imp_extend_guarantees, |
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
724 |
extend_guarantees_imp_guarantees]) 1); |
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
725 |
qed "extend_guarantees_eq"; |
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
726 |
|
9be357df93d4
New treatment of "guarantees" with polymorphic components and bijections.
paulson
parents:
8216
diff
changeset
|
727 |
|
6297 | 728 |
Close_locale "Extend"; |
7482 | 729 |
|
730 |
(*Close_locale should do this! |
|
731 |
Delsimps [f_h_eq, extend_set_inverse, f_image_extend_set, extend_act_inverse, |
|
732 |
extend_act_Image]; |
|
733 |
Delrules [make_elim h_inject1]; |
|
734 |
*) |