author | wenzelm |
Wed, 29 Nov 2006 15:44:46 +0100 | |
changeset 21587 | a3561bfe0ada |
parent 21554 | 0625898865a9 |
child 22418 | 49e2d9744ae1 |
permissions | -rw-r--r-- |
18266
55c201fe4c95
added an authors section (please let me know if somebody is left out or unhappy)
urbanc
parents:
18263
diff
changeset
|
1 |
(* $Id$ *) |
55c201fe4c95
added an authors section (please let me know if somebody is left out or unhappy)
urbanc
parents:
18263
diff
changeset
|
2 |
|
18577
a636846a02c7
added more documentation; will now try out a modification
urbanc
parents:
18424
diff
changeset
|
3 |
(*<*) |
19501 | 4 |
theory Fsub |
5 |
imports "../Nominal" |
|
18269 | 6 |
begin |
18577
a636846a02c7
added more documentation; will now try out a modification
urbanc
parents:
18424
diff
changeset
|
7 |
(*>*) |
18269 | 8 |
|
18577
a636846a02c7
added more documentation; will now try out a modification
urbanc
parents:
18424
diff
changeset
|
9 |
text{* Authors: Christian Urban, |
a636846a02c7
added more documentation; will now try out a modification
urbanc
parents:
18424
diff
changeset
|
10 |
Benjamin Pierce, |
18650 | 11 |
Dimitrios Vytiniotis |
12 |
Stephanie Weirich and |
|
13 |
Steve Zdancewic |
|
18266
55c201fe4c95
added an authors section (please let me know if somebody is left out or unhappy)
urbanc
parents:
18263
diff
changeset
|
14 |
|
18577
a636846a02c7
added more documentation; will now try out a modification
urbanc
parents:
18424
diff
changeset
|
15 |
with great help from Stefan Berghofer and Markus Wenzel. *} |
18246 | 16 |
|
18621 | 17 |
section {* Types for Names, Nominal Datatype Declaration for Types and Terms *} |
18424 | 18 |
|
18577
a636846a02c7
added more documentation; will now try out a modification
urbanc
parents:
18424
diff
changeset
|
19 |
text {* The main point of this solution is to use names everywhere (be they bound, |
18621 | 20 |
binding or free). In System \FSUB{} there are two kinds of names corresponding to |
21 |
type-variables and to term-variables. These two kinds of names are represented in |
|
18577
a636846a02c7
added more documentation; will now try out a modification
urbanc
parents:
18424
diff
changeset
|
22 |
the nominal datatype package as atom-types @{text "tyvrs"} and @{text "vrs"}: *} |
a636846a02c7
added more documentation; will now try out a modification
urbanc
parents:
18424
diff
changeset
|
23 |
|
18246 | 24 |
atom_decl tyvrs vrs |
25 |
||
18577
a636846a02c7
added more documentation; will now try out a modification
urbanc
parents:
18424
diff
changeset
|
26 |
text{* There are numerous facts that come with this declaration: for example that |
a636846a02c7
added more documentation; will now try out a modification
urbanc
parents:
18424
diff
changeset
|
27 |
there are infinitely many elements in @{text "tyvrs"} and @{text "vrs"}. *} |
a636846a02c7
added more documentation; will now try out a modification
urbanc
parents:
18424
diff
changeset
|
28 |
|
a636846a02c7
added more documentation; will now try out a modification
urbanc
parents:
18424
diff
changeset
|
29 |
text{* The constructors for types and terms in System \FSUB{} contain abstractions |
a636846a02c7
added more documentation; will now try out a modification
urbanc
parents:
18424
diff
changeset
|
30 |
over type-variables and term-variables. The nominal datatype-package uses |
a636846a02c7
added more documentation; will now try out a modification
urbanc
parents:
18424
diff
changeset
|
31 |
@{text "\<guillemotleft>\<dots>\<guillemotright>\<dots>"} to indicate where abstractions occur. *} |
a636846a02c7
added more documentation; will now try out a modification
urbanc
parents:
18424
diff
changeset
|
32 |
|
18424 | 33 |
nominal_datatype ty = |
18577
a636846a02c7
added more documentation; will now try out a modification
urbanc
parents:
18424
diff
changeset
|
34 |
Tvar "tyvrs" |
18424 | 35 |
| Top |
18577
a636846a02c7
added more documentation; will now try out a modification
urbanc
parents:
18424
diff
changeset
|
36 |
| Arrow "ty" "ty" ("_ \<rightarrow> _" [100,100] 100) |
a636846a02c7
added more documentation; will now try out a modification
urbanc
parents:
18424
diff
changeset
|
37 |
| Forall "\<guillemotleft>tyvrs\<guillemotright>ty" "ty" |
18246 | 38 |
|
18424 | 39 |
nominal_datatype trm = |
40 |
Var "vrs" |
|
18577
a636846a02c7
added more documentation; will now try out a modification
urbanc
parents:
18424
diff
changeset
|
41 |
| Lam "\<guillemotleft>vrs\<guillemotright>trm" "ty" |
a636846a02c7
added more documentation; will now try out a modification
urbanc
parents:
18424
diff
changeset
|
42 |
| Tabs "\<guillemotleft>tyvrs\<guillemotright>trm" "ty" |
18424 | 43 |
| App "trm" "trm" |
18577
a636846a02c7
added more documentation; will now try out a modification
urbanc
parents:
18424
diff
changeset
|
44 |
| Tapp "trm" "ty" |
a636846a02c7
added more documentation; will now try out a modification
urbanc
parents:
18424
diff
changeset
|
45 |
|
a636846a02c7
added more documentation; will now try out a modification
urbanc
parents:
18424
diff
changeset
|
46 |
text {* To be polite to the eye, some more familiar notation is introduced. |
18621 | 47 |
Because of the change in the order of arguments, one needs to use |
18577
a636846a02c7
added more documentation; will now try out a modification
urbanc
parents:
18424
diff
changeset
|
48 |
translation rules, instead of syntax annotations at the term-constructors |
18650 | 49 |
as given above for @{term "Arrow"}. *} |
18246 | 50 |
|
51 |
syntax |
|
18577
a636846a02c7
added more documentation; will now try out a modification
urbanc
parents:
18424
diff
changeset
|
52 |
Forall_syn :: "tyvrs \<Rightarrow> ty \<Rightarrow> ty \<Rightarrow> ty" ("\<forall>[_<:_]._" [100,100,100] 100) |
a636846a02c7
added more documentation; will now try out a modification
urbanc
parents:
18424
diff
changeset
|
53 |
Lam_syn :: "vrs \<Rightarrow> ty \<Rightarrow> trm \<Rightarrow> trm" ("Lam [_:_]._" [100,100,100] 100) |
a636846a02c7
added more documentation; will now try out a modification
urbanc
parents:
18424
diff
changeset
|
54 |
Tabs_syn :: "tyvrs \<Rightarrow> ty \<Rightarrow> trm \<Rightarrow> trm" ("Tabs [_<:_]._" [100,100,100] 100) |
18424 | 55 |
|
18246 | 56 |
translations |
18577
a636846a02c7
added more documentation; will now try out a modification
urbanc
parents:
18424
diff
changeset
|
57 |
"\<forall>[X<:T\<^isub>1].T\<^isub>2" \<rightleftharpoons> "ty.Forall X T\<^isub>2 T\<^isub>1" |
a636846a02c7
added more documentation; will now try out a modification
urbanc
parents:
18424
diff
changeset
|
58 |
"Lam [x:T].t" \<rightleftharpoons> "trm.Lam x t T" |
a636846a02c7
added more documentation; will now try out a modification
urbanc
parents:
18424
diff
changeset
|
59 |
"Tabs [X<:T].t" \<rightleftharpoons> "trm.Tabs X t T" |
18246 | 60 |
|
18621 | 61 |
text {* Again there are numerous facts that are proved automatically for @{typ "ty"} |
18650 | 62 |
and @{typ "trm"}: for example that the set of free variables, i.e.~the @{text "support"}, |
63 |
is finite. However note that nominal-datatype declarations do \emph{not} define |
|
64 |
``classical" constructor-based datatypes, but rather define $\alpha$-equivalence |
|
18621 | 65 |
classes---we can for example show that $\alpha$-equivalent @{typ "ty"}s |
18577
a636846a02c7
added more documentation; will now try out a modification
urbanc
parents:
18424
diff
changeset
|
66 |
and @{typ "trm"}s are equal: *} |
a636846a02c7
added more documentation; will now try out a modification
urbanc
parents:
18424
diff
changeset
|
67 |
|
a636846a02c7
added more documentation; will now try out a modification
urbanc
parents:
18424
diff
changeset
|
68 |
lemma alpha_illustration: |
a636846a02c7
added more documentation; will now try out a modification
urbanc
parents:
18424
diff
changeset
|
69 |
shows "\<forall>[X<:T].(Tvar X) = \<forall>[Y<:T].(Tvar Y)" |
a636846a02c7
added more documentation; will now try out a modification
urbanc
parents:
18424
diff
changeset
|
70 |
and "Lam [x:T].(Var x) = Lam [y:T].(Var y)" |
a636846a02c7
added more documentation; will now try out a modification
urbanc
parents:
18424
diff
changeset
|
71 |
by (simp_all add: ty.inject trm.inject alpha calc_atm fresh_atm) |
a636846a02c7
added more documentation; will now try out a modification
urbanc
parents:
18424
diff
changeset
|
72 |
|
18621 | 73 |
section {* SubTyping Contexts *} |
18246 | 74 |
|
75 |
types ty_context = "(tyvrs\<times>ty) list" |
|
76 |
||
18650 | 77 |
text {* Typing contexts are represented as lists that ``grow" on the left; we |
18621 | 78 |
thereby deviating from the convention in the POPLmark-paper. The lists contain |
18650 | 79 |
pairs of type-variables and types (this is sufficient for Part 1A). *} |
18577
a636846a02c7
added more documentation; will now try out a modification
urbanc
parents:
18424
diff
changeset
|
80 |
|
18628 | 81 |
text {* In order to state validity-conditions for typing-contexts, the notion of |
18621 | 82 |
a @{text "domain"} of a typing-context is handy. *} |
18577
a636846a02c7
added more documentation; will now try out a modification
urbanc
parents:
18424
diff
changeset
|
83 |
|
18246 | 84 |
consts |
85 |
"domain" :: "ty_context \<Rightarrow> tyvrs set" |
|
86 |
primrec |
|
87 |
"domain [] = {}" |
|
88 |
"domain (X#\<Gamma>) = {fst X}\<union>(domain \<Gamma>)" |
|
89 |
||
90 |
lemma domain_eqvt: |
|
91 |
fixes pi::"tyvrs prm" |
|
92 |
shows "pi\<bullet>(domain \<Gamma>) = domain (pi\<bullet>\<Gamma>)" |
|
18655
73cebafb9a89
merged the silly lemmas into the eqvt proof of subtype
urbanc
parents:
18650
diff
changeset
|
93 |
by (induct \<Gamma>, simp_all add: perm_empty perm_insert perm_fst) |
18246 | 94 |
|
95 |
lemma finite_domain: |
|
96 |
shows "finite (domain \<Gamma>)" |
|
97 |
by (induct \<Gamma>, auto) |
|
98 |
||
18621 | 99 |
lemma domain_supp: |
100 |
shows "(supp (domain \<Gamma>)) = (domain \<Gamma>)" |
|
101 |
by (simp only: at_fin_set_supp at_tyvrs_inst finite_domain) |
|
102 |
||
18424 | 103 |
lemma domain_inclusion: |
104 |
assumes a: "(X,T)\<in>set \<Gamma>" |
|
105 |
shows "X\<in>(domain \<Gamma>)" |
|
106 |
using a by (induct \<Gamma>, auto) |
|
18246 | 107 |
|
18424 | 108 |
lemma domain_existence: |
109 |
assumes a: "X\<in>(domain \<Gamma>)" |
|
110 |
shows "\<exists>T.(X,T)\<in>set \<Gamma>" |
|
111 |
using a by (induct \<Gamma>, auto) |
|
18246 | 112 |
|
113 |
lemma domain_append: |
|
114 |
shows "domain (\<Gamma>@\<Delta>) = ((domain \<Gamma>) \<union> (domain \<Delta>))" |
|
115 |
by (induct \<Gamma>, auto) |
|
116 |
||
18621 | 117 |
lemma fresh_domain_cons: |
118 |
fixes X::"tyvrs" |
|
119 |
shows "X\<sharp>(domain (Y#\<Gamma>)) = (X\<sharp>(fst Y) \<and> X\<sharp>(domain \<Gamma>))" |
|
120 |
by (simp add: fresh_fin_insert pt_tyvrs_inst at_tyvrs_inst fs_tyvrs_inst finite_domain) |
|
121 |
||
122 |
lemma fresh_domain: |
|
123 |
fixes X::"tyvrs" |
|
124 |
assumes a: "X\<sharp>\<Gamma>" |
|
125 |
shows "X\<sharp>(domain \<Gamma>)" |
|
126 |
using a |
|
127 |
apply(induct \<Gamma>) |
|
128 |
apply(simp add: fresh_set_empty) |
|
129 |
apply(simp only: fresh_domain_cons) |
|
130 |
apply(auto simp add: fresh_prod fresh_list_cons) |
|
131 |
done |
|
132 |
||
18577
a636846a02c7
added more documentation; will now try out a modification
urbanc
parents:
18424
diff
changeset
|
133 |
text {* Not all lists of type @{typ "ty_context"} are well-formed. One condition |
a636846a02c7
added more documentation; will now try out a modification
urbanc
parents:
18424
diff
changeset
|
134 |
requires that in @{term "(X,S)#\<Gamma>"} all free variables of @{term "S"} must be |
18621 | 135 |
in the @{term "domain"} of @{term "\<Gamma>"}, that is @{term "S"} must be @{text "closed"} |
18650 | 136 |
in @{term "\<Gamma>"}. The set of free variables of @{term "S"} is the |
18621 | 137 |
@{text "support"} of @{term "S"}. *} |
18246 | 138 |
|
139 |
constdefs |
|
140 |
"closed_in" :: "ty \<Rightarrow> ty_context \<Rightarrow> bool" ("_ closed'_in _" [100,100] 100) |
|
141 |
"S closed_in \<Gamma> \<equiv> (supp S)\<subseteq>(domain \<Gamma>)" |
|
142 |
||
143 |
lemma closed_in_eqvt: |
|
144 |
fixes pi::"tyvrs prm" |
|
145 |
assumes a: "S closed_in \<Gamma>" |
|
146 |
shows "(pi\<bullet>S) closed_in (pi\<bullet>\<Gamma>)" |
|
147 |
using a |
|
148 |
proof (unfold "closed_in_def") |
|
18424 | 149 |
assume "supp S \<subseteq> (domain \<Gamma>)" |
18246 | 150 |
hence "pi\<bullet>(supp S) \<subseteq> pi\<bullet>(domain \<Gamma>)" |
151 |
by (simp add: pt_subseteq_eqvt[OF pt_tyvrs_inst, OF at_tyvrs_inst]) |
|
152 |
thus "(supp (pi\<bullet>S)) \<subseteq> (domain (pi\<bullet>\<Gamma>))" |
|
153 |
by (simp add: domain_eqvt pt_perm_supp[OF pt_tyvrs_inst, OF at_tyvrs_inst]) |
|
154 |
qed |
|
155 |
||
18621 | 156 |
text {* Now validity of a context is a straightforward inductive definition. *} |
157 |
||
18246 | 158 |
consts |
159 |
valid_rel :: "ty_context set" |
|
160 |
valid_sym :: "ty_context \<Rightarrow> bool" ("\<turnstile> _ ok" [100] 100) |
|
161 |
translations |
|
162 |
"\<turnstile> \<Gamma> ok" \<rightleftharpoons> "\<Gamma> \<in> valid_rel" |
|
163 |
inductive valid_rel |
|
164 |
intros |
|
18621 | 165 |
valid_nil[simp]: "\<turnstile> [] ok" |
166 |
valid_cons[simp]: "\<lbrakk>\<turnstile> \<Gamma> ok; X\<sharp>(domain \<Gamma>); T closed_in \<Gamma>\<rbrakk> \<Longrightarrow> \<turnstile> ((X,T)#\<Gamma>) ok" |
|
18246 | 167 |
|
168 |
lemma valid_eqvt: |
|
169 |
fixes pi::"tyvrs prm" |
|
170 |
assumes a: "\<turnstile> \<Gamma> ok" |
|
171 |
shows "\<turnstile> (pi\<bullet>\<Gamma>) ok" |
|
172 |
using a |
|
173 |
proof (induct) |
|
18621 | 174 |
case valid_nil |
175 |
show "\<turnstile> (pi\<bullet>[]) ok" by simp |
|
18246 | 176 |
next |
18621 | 177 |
case (valid_cons T X \<Gamma>) |
178 |
have "\<turnstile> (pi\<bullet>\<Gamma>) ok" by fact |
|
18577
a636846a02c7
added more documentation; will now try out a modification
urbanc
parents:
18424
diff
changeset
|
179 |
moreover |
18621 | 180 |
have "X\<sharp>(domain \<Gamma>)" by fact |
19972
89c5afe4139a
added more infrastructure for the recursion combinator
urbanc
parents:
19501
diff
changeset
|
181 |
hence "(pi\<bullet>X)\<sharp>(domain (pi\<bullet>\<Gamma>))" by (simp add: fresh_bij domain_eqvt[symmetric]) |
18577
a636846a02c7
added more documentation; will now try out a modification
urbanc
parents:
18424
diff
changeset
|
182 |
moreover |
a636846a02c7
added more documentation; will now try out a modification
urbanc
parents:
18424
diff
changeset
|
183 |
have "T closed_in \<Gamma>" by fact |
18621 | 184 |
hence "(pi\<bullet>T) closed_in (pi\<bullet>\<Gamma>)" by (simp add: closed_in_eqvt) |
185 |
ultimately show "\<turnstile> (pi\<bullet>((X,T)#\<Gamma>)) ok" by simp |
|
18246 | 186 |
qed |
187 |
||
188 |
lemma validE: |
|
189 |
assumes a: "\<turnstile> ((X,T)#\<Gamma>) ok" |
|
18621 | 190 |
shows "\<turnstile> \<Gamma> ok \<and> X\<sharp>(domain \<Gamma>) \<and> T closed_in \<Gamma>" |
18246 | 191 |
using a by (cases, auto) |
192 |
||
18424 | 193 |
lemma validE_append: |
194 |
assumes a: "\<turnstile> (\<Delta>@\<Gamma>) ok" |
|
195 |
shows "\<turnstile> \<Gamma> ok" |
|
196 |
using a by (induct \<Delta>, auto dest: validE) |
|
18246 | 197 |
|
18424 | 198 |
lemma replace_type: |
199 |
assumes a: "\<turnstile> (\<Delta>@(X,T)#\<Gamma>) ok" |
|
200 |
and b: "S closed_in \<Gamma>" |
|
201 |
shows "\<turnstile> (\<Delta>@(X,S)#\<Gamma>) ok" |
|
18621 | 202 |
using a b |
18246 | 203 |
apply(induct \<Delta>) |
18621 | 204 |
apply(auto dest!: validE intro!: valid_cons simp add: domain_append closed_in_def) |
18246 | 205 |
done |
206 |
||
18650 | 207 |
text {* Well-formed contexts have a unique type-binding for a type-variable. *} |
208 |
||
18246 | 209 |
lemma uniqueness_of_ctxt: |
210 |
fixes \<Gamma>::"ty_context" |
|
18412 | 211 |
assumes a: "\<turnstile> \<Gamma> ok" |
212 |
and b: "(X,T)\<in>set \<Gamma>" |
|
213 |
and c: "(X,S)\<in>set \<Gamma>" |
|
214 |
shows "T=S" |
|
18621 | 215 |
using a b c |
216 |
proof (induct) |
|
217 |
case valid_nil thus "T=S" by simp |
|
218 |
next |
|
219 |
case (valid_cons U Y \<Gamma>) |
|
220 |
moreover |
|
221 |
{ fix \<Gamma>::"ty_context" |
|
222 |
assume a: "X\<sharp>(domain \<Gamma>)" |
|
223 |
have "\<not>(\<exists>T.(X,T)\<in>(set \<Gamma>))" using a |
|
224 |
proof (induct \<Gamma>) |
|
225 |
case (Cons Y \<Gamma>) |
|
226 |
thus "\<not> (\<exists>T.(X,T)\<in>set(Y#\<Gamma>))" |
|
227 |
by (simp only: fresh_domain_cons, auto simp add: fresh_atm) |
|
228 |
qed (simp) |
|
229 |
} |
|
230 |
ultimately show "T=S" by auto |
|
231 |
qed |
|
18577
a636846a02c7
added more documentation; will now try out a modification
urbanc
parents:
18424
diff
changeset
|
232 |
|
18628 | 233 |
section {* Size and Capture-Avoiding Substitution for Types *} |
18621 | 234 |
|
21554 | 235 |
consts size_ty :: "ty \<Rightarrow> nat" |
20395
9a60e3151244
added definition for size and substitution using the recursion
urbanc
parents:
19972
diff
changeset
|
236 |
|
21554 | 237 |
nominal_primrec |
238 |
"size_ty (Tvar X) = 1" |
|
239 |
"size_ty (Top) = 1" |
|
240 |
"size_ty (T1 \<rightarrow> T2) = (size_ty T1) + (size_ty T2) + 1" |
|
241 |
"X\<sharp>T1 \<Longrightarrow> size_ty (\<forall>[X<:T1].T2) = (size_ty T1) + (size_ty T2) + 1" |
|
242 |
apply (finite_guess add: perm_nat_def)+ |
|
243 |
apply (rule TrueI)+ |
|
244 |
apply (simp add: fresh_def supp_nat) |
|
245 |
apply (assumption | fresh_guess add: perm_nat_def)+ |
|
246 |
done |
|
20395
9a60e3151244
added definition for size and substitution using the recursion
urbanc
parents:
19972
diff
changeset
|
247 |
|
21554 | 248 |
lemma eq_eqvt: |
249 |
fixes pi::"tyvrs prm" |
|
250 |
and x::"'a::pt_tyvrs" |
|
251 |
shows "pi\<bullet>(x=y) = ((pi\<bullet>x)=(pi\<bullet>y))" |
|
252 |
apply(simp add: perm_bool perm_bij) |
|
253 |
done |
|
20395
9a60e3151244
added definition for size and substitution using the recursion
urbanc
parents:
19972
diff
changeset
|
254 |
|
21554 | 255 |
consts subst_ty :: "tyvrs \<Rightarrow> ty \<Rightarrow> ty \<Rightarrow> ty" |
20395
9a60e3151244
added definition for size and substitution using the recursion
urbanc
parents:
19972
diff
changeset
|
256 |
|
9a60e3151244
added definition for size and substitution using the recursion
urbanc
parents:
19972
diff
changeset
|
257 |
syntax |
9a60e3151244
added definition for size and substitution using the recursion
urbanc
parents:
19972
diff
changeset
|
258 |
subst_ty_syn :: "ty \<Rightarrow> tyvrs \<Rightarrow> ty \<Rightarrow> ty" ("_[_:=_]\<^isub>t\<^isub>y" [100,100,100] 100) |
9a60e3151244
added definition for size and substitution using the recursion
urbanc
parents:
19972
diff
changeset
|
259 |
|
9a60e3151244
added definition for size and substitution using the recursion
urbanc
parents:
19972
diff
changeset
|
260 |
translations |
9a60e3151244
added definition for size and substitution using the recursion
urbanc
parents:
19972
diff
changeset
|
261 |
"T1[Y:=T2]\<^isub>t\<^isub>y" \<rightleftharpoons> "subst_ty Y T2 T1" |
18577
a636846a02c7
added more documentation; will now try out a modification
urbanc
parents:
18424
diff
changeset
|
262 |
|
21554 | 263 |
nominal_primrec |
264 |
"(Tvar X)[Y:=T]\<^isub>t\<^isub>y= (if X=Y then T else (Tvar X))" |
|
265 |
"(Top)[Y:=T]\<^isub>t\<^isub>y = Top" |
|
266 |
"(T\<^isub>1 \<rightarrow> T\<^isub>2)[Y:=T]\<^isub>t\<^isub>y = (T\<^isub>1[Y:=T]\<^isub>t\<^isub>y) \<rightarrow> (T\<^isub>2[Y:=T]\<^isub>t\<^isub>y)" |
|
267 |
"\<lbrakk>X\<sharp>(Y,T); X\<sharp>T\<^isub>1\<rbrakk> \<Longrightarrow> (\<forall>[X<:T\<^isub>1].T\<^isub>2)[Y:=T]\<^isub>t\<^isub>y = (\<forall>[X<:(T\<^isub>1[Y:=T]\<^isub>t\<^isub>y)].(T\<^isub>2[Y:=T]\<^isub>t\<^isub>y))" |
|
268 |
apply (finite_guess add: perm_if eq_eqvt fs_tyvrs1) |
|
269 |
apply finite_guess |
|
270 |
apply finite_guess |
|
271 |
apply finite_guess |
|
272 |
apply perm_full_simp |
|
273 |
apply (simp add: supp_unit) |
|
274 |
apply (rule TrueI)+ |
|
275 |
apply (simp add: abs_fresh) |
|
276 |
apply (fresh_guess add: fs_tyvrs1 perm_if eq_eqvt) |
|
277 |
apply fresh_guess |
|
278 |
apply fresh_guess |
|
279 |
apply fresh_guess |
|
280 |
apply perm_full_simp |
|
281 |
apply assumption |
|
282 |
done |
|
18577
a636846a02c7
added more documentation; will now try out a modification
urbanc
parents:
18424
diff
changeset
|
283 |
|
18621 | 284 |
consts subst_tyc :: "ty_context \<Rightarrow> tyvrs \<Rightarrow> ty \<Rightarrow> ty_context" ("_[_:=_]\<^isub>t\<^isub>y\<^isub>c" [100,100,100] 100) |
18577
a636846a02c7
added more documentation; will now try out a modification
urbanc
parents:
18424
diff
changeset
|
285 |
primrec |
a636846a02c7
added more documentation; will now try out a modification
urbanc
parents:
18424
diff
changeset
|
286 |
"([])[Y:=T]\<^isub>t\<^isub>y\<^isub>c= []" |
a636846a02c7
added more documentation; will now try out a modification
urbanc
parents:
18424
diff
changeset
|
287 |
"(XT#\<Gamma>)[Y:=T]\<^isub>t\<^isub>y\<^isub>c = (fst XT,(snd XT)[Y:=T]\<^isub>t\<^isub>y)#(\<Gamma>[Y:=T]\<^isub>t\<^isub>y\<^isub>c)" |
18246 | 288 |
|
18577
a636846a02c7
added more documentation; will now try out a modification
urbanc
parents:
18424
diff
changeset
|
289 |
section {* Subtyping-Relation *} |
18246 | 290 |
|
18650 | 291 |
text {* The definition for the subtyping-relation follows quite closely what is written |
292 |
in the POPLmark-paper, except for the premises dealing with well-formed contexts and |
|
293 |
the freshness constraint @{term "X\<sharp>\<Gamma>"} in the @{text "S_Forall"}-rule. (The freshness |
|
294 |
constraint is specific to the \emph{nominal approach}. Note, however, that the constraint |
|
295 |
does \emph{not} make the subtyping-relation ``partial"\ldots because we work over |
|
296 |
$\alpha$-equivalence classes.) *} |
|
18628 | 297 |
|
18246 | 298 |
consts |
18577
a636846a02c7
added more documentation; will now try out a modification
urbanc
parents:
18424
diff
changeset
|
299 |
subtype_of :: "(ty_context \<times> ty \<times> ty) set" |
a636846a02c7
added more documentation; will now try out a modification
urbanc
parents:
18424
diff
changeset
|
300 |
syntax |
18621 | 301 |
subtype_of_syn :: "ty_context \<Rightarrow> ty \<Rightarrow> ty \<Rightarrow> bool" ("_\<turnstile>_<:_" [100,100,100] 100) |
18577
a636846a02c7
added more documentation; will now try out a modification
urbanc
parents:
18424
diff
changeset
|
302 |
|
18246 | 303 |
translations |
18577
a636846a02c7
added more documentation; will now try out a modification
urbanc
parents:
18424
diff
changeset
|
304 |
"\<Gamma> \<turnstile> S <: T" \<rightleftharpoons> "(\<Gamma>,S,T) \<in> subtype_of" |
a636846a02c7
added more documentation; will now try out a modification
urbanc
parents:
18424
diff
changeset
|
305 |
inductive subtype_of |
18246 | 306 |
intros |
18621 | 307 |
S_Top[intro]: "\<lbrakk>\<turnstile> \<Gamma> ok; S closed_in \<Gamma>\<rbrakk> \<Longrightarrow> \<Gamma> \<turnstile> S <: Top" |
308 |
S_Var[intro]: "\<lbrakk>(X,S) \<in> set \<Gamma>; \<Gamma> \<turnstile> S <: T\<rbrakk> \<Longrightarrow> \<Gamma> \<turnstile> (Tvar X) <: T" |
|
309 |
S_Refl[intro]: "\<lbrakk>\<turnstile> \<Gamma> ok; X \<in> domain \<Gamma>\<rbrakk>\<Longrightarrow> \<Gamma> \<turnstile> Tvar X <: Tvar X" |
|
310 |
S_Arrow[intro]: "\<lbrakk>\<Gamma> \<turnstile> T\<^isub>1 <: S\<^isub>1; \<Gamma> \<turnstile> S\<^isub>2 <: T\<^isub>2\<rbrakk> \<Longrightarrow> \<Gamma> \<turnstile> (S\<^isub>1 \<rightarrow> S\<^isub>2) <: (T\<^isub>1 \<rightarrow> T\<^isub>2)" |
|
311 |
S_Forall[intro]: "\<lbrakk>\<Gamma> \<turnstile> T\<^isub>1 <: S\<^isub>1; X\<sharp>\<Gamma>; ((X,T\<^isub>1)#\<Gamma>) \<turnstile> S\<^isub>2 <: T\<^isub>2\<rbrakk> |
|
312 |
\<Longrightarrow> \<Gamma> \<turnstile> \<forall>[X<:S\<^isub>1].S\<^isub>2 <: \<forall>[X<:T\<^isub>1].T\<^isub>2" |
|
18246 | 313 |
|
314 |
lemma subtype_implies_closed: |
|
315 |
assumes a: "\<Gamma> \<turnstile> S <: T" |
|
316 |
shows "S closed_in \<Gamma> \<and> T closed_in \<Gamma>" |
|
317 |
using a |
|
318 |
proof (induct) |
|
319 |
case (S_Top S \<Gamma>) |
|
18424 | 320 |
have "Top closed_in \<Gamma>" by (simp add: closed_in_def ty.supp) |
18246 | 321 |
moreover |
322 |
have "S closed_in \<Gamma>" by fact |
|
323 |
ultimately show "S closed_in \<Gamma> \<and> Top closed_in \<Gamma>" by simp |
|
324 |
next |
|
325 |
case (S_Var S T X \<Gamma>) |
|
326 |
have "(X,S)\<in>set \<Gamma>" by fact |
|
18424 | 327 |
hence "X \<in> domain \<Gamma>" by (rule domain_inclusion) |
18577
a636846a02c7
added more documentation; will now try out a modification
urbanc
parents:
18424
diff
changeset
|
328 |
hence "(Tvar X) closed_in \<Gamma>" by (simp add: closed_in_def ty.supp supp_atm) |
18246 | 329 |
moreover |
330 |
have "S closed_in \<Gamma> \<and> T closed_in \<Gamma>" by fact |
|
331 |
hence "T closed_in \<Gamma>" by force |
|
18577
a636846a02c7
added more documentation; will now try out a modification
urbanc
parents:
18424
diff
changeset
|
332 |
ultimately show "(Tvar X) closed_in \<Gamma> \<and> T closed_in \<Gamma>" by simp |
18424 | 333 |
qed (auto simp add: closed_in_def ty.supp supp_atm abs_supp) |
18246 | 334 |
|
335 |
lemma subtype_implies_ok: |
|
336 |
fixes X::"tyvrs" |
|
337 |
assumes a1: "\<Gamma> \<turnstile> S <: T" |
|
338 |
shows "\<turnstile> \<Gamma> ok" |
|
339 |
using a1 by (induct, auto) |
|
340 |
||
341 |
lemma subtype_implies_fresh: |
|
342 |
fixes X::"tyvrs" |
|
343 |
assumes a1: "\<Gamma> \<turnstile> S <: T" |
|
344 |
and a2: "X\<sharp>\<Gamma>" |
|
18424 | 345 |
shows "X\<sharp>S \<and> X\<sharp>T" |
18246 | 346 |
proof - |
347 |
from a1 have "\<turnstile> \<Gamma> ok" by (rule subtype_implies_ok) |
|
18621 | 348 |
with a2 have "X\<sharp>domain(\<Gamma>)" by (simp add: fresh_domain) |
18424 | 349 |
moreover |
18246 | 350 |
from a1 have "S closed_in \<Gamma> \<and> T closed_in \<Gamma>" by (rule subtype_implies_closed) |
18424 | 351 |
hence "supp S \<subseteq> ((supp (domain \<Gamma>))::tyvrs set)" |
18621 | 352 |
and "supp T \<subseteq> ((supp (domain \<Gamma>))::tyvrs set)" by (simp_all add: domain_supp closed_in_def) |
18424 | 353 |
ultimately show "X\<sharp>S \<and> X\<sharp>T" by (force simp add: supp_prod fresh_def) |
18246 | 354 |
qed |
355 |
||
356 |
lemma subtype_eqvt: |
|
357 |
fixes pi::"tyvrs prm" |
|
358 |
shows "\<Gamma> \<turnstile> S <: T \<Longrightarrow> (pi\<bullet>\<Gamma>) \<turnstile> (pi\<bullet>S) <: (pi\<bullet>T)" |
|
18577
a636846a02c7
added more documentation; will now try out a modification
urbanc
parents:
18424
diff
changeset
|
359 |
apply(erule subtype_of.induct) |
18246 | 360 |
apply(force intro: valid_eqvt closed_in_eqvt) |
18655
73cebafb9a89
merged the silly lemmas into the eqvt proof of subtype
urbanc
parents:
18650
diff
changeset
|
361 |
apply(force intro!: S_Var |
73cebafb9a89
merged the silly lemmas into the eqvt proof of subtype
urbanc
parents:
18650
diff
changeset
|
362 |
intro: closed_in_eqvt valid_eqvt |
73cebafb9a89
merged the silly lemmas into the eqvt proof of subtype
urbanc
parents:
18650
diff
changeset
|
363 |
dest: pt_set_bij2[OF pt_tyvrs_inst, OF at_tyvrs_inst] |
73cebafb9a89
merged the silly lemmas into the eqvt proof of subtype
urbanc
parents:
18650
diff
changeset
|
364 |
simp add: pt_list_set_pi[OF pt_tyvrs_inst, symmetric]) |
73cebafb9a89
merged the silly lemmas into the eqvt proof of subtype
urbanc
parents:
18650
diff
changeset
|
365 |
apply(force intro: valid_eqvt |
73cebafb9a89
merged the silly lemmas into the eqvt proof of subtype
urbanc
parents:
18650
diff
changeset
|
366 |
dest: pt_set_bij2[OF pt_tyvrs_inst, OF at_tyvrs_inst] |
73cebafb9a89
merged the silly lemmas into the eqvt proof of subtype
urbanc
parents:
18650
diff
changeset
|
367 |
simp add: domain_eqvt) |
18246 | 368 |
apply(force) |
19972
89c5afe4139a
added more infrastructure for the recursion combinator
urbanc
parents:
19501
diff
changeset
|
369 |
apply(force intro!: S_Forall simp add: fresh_prod fresh_bij) |
18246 | 370 |
done |
371 |
||
18628 | 372 |
text {* The most painful part of the subtyping definition is the strengthening of the |
373 |
induction principle. The induction principle that comes for free with the definition of |
|
18650 | 374 |
@{term "subtype_of"} requires to prove the @{text "S_Forall"}-case for \emph{all} binders |
375 |
@{text "X"}. This will often cause some renaming-manoeuvres in the reasoning. To avoid this, |
|
18628 | 376 |
we strengthening the induction-principle so that we only have to establish |
18650 | 377 |
the @{text "S_Forall"}-case for \emph{fresh} binders @{text "X"}. The property that allows |
378 |
us to strengthen the induction-principle is that the equivariance of @{text "subtype_of"}. *} |
|
18628 | 379 |
|
18621 | 380 |
lemma subtype_of_induct[consumes 1, case_names S_Top S_Var S_Refl S_Arrow S_Forall]: |
18305
a780f9c1538b
changed everything until the interesting transitivity_narrowing
urbanc
parents:
18269
diff
changeset
|
381 |
fixes P :: "'a::fs_tyvrs\<Rightarrow>ty_context \<Rightarrow> ty \<Rightarrow> ty \<Rightarrow>bool" |
18246 | 382 |
assumes a: "\<Gamma> \<turnstile> S <: T" |
18621 | 383 |
and a1: "\<And>\<Gamma> S x. \<lbrakk>\<turnstile> \<Gamma> ok; S closed_in \<Gamma>\<rbrakk> \<Longrightarrow> P x \<Gamma> S Top" |
384 |
and a2: "\<And>\<Gamma> X S T x. \<lbrakk>(X,S)\<in>set \<Gamma>; \<Gamma> \<turnstile> S <: T; \<And>z. P z \<Gamma> S T\<rbrakk> \<Longrightarrow> P x \<Gamma> (Tvar X) T" |
|
385 |
and a3: "\<And>\<Gamma> X x. \<lbrakk>\<turnstile> \<Gamma> ok; X\<in>domain \<Gamma>\<rbrakk> \<Longrightarrow> P x \<Gamma> (Tvar X) (Tvar X)" |
|
18628 | 386 |
and a4: "\<And>\<Gamma> S\<^isub>1 S\<^isub>2 T\<^isub>1 T\<^isub>2 x. |
387 |
\<lbrakk>\<Gamma> \<turnstile> T\<^isub>1 <: S\<^isub>1; \<And>z. P z \<Gamma> T\<^isub>1 S\<^isub>1; \<Gamma> \<turnstile> S\<^isub>2 <: T\<^isub>2; \<And>z. P z \<Gamma> S\<^isub>2 T\<^isub>2\<rbrakk> |
|
18621 | 388 |
\<Longrightarrow> P x \<Gamma> (S\<^isub>1 \<rightarrow> S\<^isub>2) (T\<^isub>1 \<rightarrow> T\<^isub>2)" |
389 |
and a5: "\<And>\<Gamma> X S\<^isub>1 S\<^isub>2 T\<^isub>1 T\<^isub>2 x. |
|
18628 | 390 |
\<lbrakk>X\<sharp>x; X\<sharp>(\<Gamma>,S\<^isub>1,T\<^isub>1); \<Gamma> \<turnstile> T\<^isub>1 <: S\<^isub>1; \<And>z. P z \<Gamma> T\<^isub>1 S\<^isub>1; |
391 |
((X,T\<^isub>1)#\<Gamma>) \<turnstile> S\<^isub>2 <: T\<^isub>2; \<And>z. P z ((X,T\<^isub>1)#\<Gamma>) S\<^isub>2 T\<^isub>2\<rbrakk> |
|
18621 | 392 |
\<Longrightarrow> P x \<Gamma> (\<forall>[X<:S\<^isub>1].S\<^isub>2) (\<forall>[X<:T\<^isub>1].T\<^isub>2)" |
18305
a780f9c1538b
changed everything until the interesting transitivity_narrowing
urbanc
parents:
18269
diff
changeset
|
393 |
shows "P x \<Gamma> S T" |
a780f9c1538b
changed everything until the interesting transitivity_narrowing
urbanc
parents:
18269
diff
changeset
|
394 |
proof - |
a780f9c1538b
changed everything until the interesting transitivity_narrowing
urbanc
parents:
18269
diff
changeset
|
395 |
from a have "\<And>(pi::tyvrs prm) (x::'a::fs_tyvrs). P x (pi\<bullet>\<Gamma>) (pi\<bullet>S) (pi\<bullet>T)" |
a780f9c1538b
changed everything until the interesting transitivity_narrowing
urbanc
parents:
18269
diff
changeset
|
396 |
proof (induct) |
18424 | 397 |
case (S_Top S \<Gamma>) |
398 |
thus "P x (pi\<bullet>\<Gamma>) (pi\<bullet>S) (pi\<bullet>Top)" by (force intro: valid_eqvt closed_in_eqvt a1) |
|
18305
a780f9c1538b
changed everything until the interesting transitivity_narrowing
urbanc
parents:
18269
diff
changeset
|
399 |
next |
a780f9c1538b
changed everything until the interesting transitivity_narrowing
urbanc
parents:
18269
diff
changeset
|
400 |
case (S_Var S T X \<Gamma>) |
18577
a636846a02c7
added more documentation; will now try out a modification
urbanc
parents:
18424
diff
changeset
|
401 |
have "(X,S) \<in> set \<Gamma>" by fact |
a636846a02c7
added more documentation; will now try out a modification
urbanc
parents:
18424
diff
changeset
|
402 |
hence "pi\<bullet>(X,S)\<in>pi\<bullet>(set \<Gamma>)" by (rule pt_set_bij2[OF pt_tyvrs_inst, OF at_tyvrs_inst]) |
a636846a02c7
added more documentation; will now try out a modification
urbanc
parents:
18424
diff
changeset
|
403 |
hence "(pi\<bullet>X,pi\<bullet>S)\<in>set (pi\<bullet>\<Gamma>)" by (simp add: pt_list_set_pi[OF pt_tyvrs_inst]) |
18246 | 404 |
moreover |
18577
a636846a02c7
added more documentation; will now try out a modification
urbanc
parents:
18424
diff
changeset
|
405 |
have "\<Gamma> \<turnstile> S <: T" by fact |
a636846a02c7
added more documentation; will now try out a modification
urbanc
parents:
18424
diff
changeset
|
406 |
hence "(pi\<bullet>\<Gamma>) \<turnstile> (pi\<bullet>S) <: (pi\<bullet>T)" by (rule subtype_eqvt) |
a636846a02c7
added more documentation; will now try out a modification
urbanc
parents:
18424
diff
changeset
|
407 |
moreover |
a636846a02c7
added more documentation; will now try out a modification
urbanc
parents:
18424
diff
changeset
|
408 |
have "\<And>(pi::tyvrs prm) x. P x (pi\<bullet>\<Gamma>) (pi\<bullet>S) (pi\<bullet>T)" by fact |
a636846a02c7
added more documentation; will now try out a modification
urbanc
parents:
18424
diff
changeset
|
409 |
hence "\<And>x. P x (pi\<bullet>\<Gamma>) (pi\<bullet>S) (pi\<bullet>T)" by simp |
18246 | 410 |
ultimately |
18577
a636846a02c7
added more documentation; will now try out a modification
urbanc
parents:
18424
diff
changeset
|
411 |
show "P x (pi\<bullet>\<Gamma>) (pi\<bullet>(Tvar X)) (pi\<bullet>T)" by (simp add: a2) |
18305
a780f9c1538b
changed everything until the interesting transitivity_narrowing
urbanc
parents:
18269
diff
changeset
|
412 |
next |
a780f9c1538b
changed everything until the interesting transitivity_narrowing
urbanc
parents:
18269
diff
changeset
|
413 |
case (S_Refl X \<Gamma>) |
18577
a636846a02c7
added more documentation; will now try out a modification
urbanc
parents:
18424
diff
changeset
|
414 |
have "\<turnstile> \<Gamma> ok" by fact |
a636846a02c7
added more documentation; will now try out a modification
urbanc
parents:
18424
diff
changeset
|
415 |
hence "\<turnstile> (pi\<bullet>\<Gamma>) ok" by (rule valid_eqvt) |
18246 | 416 |
moreover |
18577
a636846a02c7
added more documentation; will now try out a modification
urbanc
parents:
18424
diff
changeset
|
417 |
have "X \<in> domain \<Gamma>" by fact |
a636846a02c7
added more documentation; will now try out a modification
urbanc
parents:
18424
diff
changeset
|
418 |
hence "(pi\<bullet>X)\<in>pi\<bullet>domain \<Gamma>" by (rule pt_set_bij2[OF pt_tyvrs_inst, OF at_tyvrs_inst]) |
18246 | 419 |
hence "(pi\<bullet>X)\<in>domain (pi\<bullet>\<Gamma>)" by (simp add: domain_eqvt pt_list_set_pi[OF pt_tyvrs_inst]) |
18577
a636846a02c7
added more documentation; will now try out a modification
urbanc
parents:
18424
diff
changeset
|
420 |
ultimately show "P x (pi\<bullet>\<Gamma>) (pi\<bullet>(Tvar X)) (pi\<bullet>(Tvar X))" by (simp add: a3) |
18305
a780f9c1538b
changed everything until the interesting transitivity_narrowing
urbanc
parents:
18269
diff
changeset
|
421 |
next |
18424 | 422 |
case S_Arrow thus ?case by (auto intro: a4 subtype_eqvt) |
18305
a780f9c1538b
changed everything until the interesting transitivity_narrowing
urbanc
parents:
18269
diff
changeset
|
423 |
next |
18621 | 424 |
case (S_Forall S1 S2 T1 T2 X \<Gamma>) |
18305
a780f9c1538b
changed everything until the interesting transitivity_narrowing
urbanc
parents:
18269
diff
changeset
|
425 |
have b1: "\<Gamma> \<turnstile> T1 <: S1" by fact |
a780f9c1538b
changed everything until the interesting transitivity_narrowing
urbanc
parents:
18269
diff
changeset
|
426 |
have b2: "\<And>(pi::tyvrs prm) x. P x (pi\<bullet>\<Gamma>) (pi\<bullet>T1) (pi\<bullet>S1)" by fact |
a780f9c1538b
changed everything until the interesting transitivity_narrowing
urbanc
parents:
18269
diff
changeset
|
427 |
have b4: "((X,T1)#\<Gamma>) \<turnstile> S2 <: T2" by fact |
a780f9c1538b
changed everything until the interesting transitivity_narrowing
urbanc
parents:
18269
diff
changeset
|
428 |
have b5: "\<And>(pi::tyvrs prm) x. P x (pi\<bullet>((X,T1)#\<Gamma>)) (pi\<bullet>S2) (pi\<bullet>T2)" by fact |
18577
a636846a02c7
added more documentation; will now try out a modification
urbanc
parents:
18424
diff
changeset
|
429 |
have b3: "X\<sharp>\<Gamma>" by fact |
a636846a02c7
added more documentation; will now try out a modification
urbanc
parents:
18424
diff
changeset
|
430 |
have b3': "X\<sharp>T1" "X\<sharp>S1" using b1 b3 by (simp_all add: subtype_implies_fresh) |
18246 | 431 |
have "\<exists>C::tyvrs. C\<sharp>(pi\<bullet>X,pi\<bullet>S2,pi\<bullet>T2,pi\<bullet>S1,pi\<bullet>T1,pi\<bullet>\<Gamma>,x)" |
21377
c29146dc14f1
replaced exists_fresh lemma with a version formulated with obtains;
urbanc
parents:
21087
diff
changeset
|
432 |
by (rule exists_fresh', simp add: fs_tyvrs1) |
18246 | 433 |
then obtain C::"tyvrs" where f1: "C\<noteq>(pi\<bullet>X)" and f2: "C\<sharp>(pi\<bullet>S1)" and f3: "C\<sharp>(pi\<bullet>T1)" |
434 |
and f4: "C\<sharp>(pi\<bullet>S2)" and f5: "C\<sharp>(pi\<bullet>T2)" and f6: "C\<sharp>(pi\<bullet>\<Gamma>)" and f7: "C\<sharp>x" |
|
435 |
by (auto simp add: fresh_prod fresh_atm) |
|
436 |
let ?pi' = "[(C,pi\<bullet>X)]@pi" |
|
18305
a780f9c1538b
changed everything until the interesting transitivity_narrowing
urbanc
parents:
18269
diff
changeset
|
437 |
from b2 have c1: "\<And>x. P x (?pi'\<bullet>\<Gamma>) (?pi'\<bullet>T1) (?pi'\<bullet>S1)" by simp |
a780f9c1538b
changed everything until the interesting transitivity_narrowing
urbanc
parents:
18269
diff
changeset
|
438 |
from b5 have "\<And>x. P x (?pi'\<bullet>((X,T1)#\<Gamma>)) (?pi'\<bullet>S2) (?pi'\<bullet>T2)" by simp |
a780f9c1538b
changed everything until the interesting transitivity_narrowing
urbanc
parents:
18269
diff
changeset
|
439 |
hence "\<And>x. P x ((?pi'\<bullet>X,?pi'\<bullet>T1)#(?pi'\<bullet>\<Gamma>)) (?pi'\<bullet>S2) (?pi'\<bullet>T2)" by simp |
a780f9c1538b
changed everything until the interesting transitivity_narrowing
urbanc
parents:
18269
diff
changeset
|
440 |
hence c2: "\<And>x. P x ((C,?pi'\<bullet>T1)#(?pi'\<bullet>\<Gamma>)) (?pi'\<bullet>S2) (?pi'\<bullet>T2)" using f1 |
18246 | 441 |
by (simp only: pt_tyvrs2 calc_atm, simp) |
442 |
from b3 have "(pi\<bullet>X)\<sharp>(pi\<bullet>\<Gamma>)" |
|
443 |
by (simp add: fresh_prod pt_fresh_bij[OF pt_tyvrs_inst, OF at_tyvrs_inst]) |
|
444 |
with f6 have f6a: "?pi'\<bullet>\<Gamma>=pi\<bullet>\<Gamma>" |
|
445 |
by (simp only: pt_tyvrs2 pt_fresh_fresh[OF pt_tyvrs_inst, OF at_tyvrs_inst]) |
|
446 |
hence f6': "C\<sharp>(?pi'\<bullet>\<Gamma>)" using f6 by simp |
|
18577
a636846a02c7
added more documentation; will now try out a modification
urbanc
parents:
18424
diff
changeset
|
447 |
from b3' have "(pi\<bullet>X)\<sharp>(pi\<bullet>S1)" |
18246 | 448 |
by (simp add: fresh_prod pt_fresh_bij[OF pt_tyvrs_inst, OF at_tyvrs_inst]) |
449 |
with f2 have f2a: "?pi'\<bullet>S1=pi\<bullet>S1" |
|
450 |
by (simp only: pt_tyvrs2 pt_fresh_fresh[OF pt_tyvrs_inst, OF at_tyvrs_inst]) |
|
451 |
hence f2': "C\<sharp>(?pi'\<bullet>S1)" using f2 by simp |
|
18577
a636846a02c7
added more documentation; will now try out a modification
urbanc
parents:
18424
diff
changeset
|
452 |
from b3' have "(pi\<bullet>X)\<sharp>(pi\<bullet>T1)" |
18246 | 453 |
by (simp add: fresh_prod pt_fresh_bij[OF pt_tyvrs_inst, OF at_tyvrs_inst]) |
454 |
with f3 have f3a: "?pi'\<bullet>T1=pi\<bullet>T1" |
|
455 |
by (simp only: pt_tyvrs2 pt_fresh_fresh[OF pt_tyvrs_inst, OF at_tyvrs_inst]) |
|
456 |
hence f3': "C\<sharp>(?pi'\<bullet>T1)" using f3 by simp |
|
457 |
from b1 have e1: "(?pi'\<bullet>\<Gamma>) \<turnstile> (?pi'\<bullet>T1) <: (?pi'\<bullet>S1)" by (rule subtype_eqvt) |
|
458 |
from b4 have "(?pi'\<bullet>((X,T1)#\<Gamma>)) \<turnstile> (?pi'\<bullet>S2) <: (?pi'\<bullet>T2)" by (rule subtype_eqvt) |
|
459 |
hence "((?pi'\<bullet>X,?pi'\<bullet>T1)#(?pi'\<bullet>\<Gamma>)) \<turnstile> (?pi'\<bullet>S2) <: (?pi'\<bullet>T2)" by simp |
|
460 |
hence e2: "((C,?pi'\<bullet>T1)#(?pi'\<bullet>\<Gamma>)) \<turnstile> (?pi'\<bullet>S2) <: (?pi'\<bullet>T2)" using f1 |
|
461 |
by (simp only: pt_tyvrs2 calc_atm, simp) |
|
462 |
have fnew: "C\<sharp>(?pi'\<bullet>\<Gamma>,?pi'\<bullet>S1,?pi'\<bullet>T1)" using f6' f2' f3' by (simp add: fresh_prod) |
|
18577
a636846a02c7
added more documentation; will now try out a modification
urbanc
parents:
18424
diff
changeset
|
463 |
have main: "P x (?pi'\<bullet>\<Gamma>) (\<forall>[C<:(?pi'\<bullet>S1)].(?pi'\<bullet>S2)) (\<forall>[C<:(?pi'\<bullet>T1)].(?pi'\<bullet>T2))" |
18246 | 464 |
using f7 fnew e1 c1 e2 c2 by (rule a5) |
18577
a636846a02c7
added more documentation; will now try out a modification
urbanc
parents:
18424
diff
changeset
|
465 |
have alpha1: "(\<forall>[C<:(?pi'\<bullet>S1)].(?pi'\<bullet>S2)) = (pi\<bullet>(\<forall>[X<:S1].S2))" |
18246 | 466 |
using f1 f4 f2a[symmetric] by (simp add: ty.inject alpha pt_tyvrs2[symmetric]) |
18577
a636846a02c7
added more documentation; will now try out a modification
urbanc
parents:
18424
diff
changeset
|
467 |
have alpha2: "(\<forall>[C<:(?pi'\<bullet>T1)].(?pi'\<bullet>T2)) = (pi\<bullet>(\<forall>[X<:T1].T2))" |
18246 | 468 |
using f1 f5 f3a[symmetric] by (simp add: ty.inject alpha pt_tyvrs2[symmetric]) |
18577
a636846a02c7
added more documentation; will now try out a modification
urbanc
parents:
18424
diff
changeset
|
469 |
show "P x (pi\<bullet>\<Gamma>) (pi\<bullet>(\<forall>[X<:S1].S2)) (pi\<bullet>(\<forall>[X<:T1].T2))" |
18246 | 470 |
using alpha1 alpha2 f6a main by simp |
471 |
qed |
|
18305
a780f9c1538b
changed everything until the interesting transitivity_narrowing
urbanc
parents:
18269
diff
changeset
|
472 |
hence "P x (([]::tyvrs prm)\<bullet>\<Gamma>) (([]::tyvrs prm)\<bullet>S) (([]::tyvrs prm)\<bullet>T)" by blast |
a780f9c1538b
changed everything until the interesting transitivity_narrowing
urbanc
parents:
18269
diff
changeset
|
473 |
thus ?thesis by simp |
18246 | 474 |
qed |
475 |
||
18621 | 476 |
section {* Reflexivity of Subtyping *} |
18246 | 477 |
|
478 |
lemma subtype_reflexivity: |
|
18353
4dd468ccfdf7
transitivity should be now in a reasonable state. But
urbanc
parents:
18306
diff
changeset
|
479 |
assumes a: "\<turnstile> \<Gamma> ok" |
18424 | 480 |
and b: "T closed_in \<Gamma>" |
18353
4dd468ccfdf7
transitivity should be now in a reasonable state. But
urbanc
parents:
18306
diff
changeset
|
481 |
shows "\<Gamma> \<turnstile> T <: T" |
4dd468ccfdf7
transitivity should be now in a reasonable state. But
urbanc
parents:
18306
diff
changeset
|
482 |
using a b |
18660
9968dc816cda
cahges to use the new induction-principle (now proved in
urbanc
parents:
18655
diff
changeset
|
483 |
proof(nominal_induct T avoiding: \<Gamma> rule: ty.induct) |
18577
a636846a02c7
added more documentation; will now try out a modification
urbanc
parents:
18424
diff
changeset
|
484 |
case (Forall X T\<^isub>1 T\<^isub>2) |
18747 | 485 |
have ih_T\<^isub>1: "\<And>\<Gamma>. \<lbrakk>\<turnstile> \<Gamma> ok; T\<^isub>1 closed_in \<Gamma>\<rbrakk> \<Longrightarrow> \<Gamma> \<turnstile> T\<^isub>1 <: T\<^isub>1" by fact |
486 |
have ih_T\<^isub>2: "\<And>\<Gamma>. \<lbrakk>\<turnstile> \<Gamma> ok; T\<^isub>2 closed_in \<Gamma>\<rbrakk> \<Longrightarrow> \<Gamma> \<turnstile> T\<^isub>2 <: T\<^isub>2" by fact |
|
18424 | 487 |
have fresh_cond: "X\<sharp>\<Gamma>" by fact |
18621 | 488 |
hence fresh_domain: "X\<sharp>(domain \<Gamma>)" by (simp add: fresh_domain) |
18424 | 489 |
have "(\<forall>[X<:T\<^isub>2].T\<^isub>1) closed_in \<Gamma>" by fact |
490 |
hence closed\<^isub>T\<^isub>2: "T\<^isub>2 closed_in \<Gamma>" and closed\<^isub>T\<^isub>1: "T\<^isub>1 closed_in ((X,T\<^isub>2)#\<Gamma>)" |
|
491 |
by (auto simp add: closed_in_def ty.supp abs_supp) |
|
492 |
have ok: "\<turnstile> \<Gamma> ok" by fact |
|
18621 | 493 |
hence ok': "\<turnstile> ((X,T\<^isub>2)#\<Gamma>) ok" using closed\<^isub>T\<^isub>2 fresh_domain by simp |
18424 | 494 |
have "\<Gamma> \<turnstile> T\<^isub>2 <: T\<^isub>2" using ih_T\<^isub>2 closed\<^isub>T\<^isub>2 ok by simp |
18353
4dd468ccfdf7
transitivity should be now in a reasonable state. But
urbanc
parents:
18306
diff
changeset
|
495 |
moreover |
18424 | 496 |
have "((X,T\<^isub>2)#\<Gamma>) \<turnstile> T\<^isub>1 <: T\<^isub>1" using ih_T\<^isub>1 closed\<^isub>T\<^isub>1 ok' by simp |
497 |
ultimately show "\<Gamma> \<turnstile> \<forall>[X<:T\<^isub>2].T\<^isub>1 <: \<forall>[X<:T\<^isub>2].T\<^isub>1" using fresh_cond |
|
18621 | 498 |
by (simp add: subtype_of.S_Forall) |
18246 | 499 |
qed (auto simp add: closed_in_def ty.supp supp_atm) |
500 |
||
18621 | 501 |
lemma subtype_reflexivity_semiautomated: |
18305
a780f9c1538b
changed everything until the interesting transitivity_narrowing
urbanc
parents:
18269
diff
changeset
|
502 |
assumes a: "\<turnstile> \<Gamma> ok" |
a780f9c1538b
changed everything until the interesting transitivity_narrowing
urbanc
parents:
18269
diff
changeset
|
503 |
and b: "T closed_in \<Gamma>" |
a780f9c1538b
changed everything until the interesting transitivity_narrowing
urbanc
parents:
18269
diff
changeset
|
504 |
shows "\<Gamma> \<turnstile> T <: T" |
a780f9c1538b
changed everything until the interesting transitivity_narrowing
urbanc
parents:
18269
diff
changeset
|
505 |
using a b |
18660
9968dc816cda
cahges to use the new induction-principle (now proved in
urbanc
parents:
18655
diff
changeset
|
506 |
apply(nominal_induct T avoiding: \<Gamma> rule: ty.induct) |
18747 | 507 |
apply(auto simp add: ty.supp abs_supp supp_atm closed_in_def) |
18577
a636846a02c7
added more documentation; will now try out a modification
urbanc
parents:
18424
diff
changeset
|
508 |
--{* Too bad that this instantiation cannot be found automatically by |
18621 | 509 |
\isakeyword{auto}; \isakeyword{blast} would find it if we had not used |
18628 | 510 |
an explicit definition for @{text "closed_in_def"}. *} |
18305
a780f9c1538b
changed everything until the interesting transitivity_narrowing
urbanc
parents:
18269
diff
changeset
|
511 |
apply(drule_tac x="(tyvrs, ty2)#\<Gamma>" in meta_spec) |
18747 | 512 |
apply(force dest: fresh_domain simp add: closed_in_def) |
18246 | 513 |
done |
514 |
||
18747 | 515 |
|
18628 | 516 |
section {* Weakening *} |
18246 | 517 |
|
18628 | 518 |
text {* In order to prove weakening we introduce the notion of a type-context extending |
519 |
another. This generalization seems to make the proof for weakening to be |
|
520 |
smoother than if we had strictly adhered to the version in the POPLmark-paper. *} |
|
18246 | 521 |
|
522 |
constdefs |
|
523 |
extends :: "ty_context \<Rightarrow> ty_context \<Rightarrow> bool" ("_ extends _" [100,100] 100) |
|
524 |
"\<Delta> extends \<Gamma> \<equiv> \<forall>X Q. (X,Q)\<in>set \<Gamma> \<longrightarrow> (X,Q)\<in>set \<Delta>" |
|
525 |
||
526 |
lemma extends_domain: |
|
527 |
assumes a: "\<Delta> extends \<Gamma>" |
|
528 |
shows "domain \<Gamma> \<subseteq> domain \<Delta>" |
|
529 |
using a |
|
530 |
apply (auto simp add: extends_def) |
|
531 |
apply (drule domain_existence) |
|
532 |
apply (force simp add: domain_inclusion) |
|
533 |
done |
|
534 |
||
535 |
lemma extends_closed: |
|
536 |
assumes a1: "T closed_in \<Gamma>" |
|
537 |
and a2: "\<Delta> extends \<Gamma>" |
|
538 |
shows "T closed_in \<Delta>" |
|
539 |
using a1 a2 |
|
540 |
by (auto dest: extends_domain simp add: closed_in_def) |
|
541 |
||
18424 | 542 |
lemma extends_memb: |
543 |
assumes a: "\<Delta> extends \<Gamma>" |
|
544 |
and b: "(X,T) \<in> set \<Gamma>" |
|
545 |
shows "(X,T) \<in> set \<Delta>" |
|
546 |
using a b by (simp add: extends_def) |
|
547 |
||
18246 | 548 |
lemma weakening: |
18353
4dd468ccfdf7
transitivity should be now in a reasonable state. But
urbanc
parents:
18306
diff
changeset
|
549 |
assumes a: "\<Gamma> \<turnstile> S <: T" |
18424 | 550 |
and b: "\<turnstile> \<Delta> ok" |
551 |
and c: "\<Delta> extends \<Gamma>" |
|
18353
4dd468ccfdf7
transitivity should be now in a reasonable state. But
urbanc
parents:
18306
diff
changeset
|
552 |
shows "\<Delta> \<turnstile> S <: T" |
4dd468ccfdf7
transitivity should be now in a reasonable state. But
urbanc
parents:
18306
diff
changeset
|
553 |
using a b c |
18577
a636846a02c7
added more documentation; will now try out a modification
urbanc
parents:
18424
diff
changeset
|
554 |
proof (nominal_induct \<Gamma> S T avoiding: \<Delta> rule: subtype_of_induct) |
18305
a780f9c1538b
changed everything until the interesting transitivity_narrowing
urbanc
parents:
18269
diff
changeset
|
555 |
case (S_Top \<Gamma> S) |
18246 | 556 |
have lh_drv_prem: "S closed_in \<Gamma>" by fact |
18353
4dd468ccfdf7
transitivity should be now in a reasonable state. But
urbanc
parents:
18306
diff
changeset
|
557 |
have "\<turnstile> \<Delta> ok" by fact |
4dd468ccfdf7
transitivity should be now in a reasonable state. But
urbanc
parents:
18306
diff
changeset
|
558 |
moreover |
4dd468ccfdf7
transitivity should be now in a reasonable state. But
urbanc
parents:
18306
diff
changeset
|
559 |
have "\<Delta> extends \<Gamma>" by fact |
18424 | 560 |
hence "S closed_in \<Delta>" using lh_drv_prem by (simp only: extends_closed) |
18353
4dd468ccfdf7
transitivity should be now in a reasonable state. But
urbanc
parents:
18306
diff
changeset
|
561 |
ultimately show "\<Delta> \<turnstile> S <: Top" by force |
18246 | 562 |
next |
18305
a780f9c1538b
changed everything until the interesting transitivity_narrowing
urbanc
parents:
18269
diff
changeset
|
563 |
case (S_Var \<Gamma> X S T) |
18246 | 564 |
have lh_drv_prem: "(X,S) \<in> set \<Gamma>" by fact |
18353
4dd468ccfdf7
transitivity should be now in a reasonable state. But
urbanc
parents:
18306
diff
changeset
|
565 |
have ih: "\<And>\<Delta>. \<turnstile> \<Delta> ok \<Longrightarrow> \<Delta> extends \<Gamma> \<Longrightarrow> \<Delta> \<turnstile> S <: T" by fact |
4dd468ccfdf7
transitivity should be now in a reasonable state. But
urbanc
parents:
18306
diff
changeset
|
566 |
have ok: "\<turnstile> \<Delta> ok" by fact |
4dd468ccfdf7
transitivity should be now in a reasonable state. But
urbanc
parents:
18306
diff
changeset
|
567 |
have extends: "\<Delta> extends \<Gamma>" by fact |
18424 | 568 |
have "(X,S) \<in> set \<Delta>" using lh_drv_prem extends by (simp only: extends_memb) |
18353
4dd468ccfdf7
transitivity should be now in a reasonable state. But
urbanc
parents:
18306
diff
changeset
|
569 |
moreover |
4dd468ccfdf7
transitivity should be now in a reasonable state. But
urbanc
parents:
18306
diff
changeset
|
570 |
have "\<Delta> \<turnstile> S <: T" using ok extends ih by simp |
18577
a636846a02c7
added more documentation; will now try out a modification
urbanc
parents:
18424
diff
changeset
|
571 |
ultimately show "\<Delta> \<turnstile> Tvar X <: T" using ok by force |
18246 | 572 |
next |
18305
a780f9c1538b
changed everything until the interesting transitivity_narrowing
urbanc
parents:
18269
diff
changeset
|
573 |
case (S_Refl \<Gamma> X) |
18246 | 574 |
have lh_drv_prem: "X \<in> domain \<Gamma>" by fact |
18353
4dd468ccfdf7
transitivity should be now in a reasonable state. But
urbanc
parents:
18306
diff
changeset
|
575 |
have "\<turnstile> \<Delta> ok" by fact |
4dd468ccfdf7
transitivity should be now in a reasonable state. But
urbanc
parents:
18306
diff
changeset
|
576 |
moreover |
4dd468ccfdf7
transitivity should be now in a reasonable state. But
urbanc
parents:
18306
diff
changeset
|
577 |
have "\<Delta> extends \<Gamma>" by fact |
4dd468ccfdf7
transitivity should be now in a reasonable state. But
urbanc
parents:
18306
diff
changeset
|
578 |
hence "X \<in> domain \<Delta>" using lh_drv_prem by (force dest: extends_domain) |
18577
a636846a02c7
added more documentation; will now try out a modification
urbanc
parents:
18424
diff
changeset
|
579 |
ultimately show "\<Delta> \<turnstile> Tvar X <: Tvar X" by force |
18246 | 580 |
next |
18424 | 581 |
case (S_Arrow \<Gamma> S\<^isub>1 S\<^isub>2 T\<^isub>1 T\<^isub>2) thus "\<Delta> \<turnstile> S\<^isub>1 \<rightarrow> S\<^isub>2 <: T\<^isub>1 \<rightarrow> T\<^isub>2" by blast |
18246 | 582 |
next |
18621 | 583 |
case (S_Forall \<Gamma> X S\<^isub>1 S\<^isub>2 T\<^isub>1 T\<^isub>2) |
18424 | 584 |
have fresh_cond: "X\<sharp>\<Delta>" by fact |
18621 | 585 |
hence fresh_domain: "X\<sharp>(domain \<Delta>)" by (simp add: fresh_domain) |
18424 | 586 |
have ih\<^isub>1: "\<And>\<Delta>. \<turnstile> \<Delta> ok \<Longrightarrow> \<Delta> extends \<Gamma> \<Longrightarrow> \<Delta> \<turnstile> T\<^isub>1 <: S\<^isub>1" by fact |
587 |
have ih\<^isub>2: "\<And>\<Delta>. \<turnstile> \<Delta> ok \<Longrightarrow> \<Delta> extends ((X,T\<^isub>1)#\<Gamma>) \<Longrightarrow> \<Delta> \<turnstile> S\<^isub>2 <: T\<^isub>2" by fact |
|
588 |
have lh_drv_prem: "\<Gamma> \<turnstile> T\<^isub>1 <: S\<^isub>1" by fact |
|
589 |
hence closed\<^isub>T\<^isub>1: "T\<^isub>1 closed_in \<Gamma>" by (simp add: subtype_implies_closed) |
|
18353
4dd468ccfdf7
transitivity should be now in a reasonable state. But
urbanc
parents:
18306
diff
changeset
|
590 |
have ok: "\<turnstile> \<Delta> ok" by fact |
18424 | 591 |
have ext: "\<Delta> extends \<Gamma>" by fact |
592 |
have "T\<^isub>1 closed_in \<Delta>" using ext closed\<^isub>T\<^isub>1 by (simp only: extends_closed) |
|
18621 | 593 |
hence "\<turnstile> ((X,T\<^isub>1)#\<Delta>) ok" using fresh_domain ok by force |
18353
4dd468ccfdf7
transitivity should be now in a reasonable state. But
urbanc
parents:
18306
diff
changeset
|
594 |
moreover |
18424 | 595 |
have "((X,T\<^isub>1)#\<Delta>) extends ((X,T\<^isub>1)#\<Gamma>)" using ext by (force simp add: extends_def) |
596 |
ultimately have "((X,T\<^isub>1)#\<Delta>) \<turnstile> S\<^isub>2 <: T\<^isub>2" using ih\<^isub>2 by simp |
|
18353
4dd468ccfdf7
transitivity should be now in a reasonable state. But
urbanc
parents:
18306
diff
changeset
|
597 |
moreover |
18424 | 598 |
have "\<Delta> \<turnstile> T\<^isub>1 <: S\<^isub>1" using ok ext ih\<^isub>1 by simp |
18621 | 599 |
ultimately show "\<Delta> \<turnstile> \<forall>[X<:S\<^isub>1].S\<^isub>2 <: \<forall>[X<:T\<^isub>1].T\<^isub>2" using ok by (force intro: S_Forall) |
18246 | 600 |
qed |
601 |
||
18650 | 602 |
text {* In fact all ``non-binding" cases can be solved automatically: *} |
18246 | 603 |
|
18628 | 604 |
lemma weakening_more_automated: |
18353
4dd468ccfdf7
transitivity should be now in a reasonable state. But
urbanc
parents:
18306
diff
changeset
|
605 |
assumes a: "\<Gamma> \<turnstile> S <: T" |
18424 | 606 |
and b: "\<turnstile> \<Delta> ok" |
607 |
and c: "\<Delta> extends \<Gamma>" |
|
18353
4dd468ccfdf7
transitivity should be now in a reasonable state. But
urbanc
parents:
18306
diff
changeset
|
608 |
shows "\<Delta> \<turnstile> S <: T" |
4dd468ccfdf7
transitivity should be now in a reasonable state. But
urbanc
parents:
18306
diff
changeset
|
609 |
using a b c |
18577
a636846a02c7
added more documentation; will now try out a modification
urbanc
parents:
18424
diff
changeset
|
610 |
proof (nominal_induct \<Gamma> S T avoiding: \<Delta> rule: subtype_of_induct) |
18621 | 611 |
case (S_Forall \<Gamma> X S\<^isub>1 S\<^isub>2 T\<^isub>1 T\<^isub>2) |
18424 | 612 |
have fresh_cond: "X\<sharp>\<Delta>" by fact |
18621 | 613 |
hence fresh_domain: "X\<sharp>(domain \<Delta>)" by (simp add: fresh_domain) |
18424 | 614 |
have ih\<^isub>1: "\<And>\<Delta>. \<turnstile> \<Delta> ok \<Longrightarrow> \<Delta> extends \<Gamma> \<Longrightarrow> \<Delta> \<turnstile> T\<^isub>1 <: S\<^isub>1" by fact |
615 |
have ih\<^isub>2: "\<And>\<Delta>. \<turnstile> \<Delta> ok \<Longrightarrow> \<Delta> extends ((X,T\<^isub>1)#\<Gamma>) \<Longrightarrow> \<Delta> \<turnstile> S\<^isub>2 <: T\<^isub>2" by fact |
|
616 |
have lh_drv_prem: "\<Gamma> \<turnstile> T\<^isub>1 <: S\<^isub>1" by fact |
|
617 |
hence closed\<^isub>T\<^isub>1: "T\<^isub>1 closed_in \<Gamma>" by (simp add: subtype_implies_closed) |
|
18353
4dd468ccfdf7
transitivity should be now in a reasonable state. But
urbanc
parents:
18306
diff
changeset
|
618 |
have ok: "\<turnstile> \<Delta> ok" by fact |
18424 | 619 |
have ext: "\<Delta> extends \<Gamma>" by fact |
620 |
have "T\<^isub>1 closed_in \<Delta>" using ext closed\<^isub>T\<^isub>1 by (simp only: extends_closed) |
|
18621 | 621 |
hence "\<turnstile> ((X,T\<^isub>1)#\<Delta>) ok" using fresh_domain ok by force |
18628 | 622 |
moreover |
18424 | 623 |
have "((X,T\<^isub>1)#\<Delta>) extends ((X,T\<^isub>1)#\<Gamma>)" using ext by (force simp add: extends_def) |
624 |
ultimately have "((X,T\<^isub>1)#\<Delta>) \<turnstile> S\<^isub>2 <: T\<^isub>2" using ih\<^isub>2 by simp |
|
18353
4dd468ccfdf7
transitivity should be now in a reasonable state. But
urbanc
parents:
18306
diff
changeset
|
625 |
moreover |
18424 | 626 |
have "\<Delta> \<turnstile> T\<^isub>1 <: S\<^isub>1" using ok ext ih\<^isub>1 by simp |
18621 | 627 |
ultimately show "\<Delta> \<turnstile> \<forall>[X<:S\<^isub>1].S\<^isub>2 <: \<forall>[X<:T\<^isub>1].T\<^isub>2" using ok by (force intro: S_Forall) |
18424 | 628 |
qed (blast intro: extends_closed extends_memb dest: extends_domain)+ |
18246 | 629 |
|
18628 | 630 |
section {* Transitivity and Narrowing *} |
631 |
||
18650 | 632 |
text {* Some inversion lemmas that are needed in the transitivity and narrowing proof.*} |
633 |
||
634 |
lemma S_TopE: |
|
635 |
assumes a: "\<Gamma> \<turnstile> Top <: T" |
|
636 |
shows "T = Top" |
|
637 |
using a by (cases, auto) |
|
638 |
||
639 |
lemma S_ArrowE_left: |
|
640 |
assumes a: "\<Gamma> \<turnstile> S\<^isub>1 \<rightarrow> S\<^isub>2 <: T" |
|
641 |
shows "T = Top \<or> (\<exists>T\<^isub>1 T\<^isub>2. T = T\<^isub>1 \<rightarrow> T\<^isub>2 \<and> \<Gamma> \<turnstile> T\<^isub>1 <: S\<^isub>1 \<and> \<Gamma> \<turnstile> S\<^isub>2 <: T\<^isub>2)" |
|
642 |
using a by (cases, auto simp add: ty.inject) |
|
643 |
||
644 |
lemma S_ForallE_left: |
|
645 |
shows "\<lbrakk>\<Gamma> \<turnstile> \<forall>[X<:S\<^isub>1].S\<^isub>2 <: T; X\<sharp>\<Gamma>; X\<sharp>S\<^isub>1\<rbrakk> |
|
646 |
\<Longrightarrow> T = Top \<or> (\<exists>T\<^isub>1 T\<^isub>2. T = \<forall>[X<:T\<^isub>1].T\<^isub>2 \<and> \<Gamma> \<turnstile> T\<^isub>1 <: S\<^isub>1 \<and> ((X,T\<^isub>1)#\<Gamma>) \<turnstile> S\<^isub>2 <: T\<^isub>2)" |
|
647 |
apply(frule subtype_implies_ok) |
|
648 |
apply(ind_cases "\<Gamma> \<turnstile> \<forall>[X<:S\<^isub>1].S\<^isub>2 <: T") |
|
649 |
apply(auto simp add: ty.inject alpha) |
|
650 |
apply(rule_tac x="[(X,Xa)]\<bullet>T\<^isub>2" in exI) |
|
651 |
apply(rule conjI) |
|
652 |
apply(rule sym) |
|
653 |
apply(rule pt_bij2[OF pt_tyvrs_inst, OF at_tyvrs_inst]) |
|
654 |
apply(rule pt_tyvrs3) |
|
655 |
apply(simp) |
|
656 |
apply(rule at_ds5[OF at_tyvrs_inst]) |
|
657 |
apply(rule conjI) |
|
658 |
apply(simp add: pt_fresh_left[OF pt_tyvrs_inst, OF at_tyvrs_inst] calc_atm) |
|
659 |
apply(drule_tac \<Gamma>="((Xa,T\<^isub>1)#\<Gamma>)" in subtype_implies_closed)+ |
|
660 |
apply(simp add: closed_in_def) |
|
661 |
apply(drule fresh_domain)+ |
|
662 |
apply(simp add: fresh_def) |
|
663 |
apply(subgoal_tac "X \<notin> (insert Xa (domain \<Gamma>))")(*A*) |
|
664 |
apply(force) |
|
665 |
(*A*)apply(simp add: at_fin_set_supp[OF at_tyvrs_inst, OF finite_domain]) |
|
666 |
(* 2nd conjunct *)apply(frule_tac X="X" in subtype_implies_fresh) |
|
667 |
apply(assumption) |
|
668 |
apply(drule_tac X="Xa" in subtype_implies_fresh) |
|
669 |
apply(assumption) |
|
670 |
apply(simp add: fresh_prod) |
|
671 |
apply(drule_tac pi="[(X,Xa)]" in subtype_eqvt) |
|
672 |
apply(simp add: calc_atm) |
|
673 |
apply(simp add: pt_fresh_fresh[OF pt_tyvrs_inst, OF at_tyvrs_inst]) |
|
674 |
done |
|
675 |
||
676 |
text {* Next we prove the transitivity and narrowing for the subtyping-relation. |
|
18621 | 677 |
The POPLmark-paper says the following: |
678 |
||
18650 | 679 |
\begin{quote} |
18621 | 680 |
\begin{lemma}[Transitivity and Narrowing] \ |
681 |
\begin{enumerate} |
|
682 |
\item If @{term "\<Gamma> \<turnstile> S<:Q"} and @{term "\<Gamma> \<turnstile> Q<:T"}, then @{term "\<Gamma> \<turnstile> S<:T"}. |
|
683 |
\item If @{text "\<Gamma>,X<:Q,\<Delta> \<turnstile> M<:N"} and @{term "\<Gamma> \<turnstile> P<:Q"} then @{text "\<Gamma>,X<:P,\<Delta> \<turnstile> M<:N"}. |
|
684 |
\end{enumerate} |
|
685 |
\end{lemma} |
|
686 |
||
687 |
The two parts are proved simultaneously, by induction on the size |
|
688 |
of @{term "Q"}. The argument for part (2) assumes that part (1) has |
|
689 |
been established already for the @{term "Q"} in question; part (1) uses |
|
690 |
part (2) only for strictly smaller @{term "Q"}. |
|
18650 | 691 |
\end{quote} |
18621 | 692 |
|
693 |
For the induction on the size of @{term "Q"}, we use the induction-rule |
|
694 |
@{text "measure_induct_rule"}: |
|
695 |
||
696 |
\begin{center} |
|
697 |
@{thm measure_induct_rule[of "size_ty",no_vars]} |
|
698 |
\end{center} |
|
18410 | 699 |
|
18628 | 700 |
That means in order to show a property @{term "P a"} for all @{term "a"}, |
18650 | 701 |
the induct-rule requires to prove that for all @{term x} @{term "P x"} holds using the |
18621 | 702 |
assumption that for all @{term y} whose size is strictly smaller than |
703 |
that of @{term x} the property @{term "P y"} holds. *} |
|
18353
4dd468ccfdf7
transitivity should be now in a reasonable state. But
urbanc
parents:
18306
diff
changeset
|
704 |
|
18621 | 705 |
lemma |
706 |
shows trans: "\<Gamma>\<turnstile>S<:Q \<Longrightarrow> \<Gamma>\<turnstile>Q<:T \<Longrightarrow> \<Gamma>\<turnstile>S<:T" |
|
707 |
and narrow: "(\<Delta>@[(X,Q)]@\<Gamma>)\<turnstile>M<:N \<Longrightarrow> \<Gamma>\<turnstile>P<:Q \<Longrightarrow> (\<Delta>@[(X,P)]@\<Gamma>)\<turnstile>M<:N" |
|
20503 | 708 |
proof (induct Q arbitrary: \<Gamma> S T \<Delta> X P M N taking: "size_ty" rule: measure_induct_rule) |
18621 | 709 |
case (less Q) |
710 |
--{* \begin{minipage}[t]{0.9\textwidth} |
|
711 |
First we mention the induction hypotheses of the outer induction for later |
|
712 |
reference:\end{minipage}*} |
|
713 |
have IH_trans: |
|
714 |
"\<And>Q' \<Gamma> S T. \<lbrakk>size_ty Q' < size_ty Q; \<Gamma>\<turnstile>S<:Q'; \<Gamma>\<turnstile>Q'<:T\<rbrakk> \<Longrightarrow> \<Gamma>\<turnstile>S<:T" by fact |
|
715 |
have IH_narrow: |
|
716 |
"\<And>Q' \<Delta> \<Gamma> X M N P. \<lbrakk>size_ty Q' < size_ty Q; (\<Delta>@[(X,Q')]@\<Gamma>)\<turnstile>M<:N; \<Gamma>\<turnstile>P<:Q'\<rbrakk> |
|
717 |
\<Longrightarrow> (\<Delta>@[(X,P)]@\<Gamma>)\<turnstile>M<:N" by fact |
|
718 |
--{* \begin{minipage}[t]{0.9\textwidth} |
|
719 |
We proceed with the transitivity proof as an auxiliary lemma, because it needs |
|
720 |
to be referenced in the narrowing proof.\end{minipage}*} |
|
721 |
have transitivity_aux: |
|
722 |
"\<And>\<Gamma> S T. \<lbrakk>\<Gamma> \<turnstile> S <: Q; \<Gamma> \<turnstile> Q <: T\<rbrakk> \<Longrightarrow> \<Gamma> \<turnstile> S <: T" |
|
18246 | 723 |
proof - |
18424 | 724 |
fix \<Gamma>' S' T |
18621 | 725 |
assume "\<Gamma>' \<turnstile> S' <: Q" --{* left-hand derivation *} |
726 |
and "\<Gamma>' \<turnstile> Q <: T" --{* right-hand derivation *} |
|
727 |
thus "\<Gamma>' \<turnstile> S' <: T" |
|
18747 | 728 |
proof (nominal_induct \<Gamma>' S' Q\<equiv>Q rule: subtype_of_induct) |
18424 | 729 |
case (S_Top \<Gamma> S) |
18621 | 730 |
--{* \begin{minipage}[t]{0.9\textwidth} |
731 |
In this case the left-hand derivation is @{term "\<Gamma> \<turnstile> S <: Top"}, giving |
|
732 |
us @{term "\<turnstile> \<Gamma> ok"} and @{term "S closed_in \<Gamma>"}. This case is straightforward, |
|
733 |
because the right-hand derivation must be of the form @{term "\<Gamma> \<turnstile> Top <: Top"} |
|
734 |
giving us the equation @{term "T = Top"}.\end{minipage}*} |
|
18424 | 735 |
hence rh_drv: "\<Gamma> \<turnstile> Top <: T" by simp |
736 |
hence T_inst: "T = Top" by (simp add: S_TopE) |
|
18621 | 737 |
have "\<turnstile> \<Gamma> ok" |
738 |
and "S closed_in \<Gamma>" by fact |
|
739 |
hence "\<Gamma> \<turnstile> S <: Top" by (simp add: subtype_of.S_Top) |
|
18424 | 740 |
thus "\<Gamma> \<turnstile> S <: T" using T_inst by simp |
18246 | 741 |
next |
18621 | 742 |
case (S_Var \<Gamma> Y U) |
743 |
-- {* \begin{minipage}[t]{0.9\textwidth} |
|
744 |
In this case the left-hand derivation is @{term "\<Gamma> \<turnstile> Tvar Y <: Q"} |
|
745 |
with @{term "S = Tvar Y"}. We have therefore @{term "(Y,U)"} |
|
18650 | 746 |
is in @{term "\<Gamma>"} and by inner induction hypothesis that @{term "\<Gamma> \<turnstile> U <: T"}. |
18621 | 747 |
By @{text "S_Var"} follows @{term "\<Gamma> \<turnstile> Tvar Y <: T"}.\end{minipage}*} |
18424 | 748 |
hence IH_inner: "\<Gamma> \<turnstile> U <: T" by simp |
18621 | 749 |
have "(Y,U) \<in> set \<Gamma>" by fact |
750 |
with IH_inner show "\<Gamma> \<turnstile> Tvar Y <: T" by (simp add: subtype_of.S_Var) |
|
18246 | 751 |
next |
18424 | 752 |
case (S_Refl \<Gamma> X) |
18621 | 753 |
--{* \begin{minipage}[t]{0.9\textwidth} |
754 |
In this case the left-hand derivation is @{term "\<Gamma>\<turnstile>(Tvar X) <: (Tvar X)"} with |
|
755 |
@{term "Q=Tvar X"}. The goal then follows immediately from the right-hand |
|
756 |
derivation.\end{minipage}*} |
|
18577
a636846a02c7
added more documentation; will now try out a modification
urbanc
parents:
18424
diff
changeset
|
757 |
thus "\<Gamma> \<turnstile> Tvar X <: T" by simp |
18246 | 758 |
next |
18621 | 759 |
case (S_Arrow \<Gamma> S\<^isub>1 S\<^isub>2 Q\<^isub>1 Q\<^isub>2) |
760 |
--{* \begin{minipage}[t]{0.9\textwidth} |
|
761 |
In this case the left-hand derivation is @{term "\<Gamma> \<turnstile> S\<^isub>1 \<rightarrow> S\<^isub>2 <: Q\<^isub>1 \<rightarrow> Q\<^isub>2"} with |
|
762 |
@{term "S\<^isub>1\<rightarrow>S\<^isub>2=S"} and @{term "Q\<^isub>1\<rightarrow>Q\<^isub>2=Q"}. We know that the @{text "size_ty"} of |
|
763 |
@{term Q\<^isub>1} and @{term Q\<^isub>2} is smaller than that of @{term Q}; |
|
764 |
so we can apply the outer induction hypotheses for @{term Q\<^isub>1} and @{term Q\<^isub>2}. |
|
765 |
We also have the sub-derivations @{term "\<Gamma>\<turnstile>Q\<^isub>1<:S\<^isub>1"} and @{term "\<Gamma>\<turnstile>S\<^isub>2<:Q\<^isub>2"}. |
|
18628 | 766 |
The right-hand derivation is @{term "\<Gamma> \<turnstile> Q\<^isub>1 \<rightarrow> Q\<^isub>2 <: T"}. There exist types |
18621 | 767 |
@{text "T\<^isub>1,T\<^isub>2"} such that @{term "T=Top \<or> T=T\<^isub>1\<rightarrow>T\<^isub>2"}. The @{term "Top"}-case is |
768 |
straightforward once we know @{term "(S\<^isub>1 \<rightarrow> S\<^isub>2) closed_in \<Gamma>"} and @{term "\<turnstile> \<Gamma> ok"}. |
|
769 |
In the other case we have the sub-derivations @{term "\<Gamma>\<turnstile>T\<^isub>1<:Q\<^isub>1"} and @{term "\<Gamma>\<turnstile>Q\<^isub>2<:T\<^isub>2"}. |
|
770 |
Using the outer induction hypothesis for transitivity we can derive @{term "\<Gamma>\<turnstile>T\<^isub>1<:S\<^isub>1"} |
|
771 |
and @{term "\<Gamma>\<turnstile>S\<^isub>2<:T\<^isub>2"}. By rule @{text "S_Arrow"} follows @{term "\<Gamma> \<turnstile> S\<^isub>1 \<rightarrow> S\<^isub>2 <: T\<^isub>1 \<rightarrow> T\<^isub>2"}, |
|
772 |
which is @{term "\<Gamma> \<turnstile> S\<^isub>1 \<rightarrow> S\<^isub>2 <: T\<^isub>"}.\end{minipage}*} |
|
773 |
hence rh_drv: "\<Gamma> \<turnstile> Q\<^isub>1 \<rightarrow> Q\<^isub>2 <: T" by simp |
|
774 |
from `Q\<^isub>1 \<rightarrow> Q\<^isub>2 = Q` |
|
775 |
have Q\<^isub>1\<^isub>2_less: "size_ty Q\<^isub>1 < size_ty Q" "size_ty Q\<^isub>2 < size_ty Q" by auto |
|
776 |
have lh_drv_prm\<^isub>1: "\<Gamma> \<turnstile> Q\<^isub>1 <: S\<^isub>1" by fact |
|
777 |
have lh_drv_prm\<^isub>2: "\<Gamma> \<turnstile> S\<^isub>2 <: Q\<^isub>2" by fact |
|
778 |
from rh_drv have "T=Top \<or> (\<exists>T\<^isub>1 T\<^isub>2. T=T\<^isub>1\<rightarrow>T\<^isub>2 \<and> \<Gamma>\<turnstile>T\<^isub>1<:Q\<^isub>1 \<and> \<Gamma>\<turnstile>Q\<^isub>2<:T\<^isub>2)" |
|
779 |
by (simp add: S_ArrowE_left) |
|
780 |
moreover |
|
781 |
have "S\<^isub>1 closed_in \<Gamma>" and "S\<^isub>2 closed_in \<Gamma>" |
|
782 |
using lh_drv_prm\<^isub>1 lh_drv_prm\<^isub>2 by (simp_all add: subtype_implies_closed) |
|
783 |
hence "(S\<^isub>1 \<rightarrow> S\<^isub>2) closed_in \<Gamma>" by (simp add: closed_in_def ty.supp) |
|
18353
4dd468ccfdf7
transitivity should be now in a reasonable state. But
urbanc
parents:
18306
diff
changeset
|
784 |
moreover |
18424 | 785 |
have "\<turnstile> \<Gamma> ok" using rh_drv by (rule subtype_implies_ok) |
18353
4dd468ccfdf7
transitivity should be now in a reasonable state. But
urbanc
parents:
18306
diff
changeset
|
786 |
moreover |
18621 | 787 |
{ assume "\<exists>T\<^isub>1 T\<^isub>2. T=T\<^isub>1\<rightarrow>T\<^isub>2 \<and> \<Gamma>\<turnstile>T\<^isub>1<:Q\<^isub>1 \<and> \<Gamma>\<turnstile>Q\<^isub>2<:T\<^isub>2" |
788 |
then obtain T\<^isub>1 T\<^isub>2 |
|
789 |
where T_inst: "T = T\<^isub>1 \<rightarrow> T\<^isub>2" |
|
790 |
and rh_drv_prm\<^isub>1: "\<Gamma> \<turnstile> T\<^isub>1 <: Q\<^isub>1" |
|
791 |
and rh_drv_prm\<^isub>2: "\<Gamma> \<turnstile> Q\<^isub>2 <: T\<^isub>2" by force |
|
792 |
from IH_trans[of "Q\<^isub>1"] |
|
793 |
have "\<Gamma> \<turnstile> T\<^isub>1 <: S\<^isub>1" using Q\<^isub>1\<^isub>2_less rh_drv_prm\<^isub>1 lh_drv_prm\<^isub>1 by simp |
|
18246 | 794 |
moreover |
18621 | 795 |
from IH_trans[of "Q\<^isub>2"] |
796 |
have "\<Gamma> \<turnstile> S\<^isub>2 <: T\<^isub>2" using Q\<^isub>1\<^isub>2_less rh_drv_prm\<^isub>2 lh_drv_prm\<^isub>2 by simp |
|
797 |
ultimately have "\<Gamma> \<turnstile> S\<^isub>1 \<rightarrow> S\<^isub>2 <: T\<^isub>1 \<rightarrow> T\<^isub>2" by (simp add: subtype_of.S_Arrow) |
|
798 |
hence "\<Gamma> \<turnstile> S\<^isub>1 \<rightarrow> S\<^isub>2 <: T" using T_inst by simp |
|
18353
4dd468ccfdf7
transitivity should be now in a reasonable state. But
urbanc
parents:
18306
diff
changeset
|
799 |
} |
18621 | 800 |
ultimately show "\<Gamma> \<turnstile> S\<^isub>1 \<rightarrow> S\<^isub>2 <: T" by blast |
18246 | 801 |
next |
18621 | 802 |
case (S_Forall \<Gamma> X S\<^isub>1 S\<^isub>2 Q\<^isub>1 Q\<^isub>2) |
803 |
--{* \begin{minipage}[t]{0.9\textwidth} |
|
804 |
In this case the left-hand derivation is @{text "\<Gamma>\<turnstile>\<forall>[X<:S\<^isub>1].S\<^isub>2 <: \<forall>[X<:Q\<^isub>1].Q\<^isub>2"} with |
|
805 |
@{text "\<forall>[X<:S\<^isub>1].S\<^isub>2=S"} and @{text "\<forall>[X<:Q\<^isub>1].Q\<^isub>2=Q"}. We therefore have the sub-derivations |
|
806 |
@{term "\<Gamma>\<turnstile>Q\<^isub>1<:S\<^isub>1"} and @{term "((X,Q\<^isub>1)#\<Gamma>)\<turnstile>S\<^isub>2<:Q\<^isub>2"}. Since @{term "X"} is a binder, we |
|
807 |
assume that it is sufficiently fresh; in particular we have the freshness conditions |
|
18650 | 808 |
@{term "X\<sharp>\<Gamma>"} and @{term "X\<sharp>Q\<^isub>1"} (these assumptions are provided by the strong |
809 |
induction-rule @{text "subtype_of_induct"}). We know that the @{text "size_ty"} of |
|
18621 | 810 |
@{term Q\<^isub>1} and @{term Q\<^isub>2} is smaller than that of @{term Q}; |
811 |
so we can apply the outer induction hypotheses for @{term Q\<^isub>1} and @{term Q\<^isub>2}. |
|
812 |
The right-hand derivation is @{text "\<Gamma> \<turnstile> \<forall>[X<:Q\<^isub>1].Q\<^isub>2 <: T"}. Since @{term "X\<sharp>\<Gamma>"} |
|
813 |
and @{term "X\<sharp>Q\<^isub>1"} there exists types @{text "T\<^isub>1,T\<^isub>2"} such that |
|
814 |
@{text "T=Top \<or> T=\<forall>[X<:T\<^isub>1].T\<^isub>2"}. The @{term "Top"}-case is straightforward once we know |
|
815 |
@{text "(\<forall>[X<:S\<^isub>1].S\<^isub>2) closed_in \<Gamma>"} and @{term "\<turnstile> \<Gamma> ok"}. In the other case we have |
|
18628 | 816 |
the sub-derivations @{term "\<Gamma>\<turnstile>T\<^isub>1<:Q\<^isub>1"} and @{term "((X,T\<^isub>1)#\<Gamma>)\<turnstile>Q\<^isub>2<:T\<^isub>2"}. Using the outer |
18621 | 817 |
induction hypothesis for transitivity we can derive @{term "\<Gamma>\<turnstile>T\<^isub>1<:S\<^isub>1"}. From the outer |
18628 | 818 |
induction for narrowing we get @{term "((X,T\<^isub>1)#\<Gamma>) \<turnstile> S\<^isub>2 <: Q\<^isub>2"} and then using again |
819 |
induction for transitivity we obtain @{term "((X,T\<^isub>1)#\<Gamma>) \<turnstile> S\<^isub>2 <: T\<^isub>2"}. By rule |
|
820 |
@{text "S_Forall"} and the freshness condition @{term "X\<sharp>\<Gamma>"} follows |
|
18650 | 821 |
@{text "\<Gamma> \<turnstile> \<forall>[X<:S\<^isub>1].S\<^isub>2 <: \<forall>[X<:T\<^isub>1].T\<^isub>2"}, which is @{text "\<Gamma> \<turnstile> \<forall>[X<:S\<^isub>1].S\<^isub>2 <: T\<^isub>"}. |
18628 | 822 |
\end{minipage}*} |
18621 | 823 |
hence rh_drv: "\<Gamma> \<turnstile> \<forall>[X<:Q\<^isub>1].Q\<^isub>2 <: T" by simp |
824 |
have lh_drv_prm\<^isub>1: "\<Gamma> \<turnstile> Q\<^isub>1 <: S\<^isub>1" by fact |
|
825 |
have lh_drv_prm\<^isub>2: "((X,Q\<^isub>1)#\<Gamma>) \<turnstile> S\<^isub>2 <: Q\<^isub>2" by fact |
|
826 |
have fresh_cond: "X\<sharp>\<Gamma>" "X\<sharp>Q\<^isub>1" by fact |
|
827 |
from `\<forall>[X<:Q\<^isub>1].Q\<^isub>2 = Q` |
|
20395
9a60e3151244
added definition for size and substitution using the recursion
urbanc
parents:
19972
diff
changeset
|
828 |
have Q\<^isub>1\<^isub>2_less: "size_ty Q\<^isub>1 < size_ty Q" "size_ty Q\<^isub>2 < size_ty Q " using fresh_cond by auto |
18621 | 829 |
from rh_drv |
830 |
have "T=Top \<or> (\<exists>T\<^isub>1 T\<^isub>2. T=\<forall>[X<:T\<^isub>1].T\<^isub>2 \<and> \<Gamma>\<turnstile>T\<^isub>1<:Q\<^isub>1 \<and> ((X,T\<^isub>1)#\<Gamma>)\<turnstile>Q\<^isub>2<:T\<^isub>2)" |
|
831 |
using fresh_cond by (simp add: S_ForallE_left) |
|
832 |
moreover |
|
833 |
have "S\<^isub>1 closed_in \<Gamma>" and "S\<^isub>2 closed_in ((X,Q\<^isub>1)#\<Gamma>)" |
|
834 |
using lh_drv_prm\<^isub>1 lh_drv_prm\<^isub>2 by (simp_all add: subtype_implies_closed) |
|
835 |
hence "(\<forall>[X<:S\<^isub>1].S\<^isub>2) closed_in \<Gamma>" by (force simp add: closed_in_def ty.supp abs_supp) |
|
18353
4dd468ccfdf7
transitivity should be now in a reasonable state. But
urbanc
parents:
18306
diff
changeset
|
836 |
moreover |
18424 | 837 |
have "\<turnstile> \<Gamma> ok" using rh_drv by (rule subtype_implies_ok) |
18353
4dd468ccfdf7
transitivity should be now in a reasonable state. But
urbanc
parents:
18306
diff
changeset
|
838 |
moreover |
18621 | 839 |
{ assume "\<exists>T\<^isub>1 T\<^isub>2. T=\<forall>[X<:T\<^isub>1].T\<^isub>2 \<and> \<Gamma>\<turnstile>T\<^isub>1<:Q\<^isub>1 \<and> ((X,T\<^isub>1)#\<Gamma>)\<turnstile>Q\<^isub>2<:T\<^isub>2" |
840 |
then obtain T\<^isub>1 T\<^isub>2 |
|
841 |
where T_inst: "T = \<forall>[X<:T\<^isub>1].T\<^isub>2" |
|
842 |
and rh_drv_prm\<^isub>1: "\<Gamma> \<turnstile> T\<^isub>1 <: Q\<^isub>1" |
|
843 |
and rh_drv_prm\<^isub>2:"((X,T\<^isub>1)#\<Gamma>) \<turnstile> Q\<^isub>2 <: T\<^isub>2" by force |
|
844 |
from IH_trans[of "Q\<^isub>1"] |
|
845 |
have "\<Gamma> \<turnstile> T\<^isub>1 <: S\<^isub>1" using lh_drv_prm\<^isub>1 rh_drv_prm\<^isub>1 Q\<^isub>1\<^isub>2_less by blast |
|
846 |
moreover |
|
847 |
from IH_narrow[of "Q\<^isub>1" "[]"] |
|
848 |
have "((X,T\<^isub>1)#\<Gamma>) \<turnstile> S\<^isub>2 <: Q\<^isub>2" using Q\<^isub>1\<^isub>2_less lh_drv_prm\<^isub>2 rh_drv_prm\<^isub>1 by simp |
|
849 |
with IH_trans[of "Q\<^isub>2"] |
|
850 |
have "((X,T\<^isub>1)#\<Gamma>) \<turnstile> S\<^isub>2 <: T\<^isub>2" using Q\<^isub>1\<^isub>2_less rh_drv_prm\<^isub>2 by simp |
|
851 |
ultimately have "\<Gamma> \<turnstile> \<forall>[X<:S\<^isub>1].S\<^isub>2 <: \<forall>[X<:T\<^isub>1].T\<^isub>2" |
|
852 |
using fresh_cond by (simp add: subtype_of.S_Forall) |
|
853 |
hence "\<Gamma> \<turnstile> \<forall>[X<:S\<^isub>1].S\<^isub>2 <: T" using T_inst by simp |
|
18353
4dd468ccfdf7
transitivity should be now in a reasonable state. But
urbanc
parents:
18306
diff
changeset
|
854 |
} |
18621 | 855 |
ultimately show "\<Gamma> \<turnstile> \<forall>[X<:S\<^isub>1].S\<^isub>2 <: T" by blast |
18246 | 856 |
qed |
857 |
qed |
|
858 |
||
18621 | 859 |
{ --{* The transitivity proof is now by the auxiliary lemma. *} |
860 |
case 1 |
|
861 |
have "\<Gamma> \<turnstile> S <: Q" |
|
862 |
and "\<Gamma> \<turnstile> Q <: T" by fact |
|
863 |
thus "\<Gamma> \<turnstile> S <: T" by (rule transitivity_aux) |
|
864 |
next |
|
865 |
--{* The narrowing proof proceeds by an induction over @{term "(\<Delta>@[(X,Q)]@\<Gamma>) \<turnstile> M <: N"}. *} |
|
866 |
case 2 |
|
867 |
have "(\<Delta>@[(X,Q)]@\<Gamma>) \<turnstile> M <: N" --{* left-hand derivation *} |
|
868 |
and "\<Gamma> \<turnstile> P<:Q" by fact --{* right-hand derivation *} |
|
869 |
thus "(\<Delta>@[(X,P)]@\<Gamma>) \<turnstile> M <: N" |
|
870 |
proof (nominal_induct \<Gamma>\<equiv>"\<Delta>@[(X,Q)]@\<Gamma>" M N avoiding: \<Delta> \<Gamma> X rule: subtype_of_induct) |
|
18424 | 871 |
case (S_Top _ S \<Delta> \<Gamma> X) |
18621 | 872 |
--{* \begin{minipage}[t]{0.9\textwidth} |
873 |
In this case the left-hand derivation is @{term "(\<Delta>@[(X,Q)]@\<Gamma>) \<turnstile> S <: Top"}. We show |
|
874 |
that the context @{term "\<Delta>@[(X,P)]@\<Gamma>"} is ok and that @{term S} is closed in |
|
875 |
@{term "\<Delta>@[(X,P)]@\<Gamma>"}. Then we can apply the @{text "S_Top"}-rule.\end{minipage}*} |
|
876 |
hence lh_drv_prm\<^isub>1: "\<turnstile> (\<Delta>@[(X,Q)]@\<Gamma>) ok" |
|
877 |
and lh_drv_prm\<^isub>2: "S closed_in (\<Delta>@[(X,Q)]@\<Gamma>)" by simp_all |
|
18424 | 878 |
have rh_drv: "\<Gamma> \<turnstile> P <: Q" by fact |
879 |
hence "P closed_in \<Gamma>" by (simp add: subtype_implies_closed) |
|
18621 | 880 |
with lh_drv_prm\<^isub>1 have "\<turnstile> (\<Delta>@[(X,P)]@\<Gamma>) ok" by (simp add: replace_type) |
18412 | 881 |
moreover |
18621 | 882 |
from lh_drv_prm\<^isub>2 have "S closed_in (\<Delta>@[(X,P)]@\<Gamma>)" |
883 |
by (simp add: closed_in_def domain_append) |
|
18577
a636846a02c7
added more documentation; will now try out a modification
urbanc
parents:
18424
diff
changeset
|
884 |
ultimately show "(\<Delta>@[(X,P)]@\<Gamma>) \<turnstile> S <: Top" by (simp add: subtype_of.S_Top) |
18246 | 885 |
next |
18424 | 886 |
case (S_Var _ Y S N \<Delta> \<Gamma> X) |
18621 | 887 |
--{* \begin{minipage}[t]{0.9\textwidth} |
18628 | 888 |
In this case the left-hand derivation is @{term "(\<Delta>@[(X,Q)]@\<Gamma>) \<turnstile> Tvar Y <: N"} and |
889 |
by inner induction hypothesis we have @{term "(\<Delta>@[(X,P)]@\<Gamma>) \<turnstile> S <: N"}. We therefore |
|
18621 | 890 |
know that the contexts @{term "\<Delta>@[(X,Q)]@\<Gamma>"} and @{term "\<Delta>@[(X,P)]@\<Gamma>"} are ok, and that |
18628 | 891 |
@{term "(Y,S)"} is in @{term "\<Delta>@[(X,Q)]@\<Gamma>"}. We need to show that |
892 |
@{term "(\<Delta>@[(X,P)]@\<Gamma>) \<turnstile> Tvar Y <: N"} holds. In case @{term "X\<noteq>Y"} we know that |
|
893 |
@{term "(Y,S)"} is in @{term "\<Delta>@[(X,P)]@\<Gamma>"} and can use the inner induction hypothesis |
|
894 |
and rule @{text "S_Var"} to conclude. In case @{term "X=Y"} we can infer that |
|
895 |
@{term "S=Q"}; moreover we have that @{term "(\<Delta>@[(X,P)]@\<Gamma>) extends \<Gamma>"} and therefore |
|
896 |
by @{text "weakening"} that @{term "(\<Delta>@[(X,P)]@\<Gamma>) \<turnstile> P <: Q"} holds. By transitivity we |
|
897 |
obtain then @{term "(\<Delta>@[(X,P)]@\<Gamma>) \<turnstile> P <: N"} and can conclude by applying rule |
|
898 |
@{text "S_Var"}.\end{minipage}*} |
|
18621 | 899 |
hence IH_inner: "(\<Delta>@[(X,P)]@\<Gamma>) \<turnstile> S <: N" |
900 |
and lh_drv_prm: "(Y,S) \<in> set (\<Delta>@[(X,Q)]@\<Gamma>)" |
|
901 |
and rh_drv: "\<Gamma> \<turnstile> P<:Q" |
|
902 |
and ok\<^isub>Q: "\<turnstile> (\<Delta>@[(X,Q)]@\<Gamma>) ok" by (simp_all add: subtype_implies_ok) |
|
903 |
hence ok\<^isub>P: "\<turnstile> (\<Delta>@[(X,P)]@\<Gamma>) ok" by (simp add: subtype_implies_ok) |
|
904 |
show "(\<Delta>@[(X,P)]@\<Gamma>) \<turnstile> Tvar Y <: N" |
|
905 |
proof (cases "X=Y") |
|
906 |
case False |
|
907 |
have "X\<noteq>Y" by fact |
|
908 |
hence "(Y,S)\<in>set (\<Delta>@[(X,P)]@\<Gamma>)" using lh_drv_prm by simp |
|
909 |
with IH_inner show "(\<Delta>@[(X,P)]@\<Gamma>) \<turnstile> Tvar Y <: N" by (simp add: subtype_of.S_Var) |
|
910 |
next |
|
911 |
case True |
|
912 |
have memb\<^isub>X\<^isub>Q: "(X,Q)\<in>set (\<Delta>@[(X,Q)]@\<Gamma>)" by simp |
|
913 |
have memb\<^isub>X\<^isub>P: "(X,P)\<in>set (\<Delta>@[(X,P)]@\<Gamma>)" by simp |
|
914 |
have eq: "X=Y" by fact |
|
915 |
hence "S=Q" using ok\<^isub>Q lh_drv_prm memb\<^isub>X\<^isub>Q by (simp only: uniqueness_of_ctxt) |
|
18424 | 916 |
hence "(\<Delta>@[(X,P)]@\<Gamma>) \<turnstile> Q <: N" using IH_inner by simp |
917 |
moreover |
|
918 |
have "(\<Delta>@[(X,P)]@\<Gamma>) extends \<Gamma>" by (simp add: extends_def) |
|
18621 | 919 |
hence "(\<Delta>@[(X,P)]@\<Gamma>) \<turnstile> P <: Q" using rh_drv ok\<^isub>P by (simp only: weakening) |
920 |
ultimately have "(\<Delta>@[(X,P)]@\<Gamma>) \<turnstile> P <: N" by (simp add: transitivity_aux) |
|
921 |
thus "(\<Delta>@[(X,P)]@\<Gamma>) \<turnstile> Tvar Y <: N" using memb\<^isub>X\<^isub>P eq by (simp only: subtype_of.S_Var) |
|
922 |
qed |
|
18246 | 923 |
next |
18424 | 924 |
case (S_Refl _ Y \<Delta> \<Gamma> X) |
18621 | 925 |
--{* \begin{minipage}[t]{0.9\textwidth} |
926 |
In this case the left-hand derivation is @{term "(\<Delta>@[(X,Q)]@\<Gamma>) \<turnstile> Tvar Y <: Tvar Y"} and we |
|
18628 | 927 |
therefore know that @{term "\<Delta>@[(X,Q)]@\<Gamma>"} is ok and that @{term "Y"} is in |
18621 | 928 |
the domain of @{term "\<Delta>@[(X,Q)]@\<Gamma>"}. We therefore know that @{term "\<Delta>@[(X,P)]@\<Gamma>"} is ok |
929 |
and that @{term Y} is in the domain of @{term "\<Delta>@[(X,P)]@\<Gamma>"}. We can conclude by applying |
|
930 |
rule @{text "S_Refl"}.\end{minipage}*} |
|
931 |
hence lh_drv_prm\<^isub>1: "\<turnstile> (\<Delta>@[(X,Q)]@\<Gamma>) ok" |
|
932 |
and lh_drv_prm\<^isub>2: "Y \<in> domain (\<Delta>@[(X,Q)]@\<Gamma>)" by simp_all |
|
18424 | 933 |
have "\<Gamma> \<turnstile> P <: Q" by fact |
934 |
hence "P closed_in \<Gamma>" by (simp add: subtype_implies_closed) |
|
18621 | 935 |
with lh_drv_prm\<^isub>1 have "\<turnstile> (\<Delta>@[(X,P)]@\<Gamma>) ok" by (simp add: replace_type) |
18424 | 936 |
moreover |
18621 | 937 |
from lh_drv_prm\<^isub>2 have "Y \<in> domain (\<Delta>@[(X,P)]@\<Gamma>)" by (simp add: domain_append) |
18577
a636846a02c7
added more documentation; will now try out a modification
urbanc
parents:
18424
diff
changeset
|
938 |
ultimately show "(\<Delta>@[(X,P)]@\<Gamma>) \<turnstile> Tvar Y <: Tvar Y" by (simp add: subtype_of.S_Refl) |
18246 | 939 |
next |
18621 | 940 |
case (S_Arrow _ Q\<^isub>1 Q\<^isub>2 S\<^isub>1 S\<^isub>2 \<Delta> \<Gamma> X) |
941 |
--{* \begin{minipage}[t]{0.9\textwidth} |
|
942 |
In this case the left-hand derivation is @{term "(\<Delta>@[(X,Q)]@\<Gamma>) \<turnstile> Q\<^isub>1 \<rightarrow> Q\<^isub>2 <: S\<^isub>1 \<rightarrow> S\<^isub>2"} |
|
943 |
and the proof is trivial.\end{minipage}*} |
|
944 |
thus "(\<Delta>@[(X,P)]@\<Gamma>) \<turnstile> Q\<^isub>1 \<rightarrow> Q\<^isub>2 <: S\<^isub>1 \<rightarrow> S\<^isub>2" by blast |
|
18424 | 945 |
next |
18621 | 946 |
case (S_Forall _ Y S\<^isub>1 S\<^isub>2 T\<^isub>1 T\<^isub>2 \<Delta> \<Gamma> X) |
947 |
--{* \begin{minipage}[t]{0.9\textwidth} |
|
18628 | 948 |
In this case the left-hand derivation is @{text "(\<Delta>@[(X,Q)]@\<Gamma>) \<turnstile> \<forall>[Y<:S\<^isub>1].S\<^isub>2 <: \<forall>[Y<:T\<^isub>1].T\<^isub>2"} |
18621 | 949 |
and therfore we know that the binder @{term Y} is fresh for @{term "\<Delta>@[(X,Q)]@\<Gamma>"}. By |
950 |
the inner induction hypothesis we have that @{term "(\<Delta>@[(X,P)]@\<Gamma>) \<turnstile> T\<^isub>1 <: S\<^isub>1"} and |
|
951 |
@{term "((Y,T\<^isub>1)#\<Delta>@[(X,P)]@\<Gamma>) \<turnstile> S\<^isub>2 <: T\<^isub>2"}. Since @{term P} is a subtype of @{term Q} |
|
952 |
we can infer that @{term Y} is fresh for @{term P} and thus also fresh for |
|
953 |
@{term "\<Delta>@[(X,P)]@\<Gamma>"}. We can then conclude by applying rule @{text "S_Forall"}. |
|
954 |
\end{minipage}*} |
|
955 |
hence IH_inner\<^isub>1: "(\<Delta>@[(X,P)]@\<Gamma>) \<turnstile> T\<^isub>1 <: S\<^isub>1" |
|
956 |
and IH_inner\<^isub>2: "((Y,T\<^isub>1)#\<Delta>@[(X,P)]@\<Gamma>) \<turnstile> S\<^isub>2 <: T\<^isub>2" |
|
957 |
and lh_drv_prm: "Y\<sharp>(\<Delta>@[(X,Q)]@\<Gamma>)" by force+ |
|
18424 | 958 |
have rh_drv: "\<Gamma> \<turnstile> P <: Q" by fact |
18621 | 959 |
hence "Y\<sharp>P" using lh_drv_prm by (simp only: fresh_list_append subtype_implies_fresh) |
960 |
hence "Y\<sharp>(\<Delta>@[(X,P)]@\<Gamma>)" using lh_drv_prm |
|
18424 | 961 |
by (simp add: fresh_list_append fresh_list_cons fresh_prod) |
18621 | 962 |
with IH_inner\<^isub>1 IH_inner\<^isub>2 |
963 |
show "(\<Delta>@[(X,P)]@\<Gamma>) \<turnstile> \<forall>[Y<:S\<^isub>1].S\<^isub>2 <: \<forall>[Y<:T\<^isub>1].T\<^isub>2" by (simp add: subtype_of.S_Forall) |
|
18246 | 964 |
qed |
18621 | 965 |
} |
18246 | 966 |
qed |
967 |
||
18416 | 968 |
end |