author | wenzelm |
Sat, 23 May 2015 17:19:37 +0200 | |
changeset 60299 | 5ae2a2e74c93 |
parent 58889 | 5b7a9633cfa8 |
child 61986 | 2461779da2b8 |
permissions | -rw-r--r-- |
39157
b98909faaea8
more explicit HOL-Proofs sessions, including former ex/Hilbert_Classical.thy which works in parallel mode without the antiquotation option "margin" (which is still critical);
wenzelm
parents:
39126
diff
changeset
|
1 |
(* Title: HOL/Proofs/Lambda/Lambda.thy |
1120 | 2 |
Author: Tobias Nipkow |
3 |
Copyright 1995 TU Muenchen |
|
4 |
*) |
|
5 |
||
58889 | 6 |
section {* Basic definitions of Lambda-calculus *} |
9811
39ffdb8cab03
HOL/Lambda: converted into new-style theory and document;
wenzelm
parents:
6453
diff
changeset
|
7 |
|
58372
bfd497f2f4c2
moved 'old_datatype' out of 'Main' (but put it in 'HOL-Proofs' because of the inductive realizer)
blanchet
parents:
58310
diff
changeset
|
8 |
theory Lambda |
58382 | 9 |
imports Main |
58372
bfd497f2f4c2
moved 'old_datatype' out of 'Main' (but put it in 'HOL-Proofs' because of the inductive realizer)
blanchet
parents:
58310
diff
changeset
|
10 |
begin |
9811
39ffdb8cab03
HOL/Lambda: converted into new-style theory and document;
wenzelm
parents:
6453
diff
changeset
|
11 |
|
46512
4f9f61f9b535
simplified configuration options for syntax ambiguity;
wenzelm
parents:
46506
diff
changeset
|
12 |
declare [[syntax_ambiguity_warning = false]] |
39126
ee117c5b3b75
configuration options Syntax.ambiguity_enabled (inverse of former Syntax.ambiguity_is_error), Syntax.ambiguity_level (with Isar attribute "syntax_ambiguity_level"), Syntax.ambiguity_limit;
wenzelm
parents:
36862
diff
changeset
|
13 |
|
1120 | 14 |
|
9811
39ffdb8cab03
HOL/Lambda: converted into new-style theory and document;
wenzelm
parents:
6453
diff
changeset
|
15 |
subsection {* Lambda-terms in de Bruijn notation and substitution *} |
39ffdb8cab03
HOL/Lambda: converted into new-style theory and document;
wenzelm
parents:
6453
diff
changeset
|
16 |
|
58310 | 17 |
datatype dB = |
9811
39ffdb8cab03
HOL/Lambda: converted into new-style theory and document;
wenzelm
parents:
6453
diff
changeset
|
18 |
Var nat |
12011 | 19 |
| App dB dB (infixl "\<degree>" 200) |
9811
39ffdb8cab03
HOL/Lambda: converted into new-style theory and document;
wenzelm
parents:
6453
diff
changeset
|
20 |
| Abs dB |
1120 | 21 |
|
25974 | 22 |
primrec |
9811
39ffdb8cab03
HOL/Lambda: converted into new-style theory and document;
wenzelm
parents:
6453
diff
changeset
|
23 |
lift :: "[dB, nat] => dB" |
25974 | 24 |
where |
25 |
"lift (Var i) k = (if i < k then Var i else Var (i + 1))" |
|
26 |
| "lift (s \<degree> t) k = lift s k \<degree> lift t k" |
|
27 |
| "lift (Abs s) k = Abs (lift s (k + 1))" |
|
1153 | 28 |
|
5184 | 29 |
primrec |
25974 | 30 |
subst :: "[dB, dB, nat] => dB" ("_[_'/_]" [300, 0, 0] 300) |
31 |
where (* FIXME base names *) |
|
32 |
subst_Var: "(Var i)[s/k] = |
|
33 |
(if k < i then Var (i - 1) else if i = k then s else Var i)" |
|
34 |
| subst_App: "(t \<degree> u)[s/k] = t[s/k] \<degree> u[s/k]" |
|
35 |
| subst_Abs: "(Abs t)[s/k] = Abs (t[lift s 0 / k+1])" |
|
9811
39ffdb8cab03
HOL/Lambda: converted into new-style theory and document;
wenzelm
parents:
6453
diff
changeset
|
36 |
|
39ffdb8cab03
HOL/Lambda: converted into new-style theory and document;
wenzelm
parents:
6453
diff
changeset
|
37 |
declare subst_Var [simp del] |
39ffdb8cab03
HOL/Lambda: converted into new-style theory and document;
wenzelm
parents:
6453
diff
changeset
|
38 |
|
39ffdb8cab03
HOL/Lambda: converted into new-style theory and document;
wenzelm
parents:
6453
diff
changeset
|
39 |
text {* Optimized versions of @{term subst} and @{term lift}. *} |
39ffdb8cab03
HOL/Lambda: converted into new-style theory and document;
wenzelm
parents:
6453
diff
changeset
|
40 |
|
25974 | 41 |
primrec |
9811
39ffdb8cab03
HOL/Lambda: converted into new-style theory and document;
wenzelm
parents:
6453
diff
changeset
|
42 |
liftn :: "[nat, dB, nat] => dB" |
25974 | 43 |
where |
44 |
"liftn n (Var i) k = (if i < k then Var i else Var (i + n))" |
|
45 |
| "liftn n (s \<degree> t) k = liftn n s k \<degree> liftn n t k" |
|
46 |
| "liftn n (Abs s) k = Abs (liftn n s (k + 1))" |
|
9811
39ffdb8cab03
HOL/Lambda: converted into new-style theory and document;
wenzelm
parents:
6453
diff
changeset
|
47 |
|
39ffdb8cab03
HOL/Lambda: converted into new-style theory and document;
wenzelm
parents:
6453
diff
changeset
|
48 |
primrec |
25974 | 49 |
substn :: "[dB, dB, nat] => dB" |
50 |
where |
|
51 |
"substn (Var i) s k = |
|
52 |
(if k < i then Var (i - 1) else if i = k then liftn k s 0 else Var i)" |
|
53 |
| "substn (t \<degree> u) s k = substn t s k \<degree> substn u s k" |
|
54 |
| "substn (Abs t) s k = Abs (substn t s (k + 1))" |
|
1120 | 55 |
|
9811
39ffdb8cab03
HOL/Lambda: converted into new-style theory and document;
wenzelm
parents:
6453
diff
changeset
|
56 |
|
39ffdb8cab03
HOL/Lambda: converted into new-style theory and document;
wenzelm
parents:
6453
diff
changeset
|
57 |
subsection {* Beta-reduction *} |
1153 | 58 |
|
23750 | 59 |
inductive beta :: "[dB, dB] => bool" (infixl "\<rightarrow>\<^sub>\<beta>" 50) |
22271 | 60 |
where |
61 |
beta [simp, intro!]: "Abs s \<degree> t \<rightarrow>\<^sub>\<beta> s[t/0]" |
|
62 |
| appL [simp, intro!]: "s \<rightarrow>\<^sub>\<beta> t ==> s \<degree> u \<rightarrow>\<^sub>\<beta> t \<degree> u" |
|
63 |
| appR [simp, intro!]: "s \<rightarrow>\<^sub>\<beta> t ==> u \<degree> s \<rightarrow>\<^sub>\<beta> u \<degree> t" |
|
64 |
| abs [simp, intro!]: "s \<rightarrow>\<^sub>\<beta> t ==> Abs s \<rightarrow>\<^sub>\<beta> Abs t" |
|
21404
eb85850d3eb7
more robust syntax for definition/abbreviation/notation;
wenzelm
parents:
21210
diff
changeset
|
65 |
|
eb85850d3eb7
more robust syntax for definition/abbreviation/notation;
wenzelm
parents:
21210
diff
changeset
|
66 |
abbreviation |
eb85850d3eb7
more robust syntax for definition/abbreviation/notation;
wenzelm
parents:
21210
diff
changeset
|
67 |
beta_reds :: "[dB, dB] => bool" (infixl "->>" 50) where |
22271 | 68 |
"s ->> t == beta^** s t" |
19086 | 69 |
|
21210 | 70 |
notation (latex) |
19656
09be06943252
tuned concrete syntax -- abbreviation/const_syntax;
wenzelm
parents:
19380
diff
changeset
|
71 |
beta_reds (infixl "\<rightarrow>\<^sub>\<beta>\<^sup>*" 50) |
1120 | 72 |
|
23750 | 73 |
inductive_cases beta_cases [elim!]: |
14065 | 74 |
"Var i \<rightarrow>\<^sub>\<beta> t" |
75 |
"Abs r \<rightarrow>\<^sub>\<beta> s" |
|
76 |
"s \<degree> t \<rightarrow>\<^sub>\<beta> u" |
|
9811
39ffdb8cab03
HOL/Lambda: converted into new-style theory and document;
wenzelm
parents:
6453
diff
changeset
|
77 |
|
39ffdb8cab03
HOL/Lambda: converted into new-style theory and document;
wenzelm
parents:
6453
diff
changeset
|
78 |
declare if_not_P [simp] not_less_eq [simp] |
39ffdb8cab03
HOL/Lambda: converted into new-style theory and document;
wenzelm
parents:
6453
diff
changeset
|
79 |
-- {* don't add @{text "r_into_rtrancl[intro!]"} *} |
39ffdb8cab03
HOL/Lambda: converted into new-style theory and document;
wenzelm
parents:
6453
diff
changeset
|
80 |
|
39ffdb8cab03
HOL/Lambda: converted into new-style theory and document;
wenzelm
parents:
6453
diff
changeset
|
81 |
|
39ffdb8cab03
HOL/Lambda: converted into new-style theory and document;
wenzelm
parents:
6453
diff
changeset
|
82 |
subsection {* Congruence rules *} |
39ffdb8cab03
HOL/Lambda: converted into new-style theory and document;
wenzelm
parents:
6453
diff
changeset
|
83 |
|
39ffdb8cab03
HOL/Lambda: converted into new-style theory and document;
wenzelm
parents:
6453
diff
changeset
|
84 |
lemma rtrancl_beta_Abs [intro!]: |
14065 | 85 |
"s \<rightarrow>\<^sub>\<beta>\<^sup>* s' ==> Abs s \<rightarrow>\<^sub>\<beta>\<^sup>* Abs s'" |
23750 | 86 |
by (induct set: rtranclp) (blast intro: rtranclp.rtrancl_into_rtrancl)+ |
9811
39ffdb8cab03
HOL/Lambda: converted into new-style theory and document;
wenzelm
parents:
6453
diff
changeset
|
87 |
|
39ffdb8cab03
HOL/Lambda: converted into new-style theory and document;
wenzelm
parents:
6453
diff
changeset
|
88 |
lemma rtrancl_beta_AppL: |
14065 | 89 |
"s \<rightarrow>\<^sub>\<beta>\<^sup>* s' ==> s \<degree> t \<rightarrow>\<^sub>\<beta>\<^sup>* s' \<degree> t" |
23750 | 90 |
by (induct set: rtranclp) (blast intro: rtranclp.rtrancl_into_rtrancl)+ |
9811
39ffdb8cab03
HOL/Lambda: converted into new-style theory and document;
wenzelm
parents:
6453
diff
changeset
|
91 |
|
39ffdb8cab03
HOL/Lambda: converted into new-style theory and document;
wenzelm
parents:
6453
diff
changeset
|
92 |
lemma rtrancl_beta_AppR: |
14065 | 93 |
"t \<rightarrow>\<^sub>\<beta>\<^sup>* t' ==> s \<degree> t \<rightarrow>\<^sub>\<beta>\<^sup>* s \<degree> t'" |
23750 | 94 |
by (induct set: rtranclp) (blast intro: rtranclp.rtrancl_into_rtrancl)+ |
9811
39ffdb8cab03
HOL/Lambda: converted into new-style theory and document;
wenzelm
parents:
6453
diff
changeset
|
95 |
|
39ffdb8cab03
HOL/Lambda: converted into new-style theory and document;
wenzelm
parents:
6453
diff
changeset
|
96 |
lemma rtrancl_beta_App [intro]: |
14065 | 97 |
"[| s \<rightarrow>\<^sub>\<beta>\<^sup>* s'; t \<rightarrow>\<^sub>\<beta>\<^sup>* t' |] ==> s \<degree> t \<rightarrow>\<^sub>\<beta>\<^sup>* s' \<degree> t'" |
23750 | 98 |
by (blast intro!: rtrancl_beta_AppL rtrancl_beta_AppR intro: rtranclp_trans) |
9811
39ffdb8cab03
HOL/Lambda: converted into new-style theory and document;
wenzelm
parents:
6453
diff
changeset
|
99 |
|
39ffdb8cab03
HOL/Lambda: converted into new-style theory and document;
wenzelm
parents:
6453
diff
changeset
|
100 |
|
39ffdb8cab03
HOL/Lambda: converted into new-style theory and document;
wenzelm
parents:
6453
diff
changeset
|
101 |
subsection {* Substitution-lemmas *} |
39ffdb8cab03
HOL/Lambda: converted into new-style theory and document;
wenzelm
parents:
6453
diff
changeset
|
102 |
|
39ffdb8cab03
HOL/Lambda: converted into new-style theory and document;
wenzelm
parents:
6453
diff
changeset
|
103 |
lemma subst_eq [simp]: "(Var k)[u/k] = u" |
18241 | 104 |
by (simp add: subst_Var) |
9811
39ffdb8cab03
HOL/Lambda: converted into new-style theory and document;
wenzelm
parents:
6453
diff
changeset
|
105 |
|
39ffdb8cab03
HOL/Lambda: converted into new-style theory and document;
wenzelm
parents:
6453
diff
changeset
|
106 |
lemma subst_gt [simp]: "i < j ==> (Var j)[u/i] = Var (j - 1)" |
18241 | 107 |
by (simp add: subst_Var) |
9811
39ffdb8cab03
HOL/Lambda: converted into new-style theory and document;
wenzelm
parents:
6453
diff
changeset
|
108 |
|
39ffdb8cab03
HOL/Lambda: converted into new-style theory and document;
wenzelm
parents:
6453
diff
changeset
|
109 |
lemma subst_lt [simp]: "j < i ==> (Var j)[u/i] = Var j" |
18241 | 110 |
by (simp add: subst_Var) |
9811
39ffdb8cab03
HOL/Lambda: converted into new-style theory and document;
wenzelm
parents:
6453
diff
changeset
|
111 |
|
18241 | 112 |
lemma lift_lift: |
113 |
"i < k + 1 \<Longrightarrow> lift (lift t i) (Suc k) = lift (lift t k) i" |
|
20503 | 114 |
by (induct t arbitrary: i k) auto |
9811
39ffdb8cab03
HOL/Lambda: converted into new-style theory and document;
wenzelm
parents:
6453
diff
changeset
|
115 |
|
39ffdb8cab03
HOL/Lambda: converted into new-style theory and document;
wenzelm
parents:
6453
diff
changeset
|
116 |
lemma lift_subst [simp]: |
18241 | 117 |
"j < i + 1 \<Longrightarrow> lift (t[s/j]) i = (lift t (i + 1)) [lift s i / j]" |
20503 | 118 |
by (induct t arbitrary: i j s) |
18241 | 119 |
(simp_all add: diff_Suc subst_Var lift_lift split: nat.split) |
9811
39ffdb8cab03
HOL/Lambda: converted into new-style theory and document;
wenzelm
parents:
6453
diff
changeset
|
120 |
|
39ffdb8cab03
HOL/Lambda: converted into new-style theory and document;
wenzelm
parents:
6453
diff
changeset
|
121 |
lemma lift_subst_lt: |
18241 | 122 |
"i < j + 1 \<Longrightarrow> lift (t[s/j]) i = (lift t i) [lift s i / j + 1]" |
20503 | 123 |
by (induct t arbitrary: i j s) (simp_all add: subst_Var lift_lift) |
9811
39ffdb8cab03
HOL/Lambda: converted into new-style theory and document;
wenzelm
parents:
6453
diff
changeset
|
124 |
|
39ffdb8cab03
HOL/Lambda: converted into new-style theory and document;
wenzelm
parents:
6453
diff
changeset
|
125 |
lemma subst_lift [simp]: |
18241 | 126 |
"(lift t k)[s/k] = t" |
20503 | 127 |
by (induct t arbitrary: k s) simp_all |
9811
39ffdb8cab03
HOL/Lambda: converted into new-style theory and document;
wenzelm
parents:
6453
diff
changeset
|
128 |
|
18241 | 129 |
lemma subst_subst: |
130 |
"i < j + 1 \<Longrightarrow> t[lift v i / Suc j][u[v/j]/i] = t[u/i][v/j]" |
|
20503 | 131 |
by (induct t arbitrary: i j u v) |
18241 | 132 |
(simp_all add: diff_Suc subst_Var lift_lift [symmetric] lift_subst_lt |
9811
39ffdb8cab03
HOL/Lambda: converted into new-style theory and document;
wenzelm
parents:
6453
diff
changeset
|
133 |
split: nat.split) |
39ffdb8cab03
HOL/Lambda: converted into new-style theory and document;
wenzelm
parents:
6453
diff
changeset
|
134 |
|
39ffdb8cab03
HOL/Lambda: converted into new-style theory and document;
wenzelm
parents:
6453
diff
changeset
|
135 |
|
39ffdb8cab03
HOL/Lambda: converted into new-style theory and document;
wenzelm
parents:
6453
diff
changeset
|
136 |
subsection {* Equivalence proof for optimized substitution *} |
39ffdb8cab03
HOL/Lambda: converted into new-style theory and document;
wenzelm
parents:
6453
diff
changeset
|
137 |
|
18241 | 138 |
lemma liftn_0 [simp]: "liftn 0 t k = t" |
20503 | 139 |
by (induct t arbitrary: k) (simp_all add: subst_Var) |
9811
39ffdb8cab03
HOL/Lambda: converted into new-style theory and document;
wenzelm
parents:
6453
diff
changeset
|
140 |
|
18241 | 141 |
lemma liftn_lift [simp]: "liftn (Suc n) t k = lift (liftn n t k) k" |
20503 | 142 |
by (induct t arbitrary: k) (simp_all add: subst_Var) |
9811
39ffdb8cab03
HOL/Lambda: converted into new-style theory and document;
wenzelm
parents:
6453
diff
changeset
|
143 |
|
18241 | 144 |
lemma substn_subst_n [simp]: "substn t s n = t[liftn n s 0 / n]" |
20503 | 145 |
by (induct t arbitrary: n) (simp_all add: subst_Var) |
9811
39ffdb8cab03
HOL/Lambda: converted into new-style theory and document;
wenzelm
parents:
6453
diff
changeset
|
146 |
|
39ffdb8cab03
HOL/Lambda: converted into new-style theory and document;
wenzelm
parents:
6453
diff
changeset
|
147 |
theorem substn_subst_0: "substn t s 0 = t[s/0]" |
18241 | 148 |
by simp |
9811
39ffdb8cab03
HOL/Lambda: converted into new-style theory and document;
wenzelm
parents:
6453
diff
changeset
|
149 |
|
39ffdb8cab03
HOL/Lambda: converted into new-style theory and document;
wenzelm
parents:
6453
diff
changeset
|
150 |
|
39ffdb8cab03
HOL/Lambda: converted into new-style theory and document;
wenzelm
parents:
6453
diff
changeset
|
151 |
subsection {* Preservation theorems *} |
39ffdb8cab03
HOL/Lambda: converted into new-style theory and document;
wenzelm
parents:
6453
diff
changeset
|
152 |
|
39ffdb8cab03
HOL/Lambda: converted into new-style theory and document;
wenzelm
parents:
6453
diff
changeset
|
153 |
text {* Not used in Church-Rosser proof, but in Strong |
39ffdb8cab03
HOL/Lambda: converted into new-style theory and document;
wenzelm
parents:
6453
diff
changeset
|
154 |
Normalization. \medskip *} |
39ffdb8cab03
HOL/Lambda: converted into new-style theory and document;
wenzelm
parents:
6453
diff
changeset
|
155 |
|
13915
28ccb51bd2f3
Eliminated most occurrences of rule_format attribute.
berghofe
parents:
13187
diff
changeset
|
156 |
theorem subst_preserves_beta [simp]: |
18257 | 157 |
"r \<rightarrow>\<^sub>\<beta> s ==> r[t/i] \<rightarrow>\<^sub>\<beta> s[t/i]" |
20503 | 158 |
by (induct arbitrary: t i set: beta) (simp_all add: subst_subst [symmetric]) |
9811
39ffdb8cab03
HOL/Lambda: converted into new-style theory and document;
wenzelm
parents:
6453
diff
changeset
|
159 |
|
14065 | 160 |
theorem subst_preserves_beta': "r \<rightarrow>\<^sub>\<beta>\<^sup>* s ==> r[t/i] \<rightarrow>\<^sub>\<beta>\<^sup>* s[t/i]" |
23750 | 161 |
apply (induct set: rtranclp) |
162 |
apply (rule rtranclp.rtrancl_refl) |
|
163 |
apply (erule rtranclp.rtrancl_into_rtrancl) |
|
14065 | 164 |
apply (erule subst_preserves_beta) |
165 |
done |
|
166 |
||
13915
28ccb51bd2f3
Eliminated most occurrences of rule_format attribute.
berghofe
parents:
13187
diff
changeset
|
167 |
theorem lift_preserves_beta [simp]: |
18257 | 168 |
"r \<rightarrow>\<^sub>\<beta> s ==> lift r i \<rightarrow>\<^sub>\<beta> lift s i" |
20503 | 169 |
by (induct arbitrary: i set: beta) auto |
9811
39ffdb8cab03
HOL/Lambda: converted into new-style theory and document;
wenzelm
parents:
6453
diff
changeset
|
170 |
|
14065 | 171 |
theorem lift_preserves_beta': "r \<rightarrow>\<^sub>\<beta>\<^sup>* s ==> lift r i \<rightarrow>\<^sub>\<beta>\<^sup>* lift s i" |
23750 | 172 |
apply (induct set: rtranclp) |
173 |
apply (rule rtranclp.rtrancl_refl) |
|
174 |
apply (erule rtranclp.rtrancl_into_rtrancl) |
|
14065 | 175 |
apply (erule lift_preserves_beta) |
176 |
done |
|
177 |
||
18241 | 178 |
theorem subst_preserves_beta2 [simp]: "r \<rightarrow>\<^sub>\<beta> s ==> t[r/i] \<rightarrow>\<^sub>\<beta>\<^sup>* t[s/i]" |
20503 | 179 |
apply (induct t arbitrary: r s i) |
23750 | 180 |
apply (simp add: subst_Var r_into_rtranclp) |
9811
39ffdb8cab03
HOL/Lambda: converted into new-style theory and document;
wenzelm
parents:
6453
diff
changeset
|
181 |
apply (simp add: rtrancl_beta_App) |
39ffdb8cab03
HOL/Lambda: converted into new-style theory and document;
wenzelm
parents:
6453
diff
changeset
|
182 |
apply (simp add: rtrancl_beta_Abs) |
39ffdb8cab03
HOL/Lambda: converted into new-style theory and document;
wenzelm
parents:
6453
diff
changeset
|
183 |
done |
39ffdb8cab03
HOL/Lambda: converted into new-style theory and document;
wenzelm
parents:
6453
diff
changeset
|
184 |
|
14065 | 185 |
theorem subst_preserves_beta2': "r \<rightarrow>\<^sub>\<beta>\<^sup>* s ==> t[r/i] \<rightarrow>\<^sub>\<beta>\<^sup>* t[s/i]" |
23750 | 186 |
apply (induct set: rtranclp) |
187 |
apply (rule rtranclp.rtrancl_refl) |
|
188 |
apply (erule rtranclp_trans) |
|
14065 | 189 |
apply (erule subst_preserves_beta2) |
190 |
done |
|
191 |
||
11638 | 192 |
end |