author | wenzelm |
Tue, 08 Oct 2024 15:02:17 +0200 | |
changeset 81127 | 12990a6dddcb |
parent 81125 | ec121999a9cb |
permissions | -rw-r--r-- |
63167 | 1 |
section \<open>Simply-typed lambda-calculus with let and tuple patterns\<close> |
33189 | 2 |
|
3 |
theory Pattern |
|
66453
cc19f7ca2ed6
session-qualified theory imports: isabelle imports -U -i -d '~~/src/Benchmarks' -a;
wenzelm
parents:
63167
diff
changeset
|
4 |
imports "HOL-Nominal.Nominal" |
33189 | 5 |
begin |
6 |
||
7 |
atom_decl name |
|
8 |
||
9 |
nominal_datatype ty = |
|
10 |
Atom nat |
|
80914
d97fdabd9e2b
standardize mixfix annotations via "isabelle update -a -u mixfix_cartouches" --- to simplify systematic editing;
wenzelm
parents:
80142
diff
changeset
|
11 |
| Arrow ty ty (infixr \<open>\<rightarrow>\<close> 200) |
d97fdabd9e2b
standardize mixfix annotations via "isabelle update -a -u mixfix_cartouches" --- to simplify systematic editing;
wenzelm
parents:
80142
diff
changeset
|
12 |
| TupleT ty ty (infixr \<open>\<otimes>\<close> 210) |
33189 | 13 |
|
14 |
lemma fresh_type [simp]: "(a::name) \<sharp> (T::ty)" |
|
15 |
by (induct T rule: ty.induct) (simp_all add: fresh_nat) |
|
16 |
||
17 |
lemma supp_type [simp]: "supp (T::ty) = ({} :: name set)" |
|
18 |
by (induct T rule: ty.induct) (simp_all add: ty.supp supp_nat) |
|
19 |
||
20 |
lemma perm_type: "(pi::name prm) \<bullet> (T::ty) = T" |
|
21 |
by (induct T rule: ty.induct) (simp_all add: perm_nat_def) |
|
22 |
||
23 |
nominal_datatype trm = |
|
24 |
Var name |
|
80914
d97fdabd9e2b
standardize mixfix annotations via "isabelle update -a -u mixfix_cartouches" --- to simplify systematic editing;
wenzelm
parents:
80142
diff
changeset
|
25 |
| Tuple trm trm (\<open>(1'\<langle>_,/ _'\<rangle>)\<close>) |
33189 | 26 |
| Abs ty "\<guillemotleft>name\<guillemotright>trm" |
80914
d97fdabd9e2b
standardize mixfix annotations via "isabelle update -a -u mixfix_cartouches" --- to simplify systematic editing;
wenzelm
parents:
80142
diff
changeset
|
27 |
| App trm trm (infixl \<open>\<cdot>\<close> 200) |
33189 | 28 |
| Let ty trm btrm |
29 |
and btrm = |
|
30 |
Base trm |
|
31 |
| Bind ty "\<guillemotleft>name\<guillemotright>btrm" |
|
32 |
||
33 |
abbreviation |
|
80914
d97fdabd9e2b
standardize mixfix annotations via "isabelle update -a -u mixfix_cartouches" --- to simplify systematic editing;
wenzelm
parents:
80142
diff
changeset
|
34 |
Abs_syn :: "name \<Rightarrow> ty \<Rightarrow> trm \<Rightarrow> trm" (\<open>(3\<lambda>_:_./ _)\<close> [0, 0, 10] 10) |
33189 | 35 |
where |
36 |
"\<lambda>x:T. t \<equiv> Abs T x t" |
|
37 |
||
58310 | 38 |
datatype pat = |
33189 | 39 |
PVar name ty |
80914
d97fdabd9e2b
standardize mixfix annotations via "isabelle update -a -u mixfix_cartouches" --- to simplify systematic editing;
wenzelm
parents:
80142
diff
changeset
|
40 |
| PTuple pat pat (\<open>(1'\<langle>\<langle>_,/ _'\<rangle>\<rangle>)\<close>) |
33189 | 41 |
|
42 |
(* FIXME: The following should be done automatically by the nominal package *) |
|
43 |
overloading pat_perm \<equiv> "perm :: name prm \<Rightarrow> pat \<Rightarrow> pat" (unchecked) |
|
44 |
begin |
|
45 |
||
46 |
primrec pat_perm |
|
47 |
where |
|
48 |
"pat_perm pi (PVar x ty) = PVar (pi \<bullet> x) (pi \<bullet> ty)" |
|
49 |
| "pat_perm pi \<langle>\<langle>p, q\<rangle>\<rangle> = \<langle>\<langle>pat_perm pi p, pat_perm pi q\<rangle>\<rangle>" |
|
50 |
||
51 |
end |
|
52 |
||
53 |
declare pat_perm.simps [eqvt] |
|
54 |
||
55 |
lemma supp_PVar [simp]: "((supp (PVar x T))::name set) = supp x" |
|
56 |
by (simp add: supp_def perm_fresh_fresh) |
|
57 |
||
58 |
lemma supp_PTuple [simp]: "((supp \<langle>\<langle>p, q\<rangle>\<rangle>)::name set) = supp p \<union> supp q" |
|
59 |
by (simp add: supp_def Collect_disj_eq del: disj_not1) |
|
60 |
||
61 |
instance pat :: pt_name |
|
80140 | 62 |
proof |
63 |
fix x :: pat |
|
64 |
show "([]::(name \<times> _) list) \<bullet> x = x" |
|
65 |
by (induct x) simp_all |
|
66 |
fix pi1 pi2 :: "(name \<times> name) list" |
|
67 |
show "(pi1 @ pi2) \<bullet> x = pi1 \<bullet> pi2 \<bullet> x" |
|
68 |
by (induct x) (simp_all add: pt_name2) |
|
69 |
assume "pi1 \<triangleq> pi2" |
|
70 |
then show "pi1 \<bullet> x = pi2 \<bullet> x" |
|
71 |
by (induct x) (simp_all add: pt_name3) |
|
33189 | 72 |
qed |
73 |
||
74 |
instance pat :: fs_name |
|
80140 | 75 |
proof |
76 |
fix x :: pat |
|
77 |
show "finite (supp x::name set)" |
|
78 |
by (induct x) (simp_all add: fin_supp) |
|
33189 | 79 |
qed |
80 |
||
81 |
(* the following function cannot be defined using nominal_primrec, *) |
|
82 |
(* since variable parameters are currently not allowed. *) |
|
80914
d97fdabd9e2b
standardize mixfix annotations via "isabelle update -a -u mixfix_cartouches" --- to simplify systematic editing;
wenzelm
parents:
80142
diff
changeset
|
83 |
primrec abs_pat :: "pat \<Rightarrow> btrm \<Rightarrow> btrm" (\<open>(3\<lambda>[_]./ _)\<close> [0, 10] 10) |
33189 | 84 |
where |
85 |
"(\<lambda>[PVar x T]. t) = Bind T x t" |
|
86 |
| "(\<lambda>[\<langle>\<langle>p, q\<rangle>\<rangle>]. t) = (\<lambda>[p]. \<lambda>[q]. t)" |
|
87 |
||
88 |
lemma abs_pat_eqvt [eqvt]: |
|
89 |
"(pi :: name prm) \<bullet> (\<lambda>[p]. t) = (\<lambda>[pi \<bullet> p]. (pi \<bullet> t))" |
|
90 |
by (induct p arbitrary: t) simp_all |
|
91 |
||
92 |
lemma abs_pat_fresh [simp]: |
|
93 |
"(x::name) \<sharp> (\<lambda>[p]. t) = (x \<in> supp p \<or> x \<sharp> t)" |
|
94 |
by (induct p arbitrary: t) (simp_all add: abs_fresh supp_atm) |
|
95 |
||
96 |
lemma abs_pat_alpha: |
|
97 |
assumes fresh: "((pi::name prm) \<bullet> supp p::name set) \<sharp>* t" |
|
98 |
and pi: "set pi \<subseteq> supp p \<times> pi \<bullet> supp p" |
|
99 |
shows "(\<lambda>[p]. t) = (\<lambda>[pi \<bullet> p]. pi \<bullet> t)" |
|
100 |
proof - |
|
101 |
note pt_name_inst at_name_inst pi |
|
102 |
moreover have "(supp p::name set) \<sharp>* (\<lambda>[p]. t)" |
|
103 |
by (simp add: fresh_star_def) |
|
104 |
moreover from fresh |
|
105 |
have "(pi \<bullet> supp p::name set) \<sharp>* (\<lambda>[p]. t)" |
|
106 |
by (simp add: fresh_star_def) |
|
107 |
ultimately have "pi \<bullet> (\<lambda>[p]. t) = (\<lambda>[p]. t)" |
|
108 |
by (rule pt_freshs_freshs) |
|
109 |
then show ?thesis by (simp add: eqvts) |
|
110 |
qed |
|
111 |
||
112 |
primrec pat_vars :: "pat \<Rightarrow> name list" |
|
113 |
where |
|
114 |
"pat_vars (PVar x T) = [x]" |
|
115 |
| "pat_vars \<langle>\<langle>p, q\<rangle>\<rangle> = pat_vars q @ pat_vars p" |
|
116 |
||
117 |
lemma pat_vars_eqvt [eqvt]: |
|
118 |
"(pi :: name prm) \<bullet> (pat_vars p) = pat_vars (pi \<bullet> p)" |
|
119 |
by (induct p rule: pat.induct) (simp_all add: eqvts) |
|
120 |
||
121 |
lemma set_pat_vars_supp: "set (pat_vars p) = supp p" |
|
122 |
by (induct p) (auto simp add: supp_atm) |
|
123 |
||
124 |
lemma distinct_eqvt [eqvt]: |
|
125 |
"(pi :: name prm) \<bullet> (distinct (xs::name list)) = distinct (pi \<bullet> xs)" |
|
126 |
by (induct xs) (simp_all add: eqvts) |
|
127 |
||
128 |
primrec pat_type :: "pat \<Rightarrow> ty" |
|
129 |
where |
|
130 |
"pat_type (PVar x T) = T" |
|
131 |
| "pat_type \<langle>\<langle>p, q\<rangle>\<rangle> = pat_type p \<otimes> pat_type q" |
|
132 |
||
133 |
lemma pat_type_eqvt [eqvt]: |
|
134 |
"(pi :: name prm) \<bullet> (pat_type p) = pat_type (pi \<bullet> p)" |
|
135 |
by (induct p) simp_all |
|
136 |
||
137 |
lemma pat_type_perm_eq: "pat_type ((pi :: name prm) \<bullet> p) = pat_type p" |
|
138 |
by (induct p) (simp_all add: perm_type) |
|
139 |
||
41798 | 140 |
type_synonym ctx = "(name \<times> ty) list" |
33189 | 141 |
|
142 |
inductive |
|
80914
d97fdabd9e2b
standardize mixfix annotations via "isabelle update -a -u mixfix_cartouches" --- to simplify systematic editing;
wenzelm
parents:
80142
diff
changeset
|
143 |
ptyping :: "pat \<Rightarrow> ty \<Rightarrow> ctx \<Rightarrow> bool" (\<open>\<turnstile> _ : _ \<Rightarrow> _\<close> [60, 60, 60] 60) |
33189 | 144 |
where |
145 |
PVar: "\<turnstile> PVar x T : T \<Rightarrow> [(x, T)]" |
|
53015
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
45129
diff
changeset
|
146 |
| PTuple: "\<turnstile> p : T \<Rightarrow> \<Delta>\<^sub>1 \<Longrightarrow> \<turnstile> q : U \<Rightarrow> \<Delta>\<^sub>2 \<Longrightarrow> \<turnstile> \<langle>\<langle>p, q\<rangle>\<rangle> : T \<otimes> U \<Rightarrow> \<Delta>\<^sub>2 @ \<Delta>\<^sub>1" |
33189 | 147 |
|
148 |
lemma pat_vars_ptyping: |
|
149 |
assumes "\<turnstile> p : T \<Rightarrow> \<Delta>" |
|
150 |
shows "pat_vars p = map fst \<Delta>" using assms |
|
151 |
by induct simp_all |
|
152 |
||
153 |
inductive |
|
154 |
valid :: "ctx \<Rightarrow> bool" |
|
155 |
where |
|
156 |
Nil [intro!]: "valid []" |
|
157 |
| Cons [intro!]: "valid \<Gamma> \<Longrightarrow> x \<sharp> \<Gamma> \<Longrightarrow> valid ((x, T) # \<Gamma>)" |
|
158 |
||
159 |
inductive_cases validE[elim!]: "valid ((x, T) # \<Gamma>)" |
|
160 |
||
161 |
lemma fresh_ctxt_set_eq: "((x::name) \<sharp> (\<Gamma>::ctx)) = (x \<notin> fst ` set \<Gamma>)" |
|
162 |
by (induct \<Gamma>) (auto simp add: fresh_list_nil fresh_list_cons fresh_prod fresh_atm) |
|
163 |
||
164 |
lemma valid_distinct: "valid \<Gamma> = distinct (map fst \<Gamma>)" |
|
165 |
by (induct \<Gamma>) (auto simp add: fresh_ctxt_set_eq [symmetric]) |
|
166 |
||
167 |
abbreviation |
|
80914
d97fdabd9e2b
standardize mixfix annotations via "isabelle update -a -u mixfix_cartouches" --- to simplify systematic editing;
wenzelm
parents:
80142
diff
changeset
|
168 |
"sub_ctx" :: "ctx \<Rightarrow> ctx \<Rightarrow> bool" (\<open>_ \<sqsubseteq> _\<close>) |
33189 | 169 |
where |
53015
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
45129
diff
changeset
|
170 |
"\<Gamma>\<^sub>1 \<sqsubseteq> \<Gamma>\<^sub>2 \<equiv> \<forall>x. x \<in> set \<Gamma>\<^sub>1 \<longrightarrow> x \<in> set \<Gamma>\<^sub>2" |
33189 | 171 |
|
172 |
abbreviation |
|
80914
d97fdabd9e2b
standardize mixfix annotations via "isabelle update -a -u mixfix_cartouches" --- to simplify systematic editing;
wenzelm
parents:
80142
diff
changeset
|
173 |
Let_syn :: "pat \<Rightarrow> trm \<Rightarrow> trm \<Rightarrow> trm" (\<open>(LET (_ =/ _)/ IN (_))\<close> 10) |
33189 | 174 |
where |
175 |
"LET p = t IN u \<equiv> Let (pat_type p) t (\<lambda>[p]. Base u)" |
|
176 |
||
80914
d97fdabd9e2b
standardize mixfix annotations via "isabelle update -a -u mixfix_cartouches" --- to simplify systematic editing;
wenzelm
parents:
80142
diff
changeset
|
177 |
inductive typing :: "ctx \<Rightarrow> trm \<Rightarrow> ty \<Rightarrow> bool" (\<open>_ \<turnstile> _ : _\<close> [60, 60, 60] 60) |
33189 | 178 |
where |
179 |
Var [intro]: "valid \<Gamma> \<Longrightarrow> (x, T) \<in> set \<Gamma> \<Longrightarrow> \<Gamma> \<turnstile> Var x : T" |
|
180 |
| Tuple [intro]: "\<Gamma> \<turnstile> t : T \<Longrightarrow> \<Gamma> \<turnstile> u : U \<Longrightarrow> \<Gamma> \<turnstile> \<langle>t, u\<rangle> : T \<otimes> U" |
|
181 |
| Abs [intro]: "(x, T) # \<Gamma> \<turnstile> t : U \<Longrightarrow> \<Gamma> \<turnstile> (\<lambda>x:T. t) : T \<rightarrow> U" |
|
182 |
| App [intro]: "\<Gamma> \<turnstile> t : T \<rightarrow> U \<Longrightarrow> \<Gamma> \<turnstile> u : T \<Longrightarrow> \<Gamma> \<turnstile> t \<cdot> u : U" |
|
183 |
| Let: "((supp p)::name set) \<sharp>* t \<Longrightarrow> |
|
184 |
\<Gamma> \<turnstile> t : T \<Longrightarrow> \<turnstile> p : T \<Rightarrow> \<Delta> \<Longrightarrow> \<Delta> @ \<Gamma> \<turnstile> u : U \<Longrightarrow> |
|
185 |
\<Gamma> \<turnstile> (LET p = t IN u) : U" |
|
186 |
||
187 |
equivariance ptyping |
|
188 |
||
189 |
equivariance valid |
|
190 |
||
191 |
equivariance typing |
|
192 |
||
193 |
lemma valid_typing: |
|
194 |
assumes "\<Gamma> \<turnstile> t : T" |
|
195 |
shows "valid \<Gamma>" using assms |
|
196 |
by induct auto |
|
197 |
||
198 |
lemma pat_var: |
|
199 |
assumes "\<turnstile> p : T \<Rightarrow> \<Delta>" |
|
200 |
shows "(supp p::name set) = supp \<Delta>" using assms |
|
201 |
by induct (auto simp add: supp_list_nil supp_list_cons supp_prod supp_list_append) |
|
202 |
||
203 |
lemma valid_app_fresh: |
|
204 |
assumes "valid (\<Delta> @ \<Gamma>)" and "(x::name) \<in> supp \<Delta>" |
|
205 |
shows "x \<sharp> \<Gamma>" using assms |
|
206 |
by (induct \<Delta>) |
|
207 |
(auto simp add: supp_list_nil supp_list_cons supp_prod supp_atm fresh_list_append) |
|
208 |
||
209 |
lemma pat_freshs: |
|
210 |
assumes "\<turnstile> p : T \<Rightarrow> \<Delta>" |
|
211 |
shows "(supp p::name set) \<sharp>* c = (supp \<Delta>::name set) \<sharp>* c" using assms |
|
212 |
by (auto simp add: fresh_star_def pat_var) |
|
213 |
||
214 |
lemma valid_app_mono: |
|
53015
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
45129
diff
changeset
|
215 |
assumes "valid (\<Delta> @ \<Gamma>\<^sub>1)" and "(supp \<Delta>::name set) \<sharp>* \<Gamma>\<^sub>2" and "valid \<Gamma>\<^sub>2" and "\<Gamma>\<^sub>1 \<sqsubseteq> \<Gamma>\<^sub>2" |
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
45129
diff
changeset
|
216 |
shows "valid (\<Delta> @ \<Gamma>\<^sub>2)" using assms |
33189 | 217 |
by (induct \<Delta>) |
218 |
(auto simp add: supp_list_cons fresh_star_Un_elim supp_prod |
|
219 |
fresh_list_append supp_atm fresh_star_insert_elim fresh_star_empty_elim) |
|
220 |
||
221 |
nominal_inductive2 typing |
|
222 |
avoids |
|
223 |
Abs: "{x}" |
|
224 |
| Let: "(supp p)::name set" |
|
225 |
by (auto simp add: fresh_star_def abs_fresh fin_supp pat_var |
|
226 |
dest!: valid_typing valid_app_fresh) |
|
227 |
||
228 |
lemma better_T_Let [intro]: |
|
229 |
assumes t: "\<Gamma> \<turnstile> t : T" and p: "\<turnstile> p : T \<Rightarrow> \<Delta>" and u: "\<Delta> @ \<Gamma> \<turnstile> u : U" |
|
230 |
shows "\<Gamma> \<turnstile> (LET p = t IN u) : U" |
|
231 |
proof - |
|
232 |
obtain pi::"name prm" where pi: "(pi \<bullet> (supp p::name set)) \<sharp>* (t, Base u, \<Gamma>)" |
|
233 |
and pi': "set pi \<subseteq> supp p \<times> (pi \<bullet> supp p)" |
|
234 |
by (rule at_set_avoiding [OF at_name_inst fin_supp fin_supp]) |
|
235 |
from p u have p_fresh: "(supp p::name set) \<sharp>* \<Gamma>" |
|
236 |
by (auto simp add: fresh_star_def pat_var dest!: valid_typing valid_app_fresh) |
|
237 |
from pi have p_fresh': "(pi \<bullet> (supp p::name set)) \<sharp>* \<Gamma>" |
|
238 |
by (simp add: fresh_star_prod_elim) |
|
239 |
from pi have p_fresh'': "(pi \<bullet> (supp p::name set)) \<sharp>* Base u" |
|
240 |
by (simp add: fresh_star_prod_elim) |
|
241 |
from pi have "(supp (pi \<bullet> p)::name set) \<sharp>* t" |
|
242 |
by (simp add: fresh_star_prod_elim eqvts) |
|
243 |
moreover note t |
|
244 |
moreover from p have "pi \<bullet> (\<turnstile> p : T \<Rightarrow> \<Delta>)" by (rule perm_boolI) |
|
245 |
then have "\<turnstile> (pi \<bullet> p) : T \<Rightarrow> (pi \<bullet> \<Delta>)" by (simp add: eqvts perm_type) |
|
246 |
moreover from u have "pi \<bullet> (\<Delta> @ \<Gamma> \<turnstile> u : U)" by (rule perm_boolI) |
|
247 |
with pt_freshs_freshs [OF pt_name_inst at_name_inst pi' p_fresh p_fresh'] |
|
248 |
have "(pi \<bullet> \<Delta>) @ \<Gamma> \<turnstile> (pi \<bullet> u) : U" by (simp add: eqvts perm_type) |
|
249 |
ultimately have "\<Gamma> \<turnstile> (LET (pi \<bullet> p) = t IN (pi \<bullet> u)) : U" |
|
250 |
by (rule Let) |
|
251 |
then show ?thesis by (simp add: abs_pat_alpha [OF p_fresh'' pi'] pat_type_perm_eq) |
|
252 |
qed |
|
253 |
||
254 |
lemma weakening: |
|
53015
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
45129
diff
changeset
|
255 |
assumes "\<Gamma>\<^sub>1 \<turnstile> t : T" and "valid \<Gamma>\<^sub>2" and "\<Gamma>\<^sub>1 \<sqsubseteq> \<Gamma>\<^sub>2" |
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
45129
diff
changeset
|
256 |
shows "\<Gamma>\<^sub>2 \<turnstile> t : T" using assms |
80140 | 257 |
proof (nominal_induct \<Gamma>\<^sub>1 t T avoiding: \<Gamma>\<^sub>2 rule: typing.strong_induct) |
258 |
case (Abs x T \<Gamma> t U) |
|
259 |
then show ?case |
|
260 |
by (simp add: typing.Abs valid.Cons) |
|
261 |
next |
|
262 |
case (Let p t \<Gamma> T \<Delta> u U) |
|
263 |
then show ?case |
|
264 |
by (smt (verit, ccfv_threshold) Un_iff pat_freshs set_append typing.simps valid_app_mono valid_typing) |
|
265 |
qed auto |
|
33189 | 266 |
|
267 |
inductive |
|
80914
d97fdabd9e2b
standardize mixfix annotations via "isabelle update -a -u mixfix_cartouches" --- to simplify systematic editing;
wenzelm
parents:
80142
diff
changeset
|
268 |
match :: "pat \<Rightarrow> trm \<Rightarrow> (name \<times> trm) list \<Rightarrow> bool" (\<open>\<turnstile> _ \<rhd> _ \<Rightarrow> _\<close> [50, 50, 50] 50) |
33189 | 269 |
where |
270 |
PVar: "\<turnstile> PVar x T \<rhd> t \<Rightarrow> [(x, t)]" |
|
271 |
| PProd: "\<turnstile> p \<rhd> t \<Rightarrow> \<theta> \<Longrightarrow> \<turnstile> q \<rhd> u \<Rightarrow> \<theta>' \<Longrightarrow> \<turnstile> \<langle>\<langle>p, q\<rangle>\<rangle> \<rhd> \<langle>t, u\<rangle> \<Rightarrow> \<theta> @ \<theta>'" |
|
272 |
||
273 |
fun |
|
274 |
lookup :: "(name \<times> trm) list \<Rightarrow> name \<Rightarrow> trm" |
|
275 |
where |
|
276 |
"lookup [] x = Var x" |
|
277 |
| "lookup ((y, e) # \<theta>) x = (if x = y then e else lookup \<theta> x)" |
|
278 |
||
279 |
lemma lookup_eqvt[eqvt]: |
|
280 |
fixes pi :: "name prm" |
|
281 |
and \<theta> :: "(name \<times> trm) list" |
|
282 |
and X :: "name" |
|
283 |
shows "pi \<bullet> (lookup \<theta> X) = lookup (pi \<bullet> \<theta>) (pi \<bullet> X)" |
|
284 |
by (induct \<theta>) (auto simp add: eqvts) |
|
285 |
||
286 |
nominal_primrec |
|
80914
d97fdabd9e2b
standardize mixfix annotations via "isabelle update -a -u mixfix_cartouches" --- to simplify systematic editing;
wenzelm
parents:
80142
diff
changeset
|
287 |
psubst :: "(name \<times> trm) list \<Rightarrow> trm \<Rightarrow> trm" (\<open>_\<lparr>_\<rparr>\<close> [95,0] 210) |
d97fdabd9e2b
standardize mixfix annotations via "isabelle update -a -u mixfix_cartouches" --- to simplify systematic editing;
wenzelm
parents:
80142
diff
changeset
|
288 |
and psubstb :: "(name \<times> trm) list \<Rightarrow> btrm \<Rightarrow> btrm" (\<open>_\<lparr>_\<rparr>\<^sub>b\<close> [95,0] 210) |
33189 | 289 |
where |
290 |
"\<theta>\<lparr>Var x\<rparr> = (lookup \<theta> x)" |
|
291 |
| "\<theta>\<lparr>t \<cdot> u\<rparr> = \<theta>\<lparr>t\<rparr> \<cdot> \<theta>\<lparr>u\<rparr>" |
|
292 |
| "\<theta>\<lparr>\<langle>t, u\<rangle>\<rparr> = \<langle>\<theta>\<lparr>t\<rparr>, \<theta>\<lparr>u\<rparr>\<rangle>" |
|
293 |
| "\<theta>\<lparr>Let T t u\<rparr> = Let T (\<theta>\<lparr>t\<rparr>) (\<theta>\<lparr>u\<rparr>\<^sub>b)" |
|
294 |
| "x \<sharp> \<theta> \<Longrightarrow> \<theta>\<lparr>\<lambda>x:T. t\<rparr> = (\<lambda>x:T. \<theta>\<lparr>t\<rparr>)" |
|
295 |
| "\<theta>\<lparr>Base t\<rparr>\<^sub>b = Base (\<theta>\<lparr>t\<rparr>)" |
|
296 |
| "x \<sharp> \<theta> \<Longrightarrow> \<theta>\<lparr>Bind T x t\<rparr>\<^sub>b = Bind T x (\<theta>\<lparr>t\<rparr>\<^sub>b)" |
|
80140 | 297 |
by (finite_guess | simp add: abs_fresh | fresh_guess)+ |
33189 | 298 |
|
299 |
lemma lookup_fresh: |
|
300 |
"x = y \<longrightarrow> x \<in> set (map fst \<theta>) \<Longrightarrow> \<forall>(y, t)\<in>set \<theta>. x \<sharp> t \<Longrightarrow> x \<sharp> lookup \<theta> y" |
|
80140 | 301 |
by (induct \<theta>) (use fresh_atm in force)+ |
33189 | 302 |
|
303 |
lemma psubst_fresh: |
|
304 |
assumes "x \<in> set (map fst \<theta>)" and "\<forall>(y, t)\<in>set \<theta>. x \<sharp> t" |
|
305 |
shows "x \<sharp> \<theta>\<lparr>t\<rparr>" and "x \<sharp> \<theta>\<lparr>t'\<rparr>\<^sub>b" using assms |
|
80140 | 306 |
proof (nominal_induct t and t' avoiding: \<theta> rule: trm_btrm.strong_inducts) |
307 |
case (Var name) |
|
308 |
then show ?case |
|
309 |
by (metis lookup_fresh simps(1)) |
|
310 |
qed (auto simp: abs_fresh) |
|
33189 | 311 |
|
312 |
lemma psubst_eqvt[eqvt]: |
|
313 |
fixes pi :: "name prm" |
|
314 |
shows "pi \<bullet> (\<theta>\<lparr>t\<rparr>) = (pi \<bullet> \<theta>)\<lparr>pi \<bullet> t\<rparr>" |
|
315 |
and "pi \<bullet> (\<theta>\<lparr>t'\<rparr>\<^sub>b) = (pi \<bullet> \<theta>)\<lparr>pi \<bullet> t'\<rparr>\<^sub>b" |
|
316 |
by (nominal_induct t and t' avoiding: \<theta> rule: trm_btrm.strong_inducts) |
|
317 |
(simp_all add: eqvts fresh_bij) |
|
318 |
||
319 |
abbreviation |
|
81127 | 320 |
subst :: "trm \<Rightarrow> name \<Rightarrow> trm \<Rightarrow> trm" (\<open>_[_\<leadsto>_]\<close> [100,0,0] 100) |
33189 | 321 |
where |
81127 | 322 |
"t[x\<leadsto>t'] \<equiv> [(x,t')]\<lparr>t\<rparr>" |
33189 | 323 |
|
324 |
abbreviation |
|
81127 | 325 |
substb :: "btrm \<Rightarrow> name \<Rightarrow> trm \<Rightarrow> btrm" (\<open>_[_\<leadsto>_]\<^sub>b\<close> [100,0,0] 100) |
33189 | 326 |
where |
81127 | 327 |
"t[x\<leadsto>t']\<^sub>b \<equiv> [(x,t')]\<lparr>t\<rparr>\<^sub>b" |
33189 | 328 |
|
329 |
lemma lookup_forget: |
|
330 |
"(supp (map fst \<theta>)::name set) \<sharp>* x \<Longrightarrow> lookup \<theta> x = Var x" |
|
331 |
by (induct \<theta>) (auto simp add: split_paired_all fresh_star_def fresh_atm supp_list_cons supp_atm) |
|
332 |
||
333 |
lemma supp_fst: "(x::name) \<in> supp (map fst (\<theta>::(name \<times> trm) list)) \<Longrightarrow> x \<in> supp \<theta>" |
|
334 |
by (induct \<theta>) (auto simp add: supp_list_nil supp_list_cons supp_prod) |
|
335 |
||
336 |
lemma psubst_forget: |
|
337 |
"(supp (map fst \<theta>)::name set) \<sharp>* t \<Longrightarrow> \<theta>\<lparr>t\<rparr> = t" |
|
338 |
"(supp (map fst \<theta>)::name set) \<sharp>* t' \<Longrightarrow> \<theta>\<lparr>t'\<rparr>\<^sub>b = t'" |
|
80140 | 339 |
proof (nominal_induct t and t' avoiding: \<theta> rule: trm_btrm.strong_inducts) |
340 |
case (Var name) |
|
341 |
then show ?case |
|
342 |
by (simp add: fresh_star_set lookup_forget) |
|
343 |
next |
|
344 |
case (Abs ty name trm) |
|
345 |
then show ?case |
|
346 |
apply (simp add: fresh_def) |
|
347 |
by (metis abs_fresh(1) fresh_star_set supp_fst trm.fresh(3)) |
|
348 |
next |
|
349 |
case (Bind ty name btrm) |
|
350 |
then show ?case |
|
351 |
apply (simp add: fresh_def) |
|
352 |
by (metis abs_fresh(1) btrm.fresh(2) fresh_star_set supp_fst) |
|
353 |
qed (auto simp: fresh_star_set) |
|
33189 | 354 |
|
80142 | 355 |
lemma psubst_nil[simp]: "[]\<lparr>t\<rparr> = t" "[]\<lparr>t'\<rparr>\<^sub>b = t'" |
33189 | 356 |
by (induct t and t' rule: trm_btrm.inducts) (simp_all add: fresh_list_nil) |
357 |
||
358 |
lemma psubst_cons: |
|
359 |
assumes "(supp (map fst \<theta>)::name set) \<sharp>* u" |
|
81127 | 360 |
shows "((x, u) # \<theta>)\<lparr>t\<rparr> = \<theta>\<lparr>t[x\<leadsto>u]\<rparr>" and "((x, u) # \<theta>)\<lparr>t'\<rparr>\<^sub>b = \<theta>\<lparr>t'[x\<leadsto>u]\<^sub>b\<rparr>\<^sub>b" |
33189 | 361 |
using assms |
362 |
by (nominal_induct t and t' avoiding: x u \<theta> rule: trm_btrm.strong_inducts) |
|
363 |
(simp_all add: fresh_list_nil fresh_list_cons psubst_forget) |
|
364 |
||
365 |
lemma psubst_append: |
|
53015
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
45129
diff
changeset
|
366 |
"(supp (map fst (\<theta>\<^sub>1 @ \<theta>\<^sub>2))::name set) \<sharp>* map snd (\<theta>\<^sub>1 @ \<theta>\<^sub>2) \<Longrightarrow> (\<theta>\<^sub>1 @ \<theta>\<^sub>2)\<lparr>t\<rparr> = \<theta>\<^sub>2\<lparr>\<theta>\<^sub>1\<lparr>t\<rparr>\<rparr>" |
80142 | 367 |
proof (induct \<theta>\<^sub>1 arbitrary: t) |
368 |
case Nil |
|
369 |
then show ?case |
|
370 |
by (auto simp: psubst_nil) |
|
371 |
next |
|
372 |
case (Cons a \<theta>\<^sub>1) |
|
373 |
then show ?case |
|
374 |
proof (cases a) |
|
375 |
case (Pair a b) |
|
376 |
with Cons show ?thesis |
|
377 |
apply (simp add: supp_list_cons fresh_star_set fresh_list_cons) |
|
378 |
by (metis Un_iff fresh_star_set map_append psubst_cons(1) supp_list_append) |
|
379 |
qed |
|
380 |
qed |
|
33189 | 381 |
|
382 |
lemma abs_pat_psubst [simp]: |
|
383 |
"(supp p::name set) \<sharp>* \<theta> \<Longrightarrow> \<theta>\<lparr>\<lambda>[p]. t\<rparr>\<^sub>b = (\<lambda>[p]. \<theta>\<lparr>t\<rparr>\<^sub>b)" |
|
384 |
by (induct p arbitrary: t) (auto simp add: fresh_star_def supp_atm) |
|
385 |
||
386 |
lemma valid_insert: |
|
387 |
assumes "valid (\<Delta> @ [(x, T)] @ \<Gamma>)" |
|
388 |
shows "valid (\<Delta> @ \<Gamma>)" using assms |
|
389 |
by (induct \<Delta>) |
|
390 |
(auto simp add: fresh_list_append fresh_list_cons) |
|
391 |
||
392 |
lemma fresh_set: |
|
393 |
shows "y \<sharp> xs = (\<forall>x\<in>set xs. y \<sharp> x)" |
|
394 |
by (induct xs) (simp_all add: fresh_list_nil fresh_list_cons) |
|
395 |
||
396 |
lemma context_unique: |
|
397 |
assumes "valid \<Gamma>" |
|
398 |
and "(x, T) \<in> set \<Gamma>" |
|
399 |
and "(x, U) \<in> set \<Gamma>" |
|
400 |
shows "T = U" using assms |
|
401 |
by induct (auto simp add: fresh_set fresh_prod fresh_atm) |
|
402 |
||
403 |
lemma subst_type_aux: |
|
404 |
assumes a: "\<Delta> @ [(x, U)] @ \<Gamma> \<turnstile> t : T" |
|
405 |
and b: "\<Gamma> \<turnstile> u : U" |
|
81127 | 406 |
shows "\<Delta> @ \<Gamma> \<turnstile> t[x\<leadsto>u] : T" using a b |
33189 | 407 |
proof (nominal_induct \<Gamma>'\<equiv>"\<Delta> @ [(x, U)] @ \<Gamma>" t T avoiding: x u \<Delta> rule: typing.strong_induct) |
34915 | 408 |
case (Var y T x u \<Delta>) |
63167 | 409 |
from \<open>valid (\<Delta> @ [(x, U)] @ \<Gamma>)\<close> |
34915 | 410 |
have valid: "valid (\<Delta> @ \<Gamma>)" by (rule valid_insert) |
81127 | 411 |
show "\<Delta> @ \<Gamma> \<turnstile> Var y[x\<leadsto>u] : T" |
33189 | 412 |
proof cases |
413 |
assume eq: "x = y" |
|
34915 | 414 |
from Var eq have "T = U" by (auto intro: context_unique) |
81127 | 415 |
with Var eq valid show "\<Delta> @ \<Gamma> \<turnstile> Var y[x\<leadsto>u] : T" by (auto intro: weakening) |
33189 | 416 |
next |
417 |
assume ineq: "x \<noteq> y" |
|
34915 | 418 |
from Var ineq have "(y, T) \<in> set (\<Delta> @ \<Gamma>)" by simp |
81127 | 419 |
then show "\<Delta> @ \<Gamma> \<turnstile> Var y[x\<leadsto>u] : T" using ineq valid by auto |
33189 | 420 |
qed |
421 |
next |
|
53015
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
45129
diff
changeset
|
422 |
case (Tuple t\<^sub>1 T\<^sub>1 t\<^sub>2 T\<^sub>2) |
63167 | 423 |
from refl \<open>\<Gamma> \<turnstile> u : U\<close> |
81127 | 424 |
have "\<Delta> @ \<Gamma> \<turnstile> t\<^sub>1[x\<leadsto>u] : T\<^sub>1" by (rule Tuple) |
63167 | 425 |
moreover from refl \<open>\<Gamma> \<turnstile> u : U\<close> |
81127 | 426 |
have "\<Delta> @ \<Gamma> \<turnstile> t\<^sub>2[x\<leadsto>u] : T\<^sub>2" by (rule Tuple) |
427 |
ultimately have "\<Delta> @ \<Gamma> \<turnstile> \<langle>t\<^sub>1[x\<leadsto>u], t\<^sub>2[x\<leadsto>u]\<rangle> : T\<^sub>1 \<otimes> T\<^sub>2" .. |
|
33189 | 428 |
then show ?case by simp |
429 |
next |
|
34915 | 430 |
case (Let p t T \<Delta>' s S) |
63167 | 431 |
from refl \<open>\<Gamma> \<turnstile> u : U\<close> |
81127 | 432 |
have "\<Delta> @ \<Gamma> \<turnstile> t[x\<leadsto>u] : T" by (rule Let) |
63167 | 433 |
moreover note \<open>\<turnstile> p : T \<Rightarrow> \<Delta>'\<close> |
34915 | 434 |
moreover have "\<Delta>' @ (\<Delta> @ [(x, U)] @ \<Gamma>) = (\<Delta>' @ \<Delta>) @ [(x, U)] @ \<Gamma>" by simp |
81127 | 435 |
then have "(\<Delta>' @ \<Delta>) @ \<Gamma> \<turnstile> s[x\<leadsto>u] : S" using \<open>\<Gamma> \<turnstile> u : U\<close> by (rule Let) |
436 |
then have "\<Delta>' @ \<Delta> @ \<Gamma> \<turnstile> s[x\<leadsto>u] : S" by simp |
|
437 |
ultimately have "\<Delta> @ \<Gamma> \<turnstile> (LET p = t[x\<leadsto>u] IN s[x\<leadsto>u]) : S" |
|
33189 | 438 |
by (rule better_T_Let) |
439 |
moreover from Let have "(supp p::name set) \<sharp>* [(x, u)]" |
|
440 |
by (simp add: fresh_star_def fresh_list_nil fresh_list_cons) |
|
441 |
ultimately show ?case by simp |
|
442 |
next |
|
34915 | 443 |
case (Abs y T t S) |
444 |
have "(y, T) # \<Delta> @ [(x, U)] @ \<Gamma> = ((y, T) # \<Delta>) @ [(x, U)] @ \<Gamma>" |
|
33189 | 445 |
by simp |
81127 | 446 |
then have "((y, T) # \<Delta>) @ \<Gamma> \<turnstile> t[x\<leadsto>u] : S" using \<open>\<Gamma> \<turnstile> u : U\<close> by (rule Abs) |
447 |
then have "(y, T) # \<Delta> @ \<Gamma> \<turnstile> t[x\<leadsto>u] : S" by simp |
|
448 |
then have "\<Delta> @ \<Gamma> \<turnstile> (\<lambda>y:T. t[x\<leadsto>u]) : T \<rightarrow> S" |
|
33189 | 449 |
by (rule typing.Abs) |
450 |
moreover from Abs have "y \<sharp> [(x, u)]" |
|
451 |
by (simp add: fresh_list_nil fresh_list_cons) |
|
452 |
ultimately show ?case by simp |
|
453 |
next |
|
53015
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
45129
diff
changeset
|
454 |
case (App t\<^sub>1 T S t\<^sub>2) |
63167 | 455 |
from refl \<open>\<Gamma> \<turnstile> u : U\<close> |
81127 | 456 |
have "\<Delta> @ \<Gamma> \<turnstile> t\<^sub>1[x\<leadsto>u] : T \<rightarrow> S" by (rule App) |
63167 | 457 |
moreover from refl \<open>\<Gamma> \<turnstile> u : U\<close> |
81127 | 458 |
have "\<Delta> @ \<Gamma> \<turnstile> t\<^sub>2[x\<leadsto>u] : T" by (rule App) |
459 |
ultimately have "\<Delta> @ \<Gamma> \<turnstile> (t\<^sub>1[x\<leadsto>u]) \<cdot> (t\<^sub>2[x\<leadsto>u]) : S" |
|
33189 | 460 |
by (rule typing.App) |
461 |
then show ?case by simp |
|
462 |
qed |
|
463 |
||
464 |
lemmas subst_type = subst_type_aux [of "[]", simplified] |
|
465 |
||
466 |
lemma match_supp_fst: |
|
467 |
assumes "\<turnstile> p \<rhd> u \<Rightarrow> \<theta>" shows "(supp (map fst \<theta>)::name set) = supp p" using assms |
|
468 |
by induct (simp_all add: supp_list_nil supp_list_cons supp_list_append) |
|
469 |
||
470 |
lemma match_supp_snd: |
|
471 |
assumes "\<turnstile> p \<rhd> u \<Rightarrow> \<theta>" shows "(supp (map snd \<theta>)::name set) = supp u" using assms |
|
472 |
by induct (simp_all add: supp_list_nil supp_list_cons supp_list_append trm.supp) |
|
473 |
||
474 |
lemma match_fresh: "\<turnstile> p \<rhd> u \<Rightarrow> \<theta> \<Longrightarrow> (supp p::name set) \<sharp>* u \<Longrightarrow> |
|
475 |
(supp (map fst \<theta>)::name set) \<sharp>* map snd \<theta>" |
|
476 |
by (simp add: fresh_star_def fresh_def match_supp_fst match_supp_snd) |
|
477 |
||
478 |
lemma match_type_aux: |
|
479 |
assumes "\<turnstile> p : U \<Rightarrow> \<Delta>" |
|
53015
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
45129
diff
changeset
|
480 |
and "\<Gamma>\<^sub>2 \<turnstile> u : U" |
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
45129
diff
changeset
|
481 |
and "\<Gamma>\<^sub>1 @ \<Delta> @ \<Gamma>\<^sub>2 \<turnstile> t : T" |
33189 | 482 |
and "\<turnstile> p \<rhd> u \<Rightarrow> \<theta>" |
483 |
and "(supp p::name set) \<sharp>* u" |
|
53015
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
45129
diff
changeset
|
484 |
shows "\<Gamma>\<^sub>1 @ \<Gamma>\<^sub>2 \<turnstile> \<theta>\<lparr>t\<rparr> : T" using assms |
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
45129
diff
changeset
|
485 |
proof (induct arbitrary: \<Gamma>\<^sub>1 \<Gamma>\<^sub>2 t u T \<theta>) |
33189 | 486 |
case (PVar x U) |
63167 | 487 |
from \<open>\<Gamma>\<^sub>1 @ [(x, U)] @ \<Gamma>\<^sub>2 \<turnstile> t : T\<close> \<open>\<Gamma>\<^sub>2 \<turnstile> u : U\<close> |
81127 | 488 |
have "\<Gamma>\<^sub>1 @ \<Gamma>\<^sub>2 \<turnstile> t[x\<leadsto>u] : T" by (rule subst_type_aux) |
63167 | 489 |
moreover from \<open>\<turnstile> PVar x U \<rhd> u \<Rightarrow> \<theta>\<close> have "\<theta> = [(x, u)]" |
33189 | 490 |
by cases simp_all |
491 |
ultimately show ?case by simp |
|
492 |
next |
|
53015
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
45129
diff
changeset
|
493 |
case (PTuple p S \<Delta>\<^sub>1 q U \<Delta>\<^sub>2) |
63167 | 494 |
from \<open>\<turnstile> \<langle>\<langle>p, q\<rangle>\<rangle> \<rhd> u \<Rightarrow> \<theta>\<close> obtain u\<^sub>1 u\<^sub>2 \<theta>\<^sub>1 \<theta>\<^sub>2 |
53015
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
45129
diff
changeset
|
495 |
where u: "u = \<langle>u\<^sub>1, u\<^sub>2\<rangle>" and \<theta>: "\<theta> = \<theta>\<^sub>1 @ \<theta>\<^sub>2" |
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
45129
diff
changeset
|
496 |
and p: "\<turnstile> p \<rhd> u\<^sub>1 \<Rightarrow> \<theta>\<^sub>1" and q: "\<turnstile> q \<rhd> u\<^sub>2 \<Rightarrow> \<theta>\<^sub>2" |
33189 | 497 |
by cases simp_all |
53015
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
45129
diff
changeset
|
498 |
with PTuple have "\<Gamma>\<^sub>2 \<turnstile> \<langle>u\<^sub>1, u\<^sub>2\<rangle> : S \<otimes> U" by simp |
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
45129
diff
changeset
|
499 |
then obtain u\<^sub>1: "\<Gamma>\<^sub>2 \<turnstile> u\<^sub>1 : S" and u\<^sub>2: "\<Gamma>\<^sub>2 \<turnstile> u\<^sub>2 : U" |
33189 | 500 |
by cases (simp_all add: ty.inject trm.inject) |
53015
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
45129
diff
changeset
|
501 |
note u\<^sub>1 |
63167 | 502 |
moreover from \<open>\<Gamma>\<^sub>1 @ (\<Delta>\<^sub>2 @ \<Delta>\<^sub>1) @ \<Gamma>\<^sub>2 \<turnstile> t : T\<close> |
53015
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
45129
diff
changeset
|
503 |
have "(\<Gamma>\<^sub>1 @ \<Delta>\<^sub>2) @ \<Delta>\<^sub>1 @ \<Gamma>\<^sub>2 \<turnstile> t : T" by simp |
33189 | 504 |
moreover note p |
63167 | 505 |
moreover from \<open>supp \<langle>\<langle>p, q\<rangle>\<rangle> \<sharp>* u\<close> and u |
53015
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
45129
diff
changeset
|
506 |
have "(supp p::name set) \<sharp>* u\<^sub>1" by (simp add: fresh_star_def) |
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
45129
diff
changeset
|
507 |
ultimately have \<theta>\<^sub>1: "(\<Gamma>\<^sub>1 @ \<Delta>\<^sub>2) @ \<Gamma>\<^sub>2 \<turnstile> \<theta>\<^sub>1\<lparr>t\<rparr> : T" |
33189 | 508 |
by (rule PTuple) |
53015
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
45129
diff
changeset
|
509 |
note u\<^sub>2 |
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
45129
diff
changeset
|
510 |
moreover from \<theta>\<^sub>1 |
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
45129
diff
changeset
|
511 |
have "\<Gamma>\<^sub>1 @ \<Delta>\<^sub>2 @ \<Gamma>\<^sub>2 \<turnstile> \<theta>\<^sub>1\<lparr>t\<rparr> : T" by simp |
33189 | 512 |
moreover note q |
63167 | 513 |
moreover from \<open>supp \<langle>\<langle>p, q\<rangle>\<rangle> \<sharp>* u\<close> and u |
53015
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
45129
diff
changeset
|
514 |
have "(supp q::name set) \<sharp>* u\<^sub>2" by (simp add: fresh_star_def) |
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
45129
diff
changeset
|
515 |
ultimately have "\<Gamma>\<^sub>1 @ \<Gamma>\<^sub>2 \<turnstile> \<theta>\<^sub>2\<lparr>\<theta>\<^sub>1\<lparr>t\<rparr>\<rparr> : T" |
33189 | 516 |
by (rule PTuple) |
63167 | 517 |
moreover from \<open>\<turnstile> \<langle>\<langle>p, q\<rangle>\<rangle> \<rhd> u \<Rightarrow> \<theta>\<close> \<open>supp \<langle>\<langle>p, q\<rangle>\<rangle> \<sharp>* u\<close> |
33189 | 518 |
have "(supp (map fst \<theta>)::name set) \<sharp>* map snd \<theta>" |
519 |
by (rule match_fresh) |
|
520 |
ultimately show ?case using \<theta> by (simp add: psubst_append) |
|
521 |
qed |
|
522 |
||
53015
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
45129
diff
changeset
|
523 |
lemmas match_type = match_type_aux [where \<Gamma>\<^sub>1="[]", simplified] |
33189 | 524 |
|
80914
d97fdabd9e2b
standardize mixfix annotations via "isabelle update -a -u mixfix_cartouches" --- to simplify systematic editing;
wenzelm
parents:
80142
diff
changeset
|
525 |
inductive eval :: "trm \<Rightarrow> trm \<Rightarrow> bool" (\<open>_ \<longmapsto> _\<close> [60,60] 60) |
33189 | 526 |
where |
527 |
TupleL: "t \<longmapsto> t' \<Longrightarrow> \<langle>t, u\<rangle> \<longmapsto> \<langle>t', u\<rangle>" |
|
528 |
| TupleR: "u \<longmapsto> u' \<Longrightarrow> \<langle>t, u\<rangle> \<longmapsto> \<langle>t, u'\<rangle>" |
|
529 |
| Abs: "t \<longmapsto> t' \<Longrightarrow> (\<lambda>x:T. t) \<longmapsto> (\<lambda>x:T. t')" |
|
530 |
| AppL: "t \<longmapsto> t' \<Longrightarrow> t \<cdot> u \<longmapsto> t' \<cdot> u" |
|
531 |
| AppR: "u \<longmapsto> u' \<Longrightarrow> t \<cdot> u \<longmapsto> t \<cdot> u'" |
|
81127 | 532 |
| Beta: "x \<sharp> u \<Longrightarrow> (\<lambda>x:T. t) \<cdot> u \<longmapsto> t[x\<leadsto>u]" |
33189 | 533 |
| Let: "((supp p)::name set) \<sharp>* t \<Longrightarrow> distinct (pat_vars p) \<Longrightarrow> |
534 |
\<turnstile> p \<rhd> t \<Rightarrow> \<theta> \<Longrightarrow> (LET p = t IN u) \<longmapsto> \<theta>\<lparr>u\<rparr>" |
|
535 |
||
536 |
equivariance match |
|
537 |
||
538 |
equivariance eval |
|
539 |
||
540 |
lemma match_vars: |
|
541 |
assumes "\<turnstile> p \<rhd> t \<Rightarrow> \<theta>" and "x \<in> supp p" |
|
542 |
shows "x \<in> set (map fst \<theta>)" using assms |
|
543 |
by induct (auto simp add: supp_atm) |
|
544 |
||
545 |
lemma match_fresh_mono: |
|
546 |
assumes "\<turnstile> p \<rhd> t \<Rightarrow> \<theta>" and "(x::name) \<sharp> t" |
|
547 |
shows "\<forall>(y, t)\<in>set \<theta>. x \<sharp> t" using assms |
|
548 |
by induct auto |
|
549 |
||
550 |
nominal_inductive2 eval |
|
551 |
avoids |
|
552 |
Abs: "{x}" |
|
553 |
| Beta: "{x}" |
|
554 |
| Let: "(supp p)::name set" |
|
80140 | 555 |
proof (simp_all add: fresh_star_def abs_fresh fin_supp) |
81127 | 556 |
show "x \<sharp> t[x\<leadsto>u]" if "x \<sharp> u" for x t u |
80140 | 557 |
by (simp add: \<open>x \<sharp> u\<close> psubst_fresh(1)) |
558 |
next |
|
559 |
show "\<forall>x\<in>supp p. (x::name) \<sharp> \<theta>\<lparr>u\<rparr>" |
|
560 |
if "\<forall>x\<in>supp p. (x::name) \<sharp> t" and "\<turnstile> p \<rhd> t \<Rightarrow> \<theta>" |
|
561 |
for p t \<theta> u |
|
562 |
by (meson that match_fresh_mono match_vars psubst_fresh(1)) |
|
563 |
qed |
|
33189 | 564 |
|
565 |
lemma typing_case_Abs: |
|
566 |
assumes ty: "\<Gamma> \<turnstile> (\<lambda>x:T. t) : S" |
|
567 |
and fresh: "x \<sharp> \<Gamma>" |
|
568 |
and R: "\<And>U. S = T \<rightarrow> U \<Longrightarrow> (x, T) # \<Gamma> \<turnstile> t : U \<Longrightarrow> P" |
|
569 |
shows P using ty |
|
570 |
proof cases |
|
34990 | 571 |
case (Abs x' T' t' U) |
33189 | 572 |
obtain y::name where y: "y \<sharp> (x, \<Gamma>, \<lambda>x':T'. t')" |
573 |
by (rule exists_fresh) (auto intro: fin_supp) |
|
63167 | 574 |
from \<open>(\<lambda>x:T. t) = (\<lambda>x':T'. t')\<close> [symmetric] |
33189 | 575 |
have x: "x \<sharp> (\<lambda>x':T'. t')" by (simp add: abs_fresh) |
576 |
have x': "x' \<sharp> (\<lambda>x':T'. t')" by (simp add: abs_fresh) |
|
63167 | 577 |
from \<open>(x', T') # \<Gamma> \<turnstile> t' : U\<close> have x'': "x' \<sharp> \<Gamma>" |
33189 | 578 |
by (auto dest: valid_typing) |
579 |
have "(\<lambda>x:T. t) = (\<lambda>x':T'. t')" by fact |
|
580 |
also from x x' y have "\<dots> = [(x, y)] \<bullet> [(x', y)] \<bullet> (\<lambda>x':T'. t')" |
|
581 |
by (simp only: perm_fresh_fresh fresh_prod) |
|
582 |
also have "\<dots> = (\<lambda>x:T'. [(x, y)] \<bullet> [(x', y)] \<bullet> t')" |
|
583 |
by (simp add: swap_simps perm_fresh_fresh) |
|
584 |
finally have "(\<lambda>x:T. t) = (\<lambda>x:T'. [(x, y)] \<bullet> [(x', y)] \<bullet> t')" . |
|
585 |
then have T: "T = T'" and t: "[(x, y)] \<bullet> [(x', y)] \<bullet> t' = t" |
|
586 |
by (simp_all add: trm.inject alpha) |
|
587 |
from Abs T have "S = T \<rightarrow> U" by simp |
|
63167 | 588 |
moreover from \<open>(x', T') # \<Gamma> \<turnstile> t' : U\<close> |
34990 | 589 |
have "[(x, y)] \<bullet> [(x', y)] \<bullet> ((x', T') # \<Gamma> \<turnstile> t' : U)" |
33189 | 590 |
by (simp add: perm_bool) |
34990 | 591 |
with T t y x'' fresh have "(x, T) # \<Gamma> \<turnstile> t : U" |
33189 | 592 |
by (simp add: eqvts swap_simps perm_fresh_fresh fresh_prod) |
593 |
ultimately show ?thesis by (rule R) |
|
594 |
qed simp_all |
|
595 |
||
596 |
nominal_primrec ty_size :: "ty \<Rightarrow> nat" |
|
597 |
where |
|
598 |
"ty_size (Atom n) = 0" |
|
599 |
| "ty_size (T \<rightarrow> U) = ty_size T + ty_size U + 1" |
|
600 |
| "ty_size (T \<otimes> U) = ty_size T + ty_size U + 1" |
|
601 |
by (rule TrueI)+ |
|
602 |
||
603 |
lemma bind_tuple_ineq: |
|
604 |
"ty_size (pat_type p) < ty_size U \<Longrightarrow> Bind U x t \<noteq> (\<lambda>[p]. u)" |
|
605 |
by (induct p arbitrary: U x t u) (auto simp add: btrm.inject) |
|
606 |
||
607 |
lemma valid_appD: assumes "valid (\<Gamma> @ \<Delta>)" |
|
608 |
shows "valid \<Gamma>" "valid \<Delta>" using assms |
|
609 |
by (induct \<Gamma>'\<equiv>"\<Gamma> @ \<Delta>" arbitrary: \<Gamma> \<Delta>) |
|
610 |
(auto simp add: Cons_eq_append_conv fresh_list_append) |
|
611 |
||
612 |
lemma valid_app_freshs: assumes "valid (\<Gamma> @ \<Delta>)" |
|
613 |
shows "(supp \<Gamma>::name set) \<sharp>* \<Delta>" "(supp \<Delta>::name set) \<sharp>* \<Gamma>" using assms |
|
614 |
by (induct \<Gamma>'\<equiv>"\<Gamma> @ \<Delta>" arbitrary: \<Gamma> \<Delta>) |
|
615 |
(auto simp add: Cons_eq_append_conv fresh_star_def |
|
616 |
fresh_list_nil fresh_list_cons supp_list_nil supp_list_cons fresh_list_append |
|
617 |
supp_prod fresh_prod supp_atm fresh_atm |
|
44687 | 618 |
dest: notE [OF iffD1 [OF fresh_def]]) |
33189 | 619 |
|
620 |
lemma perm_mem_left: "(x::name) \<in> ((pi::name prm) \<bullet> A) \<Longrightarrow> (rev pi \<bullet> x) \<in> A" |
|
621 |
by (drule perm_boolI [of _ "rev pi"]) (simp add: eqvts perm_pi_simp) |
|
622 |
||
623 |
lemma perm_mem_right: "(rev (pi::name prm) \<bullet> (x::name)) \<in> A \<Longrightarrow> x \<in> (pi \<bullet> A)" |
|
624 |
by (drule perm_boolI [of _ pi]) (simp add: eqvts perm_pi_simp) |
|
625 |
||
626 |
lemma perm_cases: |
|
627 |
assumes pi: "set pi \<subseteq> A \<times> A" |
|
628 |
shows "((pi::name prm) \<bullet> B) \<subseteq> A \<union> B" |
|
629 |
proof |
|
630 |
fix x assume "x \<in> pi \<bullet> B" |
|
631 |
then show "x \<in> A \<union> B" using pi |
|
80140 | 632 |
proof (induct pi arbitrary: x B rule: rev_induct) |
633 |
case Nil |
|
634 |
then show ?case |
|
635 |
by simp |
|
636 |
next |
|
637 |
case (snoc y xs) |
|
638 |
then show ?case |
|
639 |
apply simp |
|
640 |
by (metis SigmaE perm_mem_left perm_pi_simp(2) pt_name2 swap_simps(3)) |
|
641 |
qed |
|
33189 | 642 |
qed |
643 |
||
644 |
lemma abs_pat_alpha': |
|
645 |
assumes eq: "(\<lambda>[p]. t) = (\<lambda>[q]. u)" |
|
646 |
and ty: "pat_type p = pat_type q" |
|
647 |
and pv: "distinct (pat_vars p)" |
|
648 |
and qv: "distinct (pat_vars q)" |
|
649 |
shows "\<exists>pi::name prm. p = pi \<bullet> q \<and> t = pi \<bullet> u \<and> |
|
650 |
set pi \<subseteq> (supp p \<union> supp q) \<times> (supp p \<union> supp q)" |
|
651 |
using assms |
|
45129
1fce03e3e8ad
tuned proofs -- eliminated vacuous "induct arbitrary: ..." situations;
wenzelm
parents:
44687
diff
changeset
|
652 |
proof (induct p arbitrary: q t u) |
33189 | 653 |
case (PVar x T) |
654 |
note PVar' = this |
|
655 |
show ?case |
|
656 |
proof (cases q) |
|
657 |
case (PVar x' T') |
|
63167 | 658 |
with \<open>(\<lambda>[PVar x T]. t) = (\<lambda>[q]. u)\<close> |
33189 | 659 |
have "x = x' \<and> t = u \<or> x \<noteq> x' \<and> t = [(x, x')] \<bullet> u \<and> x \<sharp> u" |
660 |
by (simp add: btrm.inject alpha) |
|
661 |
then show ?thesis |
|
662 |
proof |
|
663 |
assume "x = x' \<and> t = u" |
|
664 |
with PVar PVar' have "PVar x T = ([]::name prm) \<bullet> q \<and> |
|
33268
02de0317f66f
eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents:
33189
diff
changeset
|
665 |
t = ([]::name prm) \<bullet> u \<and> |
02de0317f66f
eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents:
33189
diff
changeset
|
666 |
set ([]::name prm) \<subseteq> (supp (PVar x T) \<union> supp q) \<times> |
33189 | 667 |
(supp (PVar x T) \<union> supp q)" by simp |
668 |
then show ?thesis .. |
|
669 |
next |
|
670 |
assume "x \<noteq> x' \<and> t = [(x, x')] \<bullet> u \<and> x \<sharp> u" |
|
671 |
with PVar PVar' have "PVar x T = [(x, x')] \<bullet> q \<and> |
|
33268
02de0317f66f
eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents:
33189
diff
changeset
|
672 |
t = [(x, x')] \<bullet> u \<and> |
02de0317f66f
eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents:
33189
diff
changeset
|
673 |
set [(x, x')] \<subseteq> (supp (PVar x T) \<union> supp q) \<times> |
33189 | 674 |
(supp (PVar x T) \<union> supp q)" |
33268
02de0317f66f
eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents:
33189
diff
changeset
|
675 |
by (simp add: perm_swap swap_simps supp_atm perm_type) |
33189 | 676 |
then show ?thesis .. |
677 |
qed |
|
678 |
next |
|
53015
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
45129
diff
changeset
|
679 |
case (PTuple p\<^sub>1 p\<^sub>2) |
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
45129
diff
changeset
|
680 |
with PVar have "ty_size (pat_type p\<^sub>1) < ty_size T" by simp |
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
45129
diff
changeset
|
681 |
then have "Bind T x t \<noteq> (\<lambda>[p\<^sub>1]. \<lambda>[p\<^sub>2]. u)" |
33189 | 682 |
by (rule bind_tuple_ineq) |
683 |
moreover from PTuple PVar |
|
53015
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
45129
diff
changeset
|
684 |
have "Bind T x t = (\<lambda>[p\<^sub>1]. \<lambda>[p\<^sub>2]. u)" by simp |
33189 | 685 |
ultimately show ?thesis .. |
686 |
qed |
|
687 |
next |
|
53015
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
45129
diff
changeset
|
688 |
case (PTuple p\<^sub>1 p\<^sub>2) |
33189 | 689 |
note PTuple' = this |
690 |
show ?case |
|
691 |
proof (cases q) |
|
692 |
case (PVar x T) |
|
53015
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
45129
diff
changeset
|
693 |
with PTuple have "ty_size (pat_type p\<^sub>1) < ty_size T" by auto |
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
45129
diff
changeset
|
694 |
then have "Bind T x u \<noteq> (\<lambda>[p\<^sub>1]. \<lambda>[p\<^sub>2]. t)" |
33189 | 695 |
by (rule bind_tuple_ineq) |
696 |
moreover from PTuple PVar |
|
53015
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
45129
diff
changeset
|
697 |
have "Bind T x u = (\<lambda>[p\<^sub>1]. \<lambda>[p\<^sub>2]. t)" by simp |
33189 | 698 |
ultimately show ?thesis .. |
699 |
next |
|
53015
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
45129
diff
changeset
|
700 |
case (PTuple p\<^sub>1' p\<^sub>2') |
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
45129
diff
changeset
|
701 |
with PTuple' have "(\<lambda>[p\<^sub>1]. \<lambda>[p\<^sub>2]. t) = (\<lambda>[p\<^sub>1']. \<lambda>[p\<^sub>2']. u)" by simp |
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
45129
diff
changeset
|
702 |
moreover from PTuple PTuple' have "pat_type p\<^sub>1 = pat_type p\<^sub>1'" |
33189 | 703 |
by (simp add: ty.inject) |
53015
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
45129
diff
changeset
|
704 |
moreover from PTuple' have "distinct (pat_vars p\<^sub>1)" by simp |
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
45129
diff
changeset
|
705 |
moreover from PTuple PTuple' have "distinct (pat_vars p\<^sub>1')" by simp |
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
45129
diff
changeset
|
706 |
ultimately have "\<exists>pi::name prm. p\<^sub>1 = pi \<bullet> p\<^sub>1' \<and> |
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
45129
diff
changeset
|
707 |
(\<lambda>[p\<^sub>2]. t) = pi \<bullet> (\<lambda>[p\<^sub>2']. u) \<and> |
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
45129
diff
changeset
|
708 |
set pi \<subseteq> (supp p\<^sub>1 \<union> supp p\<^sub>1') \<times> (supp p\<^sub>1 \<union> supp p\<^sub>1')" |
33189 | 709 |
by (rule PTuple') |
710 |
then obtain pi::"name prm" where |
|
53015
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
45129
diff
changeset
|
711 |
"p\<^sub>1 = pi \<bullet> p\<^sub>1'" "(\<lambda>[p\<^sub>2]. t) = pi \<bullet> (\<lambda>[p\<^sub>2']. u)" and |
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
45129
diff
changeset
|
712 |
pi: "set pi \<subseteq> (supp p\<^sub>1 \<union> supp p\<^sub>1') \<times> (supp p\<^sub>1 \<union> supp p\<^sub>1')" by auto |
63167 | 713 |
from \<open>(\<lambda>[p\<^sub>2]. t) = pi \<bullet> (\<lambda>[p\<^sub>2']. u)\<close> |
53015
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
45129
diff
changeset
|
714 |
have "(\<lambda>[p\<^sub>2]. t) = (\<lambda>[pi \<bullet> p\<^sub>2']. pi \<bullet> u)" |
33189 | 715 |
by (simp add: eqvts) |
53015
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
45129
diff
changeset
|
716 |
moreover from PTuple PTuple' have "pat_type p\<^sub>2 = pat_type (pi \<bullet> p\<^sub>2')" |
33189 | 717 |
by (simp add: ty.inject pat_type_perm_eq) |
53015
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
45129
diff
changeset
|
718 |
moreover from PTuple' have "distinct (pat_vars p\<^sub>2)" by simp |
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
45129
diff
changeset
|
719 |
moreover from PTuple PTuple' have "distinct (pat_vars (pi \<bullet> p\<^sub>2'))" |
33189 | 720 |
by (simp add: pat_vars_eqvt [symmetric] distinct_eqvt [symmetric]) |
53015
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
45129
diff
changeset
|
721 |
ultimately have "\<exists>pi'::name prm. p\<^sub>2 = pi' \<bullet> pi \<bullet> p\<^sub>2' \<and> |
33189 | 722 |
t = pi' \<bullet> pi \<bullet> u \<and> |
53015
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
45129
diff
changeset
|
723 |
set pi' \<subseteq> (supp p\<^sub>2 \<union> supp (pi \<bullet> p\<^sub>2')) \<times> (supp p\<^sub>2 \<union> supp (pi \<bullet> p\<^sub>2'))" |
33189 | 724 |
by (rule PTuple') |
725 |
then obtain pi'::"name prm" where |
|
53015
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
45129
diff
changeset
|
726 |
"p\<^sub>2 = pi' \<bullet> pi \<bullet> p\<^sub>2'" "t = pi' \<bullet> pi \<bullet> u" and |
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
45129
diff
changeset
|
727 |
pi': "set pi' \<subseteq> (supp p\<^sub>2 \<union> supp (pi \<bullet> p\<^sub>2')) \<times> |
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
45129
diff
changeset
|
728 |
(supp p\<^sub>2 \<union> supp (pi \<bullet> p\<^sub>2'))" by auto |
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
45129
diff
changeset
|
729 |
from PTuple PTuple' have "pi \<bullet> distinct (pat_vars \<langle>\<langle>p\<^sub>1', p\<^sub>2'\<rangle>\<rangle>)" by simp |
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
45129
diff
changeset
|
730 |
then have "distinct (pat_vars \<langle>\<langle>pi \<bullet> p\<^sub>1', pi \<bullet> p\<^sub>2'\<rangle>\<rangle>)" by (simp only: eqvts) |
63167 | 731 |
with \<open>p\<^sub>1 = pi \<bullet> p\<^sub>1'\<close> PTuple' |
53015
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
45129
diff
changeset
|
732 |
have fresh: "(supp p\<^sub>2 \<union> supp (pi \<bullet> p\<^sub>2') :: name set) \<sharp>* p\<^sub>1" |
33189 | 733 |
by (auto simp add: set_pat_vars_supp fresh_star_def fresh_def eqvts) |
63167 | 734 |
from \<open>p\<^sub>1 = pi \<bullet> p\<^sub>1'\<close> have "pi' \<bullet> (p\<^sub>1 = pi \<bullet> p\<^sub>1')" by (rule perm_boolI) |
33189 | 735 |
with pt_freshs_freshs [OF pt_name_inst at_name_inst pi' fresh fresh] |
53015
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
45129
diff
changeset
|
736 |
have "p\<^sub>1 = pi' \<bullet> pi \<bullet> p\<^sub>1'" by (simp add: eqvts) |
63167 | 737 |
with \<open>p\<^sub>2 = pi' \<bullet> pi \<bullet> p\<^sub>2'\<close> have "\<langle>\<langle>p\<^sub>1, p\<^sub>2\<rangle>\<rangle> = (pi' @ pi) \<bullet> \<langle>\<langle>p\<^sub>1', p\<^sub>2'\<rangle>\<rangle>" |
33189 | 738 |
by (simp add: pt_name2) |
739 |
moreover |
|
53015
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
45129
diff
changeset
|
740 |
have "((supp p\<^sub>2 \<union> (pi \<bullet> supp p\<^sub>2')) \<times> (supp p\<^sub>2 \<union> (pi \<bullet> supp p\<^sub>2'))::(name \<times> name) set) \<subseteq> |
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
45129
diff
changeset
|
741 |
(supp p\<^sub>2 \<union> (supp p\<^sub>1 \<union> supp p\<^sub>1' \<union> supp p\<^sub>2')) \<times> (supp p\<^sub>2 \<union> (supp p\<^sub>1 \<union> supp p\<^sub>1' \<union> supp p\<^sub>2'))" |
33189 | 742 |
by (rule subset_refl Sigma_mono Un_mono perm_cases [OF pi])+ |
743 |
with pi' have "set pi' \<subseteq> \<dots>" by (simp add: supp_eqvt [symmetric]) |
|
53015
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
45129
diff
changeset
|
744 |
with pi have "set (pi' @ pi) \<subseteq> (supp \<langle>\<langle>p\<^sub>1, p\<^sub>2\<rangle>\<rangle> \<union> supp \<langle>\<langle>p\<^sub>1', p\<^sub>2'\<rangle>\<rangle>) \<times> |
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
45129
diff
changeset
|
745 |
(supp \<langle>\<langle>p\<^sub>1, p\<^sub>2\<rangle>\<rangle> \<union> supp \<langle>\<langle>p\<^sub>1', p\<^sub>2'\<rangle>\<rangle>)" |
33189 | 746 |
by (simp add: Sigma_Un_distrib1 Sigma_Un_distrib2 Un_ac) blast |
63167 | 747 |
moreover note \<open>t = pi' \<bullet> pi \<bullet> u\<close> |
53015
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
45129
diff
changeset
|
748 |
ultimately have "\<langle>\<langle>p\<^sub>1, p\<^sub>2\<rangle>\<rangle> = (pi' @ pi) \<bullet> q \<and> t = (pi' @ pi) \<bullet> u \<and> |
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
45129
diff
changeset
|
749 |
set (pi' @ pi) \<subseteq> (supp \<langle>\<langle>p\<^sub>1, p\<^sub>2\<rangle>\<rangle> \<union> supp q) \<times> |
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
45129
diff
changeset
|
750 |
(supp \<langle>\<langle>p\<^sub>1, p\<^sub>2\<rangle>\<rangle> \<union> supp q)" using PTuple |
33189 | 751 |
by (simp add: pt_name2) |
752 |
then show ?thesis .. |
|
753 |
qed |
|
754 |
qed |
|
755 |
||
756 |
lemma typing_case_Let: |
|
757 |
assumes ty: "\<Gamma> \<turnstile> (LET p = t IN u) : U" |
|
758 |
and fresh: "(supp p::name set) \<sharp>* \<Gamma>" |
|
759 |
and distinct: "distinct (pat_vars p)" |
|
760 |
and R: "\<And>T \<Delta>. \<Gamma> \<turnstile> t : T \<Longrightarrow> \<turnstile> p : T \<Rightarrow> \<Delta> \<Longrightarrow> \<Delta> @ \<Gamma> \<turnstile> u : U \<Longrightarrow> P" |
|
761 |
shows P using ty |
|
762 |
proof cases |
|
34990 | 763 |
case (Let p' t' T \<Delta> u') |
33189 | 764 |
then have "(supp \<Delta>::name set) \<sharp>* \<Gamma>" |
765 |
by (auto intro: valid_typing valid_app_freshs) |
|
766 |
with Let have "(supp p'::name set) \<sharp>* \<Gamma>" |
|
767 |
by (simp add: pat_var) |
|
768 |
with fresh have fresh': "(supp p \<union> supp p' :: name set) \<sharp>* \<Gamma>" |
|
769 |
by (auto simp add: fresh_star_def) |
|
770 |
from Let have "(\<lambda>[p]. Base u) = (\<lambda>[p']. Base u')" |
|
771 |
by (simp add: trm.inject) |
|
772 |
moreover from Let have "pat_type p = pat_type p'" |
|
773 |
by (simp add: trm.inject) |
|
774 |
moreover note distinct |
|
63167 | 775 |
moreover from \<open>\<Delta> @ \<Gamma> \<turnstile> u' : U\<close> have "valid (\<Delta> @ \<Gamma>)" |
33189 | 776 |
by (rule valid_typing) |
777 |
then have "valid \<Delta>" by (rule valid_appD) |
|
63167 | 778 |
with \<open>\<turnstile> p' : T \<Rightarrow> \<Delta>\<close> have "distinct (pat_vars p')" |
33189 | 779 |
by (simp add: valid_distinct pat_vars_ptyping) |
780 |
ultimately have "\<exists>pi::name prm. p = pi \<bullet> p' \<and> Base u = pi \<bullet> Base u' \<and> |
|
781 |
set pi \<subseteq> (supp p \<union> supp p') \<times> (supp p \<union> supp p')" |
|
782 |
by (rule abs_pat_alpha') |
|
783 |
then obtain pi::"name prm" where pi: "p = pi \<bullet> p'" "u = pi \<bullet> u'" |
|
784 |
and pi': "set pi \<subseteq> (supp p \<union> supp p') \<times> (supp p \<union> supp p')" |
|
785 |
by (auto simp add: btrm.inject) |
|
786 |
from Let have "\<Gamma> \<turnstile> t : T" by (simp add: trm.inject) |
|
63167 | 787 |
moreover from \<open>\<turnstile> p' : T \<Rightarrow> \<Delta>\<close> have "\<turnstile> (pi \<bullet> p') : (pi \<bullet> T) \<Rightarrow> (pi \<bullet> \<Delta>)" |
33189 | 788 |
by (simp add: ptyping.eqvt) |
789 |
with pi have "\<turnstile> p : T \<Rightarrow> (pi \<bullet> \<Delta>)" by (simp add: perm_type) |
|
790 |
moreover from Let |
|
791 |
have "(pi \<bullet> \<Delta>) @ (pi \<bullet> \<Gamma>) \<turnstile> (pi \<bullet> u') : (pi \<bullet> U)" |
|
792 |
by (simp add: append_eqvt [symmetric] typing.eqvt) |
|
793 |
with pi have "(pi \<bullet> \<Delta>) @ \<Gamma> \<turnstile> u : U" |
|
794 |
by (simp add: perm_type pt_freshs_freshs |
|
795 |
[OF pt_name_inst at_name_inst pi' fresh' fresh']) |
|
796 |
ultimately show ?thesis by (rule R) |
|
797 |
qed simp_all |
|
798 |
||
799 |
lemma preservation: |
|
800 |
assumes "t \<longmapsto> t'" and "\<Gamma> \<turnstile> t : T" |
|
801 |
shows "\<Gamma> \<turnstile> t' : T" using assms |
|
802 |
proof (nominal_induct avoiding: \<Gamma> T rule: eval.strong_induct) |
|
803 |
case (TupleL t t' u) |
|
63167 | 804 |
from \<open>\<Gamma> \<turnstile> \<langle>t, u\<rangle> : T\<close> obtain T\<^sub>1 T\<^sub>2 |
53015
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
45129
diff
changeset
|
805 |
where "T = T\<^sub>1 \<otimes> T\<^sub>2" "\<Gamma> \<turnstile> t : T\<^sub>1" "\<Gamma> \<turnstile> u : T\<^sub>2" |
33189 | 806 |
by cases (simp_all add: trm.inject) |
63167 | 807 |
from \<open>\<Gamma> \<turnstile> t : T\<^sub>1\<close> have "\<Gamma> \<turnstile> t' : T\<^sub>1" by (rule TupleL) |
808 |
then have "\<Gamma> \<turnstile> \<langle>t', u\<rangle> : T\<^sub>1 \<otimes> T\<^sub>2" using \<open>\<Gamma> \<turnstile> u : T\<^sub>2\<close> |
|
33189 | 809 |
by (rule Tuple) |
63167 | 810 |
with \<open>T = T\<^sub>1 \<otimes> T\<^sub>2\<close> show ?case by simp |
33189 | 811 |
next |
812 |
case (TupleR u u' t) |
|
63167 | 813 |
from \<open>\<Gamma> \<turnstile> \<langle>t, u\<rangle> : T\<close> obtain T\<^sub>1 T\<^sub>2 |
53015
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
45129
diff
changeset
|
814 |
where "T = T\<^sub>1 \<otimes> T\<^sub>2" "\<Gamma> \<turnstile> t : T\<^sub>1" "\<Gamma> \<turnstile> u : T\<^sub>2" |
33189 | 815 |
by cases (simp_all add: trm.inject) |
63167 | 816 |
from \<open>\<Gamma> \<turnstile> u : T\<^sub>2\<close> have "\<Gamma> \<turnstile> u' : T\<^sub>2" by (rule TupleR) |
817 |
with \<open>\<Gamma> \<turnstile> t : T\<^sub>1\<close> have "\<Gamma> \<turnstile> \<langle>t, u'\<rangle> : T\<^sub>1 \<otimes> T\<^sub>2" |
|
33189 | 818 |
by (rule Tuple) |
63167 | 819 |
with \<open>T = T\<^sub>1 \<otimes> T\<^sub>2\<close> show ?case by simp |
33189 | 820 |
next |
821 |
case (Abs t t' x S) |
|
63167 | 822 |
from \<open>\<Gamma> \<turnstile> (\<lambda>x:S. t) : T\<close> \<open>x \<sharp> \<Gamma>\<close> obtain U where |
33189 | 823 |
T: "T = S \<rightarrow> U" and U: "(x, S) # \<Gamma> \<turnstile> t : U" |
824 |
by (rule typing_case_Abs) |
|
825 |
from U have "(x, S) # \<Gamma> \<turnstile> t' : U" by (rule Abs) |
|
826 |
then have "\<Gamma> \<turnstile> (\<lambda>x:S. t') : S \<rightarrow> U" |
|
827 |
by (rule typing.Abs) |
|
828 |
with T show ?case by simp |
|
829 |
next |
|
830 |
case (Beta x u S t) |
|
63167 | 831 |
from \<open>\<Gamma> \<turnstile> (\<lambda>x:S. t) \<cdot> u : T\<close> \<open>x \<sharp> \<Gamma>\<close> |
33189 | 832 |
obtain "(x, S) # \<Gamma> \<turnstile> t : T" and "\<Gamma> \<turnstile> u : S" |
833 |
by cases (auto simp add: trm.inject ty.inject elim: typing_case_Abs) |
|
834 |
then show ?case by (rule subst_type) |
|
835 |
next |
|
836 |
case (Let p t \<theta> u) |
|
63167 | 837 |
from \<open>\<Gamma> \<turnstile> (LET p = t IN u) : T\<close> \<open>supp p \<sharp>* \<Gamma>\<close> \<open>distinct (pat_vars p)\<close> |
33189 | 838 |
obtain U \<Delta> where "\<turnstile> p : U \<Rightarrow> \<Delta>" "\<Gamma> \<turnstile> t : U" "\<Delta> @ \<Gamma> \<turnstile> u : T" |
839 |
by (rule typing_case_Let) |
|
63167 | 840 |
then show ?case using \<open>\<turnstile> p \<rhd> t \<Rightarrow> \<theta>\<close> \<open>supp p \<sharp>* t\<close> |
33189 | 841 |
by (rule match_type) |
842 |
next |
|
843 |
case (AppL t t' u) |
|
63167 | 844 |
from \<open>\<Gamma> \<turnstile> t \<cdot> u : T\<close> obtain U where |
33189 | 845 |
t: "\<Gamma> \<turnstile> t : U \<rightarrow> T" and u: "\<Gamma> \<turnstile> u : U" |
846 |
by cases (auto simp add: trm.inject) |
|
847 |
from t have "\<Gamma> \<turnstile> t' : U \<rightarrow> T" by (rule AppL) |
|
848 |
then show ?case using u by (rule typing.App) |
|
849 |
next |
|
850 |
case (AppR u u' t) |
|
63167 | 851 |
from \<open>\<Gamma> \<turnstile> t \<cdot> u : T\<close> obtain U where |
33189 | 852 |
t: "\<Gamma> \<turnstile> t : U \<rightarrow> T" and u: "\<Gamma> \<turnstile> u : U" |
853 |
by cases (auto simp add: trm.inject) |
|
854 |
from u have "\<Gamma> \<turnstile> u' : U" by (rule AppR) |
|
855 |
with t show ?case by (rule typing.App) |
|
856 |
qed |
|
857 |
||
858 |
end |