author | wenzelm |
Tue, 13 Sep 2022 09:38:02 +0200 | |
changeset 76129 | 5979f73b9db1 |
parent 71085 | 950e1cfe0fe4 |
child 76213 | e44d86131648 |
permissions | -rw-r--r-- |
13165 | 1 |
(* Title: ZF/WF.thy |
1478 | 2 |
Author: Tobias Nipkow and Lawrence C Paulson |
435 | 3 |
Copyright 1994 University of Cambridge |
0 | 4 |
|
13165 | 5 |
Derived first for transitive relations, and finally for arbitrary WF relations |
6 |
via wf_trancl and trans_trancl. |
|
7 |
||
8 |
It is difficult to derive this general case directly, using r^+ instead of |
|
9 |
r. In is_recfun, the two occurrences of the relation must have the same |
|
10 |
form. Inserting r^+ in the_recfun or wftrec yields a recursion rule with |
|
11 |
r^+ -`` {a} instead of r-``{a}. This recursion rule is stronger in |
|
12 |
principle, but harder to use, especially to prove wfrec_eclose_eq in |
|
13 |
epsilon.ML. Expanding out the definition of wftrec in wfrec would yield |
|
14 |
a mess. |
|
0 | 15 |
*) |
16 |
||
60770 | 17 |
section\<open>Well-Founded Recursion\<close> |
13356 | 18 |
|
16417 | 19 |
theory WF imports Trancl begin |
13165 | 20 |
|
24893 | 21 |
definition |
22 |
wf :: "i=>o" where |
|
13165 | 23 |
(*r is a well-founded relation*) |
46953 | 24 |
"wf(r) == \<forall>Z. Z=0 | (\<exists>x\<in>Z. \<forall>y. <y,x>:r \<longrightarrow> ~ y \<in> Z)" |
13165 | 25 |
|
24893 | 26 |
definition |
69587 | 27 |
wf_on :: "[i,i]=>o" (\<open>wf[_]'(_')\<close>) where |
13165 | 28 |
(*r is well-founded on A*) |
46820 | 29 |
"wf_on(A,r) == wf(r \<inter> A*A)" |
13165 | 30 |
|
24893 | 31 |
definition |
32 |
is_recfun :: "[i, i, [i,i]=>i, i] =>o" where |
|
46820 | 33 |
"is_recfun(r,a,H,f) == (f = (\<lambda>x\<in>r-``{a}. H(x, restrict(f, r-``{x}))))" |
13165 | 34 |
|
24893 | 35 |
definition |
36 |
the_recfun :: "[i, i, [i,i]=>i] =>i" where |
|
13165 | 37 |
"the_recfun(r,a,H) == (THE f. is_recfun(r,a,H,f))" |
38 |
||
24893 | 39 |
definition |
40 |
wftrec :: "[i, i, [i,i]=>i] =>i" where |
|
13165 | 41 |
"wftrec(r,a,H) == H(a, the_recfun(r,a,H))" |
42 |
||
24893 | 43 |
definition |
44 |
wfrec :: "[i, i, [i,i]=>i] =>i" where |
|
13165 | 45 |
(*public version. Does not require r to be transitive*) |
46 |
"wfrec(r,a,H) == wftrec(r^+, a, %x f. H(x, restrict(f,r-``{x})))" |
|
47 |
||
24893 | 48 |
definition |
69587 | 49 |
wfrec_on :: "[i, i, i, [i,i]=>i] =>i" (\<open>wfrec[_]'(_,_,_')\<close>) where |
46820 | 50 |
"wfrec[A](r,a,H) == wfrec(r \<inter> A*A, a, H)" |
13165 | 51 |
|
52 |
||
60770 | 53 |
subsection\<open>Well-Founded Relations\<close> |
13165 | 54 |
|
69593 | 55 |
subsubsection\<open>Equivalences between \<^term>\<open>wf\<close> and \<^term>\<open>wf_on\<close>\<close> |
13165 | 56 |
|
57 |
lemma wf_imp_wf_on: "wf(r) ==> wf[A](r)" |
|
46820 | 58 |
by (unfold wf_def wf_on_def, force) |
13165 | 59 |
|
46993 | 60 |
lemma wf_on_imp_wf: "[|wf[A](r); r \<subseteq> A*A|] ==> wf(r)" |
13248 | 61 |
by (simp add: wf_on_def subset_Int_iff) |
62 |
||
13165 | 63 |
lemma wf_on_field_imp_wf: "wf[field(r)](r) ==> wf(r)" |
64 |
by (unfold wf_def wf_on_def, fast) |
|
65 |
||
46821
ff6b0c1087f2
Using mathematical notation for <-> and cardinal arithmetic
paulson
parents:
46820
diff
changeset
|
66 |
lemma wf_iff_wf_on_field: "wf(r) \<longleftrightarrow> wf[field(r)](r)" |
13165 | 67 |
by (blast intro: wf_imp_wf_on wf_on_field_imp_wf) |
68 |
||
69 |
lemma wf_on_subset_A: "[| wf[A](r); B<=A |] ==> wf[B](r)" |
|
70 |
by (unfold wf_on_def wf_def, fast) |
|
71 |
||
72 |
lemma wf_on_subset_r: "[| wf[A](r); s<=r |] ==> wf[A](s)" |
|
73 |
by (unfold wf_on_def wf_def, fast) |
|
74 |
||
13217 | 75 |
lemma wf_subset: "[|wf(s); r<=s|] ==> wf(r)" |
76 |
by (simp add: wf_def, fast) |
|
77 |
||
69593 | 78 |
subsubsection\<open>Introduction Rules for \<^term>\<open>wf_on\<close>\<close> |
13165 | 79 |
|
69593 | 80 |
text\<open>If every non-empty subset of \<^term>\<open>A\<close> has an \<^term>\<open>r\<close>-minimal element |
81 |
then we have \<^term>\<open>wf[A](r)\<close>.\<close> |
|
13165 | 82 |
lemma wf_onI: |
46953 | 83 |
assumes prem: "!!Z u. [| Z<=A; u \<in> Z; \<forall>x\<in>Z. \<exists>y\<in>Z. <y,x>:r |] ==> False" |
13165 | 84 |
shows "wf[A](r)" |
85 |
apply (unfold wf_on_def wf_def) |
|
86 |
apply (rule equals0I [THEN disjCI, THEN allI]) |
|
13784 | 87 |
apply (rule_tac Z = Z in prem, blast+) |
13165 | 88 |
done |
89 |
||
69593 | 90 |
text\<open>If \<^term>\<open>r\<close> allows well-founded induction over \<^term>\<open>A\<close> |
91 |
then we have \<^term>\<open>wf[A](r)\<close>. Premise is equivalent to |
|
92 |
\<^prop>\<open>!!B. \<forall>x\<in>A. (\<forall>y. <y,x>: r \<longrightarrow> y \<in> B) \<longrightarrow> x \<in> B ==> A<=B\<close>\<close> |
|
13165 | 93 |
lemma wf_onI2: |
46953 | 94 |
assumes prem: "!!y B. [| \<forall>x\<in>A. (\<forall>y\<in>A. <y,x>:r \<longrightarrow> y \<in> B) \<longrightarrow> x \<in> B; y \<in> A |] |
95 |
==> y \<in> B" |
|
13165 | 96 |
shows "wf[A](r)" |
97 |
apply (rule wf_onI) |
|
98 |
apply (rule_tac c=u in prem [THEN DiffE]) |
|
46820 | 99 |
prefer 3 apply blast |
13165 | 100 |
apply fast+ |
101 |
done |
|
102 |
||
103 |
||
60770 | 104 |
subsubsection\<open>Well-founded Induction\<close> |
13165 | 105 |
|
69593 | 106 |
text\<open>Consider the least \<^term>\<open>z\<close> in \<^term>\<open>domain(r)\<close> such that |
107 |
\<^term>\<open>P(z)\<close> does not hold...\<close> |
|
46993 | 108 |
lemma wf_induct_raw: |
13165 | 109 |
"[| wf(r); |
46820 | 110 |
!!x.[| \<forall>y. <y,x>: r \<longrightarrow> P(y) |] ==> P(x) |] |
13634 | 111 |
==> P(a)" |
46820 | 112 |
apply (unfold wf_def) |
113 |
apply (erule_tac x = "{z \<in> domain(r). ~ P(z)}" in allE) |
|
114 |
apply blast |
|
13165 | 115 |
done |
435 | 116 |
|
46993 | 117 |
lemmas wf_induct = wf_induct_raw [rule_format, consumes 1, case_names step, induct set: wf] |
13203
fac77a839aa2
Tidying up. Mainly moving proofs from Main.thy to other (Isar) theory files.
paulson
parents:
13175
diff
changeset
|
118 |
|
61798 | 119 |
text\<open>The form of this rule is designed to match \<open>wfI\<close>\<close> |
13165 | 120 |
lemma wf_induct2: |
46953 | 121 |
"[| wf(r); a \<in> A; field(r)<=A; |
122 |
!!x.[| x \<in> A; \<forall>y. <y,x>: r \<longrightarrow> P(y) |] ==> P(x) |] |
|
13165 | 123 |
==> P(a)" |
46953 | 124 |
apply (erule_tac P="a \<in> A" in rev_mp) |
46820 | 125 |
apply (erule_tac a=a in wf_induct, blast) |
13165 | 126 |
done |
127 |
||
46820 | 128 |
lemma field_Int_square: "field(r \<inter> A*A) \<subseteq> A" |
13165 | 129 |
by blast |
130 |
||
46993 | 131 |
lemma wf_on_induct_raw [consumes 2, induct set: wf_on]: |
46953 | 132 |
"[| wf[A](r); a \<in> A; |
133 |
!!x.[| x \<in> A; \<forall>y\<in>A. <y,x>: r \<longrightarrow> P(y) |] ==> P(x) |
|
13165 | 134 |
|] ==> P(a)" |
46820 | 135 |
apply (unfold wf_on_def) |
13165 | 136 |
apply (erule wf_induct2, assumption) |
137 |
apply (rule field_Int_square, blast) |
|
138 |
done |
|
139 |
||
71085
950e1cfe0fe4
tuned proofs -- more stable proof terms without [rule_format];
wenzelm
parents:
69593
diff
changeset
|
140 |
lemma wf_on_induct [consumes 2, case_names step, induct set: wf_on]: |
950e1cfe0fe4
tuned proofs -- more stable proof terms without [rule_format];
wenzelm
parents:
69593
diff
changeset
|
141 |
"wf[A](r) \<Longrightarrow> a \<in> A \<Longrightarrow> (\<And>x. x \<in> A \<Longrightarrow> (\<And>y. y \<in> A \<Longrightarrow> \<langle>y, x\<rangle> \<in> r \<Longrightarrow> P(y)) \<Longrightarrow> P(x)) \<Longrightarrow> P(a)" |
950e1cfe0fe4
tuned proofs -- more stable proof terms without [rule_format];
wenzelm
parents:
69593
diff
changeset
|
142 |
using wf_on_induct_raw [of A r a P] by simp |
13203
fac77a839aa2
Tidying up. Mainly moving proofs from Main.thy to other (Isar) theory files.
paulson
parents:
13175
diff
changeset
|
143 |
|
69593 | 144 |
text\<open>If \<^term>\<open>r\<close> allows well-founded induction |
145 |
then we have \<^term>\<open>wf(r)\<close>.\<close> |
|
13165 | 146 |
lemma wfI: |
147 |
"[| field(r)<=A; |
|
46953 | 148 |
!!y B. [| \<forall>x\<in>A. (\<forall>y\<in>A. <y,x>:r \<longrightarrow> y \<in> B) \<longrightarrow> x \<in> B; y \<in> A|] |
149 |
==> y \<in> B |] |
|
13165 | 150 |
==> wf(r)" |
151 |
apply (rule wf_on_subset_A [THEN wf_on_field_imp_wf]) |
|
152 |
apply (rule wf_onI2) |
|
46820 | 153 |
prefer 2 apply blast |
154 |
apply blast |
|
13165 | 155 |
done |
156 |
||
157 |
||
60770 | 158 |
subsection\<open>Basic Properties of Well-Founded Relations\<close> |
13165 | 159 |
|
46820 | 160 |
lemma wf_not_refl: "wf(r) ==> <a,a> \<notin> r" |
13165 | 161 |
by (erule_tac a=a in wf_induct, blast) |
162 |
||
46820 | 163 |
lemma wf_not_sym [rule_format]: "wf(r) ==> \<forall>x. <a,x>:r \<longrightarrow> <x,a> \<notin> r" |
13165 | 164 |
by (erule_tac a=a in wf_induct, blast) |
165 |
||
46820 | 166 |
(* @{term"[| wf(r); <a,x> \<in> r; ~P ==> <x,a> \<in> r |] ==> P"} *) |
45602 | 167 |
lemmas wf_asym = wf_not_sym [THEN swap] |
13165 | 168 |
|
46953 | 169 |
lemma wf_on_not_refl: "[| wf[A](r); a \<in> A |] ==> <a,a> \<notin> r" |
13269 | 170 |
by (erule_tac a=a in wf_on_induct, assumption, blast) |
0 | 171 |
|
71085
950e1cfe0fe4
tuned proofs -- more stable proof terms without [rule_format];
wenzelm
parents:
69593
diff
changeset
|
172 |
lemma wf_on_not_sym: |
950e1cfe0fe4
tuned proofs -- more stable proof terms without [rule_format];
wenzelm
parents:
69593
diff
changeset
|
173 |
"[| wf[A](r); a \<in> A |] ==> (\<And>b. b\<in>A \<Longrightarrow> <a,b>:r \<Longrightarrow> <b,a>\<notin>r)" |
950e1cfe0fe4
tuned proofs -- more stable proof terms without [rule_format];
wenzelm
parents:
69593
diff
changeset
|
174 |
apply (atomize (full), intro impI) |
13269 | 175 |
apply (erule_tac a=a in wf_on_induct, assumption, blast) |
13165 | 176 |
done |
177 |
||
178 |
lemma wf_on_asym: |
|
46820 | 179 |
"[| wf[A](r); ~Z ==> <a,b> \<in> r; |
180 |
<b,a> \<notin> r ==> Z; ~Z ==> a \<in> A; ~Z ==> b \<in> A |] ==> Z" |
|
181 |
by (blast dest: wf_on_not_sym) |
|
13165 | 182 |
|
183 |
||
184 |
(*Needed to prove well_ordI. Could also reason that wf[A](r) means |
|
46820 | 185 |
wf(r \<inter> A*A); thus wf( (r \<inter> A*A)^+ ) and use wf_not_refl *) |
13165 | 186 |
lemma wf_on_chain3: |
46953 | 187 |
"[| wf[A](r); <a,b>:r; <b,c>:r; <c,a>:r; a \<in> A; b \<in> A; c \<in> A |] ==> P" |
46820 | 188 |
apply (subgoal_tac "\<forall>y\<in>A. \<forall>z\<in>A. <a,y>:r \<longrightarrow> <y,z>:r \<longrightarrow> <z,a>:r \<longrightarrow> P", |
189 |
blast) |
|
13269 | 190 |
apply (erule_tac a=a in wf_on_induct, assumption, blast) |
13165 | 191 |
done |
192 |
||
193 |
||
194 |
||
60770 | 195 |
text\<open>transitive closure of a WF relation is WF provided |
69593 | 196 |
\<^term>\<open>A\<close> is downward closed\<close> |
13165 | 197 |
lemma wf_on_trancl: |
46820 | 198 |
"[| wf[A](r); r-``A \<subseteq> A |] ==> wf[A](r^+)" |
13165 | 199 |
apply (rule wf_onI2) |
200 |
apply (frule bspec [THEN mp], assumption+) |
|
13784 | 201 |
apply (erule_tac a = y in wf_on_induct, assumption) |
46820 | 202 |
apply (blast elim: tranclE, blast) |
13165 | 203 |
done |
204 |
||
205 |
lemma wf_trancl: "wf(r) ==> wf(r^+)" |
|
206 |
apply (simp add: wf_iff_wf_on_field) |
|
46820 | 207 |
apply (rule wf_on_subset_A) |
13165 | 208 |
apply (erule wf_on_trancl) |
46820 | 209 |
apply blast |
13165 | 210 |
apply (rule trancl_type [THEN field_rel_subset]) |
211 |
done |
|
212 |
||
213 |
||
69593 | 214 |
text\<open>\<^term>\<open>r-``{a}\<close> is the set of everything under \<^term>\<open>a\<close> in \<^term>\<open>r\<close>\<close> |
13165 | 215 |
|
45602 | 216 |
lemmas underI = vimage_singleton_iff [THEN iffD2] |
217 |
lemmas underD = vimage_singleton_iff [THEN iffD1] |
|
13165 | 218 |
|
13634 | 219 |
|
69593 | 220 |
subsection\<open>The Predicate \<^term>\<open>is_recfun\<close>\<close> |
0 | 221 |
|
46953 | 222 |
lemma is_recfun_type: "is_recfun(r,a,H,f) ==> f \<in> r-``{a} -> range(f)" |
13165 | 223 |
apply (unfold is_recfun_def) |
224 |
apply (erule ssubst) |
|
225 |
apply (rule lamI [THEN rangeI, THEN lam_type], assumption) |
|
226 |
done |
|
227 |
||
13269 | 228 |
lemmas is_recfun_imp_function = is_recfun_type [THEN fun_is_function] |
229 |
||
13165 | 230 |
lemma apply_recfun: |
231 |
"[| is_recfun(r,a,H,f); <x,a>:r |] ==> f`x = H(x, restrict(f,r-``{x}))" |
|
46820 | 232 |
apply (unfold is_recfun_def) |
60770 | 233 |
txt\<open>replace f only on the left-hand side\<close> |
59788 | 234 |
apply (erule_tac P = "%x. t(x) = u" for t u in ssubst) |
46820 | 235 |
apply (simp add: underI) |
13165 | 236 |
done |
237 |
||
238 |
lemma is_recfun_equal [rule_format]: |
|
239 |
"[| wf(r); trans(r); is_recfun(r,a,H,f); is_recfun(r,b,H,g) |] |
|
46820 | 240 |
==> <x,a>:r \<longrightarrow> <x,b>:r \<longrightarrow> f`x=g`x" |
13784 | 241 |
apply (frule_tac f = f in is_recfun_type) |
242 |
apply (frule_tac f = g in is_recfun_type) |
|
13165 | 243 |
apply (simp add: is_recfun_def) |
244 |
apply (erule_tac a=x in wf_induct) |
|
245 |
apply (intro impI) |
|
246 |
apply (elim ssubst) |
|
247 |
apply (simp (no_asm_simp) add: vimage_singleton_iff restrict_def) |
|
59788 | 248 |
apply (rule_tac t = "%z. H (x, z)" for x in subst_context) |
46821
ff6b0c1087f2
Using mathematical notation for <-> and cardinal arithmetic
paulson
parents:
46820
diff
changeset
|
249 |
apply (subgoal_tac "\<forall>y\<in>r-``{x}. \<forall>z. <y,z>:f \<longleftrightarrow> <y,z>:g") |
13165 | 250 |
apply (blast dest: transD) |
251 |
apply (simp add: apply_iff) |
|
252 |
apply (blast dest: transD intro: sym) |
|
253 |
done |
|
254 |
||
255 |
lemma is_recfun_cut: |
|
256 |
"[| wf(r); trans(r); |
|
257 |
is_recfun(r,a,H,f); is_recfun(r,b,H,g); <b,a>:r |] |
|
258 |
==> restrict(f, r-``{b}) = g" |
|
13784 | 259 |
apply (frule_tac f = f in is_recfun_type) |
13165 | 260 |
apply (rule fun_extension) |
261 |
apply (blast dest: transD intro: restrict_type2) |
|
262 |
apply (erule is_recfun_type, simp) |
|
263 |
apply (blast dest: transD intro: is_recfun_equal) |
|
264 |
done |
|
265 |
||
60770 | 266 |
subsection\<open>Recursion: Main Existence Lemma\<close> |
435 | 267 |
|
13165 | 268 |
lemma is_recfun_functional: |
269 |
"[| wf(r); trans(r); is_recfun(r,a,H,f); is_recfun(r,a,H,g) |] ==> f=g" |
|
270 |
by (blast intro: fun_extension is_recfun_type is_recfun_equal) |
|
271 |
||
13248 | 272 |
lemma the_recfun_eq: |
273 |
"[| is_recfun(r,a,H,f); wf(r); trans(r) |] ==> the_recfun(r,a,H) = f" |
|
274 |
apply (unfold the_recfun_def) |
|
275 |
apply (blast intro: is_recfun_functional) |
|
276 |
done |
|
277 |
||
13165 | 278 |
(*If some f satisfies is_recfun(r,a,H,-) then so does the_recfun(r,a,H) *) |
279 |
lemma is_the_recfun: |
|
280 |
"[| is_recfun(r,a,H,f); wf(r); trans(r) |] |
|
281 |
==> is_recfun(r, a, H, the_recfun(r,a,H))" |
|
13248 | 282 |
by (simp add: the_recfun_eq) |
13165 | 283 |
|
284 |
lemma unfold_the_recfun: |
|
285 |
"[| wf(r); trans(r) |] ==> is_recfun(r, a, H, the_recfun(r,a,H))" |
|
286 |
apply (rule_tac a=a in wf_induct, assumption) |
|
46820 | 287 |
apply (rename_tac a1) |
288 |
apply (rule_tac f = "\<lambda>y\<in>r-``{a1}. wftrec (r,y,H)" in is_the_recfun) |
|
13165 | 289 |
apply typecheck |
290 |
apply (unfold is_recfun_def wftrec_def) |
|
67443
3abf6a722518
standardized towards new-style formal comments: isabelle update_comments;
wenzelm
parents:
61798
diff
changeset
|
291 |
\<comment> \<open>Applying the substitution: must keep the quantified assumption!\<close> |
46820 | 292 |
apply (rule lam_cong [OF refl]) |
293 |
apply (drule underD) |
|
13165 | 294 |
apply (fold is_recfun_def) |
59788 | 295 |
apply (rule_tac t = "%z. H(x, z)" for x in subst_context) |
13165 | 296 |
apply (rule fun_extension) |
297 |
apply (blast intro: is_recfun_type) |
|
298 |
apply (rule lam_type [THEN restrict_type2]) |
|
299 |
apply blast |
|
300 |
apply (blast dest: transD) |
|
46993 | 301 |
apply atomize |
13165 | 302 |
apply (frule spec [THEN mp], assumption) |
46820 | 303 |
apply (subgoal_tac "<xa,a1> \<in> r") |
13784 | 304 |
apply (drule_tac x1 = xa in spec [THEN mp], assumption) |
46820 | 305 |
apply (simp add: vimage_singleton_iff |
13165 | 306 |
apply_recfun is_recfun_cut) |
307 |
apply (blast dest: transD) |
|
308 |
done |
|
309 |
||
310 |
||
69593 | 311 |
subsection\<open>Unfolding \<^term>\<open>wftrec(r,a,H)\<close>\<close> |
13165 | 312 |
|
313 |
lemma the_recfun_cut: |
|
314 |
"[| wf(r); trans(r); <b,a>:r |] |
|
315 |
==> restrict(the_recfun(r,a,H), r-``{b}) = the_recfun(r,b,H)" |
|
13269 | 316 |
by (blast intro: is_recfun_cut unfold_the_recfun) |
0 | 317 |
|
13165 | 318 |
(*NOT SUITABLE FOR REWRITING: it is recursive!*) |
319 |
lemma wftrec: |
|
320 |
"[| wf(r); trans(r) |] ==> |
|
46820 | 321 |
wftrec(r,a,H) = H(a, \<lambda>x\<in>r-``{a}. wftrec(r,x,H))" |
13165 | 322 |
apply (unfold wftrec_def) |
323 |
apply (subst unfold_the_recfun [unfolded is_recfun_def]) |
|
324 |
apply (simp_all add: vimage_singleton_iff [THEN iff_sym] the_recfun_cut) |
|
325 |
done |
|
326 |
||
13634 | 327 |
|
69593 | 328 |
subsubsection\<open>Removal of the Premise \<^term>\<open>trans(r)\<close>\<close> |
13165 | 329 |
|
330 |
(*NOT SUITABLE FOR REWRITING: it is recursive!*) |
|
331 |
lemma wfrec: |
|
46820 | 332 |
"wf(r) ==> wfrec(r,a,H) = H(a, \<lambda>x\<in>r-``{a}. wfrec(r,x,H))" |
333 |
apply (unfold wfrec_def) |
|
13165 | 334 |
apply (erule wf_trancl [THEN wftrec, THEN ssubst]) |
335 |
apply (rule trans_trancl) |
|
336 |
apply (rule vimage_pair_mono [THEN restrict_lam_eq, THEN subst_context]) |
|
337 |
apply (erule r_into_trancl) |
|
338 |
apply (rule subset_refl) |
|
339 |
done |
|
0 | 340 |
|
13165 | 341 |
(*This form avoids giant explosions in proofs. NOTE USE OF == *) |
342 |
lemma def_wfrec: |
|
343 |
"[| !!x. h(x)==wfrec(r,x,H); wf(r) |] ==> |
|
46820 | 344 |
h(a) = H(a, \<lambda>x\<in>r-``{a}. h(x))" |
13165 | 345 |
apply simp |
46820 | 346 |
apply (elim wfrec) |
13165 | 347 |
done |
348 |
||
349 |
lemma wfrec_type: |
|
46953 | 350 |
"[| wf(r); a \<in> A; field(r)<=A; |
351 |
!!x u. [| x \<in> A; u \<in> Pi(r-``{x}, B) |] ==> H(x,u) \<in> B(x) |
|
46820 | 352 |
|] ==> wfrec(r,a,H) \<in> B(a)" |
13784 | 353 |
apply (rule_tac a = a in wf_induct2, assumption+) |
13165 | 354 |
apply (subst wfrec, assumption) |
46820 | 355 |
apply (simp add: lam_type underD) |
13165 | 356 |
done |
357 |
||
358 |
||
359 |
lemma wfrec_on: |
|
46953 | 360 |
"[| wf[A](r); a \<in> A |] ==> |
46820 | 361 |
wfrec[A](r,a,H) = H(a, \<lambda>x\<in>(r-``{a}) \<inter> A. wfrec[A](r,x,H))" |
13165 | 362 |
apply (unfold wf_on_def wfrec_on_def) |
363 |
apply (erule wfrec [THEN trans]) |
|
364 |
apply (simp add: vimage_Int_square cons_subset_iff) |
|
365 |
done |
|
0 | 366 |
|
60770 | 367 |
text\<open>Minimal-element characterization of well-foundedness\<close> |
13165 | 368 |
lemma wf_eq_minimal: |
46953 | 369 |
"wf(r) \<longleftrightarrow> (\<forall>Q x. x \<in> Q \<longrightarrow> (\<exists>z\<in>Q. \<forall>y. <y,z>:r \<longrightarrow> y\<notin>Q))" |
13634 | 370 |
by (unfold wf_def, blast) |
371 |
||
0 | 372 |
end |