| author | wenzelm |
| Tue, 02 Jul 2024 23:29:46 +0200 | |
| changeset 80482 | 2136ecf06a4c |
| parent 80397 | 7e0cbc6600b9 |
| child 80572 | 6ab6431864b6 |
| permissions | -rw-r--r-- |
|
32960
69916a850301
eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents:
32704
diff
changeset
|
1 |
(* Title: HOL/Wellfounded.thy |
|
69916a850301
eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents:
32704
diff
changeset
|
2 |
Author: Tobias Nipkow |
|
69916a850301
eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents:
32704
diff
changeset
|
3 |
Author: Lawrence C Paulson |
|
69916a850301
eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents:
32704
diff
changeset
|
4 |
Author: Konrad Slind |
|
69916a850301
eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents:
32704
diff
changeset
|
5 |
Author: Alexander Krauss |
| 55027 | 6 |
Author: Andrei Popescu, TU Muenchen |
|
80046
38803a6b3357
added lemma wfp_on_image and author name to theory
desharna
parents:
80019
diff
changeset
|
7 |
Author: Martin Desharnais, MPI-INF Saarbruecken |
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
8 |
*) |
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
9 |
|
| 60758 | 10 |
section \<open>Well-founded Recursion\<close> |
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
11 |
|
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
12 |
theory Wellfounded |
| 63572 | 13 |
imports Transitive_Closure |
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
14 |
begin |
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
15 |
|
| 60758 | 16 |
subsection \<open>Basic Definitions\<close> |
| 26976 | 17 |
|
|
79971
033f90dc441d
redefined wf as an abbreviation for "wf_on UNIV"
desharna
parents:
79965
diff
changeset
|
18 |
definition wf_on :: "'a set \<Rightarrow> 'a rel \<Rightarrow> bool" where |
|
033f90dc441d
redefined wf as an abbreviation for "wf_on UNIV"
desharna
parents:
79965
diff
changeset
|
19 |
"wf_on A r \<longleftrightarrow> (\<forall>P. (\<forall>x \<in> A. (\<forall>y \<in> A. (y, x) \<in> r \<longrightarrow> P y) \<longrightarrow> P x) \<longrightarrow> (\<forall>x \<in> A. P x))" |
|
79917
d0205dde00bb
added definitions wf_on and wfp_on as restricted versions of wf and wfP respectively
desharna
parents:
77172
diff
changeset
|
20 |
|
|
79971
033f90dc441d
redefined wf as an abbreviation for "wf_on UNIV"
desharna
parents:
79965
diff
changeset
|
21 |
abbreviation wf :: "('a \<times> 'a) set \<Rightarrow> bool" where
|
|
033f90dc441d
redefined wf as an abbreviation for "wf_on UNIV"
desharna
parents:
79965
diff
changeset
|
22 |
"wf \<equiv> wf_on UNIV" |
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
23 |
|
|
79917
d0205dde00bb
added definitions wf_on and wfp_on as restricted versions of wf and wfP respectively
desharna
parents:
77172
diff
changeset
|
24 |
definition wfp_on :: "'a set \<Rightarrow> ('a \<Rightarrow> 'a \<Rightarrow> bool) \<Rightarrow> bool" where
|
|
d0205dde00bb
added definitions wf_on and wfp_on as restricted versions of wf and wfP respectively
desharna
parents:
77172
diff
changeset
|
25 |
"wfp_on A R \<longleftrightarrow> (\<forall>P. (\<forall>x \<in> A. (\<forall>y \<in> A. R y x \<longrightarrow> P y) \<longrightarrow> P x) \<longrightarrow> (\<forall>x \<in> A. P x))" |
|
d0205dde00bb
added definitions wf_on and wfp_on as restricted versions of wf and wfP respectively
desharna
parents:
77172
diff
changeset
|
26 |
|
|
79965
233d70cad0cf
redefined wfP as an abbreviation for "wfp_on UNIV"
desharna
parents:
79963
diff
changeset
|
27 |
abbreviation wfP :: "('a \<Rightarrow> 'a \<Rightarrow> bool) \<Rightarrow> bool" where
|
|
233d70cad0cf
redefined wfP as an abbreviation for "wfp_on UNIV"
desharna
parents:
79963
diff
changeset
|
28 |
"wfP \<equiv> wfp_on UNIV" |
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
29 |
|
| 79924 | 30 |
alias wfp = wfP |
31 |
||
32 |
text \<open>We keep old name \<^const>\<open>wfP\<close> for backward compatibility, but offer new name \<^const>\<open>wfp\<close> to be |
|
33 |
consistent with similar predicates, e.g., \<^const>\<open>asymp\<close>, \<^const>\<open>transp\<close>, \<^const>\<open>totalp\<close>.\<close> |
|
34 |
||
|
79917
d0205dde00bb
added definitions wf_on and wfp_on as restricted versions of wf and wfP respectively
desharna
parents:
77172
diff
changeset
|
35 |
|
|
d0205dde00bb
added definitions wf_on and wfp_on as restricted versions of wf and wfP respectively
desharna
parents:
77172
diff
changeset
|
36 |
subsection \<open>Equivalence of Definitions\<close> |
|
d0205dde00bb
added definitions wf_on and wfp_on as restricted versions of wf and wfP respectively
desharna
parents:
77172
diff
changeset
|
37 |
|
|
d0205dde00bb
added definitions wf_on and wfp_on as restricted versions of wf and wfP respectively
desharna
parents:
77172
diff
changeset
|
38 |
lemma wfp_on_wf_on_eq[pred_set_conv]: "wfp_on A (\<lambda>x y. (x, y) \<in> r) \<longleftrightarrow> wf_on A r" |
|
d0205dde00bb
added definitions wf_on and wfp_on as restricted versions of wf and wfP respectively
desharna
parents:
77172
diff
changeset
|
39 |
by (simp add: wfp_on_def wf_on_def) |
|
d0205dde00bb
added definitions wf_on and wfp_on as restricted versions of wf and wfP respectively
desharna
parents:
77172
diff
changeset
|
40 |
|
|
79971
033f90dc441d
redefined wf as an abbreviation for "wf_on UNIV"
desharna
parents:
79965
diff
changeset
|
41 |
lemma wf_def: "wf r \<longleftrightarrow> (\<forall>P. (\<forall>x. (\<forall>y. (y, x) \<in> r \<longrightarrow> P y) \<longrightarrow> P x) \<longrightarrow> (\<forall>x. P x))" |
|
033f90dc441d
redefined wf as an abbreviation for "wf_on UNIV"
desharna
parents:
79965
diff
changeset
|
42 |
unfolding wf_on_def by simp |
|
033f90dc441d
redefined wf as an abbreviation for "wf_on UNIV"
desharna
parents:
79965
diff
changeset
|
43 |
|
| 80322 | 44 |
lemma wfp_def: "wfp r \<longleftrightarrow> wf {(x, y). r x y}"
|
|
79965
233d70cad0cf
redefined wfP as an abbreviation for "wfp_on UNIV"
desharna
parents:
79963
diff
changeset
|
45 |
unfolding wf_def wfp_on_def by simp |
|
233d70cad0cf
redefined wfP as an abbreviation for "wfp_on UNIV"
desharna
parents:
79963
diff
changeset
|
46 |
|
| 80322 | 47 |
lemma wfp_wf_eq: "wfp (\<lambda>x y. (x, y) \<in> r) = wf r" |
|
79971
033f90dc441d
redefined wf as an abbreviation for "wf_on UNIV"
desharna
parents:
79965
diff
changeset
|
48 |
using wfp_on_wf_on_eq . |
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
49 |
|
|
79917
d0205dde00bb
added definitions wf_on and wfp_on as restricted versions of wf and wfP respectively
desharna
parents:
77172
diff
changeset
|
50 |
|
|
d0205dde00bb
added definitions wf_on and wfp_on as restricted versions of wf and wfP respectively
desharna
parents:
77172
diff
changeset
|
51 |
subsection \<open>Induction Principles\<close> |
|
d0205dde00bb
added definitions wf_on and wfp_on as restricted versions of wf and wfP respectively
desharna
parents:
77172
diff
changeset
|
52 |
|
|
79996
4f803ae64781
changed number of consumed assumptions of wf_on_induct and wfp_on_induct
desharna
parents:
79971
diff
changeset
|
53 |
lemma wf_on_induct[consumes 1, case_names in_set less, induct set: wf_on]: |
|
79917
d0205dde00bb
added definitions wf_on and wfp_on as restricted versions of wf and wfP respectively
desharna
parents:
77172
diff
changeset
|
54 |
assumes "wf_on A r" and "x \<in> A" and "\<And>x. x \<in> A \<Longrightarrow> (\<And>y. y \<in> A \<Longrightarrow> (y, x) \<in> r \<Longrightarrow> P y) \<Longrightarrow> P x" |
|
d0205dde00bb
added definitions wf_on and wfp_on as restricted versions of wf and wfP respectively
desharna
parents:
77172
diff
changeset
|
55 |
shows "P x" |
|
d0205dde00bb
added definitions wf_on and wfp_on as restricted versions of wf and wfP respectively
desharna
parents:
77172
diff
changeset
|
56 |
using assms(2,3) by (auto intro: \<open>wf_on A r\<close>[unfolded wf_on_def, rule_format]) |
|
d0205dde00bb
added definitions wf_on and wfp_on as restricted versions of wf and wfP respectively
desharna
parents:
77172
diff
changeset
|
57 |
|
|
79996
4f803ae64781
changed number of consumed assumptions of wf_on_induct and wfp_on_induct
desharna
parents:
79971
diff
changeset
|
58 |
lemma wfp_on_induct[consumes 1, case_names in_set less, induct pred: wfp_on]: |
|
79917
d0205dde00bb
added definitions wf_on and wfp_on as restricted versions of wf and wfP respectively
desharna
parents:
77172
diff
changeset
|
59 |
assumes "wfp_on A r" and "x \<in> A" and "\<And>x. x \<in> A \<Longrightarrow> (\<And>y. y \<in> A \<Longrightarrow> r y x \<Longrightarrow> P y) \<Longrightarrow> P x" |
|
d0205dde00bb
added definitions wf_on and wfp_on as restricted versions of wf and wfP respectively
desharna
parents:
77172
diff
changeset
|
60 |
shows "P x" |
|
d0205dde00bb
added definitions wf_on and wfp_on as restricted versions of wf and wfP respectively
desharna
parents:
77172
diff
changeset
|
61 |
using assms by (fact wf_on_induct[to_pred]) |
|
d0205dde00bb
added definitions wf_on and wfp_on as restricted versions of wf and wfP respectively
desharna
parents:
77172
diff
changeset
|
62 |
|
|
d0205dde00bb
added definitions wf_on and wfp_on as restricted versions of wf and wfP respectively
desharna
parents:
77172
diff
changeset
|
63 |
lemma wf_induct: |
|
d0205dde00bb
added definitions wf_on and wfp_on as restricted versions of wf and wfP respectively
desharna
parents:
77172
diff
changeset
|
64 |
assumes "wf r" |
|
d0205dde00bb
added definitions wf_on and wfp_on as restricted versions of wf and wfP respectively
desharna
parents:
77172
diff
changeset
|
65 |
and "\<And>x. \<forall>y. (y, x) \<in> r \<longrightarrow> P y \<Longrightarrow> P x" |
|
d0205dde00bb
added definitions wf_on and wfp_on as restricted versions of wf and wfP respectively
desharna
parents:
77172
diff
changeset
|
66 |
shows "P a" |
|
79971
033f90dc441d
redefined wf as an abbreviation for "wf_on UNIV"
desharna
parents:
79965
diff
changeset
|
67 |
using assms by (auto intro: wf_on_induct[of UNIV]) |
|
79917
d0205dde00bb
added definitions wf_on and wfp_on as restricted versions of wf and wfP respectively
desharna
parents:
77172
diff
changeset
|
68 |
|
| 80322 | 69 |
lemmas wfp_induct = wf_induct [to_pred] |
|
79917
d0205dde00bb
added definitions wf_on and wfp_on as restricted versions of wf and wfP respectively
desharna
parents:
77172
diff
changeset
|
70 |
|
|
d0205dde00bb
added definitions wf_on and wfp_on as restricted versions of wf and wfP respectively
desharna
parents:
77172
diff
changeset
|
71 |
lemmas wf_induct_rule = wf_induct [rule_format, consumes 1, case_names less, induct set: wf] |
|
d0205dde00bb
added definitions wf_on and wfp_on as restricted versions of wf and wfP respectively
desharna
parents:
77172
diff
changeset
|
72 |
|
| 80322 | 73 |
lemmas wfp_induct_rule = wf_induct_rule [to_pred, induct set: wfp] |
|
79917
d0205dde00bb
added definitions wf_on and wfp_on as restricted versions of wf and wfP respectively
desharna
parents:
77172
diff
changeset
|
74 |
|
| 79997 | 75 |
lemma wf_on_iff_wf: "wf_on A r \<longleftrightarrow> wf {(x, y) \<in> r. x \<in> A \<and> y \<in> A}"
|
76 |
proof (rule iffI) |
|
77 |
assume wf: "wf_on A r" |
|
78 |
show "wf {(x, y) \<in> r. x \<in> A \<and> y \<in> A}"
|
|
79 |
unfolding wf_def |
|
80 |
proof (intro allI impI ballI) |
|
81 |
fix P x |
|
82 |
assume IH: "\<forall>x. (\<forall>y. (y, x) \<in> {(x, y). (x, y) \<in> r \<and> x \<in> A \<and> y \<in> A} \<longrightarrow> P y) \<longrightarrow> P x"
|
|
83 |
show "P x" |
|
84 |
proof (cases "x \<in> A") |
|
85 |
case True |
|
86 |
show ?thesis |
|
87 |
using wf |
|
88 |
proof (induction x rule: wf_on_induct) |
|
89 |
case in_set |
|
90 |
thus ?case |
|
91 |
using True . |
|
92 |
next |
|
93 |
case (less x) |
|
94 |
thus ?case |
|
95 |
by (auto intro: IH[rule_format]) |
|
96 |
qed |
|
97 |
next |
|
98 |
case False |
|
99 |
then show ?thesis |
|
100 |
by (auto intro: IH[rule_format]) |
|
101 |
qed |
|
102 |
qed |
|
103 |
next |
|
104 |
assume wf: "wf {(x, y). (x, y) \<in> r \<and> x \<in> A \<and> y \<in> A}"
|
|
105 |
show "wf_on A r" |
|
106 |
unfolding wf_on_def |
|
107 |
proof (intro allI impI ballI) |
|
108 |
fix P x |
|
109 |
assume IH: "\<forall>x\<in>A. (\<forall>y\<in>A. (y, x) \<in> r \<longrightarrow> P y) \<longrightarrow> P x" and "x \<in> A" |
|
110 |
show "P x" |
|
111 |
using wf \<open>x \<in> A\<close> |
|
112 |
proof (induction x rule: wf_on_induct) |
|
113 |
case in_set |
|
114 |
show ?case |
|
115 |
by simp |
|
116 |
next |
|
117 |
case (less y) |
|
118 |
hence "\<And>z. (z, y) \<in> r \<Longrightarrow> z \<in> A \<Longrightarrow> P z" |
|
119 |
by simp |
|
120 |
thus ?case |
|
121 |
using IH[rule_format, OF \<open>y \<in> A\<close>] by simp |
|
122 |
qed |
|
123 |
qed |
|
124 |
qed |
|
125 |
||
|
79917
d0205dde00bb
added definitions wf_on and wfp_on as restricted versions of wf and wfP respectively
desharna
parents:
77172
diff
changeset
|
126 |
|
|
d0205dde00bb
added definitions wf_on and wfp_on as restricted versions of wf and wfP respectively
desharna
parents:
77172
diff
changeset
|
127 |
subsection \<open>Introduction Rules\<close> |
|
d0205dde00bb
added definitions wf_on and wfp_on as restricted versions of wf and wfP respectively
desharna
parents:
77172
diff
changeset
|
128 |
|
| 63108 | 129 |
lemma wfUNIVI: "(\<And>P x. (\<forall>x. (\<forall>y. (y, x) \<in> r \<longrightarrow> P y) \<longrightarrow> P x) \<Longrightarrow> P x) \<Longrightarrow> wf r" |
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
130 |
unfolding wf_def by blast |
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
131 |
|
| 80322 | 132 |
lemmas wfpUNIVI = wfUNIVI [to_pred] |
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
133 |
|
| 63108 | 134 |
text \<open>Restriction to domain \<open>A\<close> and range \<open>B\<close>. |
135 |
If \<open>r\<close> is well-founded over their intersection, then \<open>wf r\<close>.\<close> |
|
136 |
lemma wfI: |
|
137 |
assumes "r \<subseteq> A \<times> B" |
|
138 |
and "\<And>x P. \<lbrakk>\<forall>x. (\<forall>y. (y, x) \<in> r \<longrightarrow> P y) \<longrightarrow> P x; x \<in> A; x \<in> B\<rbrakk> \<Longrightarrow> P x" |
|
139 |
shows "wf r" |
|
140 |
using assms unfolding wf_def by blast |
|
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
141 |
|
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
142 |
|
|
79917
d0205dde00bb
added definitions wf_on and wfp_on as restricted versions of wf and wfP respectively
desharna
parents:
77172
diff
changeset
|
143 |
subsection \<open>Ordering Properties\<close> |
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
144 |
|
| 63108 | 145 |
lemma wf_not_sym: "wf r \<Longrightarrow> (a, x) \<in> r \<Longrightarrow> (x, a) \<notin> r" |
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
146 |
by (induct a arbitrary: x set: wf) blast |
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
147 |
|
|
33215
6fd85372981e
replaced (outdated) comments by explicit statements
krauss
parents:
32960
diff
changeset
|
148 |
lemma wf_asym: |
|
6fd85372981e
replaced (outdated) comments by explicit statements
krauss
parents:
32960
diff
changeset
|
149 |
assumes "wf r" "(a, x) \<in> r" |
|
6fd85372981e
replaced (outdated) comments by explicit statements
krauss
parents:
32960
diff
changeset
|
150 |
obtains "(x, a) \<notin> r" |
|
6fd85372981e
replaced (outdated) comments by explicit statements
krauss
parents:
32960
diff
changeset
|
151 |
by (drule wf_not_sym[OF assms]) |
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
152 |
|
|
74971
16eaa56f69f7
added lemmas wf_imp_asym, wfP_imp_asymp, and wfP_imp_irreflp
desharna
parents:
74868
diff
changeset
|
153 |
lemma wf_imp_asym: "wf r \<Longrightarrow> asym r" |
|
16eaa56f69f7
added lemmas wf_imp_asym, wfP_imp_asymp, and wfP_imp_irreflp
desharna
parents:
74868
diff
changeset
|
154 |
by (auto intro: asymI elim: wf_asym) |
|
16eaa56f69f7
added lemmas wf_imp_asym, wfP_imp_asymp, and wfP_imp_irreflp
desharna
parents:
74868
diff
changeset
|
155 |
|
| 80322 | 156 |
lemma wfp_imp_asymp: "wfp r \<Longrightarrow> asymp r" |
|
74971
16eaa56f69f7
added lemmas wf_imp_asym, wfP_imp_asymp, and wfP_imp_irreflp
desharna
parents:
74868
diff
changeset
|
157 |
by (rule wf_imp_asym[to_pred]) |
|
16eaa56f69f7
added lemmas wf_imp_asym, wfP_imp_asymp, and wfP_imp_irreflp
desharna
parents:
74868
diff
changeset
|
158 |
|
| 63108 | 159 |
lemma wf_not_refl [simp]: "wf r \<Longrightarrow> (a, a) \<notin> r" |
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
160 |
by (blast elim: wf_asym) |
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
161 |
|
| 63572 | 162 |
lemma wf_irrefl: |
163 |
assumes "wf r" |
|
164 |
obtains "(a, a) \<notin> r" |
|
| 63108 | 165 |
by (drule wf_not_refl[OF assms]) |
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
166 |
|
|
72170
7fa9605b226c
Another go with lex: now lexordp back in class ord
paulson <lp15@cam.ac.uk>
parents:
72168
diff
changeset
|
167 |
lemma wf_imp_irrefl: |
|
7fa9605b226c
Another go with lex: now lexordp back in class ord
paulson <lp15@cam.ac.uk>
parents:
72168
diff
changeset
|
168 |
assumes "wf r" shows "irrefl r" |
|
7fa9605b226c
Another go with lex: now lexordp back in class ord
paulson <lp15@cam.ac.uk>
parents:
72168
diff
changeset
|
169 |
using wf_irrefl [OF assms] by (auto simp add: irrefl_def) |
|
7fa9605b226c
Another go with lex: now lexordp back in class ord
paulson <lp15@cam.ac.uk>
parents:
72168
diff
changeset
|
170 |
|
| 80322 | 171 |
lemma wfp_imp_irreflp: "wfp r \<Longrightarrow> irreflp r" |
|
76588
82a36e3d1b55
rewrite proofs using to_pred attribute on existing lemmas
desharna
parents:
76559
diff
changeset
|
172 |
by (rule wf_imp_irrefl[to_pred]) |
|
74971
16eaa56f69f7
added lemmas wf_imp_asym, wfP_imp_asymp, and wfP_imp_irreflp
desharna
parents:
74868
diff
changeset
|
173 |
|
| 27823 | 174 |
lemma wf_wellorderI: |
175 |
assumes wf: "wf {(x::'a::ord, y). x < y}"
|
|
| 63572 | 176 |
and lin: "OFCLASS('a::ord, linorder_class)"
|
| 27823 | 177 |
shows "OFCLASS('a::ord, wellorder_class)"
|
| 71410 | 178 |
apply (rule wellorder_class.intro [OF lin]) |
179 |
apply (simp add: wellorder_class.intro class.wellorder_axioms.intro wf_induct_rule [OF wf]) |
|
| 63108 | 180 |
done |
| 27823 | 181 |
|
| 63108 | 182 |
lemma (in wellorder) wf: "wf {(x, y). x < y}"
|
183 |
unfolding wf_def by (blast intro: less_induct) |
|
| 27823 | 184 |
|
| 79963 | 185 |
lemma (in wellorder) wfp_on_less[simp]: "wfp_on A (<)" |
186 |
unfolding wfp_on_def |
|
187 |
proof (intro allI impI ballI) |
|
188 |
fix P x |
|
189 |
assume hyps: "\<forall>x\<in>A. (\<forall>y\<in>A. y < x \<longrightarrow> P y) \<longrightarrow> P x" |
|
190 |
show "x \<in> A \<Longrightarrow> P x" |
|
191 |
proof (induction x rule: less_induct) |
|
192 |
case (less x) |
|
193 |
show ?case |
|
194 |
proof (rule hyps[rule_format]) |
|
195 |
show "x \<in> A" |
|
196 |
using \<open>x \<in> A\<close> . |
|
197 |
next |
|
198 |
show "\<And>y. y \<in> A \<Longrightarrow> y < x \<Longrightarrow> P y" |
|
199 |
using less.IH . |
|
200 |
qed |
|
201 |
qed |
|
202 |
qed |
|
203 |
||
| 27823 | 204 |
|
| 60758 | 205 |
subsection \<open>Basic Results\<close> |
| 26976 | 206 |
|
| 60758 | 207 |
text \<open>Point-free characterization of well-foundedness\<close> |
| 33216 | 208 |
|
|
79919
65e0682cca63
added lemmas wfP_iff_ex_minimal, wf_iff_ex_minimal, wf_onE_pf, wf_onI_pf, wf_on_iff_ex_minimal, and wfp_on_iff_ex_minimal
desharna
parents:
79917
diff
changeset
|
209 |
lemma wf_onE_pf: |
|
65e0682cca63
added lemmas wfP_iff_ex_minimal, wf_iff_ex_minimal, wf_onE_pf, wf_onI_pf, wf_on_iff_ex_minimal, and wfp_on_iff_ex_minimal
desharna
parents:
79917
diff
changeset
|
210 |
assumes wf: "wf_on A r" and "B \<subseteq> A" and "B \<subseteq> r `` B" |
|
65e0682cca63
added lemmas wfP_iff_ex_minimal, wf_iff_ex_minimal, wf_onE_pf, wf_onI_pf, wf_on_iff_ex_minimal, and wfp_on_iff_ex_minimal
desharna
parents:
79917
diff
changeset
|
211 |
shows "B = {}"
|
|
65e0682cca63
added lemmas wfP_iff_ex_minimal, wf_iff_ex_minimal, wf_onE_pf, wf_onI_pf, wf_on_iff_ex_minimal, and wfp_on_iff_ex_minimal
desharna
parents:
79917
diff
changeset
|
212 |
proof - |
|
65e0682cca63
added lemmas wfP_iff_ex_minimal, wf_iff_ex_minimal, wf_onE_pf, wf_onI_pf, wf_on_iff_ex_minimal, and wfp_on_iff_ex_minimal
desharna
parents:
79917
diff
changeset
|
213 |
have "x \<notin> B" if "x \<in> A" for x |
|
79996
4f803ae64781
changed number of consumed assumptions of wf_on_induct and wfp_on_induct
desharna
parents:
79971
diff
changeset
|
214 |
using wf |
|
79919
65e0682cca63
added lemmas wfP_iff_ex_minimal, wf_iff_ex_minimal, wf_onE_pf, wf_onI_pf, wf_on_iff_ex_minimal, and wfp_on_iff_ex_minimal
desharna
parents:
79917
diff
changeset
|
215 |
proof (induction x rule: wf_on_induct) |
|
79996
4f803ae64781
changed number of consumed assumptions of wf_on_induct and wfp_on_induct
desharna
parents:
79971
diff
changeset
|
216 |
case in_set |
|
4f803ae64781
changed number of consumed assumptions of wf_on_induct and wfp_on_induct
desharna
parents:
79971
diff
changeset
|
217 |
show ?case |
|
4f803ae64781
changed number of consumed assumptions of wf_on_induct and wfp_on_induct
desharna
parents:
79971
diff
changeset
|
218 |
using that . |
|
4f803ae64781
changed number of consumed assumptions of wf_on_induct and wfp_on_induct
desharna
parents:
79971
diff
changeset
|
219 |
next |
|
79919
65e0682cca63
added lemmas wfP_iff_ex_minimal, wf_iff_ex_minimal, wf_onE_pf, wf_onI_pf, wf_on_iff_ex_minimal, and wfp_on_iff_ex_minimal
desharna
parents:
79917
diff
changeset
|
220 |
case (less x) |
|
65e0682cca63
added lemmas wfP_iff_ex_minimal, wf_iff_ex_minimal, wf_onE_pf, wf_onI_pf, wf_on_iff_ex_minimal, and wfp_on_iff_ex_minimal
desharna
parents:
79917
diff
changeset
|
221 |
have "x \<notin> r `` B" |
|
65e0682cca63
added lemmas wfP_iff_ex_minimal, wf_iff_ex_minimal, wf_onE_pf, wf_onI_pf, wf_on_iff_ex_minimal, and wfp_on_iff_ex_minimal
desharna
parents:
79917
diff
changeset
|
222 |
using less.IH \<open>B \<subseteq> A\<close> by blast |
|
65e0682cca63
added lemmas wfP_iff_ex_minimal, wf_iff_ex_minimal, wf_onE_pf, wf_onI_pf, wf_on_iff_ex_minimal, and wfp_on_iff_ex_minimal
desharna
parents:
79917
diff
changeset
|
223 |
thus ?case |
|
65e0682cca63
added lemmas wfP_iff_ex_minimal, wf_iff_ex_minimal, wf_onE_pf, wf_onI_pf, wf_on_iff_ex_minimal, and wfp_on_iff_ex_minimal
desharna
parents:
79917
diff
changeset
|
224 |
using \<open>B \<subseteq> r `` B\<close> by blast |
|
65e0682cca63
added lemmas wfP_iff_ex_minimal, wf_iff_ex_minimal, wf_onE_pf, wf_onI_pf, wf_on_iff_ex_minimal, and wfp_on_iff_ex_minimal
desharna
parents:
79917
diff
changeset
|
225 |
qed |
|
65e0682cca63
added lemmas wfP_iff_ex_minimal, wf_iff_ex_minimal, wf_onE_pf, wf_onI_pf, wf_on_iff_ex_minimal, and wfp_on_iff_ex_minimal
desharna
parents:
79917
diff
changeset
|
226 |
with \<open>B \<subseteq> A\<close> show ?thesis |
|
65e0682cca63
added lemmas wfP_iff_ex_minimal, wf_iff_ex_minimal, wf_onE_pf, wf_onI_pf, wf_on_iff_ex_minimal, and wfp_on_iff_ex_minimal
desharna
parents:
79917
diff
changeset
|
227 |
by blast |
|
65e0682cca63
added lemmas wfP_iff_ex_minimal, wf_iff_ex_minimal, wf_onE_pf, wf_onI_pf, wf_on_iff_ex_minimal, and wfp_on_iff_ex_minimal
desharna
parents:
79917
diff
changeset
|
228 |
qed |
|
65e0682cca63
added lemmas wfP_iff_ex_minimal, wf_iff_ex_minimal, wf_onE_pf, wf_onI_pf, wf_on_iff_ex_minimal, and wfp_on_iff_ex_minimal
desharna
parents:
79917
diff
changeset
|
229 |
|
| 79920 | 230 |
lemma wfE_pf: "wf R \<Longrightarrow> A \<subseteq> R `` A \<Longrightarrow> A = {}"
|
|
79971
033f90dc441d
redefined wf as an abbreviation for "wf_on UNIV"
desharna
parents:
79965
diff
changeset
|
231 |
using wf_onE_pf[of UNIV, simplified] . |
| 33216 | 232 |
|
|
79919
65e0682cca63
added lemmas wfP_iff_ex_minimal, wf_iff_ex_minimal, wf_onE_pf, wf_onI_pf, wf_on_iff_ex_minimal, and wfp_on_iff_ex_minimal
desharna
parents:
79917
diff
changeset
|
233 |
lemma wf_onI_pf: |
|
65e0682cca63
added lemmas wfP_iff_ex_minimal, wf_iff_ex_minimal, wf_onE_pf, wf_onI_pf, wf_on_iff_ex_minimal, and wfp_on_iff_ex_minimal
desharna
parents:
79917
diff
changeset
|
234 |
assumes "\<And>B. B \<subseteq> A \<Longrightarrow> B \<subseteq> R `` B \<Longrightarrow> B = {}"
|
|
65e0682cca63
added lemmas wfP_iff_ex_minimal, wf_iff_ex_minimal, wf_onE_pf, wf_onI_pf, wf_on_iff_ex_minimal, and wfp_on_iff_ex_minimal
desharna
parents:
79917
diff
changeset
|
235 |
shows "wf_on A R" |
|
65e0682cca63
added lemmas wfP_iff_ex_minimal, wf_iff_ex_minimal, wf_onE_pf, wf_onI_pf, wf_on_iff_ex_minimal, and wfp_on_iff_ex_minimal
desharna
parents:
79917
diff
changeset
|
236 |
unfolding wf_on_def |
|
65e0682cca63
added lemmas wfP_iff_ex_minimal, wf_iff_ex_minimal, wf_onE_pf, wf_onI_pf, wf_on_iff_ex_minimal, and wfp_on_iff_ex_minimal
desharna
parents:
79917
diff
changeset
|
237 |
proof (intro allI impI ballI) |
|
65e0682cca63
added lemmas wfP_iff_ex_minimal, wf_iff_ex_minimal, wf_onE_pf, wf_onI_pf, wf_on_iff_ex_minimal, and wfp_on_iff_ex_minimal
desharna
parents:
79917
diff
changeset
|
238 |
fix P :: "'a \<Rightarrow> bool" and x :: 'a |
|
65e0682cca63
added lemmas wfP_iff_ex_minimal, wf_iff_ex_minimal, wf_onE_pf, wf_onI_pf, wf_on_iff_ex_minimal, and wfp_on_iff_ex_minimal
desharna
parents:
79917
diff
changeset
|
239 |
let ?B = "{x \<in> A. \<not> P x}"
|
|
65e0682cca63
added lemmas wfP_iff_ex_minimal, wf_iff_ex_minimal, wf_onE_pf, wf_onI_pf, wf_on_iff_ex_minimal, and wfp_on_iff_ex_minimal
desharna
parents:
79917
diff
changeset
|
240 |
assume "\<forall>x\<in>A. (\<forall>y\<in>A. (y, x) \<in> R \<longrightarrow> P y) \<longrightarrow> P x" |
|
65e0682cca63
added lemmas wfP_iff_ex_minimal, wf_iff_ex_minimal, wf_onE_pf, wf_onI_pf, wf_on_iff_ex_minimal, and wfp_on_iff_ex_minimal
desharna
parents:
79917
diff
changeset
|
241 |
hence "?B \<subseteq> R `` ?B" by blast |
|
65e0682cca63
added lemmas wfP_iff_ex_minimal, wf_iff_ex_minimal, wf_onE_pf, wf_onI_pf, wf_on_iff_ex_minimal, and wfp_on_iff_ex_minimal
desharna
parents:
79917
diff
changeset
|
242 |
hence "{x \<in> A. \<not> P x} = {}"
|
|
65e0682cca63
added lemmas wfP_iff_ex_minimal, wf_iff_ex_minimal, wf_onE_pf, wf_onI_pf, wf_on_iff_ex_minimal, and wfp_on_iff_ex_minimal
desharna
parents:
79917
diff
changeset
|
243 |
using assms(1)[of ?B] by simp |
|
65e0682cca63
added lemmas wfP_iff_ex_minimal, wf_iff_ex_minimal, wf_onE_pf, wf_onI_pf, wf_on_iff_ex_minimal, and wfp_on_iff_ex_minimal
desharna
parents:
79917
diff
changeset
|
244 |
moreover assume "x \<in> A" |
|
65e0682cca63
added lemmas wfP_iff_ex_minimal, wf_iff_ex_minimal, wf_onE_pf, wf_onI_pf, wf_on_iff_ex_minimal, and wfp_on_iff_ex_minimal
desharna
parents:
79917
diff
changeset
|
245 |
ultimately show "P x" |
|
65e0682cca63
added lemmas wfP_iff_ex_minimal, wf_iff_ex_minimal, wf_onE_pf, wf_onI_pf, wf_on_iff_ex_minimal, and wfp_on_iff_ex_minimal
desharna
parents:
79917
diff
changeset
|
246 |
by simp |
|
65e0682cca63
added lemmas wfP_iff_ex_minimal, wf_iff_ex_minimal, wf_onE_pf, wf_onI_pf, wf_on_iff_ex_minimal, and wfp_on_iff_ex_minimal
desharna
parents:
79917
diff
changeset
|
247 |
qed |
|
65e0682cca63
added lemmas wfP_iff_ex_minimal, wf_iff_ex_minimal, wf_onE_pf, wf_onI_pf, wf_on_iff_ex_minimal, and wfp_on_iff_ex_minimal
desharna
parents:
79917
diff
changeset
|
248 |
|
| 79920 | 249 |
lemma wfI_pf: "(\<And>A. A \<subseteq> R `` A \<Longrightarrow> A = {}) \<Longrightarrow> wf R"
|
|
79971
033f90dc441d
redefined wf as an abbreviation for "wf_on UNIV"
desharna
parents:
79965
diff
changeset
|
250 |
using wf_onI_pf[of UNIV, simplified] . |
| 33216 | 251 |
|
| 63108 | 252 |
|
253 |
subsubsection \<open>Minimal-element characterization of well-foundedness\<close> |
|
| 33216 | 254 |
|
|
79919
65e0682cca63
added lemmas wfP_iff_ex_minimal, wf_iff_ex_minimal, wf_onE_pf, wf_onI_pf, wf_on_iff_ex_minimal, and wfp_on_iff_ex_minimal
desharna
parents:
79917
diff
changeset
|
255 |
lemma wf_on_iff_ex_minimal: "wf_on A R \<longleftrightarrow> (\<forall>B \<subseteq> A. B \<noteq> {} \<longrightarrow> (\<exists>z \<in> B. \<forall>y. (y, z) \<in> R \<longrightarrow> y \<notin> B))"
|
|
65e0682cca63
added lemmas wfP_iff_ex_minimal, wf_iff_ex_minimal, wf_onE_pf, wf_onI_pf, wf_on_iff_ex_minimal, and wfp_on_iff_ex_minimal
desharna
parents:
79917
diff
changeset
|
256 |
proof (intro iffI allI impI) |
|
65e0682cca63
added lemmas wfP_iff_ex_minimal, wf_iff_ex_minimal, wf_onE_pf, wf_onI_pf, wf_on_iff_ex_minimal, and wfp_on_iff_ex_minimal
desharna
parents:
79917
diff
changeset
|
257 |
fix B |
|
65e0682cca63
added lemmas wfP_iff_ex_minimal, wf_iff_ex_minimal, wf_onE_pf, wf_onI_pf, wf_on_iff_ex_minimal, and wfp_on_iff_ex_minimal
desharna
parents:
79917
diff
changeset
|
258 |
assume "wf_on A R" and "B \<subseteq> A" and "B \<noteq> {}"
|
|
65e0682cca63
added lemmas wfP_iff_ex_minimal, wf_iff_ex_minimal, wf_onE_pf, wf_onI_pf, wf_on_iff_ex_minimal, and wfp_on_iff_ex_minimal
desharna
parents:
79917
diff
changeset
|
259 |
show "\<exists>z \<in> B. \<forall>y. (y, z) \<in> R \<longrightarrow> y \<notin> B" |
|
65e0682cca63
added lemmas wfP_iff_ex_minimal, wf_iff_ex_minimal, wf_onE_pf, wf_onI_pf, wf_on_iff_ex_minimal, and wfp_on_iff_ex_minimal
desharna
parents:
79917
diff
changeset
|
260 |
using wf_onE_pf[OF \<open>wf_on A R\<close> \<open>B \<subseteq> A\<close>] \<open>B \<noteq> {}\<close> by blast
|
|
65e0682cca63
added lemmas wfP_iff_ex_minimal, wf_iff_ex_minimal, wf_onE_pf, wf_onI_pf, wf_on_iff_ex_minimal, and wfp_on_iff_ex_minimal
desharna
parents:
79917
diff
changeset
|
261 |
next |
|
65e0682cca63
added lemmas wfP_iff_ex_minimal, wf_iff_ex_minimal, wf_onE_pf, wf_onI_pf, wf_on_iff_ex_minimal, and wfp_on_iff_ex_minimal
desharna
parents:
79917
diff
changeset
|
262 |
assume ex_min: "\<forall>B\<subseteq>A. B \<noteq> {} \<longrightarrow> (\<exists>z\<in>B. \<forall>y. (y, z) \<in> R \<longrightarrow> y \<notin> B)"
|
|
65e0682cca63
added lemmas wfP_iff_ex_minimal, wf_iff_ex_minimal, wf_onE_pf, wf_onI_pf, wf_on_iff_ex_minimal, and wfp_on_iff_ex_minimal
desharna
parents:
79917
diff
changeset
|
263 |
show "wf_on A R " |
|
65e0682cca63
added lemmas wfP_iff_ex_minimal, wf_iff_ex_minimal, wf_onE_pf, wf_onI_pf, wf_on_iff_ex_minimal, and wfp_on_iff_ex_minimal
desharna
parents:
79917
diff
changeset
|
264 |
proof (rule wf_onI_pf) |
|
65e0682cca63
added lemmas wfP_iff_ex_minimal, wf_iff_ex_minimal, wf_onE_pf, wf_onI_pf, wf_on_iff_ex_minimal, and wfp_on_iff_ex_minimal
desharna
parents:
79917
diff
changeset
|
265 |
fix B |
|
65e0682cca63
added lemmas wfP_iff_ex_minimal, wf_iff_ex_minimal, wf_onE_pf, wf_onI_pf, wf_on_iff_ex_minimal, and wfp_on_iff_ex_minimal
desharna
parents:
79917
diff
changeset
|
266 |
assume "B \<subseteq> A" and "B \<subseteq> R `` B" |
|
65e0682cca63
added lemmas wfP_iff_ex_minimal, wf_iff_ex_minimal, wf_onE_pf, wf_onI_pf, wf_on_iff_ex_minimal, and wfp_on_iff_ex_minimal
desharna
parents:
79917
diff
changeset
|
267 |
have False if "B \<noteq> {}"
|
|
65e0682cca63
added lemmas wfP_iff_ex_minimal, wf_iff_ex_minimal, wf_onE_pf, wf_onI_pf, wf_on_iff_ex_minimal, and wfp_on_iff_ex_minimal
desharna
parents:
79917
diff
changeset
|
268 |
using ex_min[rule_format, OF \<open>B \<subseteq> A\<close> \<open>B \<noteq> {}\<close>]
|
|
65e0682cca63
added lemmas wfP_iff_ex_minimal, wf_iff_ex_minimal, wf_onE_pf, wf_onI_pf, wf_on_iff_ex_minimal, and wfp_on_iff_ex_minimal
desharna
parents:
79917
diff
changeset
|
269 |
using \<open>B \<subseteq> R `` B\<close> by blast |
|
65e0682cca63
added lemmas wfP_iff_ex_minimal, wf_iff_ex_minimal, wf_onE_pf, wf_onI_pf, wf_on_iff_ex_minimal, and wfp_on_iff_ex_minimal
desharna
parents:
79917
diff
changeset
|
270 |
thus "B = {}"
|
|
65e0682cca63
added lemmas wfP_iff_ex_minimal, wf_iff_ex_minimal, wf_onE_pf, wf_onI_pf, wf_on_iff_ex_minimal, and wfp_on_iff_ex_minimal
desharna
parents:
79917
diff
changeset
|
271 |
by blast |
|
65e0682cca63
added lemmas wfP_iff_ex_minimal, wf_iff_ex_minimal, wf_onE_pf, wf_onI_pf, wf_on_iff_ex_minimal, and wfp_on_iff_ex_minimal
desharna
parents:
79917
diff
changeset
|
272 |
qed |
|
65e0682cca63
added lemmas wfP_iff_ex_minimal, wf_iff_ex_minimal, wf_onE_pf, wf_onI_pf, wf_on_iff_ex_minimal, and wfp_on_iff_ex_minimal
desharna
parents:
79917
diff
changeset
|
273 |
qed |
|
65e0682cca63
added lemmas wfP_iff_ex_minimal, wf_iff_ex_minimal, wf_onE_pf, wf_onI_pf, wf_on_iff_ex_minimal, and wfp_on_iff_ex_minimal
desharna
parents:
79917
diff
changeset
|
274 |
|
|
65e0682cca63
added lemmas wfP_iff_ex_minimal, wf_iff_ex_minimal, wf_onE_pf, wf_onI_pf, wf_on_iff_ex_minimal, and wfp_on_iff_ex_minimal
desharna
parents:
79917
diff
changeset
|
275 |
lemma wf_iff_ex_minimal: "wf R \<longleftrightarrow> (\<forall>B. B \<noteq> {} \<longrightarrow> (\<exists>z \<in> B. \<forall>y. (y, z) \<in> R \<longrightarrow> y \<notin> B))"
|
|
79971
033f90dc441d
redefined wf as an abbreviation for "wf_on UNIV"
desharna
parents:
79965
diff
changeset
|
276 |
using wf_on_iff_ex_minimal[of UNIV, simplified] . |
|
79919
65e0682cca63
added lemmas wfP_iff_ex_minimal, wf_iff_ex_minimal, wf_onE_pf, wf_onI_pf, wf_on_iff_ex_minimal, and wfp_on_iff_ex_minimal
desharna
parents:
79917
diff
changeset
|
277 |
|
|
65e0682cca63
added lemmas wfP_iff_ex_minimal, wf_iff_ex_minimal, wf_onE_pf, wf_onI_pf, wf_on_iff_ex_minimal, and wfp_on_iff_ex_minimal
desharna
parents:
79917
diff
changeset
|
278 |
lemma wfp_on_iff_ex_minimal: "wfp_on A R \<longleftrightarrow> (\<forall>B \<subseteq> A. B \<noteq> {} \<longrightarrow> (\<exists>z \<in> B. \<forall>y. R y z \<longrightarrow> y \<notin> B))"
|
|
65e0682cca63
added lemmas wfP_iff_ex_minimal, wf_iff_ex_minimal, wf_onE_pf, wf_onI_pf, wf_on_iff_ex_minimal, and wfp_on_iff_ex_minimal
desharna
parents:
79917
diff
changeset
|
279 |
using wf_on_iff_ex_minimal[of A, to_pred] by simp |
|
65e0682cca63
added lemmas wfP_iff_ex_minimal, wf_iff_ex_minimal, wf_onE_pf, wf_onI_pf, wf_on_iff_ex_minimal, and wfp_on_iff_ex_minimal
desharna
parents:
79917
diff
changeset
|
280 |
|
|
80019
991557e01814
renamed lemma wfP_iff_ex_minimal to wfp_iff_ex_minimal
desharna
parents:
79999
diff
changeset
|
281 |
lemma wfp_iff_ex_minimal: "wfp R \<longleftrightarrow> (\<forall>B. B \<noteq> {} \<longrightarrow> (\<exists>z \<in> B. \<forall>y. R y z \<longrightarrow> y \<notin> B))"
|
|
79965
233d70cad0cf
redefined wfP as an abbreviation for "wfp_on UNIV"
desharna
parents:
79963
diff
changeset
|
282 |
using wfp_on_iff_ex_minimal[of UNIV, simplified] . |
|
79919
65e0682cca63
added lemmas wfP_iff_ex_minimal, wf_iff_ex_minimal, wf_onE_pf, wf_onI_pf, wf_on_iff_ex_minimal, and wfp_on_iff_ex_minimal
desharna
parents:
79917
diff
changeset
|
283 |
|
| 33216 | 284 |
lemma wfE_min: |
285 |
assumes wf: "wf R" and Q: "x \<in> Q" |
|
286 |
obtains z where "z \<in> Q" "\<And>y. (y, z) \<in> R \<Longrightarrow> y \<notin> Q" |
|
287 |
using Q wfE_pf[OF wf, of Q] by blast |
|
288 |
||
|
63099
af0e964aad7b
Moved material from AFP/Randomised_Social_Choice to distribution
eberlm
parents:
63088
diff
changeset
|
289 |
lemma wfE_min': |
|
af0e964aad7b
Moved material from AFP/Randomised_Social_Choice to distribution
eberlm
parents:
63088
diff
changeset
|
290 |
"wf R \<Longrightarrow> Q \<noteq> {} \<Longrightarrow> (\<And>z. z \<in> Q \<Longrightarrow> (\<And>y. (y, z) \<in> R \<Longrightarrow> y \<notin> Q) \<Longrightarrow> thesis) \<Longrightarrow> thesis"
|
|
af0e964aad7b
Moved material from AFP/Randomised_Social_Choice to distribution
eberlm
parents:
63088
diff
changeset
|
291 |
using wfE_min[of R _ Q] by blast |
|
af0e964aad7b
Moved material from AFP/Randomised_Social_Choice to distribution
eberlm
parents:
63088
diff
changeset
|
292 |
|
| 33216 | 293 |
lemma wfI_min: |
294 |
assumes a: "\<And>x Q. x \<in> Q \<Longrightarrow> \<exists>z\<in>Q. \<forall>y. (y, z) \<in> R \<longrightarrow> y \<notin> Q" |
|
295 |
shows "wf R" |
|
296 |
proof (rule wfI_pf) |
|
| 63108 | 297 |
fix A |
298 |
assume b: "A \<subseteq> R `` A" |
|
299 |
have False if "x \<in> A" for x |
|
300 |
using a[OF that] b by blast |
|
301 |
then show "A = {}" by blast
|
|
| 33216 | 302 |
qed |
303 |
||
| 63108 | 304 |
lemma wf_eq_minimal: "wf r \<longleftrightarrow> (\<forall>Q x. x \<in> Q \<longrightarrow> (\<exists>z\<in>Q. \<forall>y. (y, z) \<in> r \<longrightarrow> y \<notin> Q))" |
| 79920 | 305 |
unfolding wf_iff_ex_minimal by blast |
| 33216 | 306 |
|
| 80322 | 307 |
lemmas wfp_eq_minimal = wf_eq_minimal [to_pred] |
| 33216 | 308 |
|
| 63108 | 309 |
|
|
79922
caa9dbffd712
added lemmas wf_on_antimono, wf_on_antimono_strong, wfp_on_antimono, wfp_on_antimono_strong, wf_on_subset, and wfp_on_subset
desharna
parents:
79920
diff
changeset
|
310 |
subsubsection \<open>Antimonotonicity\<close> |
|
caa9dbffd712
added lemmas wf_on_antimono, wf_on_antimono_strong, wfp_on_antimono, wfp_on_antimono_strong, wf_on_subset, and wfp_on_subset
desharna
parents:
79920
diff
changeset
|
311 |
|
|
caa9dbffd712
added lemmas wf_on_antimono, wf_on_antimono_strong, wfp_on_antimono, wfp_on_antimono_strong, wf_on_subset, and wfp_on_subset
desharna
parents:
79920
diff
changeset
|
312 |
lemma wf_on_antimono_strong: |
|
caa9dbffd712
added lemmas wf_on_antimono, wf_on_antimono_strong, wfp_on_antimono, wfp_on_antimono_strong, wf_on_subset, and wfp_on_subset
desharna
parents:
79920
diff
changeset
|
313 |
assumes "wf_on B r" and "A \<subseteq> B" and "(\<And>x y. x \<in> A \<Longrightarrow> y \<in> A \<Longrightarrow> (x, y) \<in> q \<Longrightarrow> (x, y) \<in> r)" |
|
caa9dbffd712
added lemmas wf_on_antimono, wf_on_antimono_strong, wfp_on_antimono, wfp_on_antimono_strong, wf_on_subset, and wfp_on_subset
desharna
parents:
79920
diff
changeset
|
314 |
shows "wf_on A q" |
|
caa9dbffd712
added lemmas wf_on_antimono, wf_on_antimono_strong, wfp_on_antimono, wfp_on_antimono_strong, wf_on_subset, and wfp_on_subset
desharna
parents:
79920
diff
changeset
|
315 |
unfolding wf_on_iff_ex_minimal |
|
caa9dbffd712
added lemmas wf_on_antimono, wf_on_antimono_strong, wfp_on_antimono, wfp_on_antimono_strong, wf_on_subset, and wfp_on_subset
desharna
parents:
79920
diff
changeset
|
316 |
proof (intro allI impI) |
|
caa9dbffd712
added lemmas wf_on_antimono, wf_on_antimono_strong, wfp_on_antimono, wfp_on_antimono_strong, wf_on_subset, and wfp_on_subset
desharna
parents:
79920
diff
changeset
|
317 |
fix AA assume "AA \<subseteq> A" and "AA \<noteq> {}"
|
|
caa9dbffd712
added lemmas wf_on_antimono, wf_on_antimono_strong, wfp_on_antimono, wfp_on_antimono_strong, wf_on_subset, and wfp_on_subset
desharna
parents:
79920
diff
changeset
|
318 |
hence "\<exists>z\<in>AA. \<forall>y. (y, z) \<in> r \<longrightarrow> y \<notin> AA" |
|
caa9dbffd712
added lemmas wf_on_antimono, wf_on_antimono_strong, wfp_on_antimono, wfp_on_antimono_strong, wf_on_subset, and wfp_on_subset
desharna
parents:
79920
diff
changeset
|
319 |
using \<open>wf_on B r\<close> \<open>A \<subseteq> B\<close> |
|
caa9dbffd712
added lemmas wf_on_antimono, wf_on_antimono_strong, wfp_on_antimono, wfp_on_antimono_strong, wf_on_subset, and wfp_on_subset
desharna
parents:
79920
diff
changeset
|
320 |
by (simp add: wf_on_iff_ex_minimal) |
|
caa9dbffd712
added lemmas wf_on_antimono, wf_on_antimono_strong, wfp_on_antimono, wfp_on_antimono_strong, wf_on_subset, and wfp_on_subset
desharna
parents:
79920
diff
changeset
|
321 |
then show "\<exists>z\<in>AA. \<forall>y. (y, z) \<in> q \<longrightarrow> y \<notin> AA" |
|
caa9dbffd712
added lemmas wf_on_antimono, wf_on_antimono_strong, wfp_on_antimono, wfp_on_antimono_strong, wf_on_subset, and wfp_on_subset
desharna
parents:
79920
diff
changeset
|
322 |
using \<open>AA \<subseteq> A\<close> assms(3) by blast |
|
caa9dbffd712
added lemmas wf_on_antimono, wf_on_antimono_strong, wfp_on_antimono, wfp_on_antimono_strong, wf_on_subset, and wfp_on_subset
desharna
parents:
79920
diff
changeset
|
323 |
qed |
|
caa9dbffd712
added lemmas wf_on_antimono, wf_on_antimono_strong, wfp_on_antimono, wfp_on_antimono_strong, wf_on_subset, and wfp_on_subset
desharna
parents:
79920
diff
changeset
|
324 |
|
|
caa9dbffd712
added lemmas wf_on_antimono, wf_on_antimono_strong, wfp_on_antimono, wfp_on_antimono_strong, wf_on_subset, and wfp_on_subset
desharna
parents:
79920
diff
changeset
|
325 |
lemma wfp_on_antimono_strong: |
|
caa9dbffd712
added lemmas wf_on_antimono, wf_on_antimono_strong, wfp_on_antimono, wfp_on_antimono_strong, wf_on_subset, and wfp_on_subset
desharna
parents:
79920
diff
changeset
|
326 |
"wfp_on B R \<Longrightarrow> A \<subseteq> B \<Longrightarrow> (\<And>x y. x \<in> A \<Longrightarrow> y \<in> A \<Longrightarrow> Q x y \<Longrightarrow> R x y) \<Longrightarrow> wfp_on A Q" |
|
caa9dbffd712
added lemmas wf_on_antimono, wf_on_antimono_strong, wfp_on_antimono, wfp_on_antimono_strong, wf_on_subset, and wfp_on_subset
desharna
parents:
79920
diff
changeset
|
327 |
using wf_on_antimono_strong[of B _ A, to_pred] . |
|
caa9dbffd712
added lemmas wf_on_antimono, wf_on_antimono_strong, wfp_on_antimono, wfp_on_antimono_strong, wf_on_subset, and wfp_on_subset
desharna
parents:
79920
diff
changeset
|
328 |
|
|
caa9dbffd712
added lemmas wf_on_antimono, wf_on_antimono_strong, wfp_on_antimono, wfp_on_antimono_strong, wf_on_subset, and wfp_on_subset
desharna
parents:
79920
diff
changeset
|
329 |
lemma wf_on_antimono: "A \<subseteq> B \<Longrightarrow> q \<subseteq> r \<Longrightarrow> wf_on B r \<le> wf_on A q" |
|
caa9dbffd712
added lemmas wf_on_antimono, wf_on_antimono_strong, wfp_on_antimono, wfp_on_antimono_strong, wf_on_subset, and wfp_on_subset
desharna
parents:
79920
diff
changeset
|
330 |
using wf_on_antimono_strong[of B r A q] by auto |
|
caa9dbffd712
added lemmas wf_on_antimono, wf_on_antimono_strong, wfp_on_antimono, wfp_on_antimono_strong, wf_on_subset, and wfp_on_subset
desharna
parents:
79920
diff
changeset
|
331 |
|
|
caa9dbffd712
added lemmas wf_on_antimono, wf_on_antimono_strong, wfp_on_antimono, wfp_on_antimono_strong, wf_on_subset, and wfp_on_subset
desharna
parents:
79920
diff
changeset
|
332 |
lemma wfp_on_antimono: "A \<subseteq> B \<Longrightarrow> Q \<le> R \<Longrightarrow> wfp_on B R \<le> wfp_on A Q" |
|
caa9dbffd712
added lemmas wf_on_antimono, wf_on_antimono_strong, wfp_on_antimono, wfp_on_antimono_strong, wf_on_subset, and wfp_on_subset
desharna
parents:
79920
diff
changeset
|
333 |
using wfp_on_antimono_strong[of B R A Q] by auto |
|
caa9dbffd712
added lemmas wf_on_antimono, wf_on_antimono_strong, wfp_on_antimono, wfp_on_antimono_strong, wf_on_subset, and wfp_on_subset
desharna
parents:
79920
diff
changeset
|
334 |
|
|
caa9dbffd712
added lemmas wf_on_antimono, wf_on_antimono_strong, wfp_on_antimono, wfp_on_antimono_strong, wf_on_subset, and wfp_on_subset
desharna
parents:
79920
diff
changeset
|
335 |
lemma wf_on_subset: "wf_on B r \<Longrightarrow> A \<subseteq> B \<Longrightarrow> wf_on A r" |
|
caa9dbffd712
added lemmas wf_on_antimono, wf_on_antimono_strong, wfp_on_antimono, wfp_on_antimono_strong, wf_on_subset, and wfp_on_subset
desharna
parents:
79920
diff
changeset
|
336 |
using wf_on_antimono_strong . |
|
caa9dbffd712
added lemmas wf_on_antimono, wf_on_antimono_strong, wfp_on_antimono, wfp_on_antimono_strong, wf_on_subset, and wfp_on_subset
desharna
parents:
79920
diff
changeset
|
337 |
|
|
caa9dbffd712
added lemmas wf_on_antimono, wf_on_antimono_strong, wfp_on_antimono, wfp_on_antimono_strong, wf_on_subset, and wfp_on_subset
desharna
parents:
79920
diff
changeset
|
338 |
lemma wfp_on_subset: "wfp_on B R \<Longrightarrow> A \<subseteq> B \<Longrightarrow> wfp_on A R" |
|
caa9dbffd712
added lemmas wf_on_antimono, wf_on_antimono_strong, wfp_on_antimono, wfp_on_antimono_strong, wf_on_subset, and wfp_on_subset
desharna
parents:
79920
diff
changeset
|
339 |
using wfp_on_antimono_strong . |
|
caa9dbffd712
added lemmas wf_on_antimono, wf_on_antimono_strong, wfp_on_antimono, wfp_on_antimono_strong, wf_on_subset, and wfp_on_subset
desharna
parents:
79920
diff
changeset
|
340 |
|
|
caa9dbffd712
added lemmas wf_on_antimono, wf_on_antimono_strong, wfp_on_antimono, wfp_on_antimono_strong, wf_on_subset, and wfp_on_subset
desharna
parents:
79920
diff
changeset
|
341 |
|
| 63108 | 342 |
subsubsection \<open>Well-foundedness of transitive closure\<close> |
| 33216 | 343 |
|
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
344 |
lemma wf_trancl: |
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
345 |
assumes "wf r" |
| 63108 | 346 |
shows "wf (r\<^sup>+)" |
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
347 |
proof - |
| 63108 | 348 |
have "P x" if induct_step: "\<And>x. (\<And>y. (y, x) \<in> r\<^sup>+ \<Longrightarrow> P y) \<Longrightarrow> P x" for P x |
349 |
proof (rule induct_step) |
|
350 |
show "P y" if "(y, x) \<in> r\<^sup>+" for y |
|
351 |
using \<open>wf r\<close> and that |
|
352 |
proof (induct x arbitrary: y) |
|
353 |
case (less x) |
|
354 |
note hyp = \<open>\<And>x' y'. (x', x) \<in> r \<Longrightarrow> (y', x') \<in> r\<^sup>+ \<Longrightarrow> P y'\<close> |
|
355 |
from \<open>(y, x) \<in> r\<^sup>+\<close> show "P y" |
|
356 |
proof cases |
|
357 |
case base |
|
358 |
show "P y" |
|
359 |
proof (rule induct_step) |
|
360 |
fix y' |
|
361 |
assume "(y', y) \<in> r\<^sup>+" |
|
362 |
with \<open>(y, x) \<in> r\<close> show "P y'" |
|
363 |
by (rule hyp [of y y']) |
|
|
32960
69916a850301
eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents:
32704
diff
changeset
|
364 |
qed |
| 63108 | 365 |
next |
366 |
case step |
|
367 |
then obtain x' where "(x', x) \<in> r" and "(y, x') \<in> r\<^sup>+" |
|
368 |
by simp |
|
369 |
then show "P y" by (rule hyp [of x' y]) |
|
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
370 |
qed |
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
371 |
qed |
| 63108 | 372 |
qed |
373 |
then show ?thesis unfolding wf_def by blast |
|
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
374 |
qed |
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
375 |
|
| 80322 | 376 |
lemmas wfp_tranclp = wf_trancl [to_pred] |
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
377 |
|
| 63108 | 378 |
lemma wf_converse_trancl: "wf (r\<inverse>) \<Longrightarrow> wf ((r\<^sup>+)\<inverse>)" |
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
379 |
apply (subst trancl_converse [symmetric]) |
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
380 |
apply (erule wf_trancl) |
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
381 |
done |
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
382 |
|
| 60758 | 383 |
text \<open>Well-foundedness of subsets\<close> |
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
384 |
|
| 63108 | 385 |
lemma wf_subset: "wf r \<Longrightarrow> p \<subseteq> r \<Longrightarrow> wf p" |
| 63612 | 386 |
by (simp add: wf_eq_minimal) fast |
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
387 |
|
| 80322 | 388 |
lemmas wfp_subset = wf_subset [to_pred] |
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
389 |
|
| 60758 | 390 |
text \<open>Well-foundedness of the empty relation\<close> |
| 33216 | 391 |
|
392 |
lemma wf_empty [iff]: "wf {}"
|
|
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
393 |
by (simp add: wf_def) |
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
394 |
|
| 80322 | 395 |
lemma wfp_empty [iff]: "wfp (\<lambda>x y. False)" |
| 32205 | 396 |
proof - |
| 80322 | 397 |
have "wfp bot" |
| 66952 | 398 |
by (fact wf_empty[to_pred bot_empty_eq2]) |
| 63612 | 399 |
then show ?thesis |
400 |
by (simp add: bot_fun_def) |
|
| 32205 | 401 |
qed |
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
402 |
|
| 63572 | 403 |
lemma wf_Int1: "wf r \<Longrightarrow> wf (r \<inter> r')" |
404 |
by (erule wf_subset) (rule Int_lower1) |
|
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
405 |
|
| 63572 | 406 |
lemma wf_Int2: "wf r \<Longrightarrow> wf (r' \<inter> r)" |
407 |
by (erule wf_subset) (rule Int_lower2) |
|
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
408 |
|
| 63572 | 409 |
text \<open>Exponentiation.\<close> |
| 33216 | 410 |
lemma wf_exp: |
411 |
assumes "wf (R ^^ n)" |
|
412 |
shows "wf R" |
|
413 |
proof (rule wfI_pf) |
|
414 |
fix A assume "A \<subseteq> R `` A" |
|
| 63612 | 415 |
then have "A \<subseteq> (R ^^ n) `` A" |
416 |
by (induct n) force+ |
|
417 |
with \<open>wf (R ^^ n)\<close> show "A = {}"
|
|
418 |
by (rule wfE_pf) |
|
| 33216 | 419 |
qed |
420 |
||
| 63572 | 421 |
text \<open>Well-foundedness of \<open>insert\<close>.\<close> |
| 68646 | 422 |
lemma wf_insert [iff]: "wf (insert (y,x) r) \<longleftrightarrow> wf r \<and> (x,y) \<notin> r\<^sup>*" (is "?lhs = ?rhs") |
423 |
proof |
|
424 |
assume ?lhs then show ?rhs |
|
425 |
by (blast elim: wf_trancl [THEN wf_irrefl] |
|
426 |
intro: rtrancl_into_trancl1 wf_subset rtrancl_mono [THEN subsetD]) |
|
427 |
next |
|
| 71410 | 428 |
assume R: ?rhs |
| 68646 | 429 |
then have R': "Q \<noteq> {} \<Longrightarrow> (\<exists>z\<in>Q. \<forall>y. (y, z) \<in> r \<longrightarrow> y \<notin> Q)" for Q
|
430 |
by (auto simp: wf_eq_minimal) |
|
431 |
show ?lhs |
|
432 |
unfolding wf_eq_minimal |
|
433 |
proof clarify |
|
434 |
fix Q :: "'a set" and q |
|
435 |
assume "q \<in> Q" |
|
436 |
then obtain a where "a \<in> Q" and a: "\<And>y. (y, a) \<in> r \<Longrightarrow> y \<notin> Q" |
|
437 |
using R by (auto simp: wf_eq_minimal) |
|
438 |
show "\<exists>z\<in>Q. \<forall>y'. (y', z) \<in> insert (y, x) r \<longrightarrow> y' \<notin> Q" |
|
439 |
proof (cases "a=x") |
|
440 |
case True |
|
441 |
show ?thesis |
|
442 |
proof (cases "y \<in> Q") |
|
443 |
case True |
|
444 |
then obtain z where "z \<in> Q" "(z, y) \<in> r\<^sup>*" |
|
445 |
"\<And>z'. (z', z) \<in> r \<longrightarrow> z' \<in> Q \<longrightarrow> (z', y) \<notin> r\<^sup>*" |
|
446 |
using R' [of "{z \<in> Q. (z,y) \<in> r\<^sup>*}"] by auto
|
|
|
75669
43f5dfb7fa35
tuned (some HOL lints, by Yecine Megdiche);
Fabian Huch <huch@in.tum.de>
parents:
74971
diff
changeset
|
447 |
then have "\<forall>y'. (y', z) \<in> insert (y, x) r \<longrightarrow> y' \<notin> Q" |
|
43f5dfb7fa35
tuned (some HOL lints, by Yecine Megdiche);
Fabian Huch <huch@in.tum.de>
parents:
74971
diff
changeset
|
448 |
using R by(blast intro: rtrancl_trans)+ |
|
43f5dfb7fa35
tuned (some HOL lints, by Yecine Megdiche);
Fabian Huch <huch@in.tum.de>
parents:
74971
diff
changeset
|
449 |
then show ?thesis |
|
43f5dfb7fa35
tuned (some HOL lints, by Yecine Megdiche);
Fabian Huch <huch@in.tum.de>
parents:
74971
diff
changeset
|
450 |
by (rule bexI) fact |
| 68646 | 451 |
next |
452 |
case False |
|
453 |
then show ?thesis |
|
454 |
using a \<open>a \<in> Q\<close> by blast |
|
455 |
qed |
|
456 |
next |
|
457 |
case False |
|
458 |
with a \<open>a \<in> Q\<close> show ?thesis |
|
459 |
by blast |
|
460 |
qed |
|
461 |
qed |
|
462 |
qed |
|
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
463 |
|
| 63108 | 464 |
|
465 |
subsubsection \<open>Well-foundedness of image\<close> |
|
| 33216 | 466 |
|
|
68259
80df7c90e315
By Andrei Popescu based on an initial version by Kasper F. Brandt
nipkow
parents:
67399
diff
changeset
|
467 |
lemma wf_map_prod_image_Dom_Ran: |
|
80df7c90e315
By Andrei Popescu based on an initial version by Kasper F. Brandt
nipkow
parents:
67399
diff
changeset
|
468 |
fixes r:: "('a \<times> 'a) set"
|
|
80df7c90e315
By Andrei Popescu based on an initial version by Kasper F. Brandt
nipkow
parents:
67399
diff
changeset
|
469 |
and f:: "'a \<Rightarrow> 'b" |
|
80df7c90e315
By Andrei Popescu based on an initial version by Kasper F. Brandt
nipkow
parents:
67399
diff
changeset
|
470 |
assumes wf_r: "wf r" |
|
80df7c90e315
By Andrei Popescu based on an initial version by Kasper F. Brandt
nipkow
parents:
67399
diff
changeset
|
471 |
and inj: "\<And> a a'. a \<in> Domain r \<Longrightarrow> a' \<in> Range r \<Longrightarrow> f a = f a' \<Longrightarrow> a = a'" |
|
80df7c90e315
By Andrei Popescu based on an initial version by Kasper F. Brandt
nipkow
parents:
67399
diff
changeset
|
472 |
shows "wf (map_prod f f ` r)" |
|
80df7c90e315
By Andrei Popescu based on an initial version by Kasper F. Brandt
nipkow
parents:
67399
diff
changeset
|
473 |
proof (unfold wf_eq_minimal, clarify) |
| 68262 | 474 |
fix B :: "'b set" and b::"'b" |
475 |
assume "b \<in> B" |
|
476 |
define A where "A = f -` B \<inter> Domain r" |
|
477 |
show "\<exists>z\<in>B. \<forall>y. (y, z) \<in> map_prod f f ` r \<longrightarrow> y \<notin> B" |
|
478 |
proof (cases "A = {}")
|
|
|
68259
80df7c90e315
By Andrei Popescu based on an initial version by Kasper F. Brandt
nipkow
parents:
67399
diff
changeset
|
479 |
case False |
| 68262 | 480 |
then obtain a0 where "a0 \<in> A" and "\<forall>a. (a, a0) \<in> r \<longrightarrow> a \<notin> A" |
|
68259
80df7c90e315
By Andrei Popescu based on an initial version by Kasper F. Brandt
nipkow
parents:
67399
diff
changeset
|
481 |
using wfE_min[OF wf_r] by auto |
| 71410 | 482 |
thus ?thesis |
| 68262 | 483 |
using inj unfolding A_def |
484 |
by (intro bexI[of _ "f a0"]) auto |
|
|
75669
43f5dfb7fa35
tuned (some HOL lints, by Yecine Megdiche);
Fabian Huch <huch@in.tum.de>
parents:
74971
diff
changeset
|
485 |
qed (use \<open>b \<in> B\<close> in \<open>unfold A_def, auto\<close>) |
|
68259
80df7c90e315
By Andrei Popescu based on an initial version by Kasper F. Brandt
nipkow
parents:
67399
diff
changeset
|
486 |
qed |
|
80df7c90e315
By Andrei Popescu based on an initial version by Kasper F. Brandt
nipkow
parents:
67399
diff
changeset
|
487 |
|
| 63108 | 488 |
lemma wf_map_prod_image: "wf r \<Longrightarrow> inj f \<Longrightarrow> wf (map_prod f f ` r)" |
|
68259
80df7c90e315
By Andrei Popescu based on an initial version by Kasper F. Brandt
nipkow
parents:
67399
diff
changeset
|
489 |
by(rule wf_map_prod_image_Dom_Ran) (auto dest: inj_onD) |
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
490 |
|
|
80046
38803a6b3357
added lemma wfp_on_image and author name to theory
desharna
parents:
80019
diff
changeset
|
491 |
lemma wfp_on_image: "wfp_on (f ` A) R \<longleftrightarrow> wfp_on A (\<lambda>a b. R (f a) (f b))" |
|
38803a6b3357
added lemma wfp_on_image and author name to theory
desharna
parents:
80019
diff
changeset
|
492 |
proof (rule iffI) |
|
38803a6b3357
added lemma wfp_on_image and author name to theory
desharna
parents:
80019
diff
changeset
|
493 |
assume hyp: "wfp_on (f ` A) R" |
|
38803a6b3357
added lemma wfp_on_image and author name to theory
desharna
parents:
80019
diff
changeset
|
494 |
show "wfp_on A (\<lambda>a b. R (f a) (f b))" |
|
38803a6b3357
added lemma wfp_on_image and author name to theory
desharna
parents:
80019
diff
changeset
|
495 |
unfolding wfp_on_iff_ex_minimal |
|
38803a6b3357
added lemma wfp_on_image and author name to theory
desharna
parents:
80019
diff
changeset
|
496 |
proof (intro allI impI) |
|
38803a6b3357
added lemma wfp_on_image and author name to theory
desharna
parents:
80019
diff
changeset
|
497 |
fix B |
|
38803a6b3357
added lemma wfp_on_image and author name to theory
desharna
parents:
80019
diff
changeset
|
498 |
assume "B \<subseteq> A" and "B \<noteq> {}"
|
|
38803a6b3357
added lemma wfp_on_image and author name to theory
desharna
parents:
80019
diff
changeset
|
499 |
hence "f ` B \<subseteq> f ` A" and "f ` B \<noteq> {}"
|
|
38803a6b3357
added lemma wfp_on_image and author name to theory
desharna
parents:
80019
diff
changeset
|
500 |
unfolding atomize_conj image_is_empty |
|
38803a6b3357
added lemma wfp_on_image and author name to theory
desharna
parents:
80019
diff
changeset
|
501 |
using image_mono by iprover |
|
38803a6b3357
added lemma wfp_on_image and author name to theory
desharna
parents:
80019
diff
changeset
|
502 |
hence "\<exists>z\<in>f ` B. \<forall>y. R y z \<longrightarrow> y \<notin> f ` B" |
|
38803a6b3357
added lemma wfp_on_image and author name to theory
desharna
parents:
80019
diff
changeset
|
503 |
using hyp[unfolded wfp_on_iff_ex_minimal, rule_format] by iprover |
|
38803a6b3357
added lemma wfp_on_image and author name to theory
desharna
parents:
80019
diff
changeset
|
504 |
then obtain fz where "fz \<in> f ` B" and fz_max: "\<forall>y. R y fz \<longrightarrow> y \<notin> f ` B" .. |
|
38803a6b3357
added lemma wfp_on_image and author name to theory
desharna
parents:
80019
diff
changeset
|
505 |
|
|
38803a6b3357
added lemma wfp_on_image and author name to theory
desharna
parents:
80019
diff
changeset
|
506 |
obtain z where "z \<in> B" and "fz = f z" |
|
38803a6b3357
added lemma wfp_on_image and author name to theory
desharna
parents:
80019
diff
changeset
|
507 |
using \<open>fz \<in> f ` B\<close> unfolding image_iff .. |
|
38803a6b3357
added lemma wfp_on_image and author name to theory
desharna
parents:
80019
diff
changeset
|
508 |
|
|
38803a6b3357
added lemma wfp_on_image and author name to theory
desharna
parents:
80019
diff
changeset
|
509 |
show "\<exists>z\<in>B. \<forall>y. R (f y) (f z) \<longrightarrow> y \<notin> B" |
|
38803a6b3357
added lemma wfp_on_image and author name to theory
desharna
parents:
80019
diff
changeset
|
510 |
proof (intro bexI allI impI) |
|
38803a6b3357
added lemma wfp_on_image and author name to theory
desharna
parents:
80019
diff
changeset
|
511 |
show "z \<in> B" |
|
38803a6b3357
added lemma wfp_on_image and author name to theory
desharna
parents:
80019
diff
changeset
|
512 |
using \<open>z \<in> B\<close> . |
|
38803a6b3357
added lemma wfp_on_image and author name to theory
desharna
parents:
80019
diff
changeset
|
513 |
next |
|
38803a6b3357
added lemma wfp_on_image and author name to theory
desharna
parents:
80019
diff
changeset
|
514 |
fix y assume "R (f y) (f z)" |
|
38803a6b3357
added lemma wfp_on_image and author name to theory
desharna
parents:
80019
diff
changeset
|
515 |
hence "f y \<notin> f ` B" |
|
38803a6b3357
added lemma wfp_on_image and author name to theory
desharna
parents:
80019
diff
changeset
|
516 |
using fz_max \<open>fz = f z\<close> by iprover |
|
38803a6b3357
added lemma wfp_on_image and author name to theory
desharna
parents:
80019
diff
changeset
|
517 |
thus "y \<notin> B" |
|
38803a6b3357
added lemma wfp_on_image and author name to theory
desharna
parents:
80019
diff
changeset
|
518 |
by (rule contrapos_nn) (rule imageI) |
|
38803a6b3357
added lemma wfp_on_image and author name to theory
desharna
parents:
80019
diff
changeset
|
519 |
qed |
|
38803a6b3357
added lemma wfp_on_image and author name to theory
desharna
parents:
80019
diff
changeset
|
520 |
qed |
|
38803a6b3357
added lemma wfp_on_image and author name to theory
desharna
parents:
80019
diff
changeset
|
521 |
next |
|
38803a6b3357
added lemma wfp_on_image and author name to theory
desharna
parents:
80019
diff
changeset
|
522 |
assume hyp: "wfp_on A (\<lambda>a b. R (f a) (f b))" |
|
38803a6b3357
added lemma wfp_on_image and author name to theory
desharna
parents:
80019
diff
changeset
|
523 |
show "wfp_on (f ` A) R" |
|
38803a6b3357
added lemma wfp_on_image and author name to theory
desharna
parents:
80019
diff
changeset
|
524 |
unfolding wfp_on_iff_ex_minimal |
|
38803a6b3357
added lemma wfp_on_image and author name to theory
desharna
parents:
80019
diff
changeset
|
525 |
proof (intro allI impI) |
|
38803a6b3357
added lemma wfp_on_image and author name to theory
desharna
parents:
80019
diff
changeset
|
526 |
fix fA |
|
38803a6b3357
added lemma wfp_on_image and author name to theory
desharna
parents:
80019
diff
changeset
|
527 |
assume "fA \<subseteq> f ` A" and "fA \<noteq> {}"
|
|
38803a6b3357
added lemma wfp_on_image and author name to theory
desharna
parents:
80019
diff
changeset
|
528 |
then obtain A' where "A' \<subseteq> A" and "A' \<noteq> {}" and "fA = f ` A'"
|
|
38803a6b3357
added lemma wfp_on_image and author name to theory
desharna
parents:
80019
diff
changeset
|
529 |
by (auto simp only: subset_image_iff) |
|
38803a6b3357
added lemma wfp_on_image and author name to theory
desharna
parents:
80019
diff
changeset
|
530 |
|
|
38803a6b3357
added lemma wfp_on_image and author name to theory
desharna
parents:
80019
diff
changeset
|
531 |
obtain z where "z \<in> A'" and z_max: "\<forall>y. R (f y) (f z) \<longrightarrow> y \<notin> A'" |
|
38803a6b3357
added lemma wfp_on_image and author name to theory
desharna
parents:
80019
diff
changeset
|
532 |
using hyp[unfolded wfp_on_iff_ex_minimal, rule_format, OF \<open>A' \<subseteq> A\<close> \<open>A' \<noteq> {}\<close>] by blast
|
|
38803a6b3357
added lemma wfp_on_image and author name to theory
desharna
parents:
80019
diff
changeset
|
533 |
|
|
38803a6b3357
added lemma wfp_on_image and author name to theory
desharna
parents:
80019
diff
changeset
|
534 |
show "\<exists>z\<in>fA. \<forall>y. R y z \<longrightarrow> y \<notin> fA" |
|
38803a6b3357
added lemma wfp_on_image and author name to theory
desharna
parents:
80019
diff
changeset
|
535 |
proof (intro bexI allI impI) |
|
38803a6b3357
added lemma wfp_on_image and author name to theory
desharna
parents:
80019
diff
changeset
|
536 |
show "f z \<in> fA" |
|
38803a6b3357
added lemma wfp_on_image and author name to theory
desharna
parents:
80019
diff
changeset
|
537 |
unfolding \<open>fA = f ` A'\<close> |
|
38803a6b3357
added lemma wfp_on_image and author name to theory
desharna
parents:
80019
diff
changeset
|
538 |
using imageI[OF \<open>z \<in> A'\<close>] . |
|
38803a6b3357
added lemma wfp_on_image and author name to theory
desharna
parents:
80019
diff
changeset
|
539 |
next |
|
38803a6b3357
added lemma wfp_on_image and author name to theory
desharna
parents:
80019
diff
changeset
|
540 |
show "\<And>y. R y (f z) \<Longrightarrow> y \<notin> fA" |
|
38803a6b3357
added lemma wfp_on_image and author name to theory
desharna
parents:
80019
diff
changeset
|
541 |
unfolding \<open>fA = f ` A'\<close> |
|
38803a6b3357
added lemma wfp_on_image and author name to theory
desharna
parents:
80019
diff
changeset
|
542 |
using z_max by auto |
|
38803a6b3357
added lemma wfp_on_image and author name to theory
desharna
parents:
80019
diff
changeset
|
543 |
qed |
|
38803a6b3357
added lemma wfp_on_image and author name to theory
desharna
parents:
80019
diff
changeset
|
544 |
qed |
|
38803a6b3357
added lemma wfp_on_image and author name to theory
desharna
parents:
80019
diff
changeset
|
545 |
qed |
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
546 |
|
| 60758 | 547 |
subsection \<open>Well-Foundedness Results for Unions\<close> |
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
548 |
|
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
549 |
lemma wf_union_compatible: |
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
550 |
assumes "wf R" "wf S" |
|
32235
8f9b8d14fc9f
"more standard" argument order of relation composition (op O)
krauss
parents:
32205
diff
changeset
|
551 |
assumes "R O S \<subseteq> R" |
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
552 |
shows "wf (R \<union> S)" |
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
553 |
proof (rule wfI_min) |
| 63108 | 554 |
fix x :: 'a and Q |
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
555 |
let ?Q' = "{x \<in> Q. \<forall>y. (y, x) \<in> R \<longrightarrow> y \<notin> Q}"
|
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
556 |
assume "x \<in> Q" |
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
557 |
obtain a where "a \<in> ?Q'" |
| 60758 | 558 |
by (rule wfE_min [OF \<open>wf R\<close> \<open>x \<in> Q\<close>]) blast |
| 63108 | 559 |
with \<open>wf S\<close> obtain z where "z \<in> ?Q'" and zmin: "\<And>y. (y, z) \<in> S \<Longrightarrow> y \<notin> ?Q'" |
560 |
by (erule wfE_min) |
|
| 63572 | 561 |
have "y \<notin> Q" if "(y, z) \<in> S" for y |
562 |
proof |
|
563 |
from that have "y \<notin> ?Q'" by (rule zmin) |
|
564 |
assume "y \<in> Q" |
|
565 |
with \<open>y \<notin> ?Q'\<close> obtain w where "(w, y) \<in> R" and "w \<in> Q" by auto |
|
566 |
from \<open>(w, y) \<in> R\<close> \<open>(y, z) \<in> S\<close> have "(w, z) \<in> R O S" by (rule relcompI) |
|
567 |
with \<open>R O S \<subseteq> R\<close> have "(w, z) \<in> R" .. |
|
568 |
with \<open>z \<in> ?Q'\<close> have "w \<notin> Q" by blast |
|
569 |
with \<open>w \<in> Q\<close> show False by contradiction |
|
570 |
qed |
|
| 60758 | 571 |
with \<open>z \<in> ?Q'\<close> show "\<exists>z\<in>Q. \<forall>y. (y, z) \<in> R \<union> S \<longrightarrow> y \<notin> Q" by blast |
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
572 |
qed |
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
573 |
|
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
574 |
|
| 63572 | 575 |
text \<open>Well-foundedness of indexed union with disjoint domains and ranges.\<close> |
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
576 |
|
| 63108 | 577 |
lemma wf_UN: |
| 68646 | 578 |
assumes r: "\<And>i. i \<in> I \<Longrightarrow> wf (r i)" |
579 |
and disj: "\<And>i j. \<lbrakk>i \<in> I; j \<in> I; r i \<noteq> r j\<rbrakk> \<Longrightarrow> Domain (r i) \<inter> Range (r j) = {}"
|
|
| 63108 | 580 |
shows "wf (\<Union>i\<in>I. r i)" |
| 68646 | 581 |
unfolding wf_eq_minimal |
582 |
proof clarify |
|
583 |
fix A and a :: "'b" |
|
584 |
assume "a \<in> A" |
|
| 69275 | 585 |
show "\<exists>z\<in>A. \<forall>y. (y, z) \<in> \<Union>(r ` I) \<longrightarrow> y \<notin> A" |
| 68646 | 586 |
proof (cases "\<exists>i\<in>I. \<exists>a\<in>A. \<exists>b\<in>A. (b, a) \<in> r i") |
587 |
case True |
|
588 |
then obtain i b c where ibc: "i \<in> I" "b \<in> A" "c \<in> A" "(c,b) \<in> r i" |
|
589 |
by blast |
|
590 |
have ri: "\<And>Q. Q \<noteq> {} \<Longrightarrow> \<exists>z\<in>Q. \<forall>y. (y, z) \<in> r i \<longrightarrow> y \<notin> Q"
|
|
591 |
using r [OF \<open>i \<in> I\<close>] unfolding wf_eq_minimal by auto |
|
592 |
show ?thesis |
|
| 71410 | 593 |
using ri [of "{a. a \<in> A \<and> (\<exists>b\<in>A. (b, a) \<in> r i) }"] ibc disj
|
| 68646 | 594 |
by blast |
595 |
next |
|
596 |
case False |
|
597 |
with \<open>a \<in> A\<close> show ?thesis |
|
598 |
by blast |
|
599 |
qed |
|
600 |
qed |
|
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
601 |
|
| 80322 | 602 |
lemma wfp_SUP: |
603 |
"\<forall>i. wfp (r i) \<Longrightarrow> \<forall>i j. r i \<noteq> r j \<longrightarrow> inf (Domainp (r i)) (Rangep (r j)) = bot \<Longrightarrow> |
|
604 |
wfp (\<Squnion>(range r))" |
|
| 63572 | 605 |
by (rule wf_UN[to_pred]) simp_all |
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
606 |
|
| 63108 | 607 |
lemma wf_Union: |
608 |
assumes "\<forall>r\<in>R. wf r" |
|
609 |
and "\<forall>r\<in>R. \<forall>s\<in>R. r \<noteq> s \<longrightarrow> Domain r \<inter> Range s = {}"
|
|
610 |
shows "wf (\<Union>R)" |
|
611 |
using assms wf_UN[of R "\<lambda>i. i"] by simp |
|
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
612 |
|
| 63109 | 613 |
text \<open> |
614 |
Intuition: We find an \<open>R \<union> S\<close>-min element of a nonempty subset \<open>A\<close> by case distinction. |
|
615 |
\<^enum> There is a step \<open>a \<midarrow>R\<rightarrow> b\<close> with \<open>a, b \<in> A\<close>. |
|
616 |
Pick an \<open>R\<close>-min element \<open>z\<close> of the (nonempty) set \<open>{a\<in>A | \<exists>b\<in>A. a \<midarrow>R\<rightarrow> b}\<close>.
|
|
617 |
By definition, there is \<open>z' \<in> A\<close> s.t. \<open>z \<midarrow>R\<rightarrow> z'\<close>. Because \<open>z\<close> is \<open>R\<close>-min in the |
|
618 |
subset, \<open>z'\<close> must be \<open>R\<close>-min in \<open>A\<close>. Because \<open>z'\<close> has an \<open>R\<close>-predecessor, it cannot |
|
619 |
have an \<open>S\<close>-successor and is thus \<open>S\<close>-min in \<open>A\<close> as well. |
|
620 |
\<^enum> There is no such step. |
|
621 |
Pick an \<open>S\<close>-min element of \<open>A\<close>. In this case it must be an \<open>R\<close>-min |
|
622 |
element of \<open>A\<close> as well. |
|
623 |
\<close> |
|
| 63108 | 624 |
lemma wf_Un: "wf r \<Longrightarrow> wf s \<Longrightarrow> Domain r \<inter> Range s = {} \<Longrightarrow> wf (r \<union> s)"
|
625 |
using wf_union_compatible[of s r] |
|
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
626 |
by (auto simp: Un_ac) |
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
627 |
|
| 63108 | 628 |
lemma wf_union_merge: "wf (R \<union> S) = wf (R O R \<union> S O R \<union> S)" |
629 |
(is "wf ?A = wf ?B") |
|
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
630 |
proof |
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
631 |
assume "wf ?A" |
| 63108 | 632 |
with wf_trancl have wfT: "wf (?A\<^sup>+)" . |
633 |
moreover have "?B \<subseteq> ?A\<^sup>+" |
|
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
634 |
by (subst trancl_unfold, subst trancl_unfold) blast |
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
635 |
ultimately show "wf ?B" by (rule wf_subset) |
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
636 |
next |
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
637 |
assume "wf ?B" |
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
638 |
show "wf ?A" |
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
639 |
proof (rule wfI_min) |
| 63108 | 640 |
fix Q :: "'a set" and x |
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
641 |
assume "x \<in> Q" |
| 63109 | 642 |
with \<open>wf ?B\<close> obtain z where "z \<in> Q" and "\<And>y. (y, z) \<in> ?B \<Longrightarrow> y \<notin> Q" |
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
643 |
by (erule wfE_min) |
| 63109 | 644 |
then have 1: "\<And>y. (y, z) \<in> R O R \<Longrightarrow> y \<notin> Q" |
645 |
and 2: "\<And>y. (y, z) \<in> S O R \<Longrightarrow> y \<notin> Q" |
|
646 |
and 3: "\<And>y. (y, z) \<in> S \<Longrightarrow> y \<notin> Q" |
|
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
647 |
by auto |
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
648 |
show "\<exists>z\<in>Q. \<forall>y. (y, z) \<in> ?A \<longrightarrow> y \<notin> Q" |
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
649 |
proof (cases "\<forall>y. (y, z) \<in> R \<longrightarrow> y \<notin> Q") |
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
650 |
case True |
| 63109 | 651 |
with \<open>z \<in> Q\<close> 3 show ?thesis by blast |
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
652 |
next |
| 63108 | 653 |
case False |
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
654 |
then obtain z' where "z'\<in>Q" "(z', z) \<in> R" by blast |
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
655 |
have "\<forall>y. (y, z') \<in> ?A \<longrightarrow> y \<notin> Q" |
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
656 |
proof (intro allI impI) |
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
657 |
fix y assume "(y, z') \<in> ?A" |
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
658 |
then show "y \<notin> Q" |
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
659 |
proof |
| 63108 | 660 |
assume "(y, z') \<in> R" |
| 60758 | 661 |
then have "(y, z) \<in> R O R" using \<open>(z', z) \<in> R\<close> .. |
| 63109 | 662 |
with 1 show "y \<notin> Q" . |
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
663 |
next |
| 63108 | 664 |
assume "(y, z') \<in> S" |
| 60758 | 665 |
then have "(y, z) \<in> S O R" using \<open>(z', z) \<in> R\<close> .. |
| 63109 | 666 |
with 2 show "y \<notin> Q" . |
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
667 |
qed |
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
668 |
qed |
| 60758 | 669 |
with \<open>z' \<in> Q\<close> show ?thesis .. |
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
670 |
qed |
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
671 |
qed |
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
672 |
qed |
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
673 |
|
| 63612 | 674 |
lemma wf_comp_self: "wf R \<longleftrightarrow> wf (R O R)" \<comment> \<open>special case\<close> |
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
675 |
by (rule wf_union_merge [where S = "{}", simplified])
|
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
676 |
|
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
677 |
|
| 60758 | 678 |
subsection \<open>Well-Foundedness of Composition\<close> |
| 60148 | 679 |
|
|
60493
866f41a869e6
New WF theorem by Tjark Weber. Replaced the proof of the subsequent theorem.
paulson <lp15@cam.ac.uk>
parents:
60148
diff
changeset
|
680 |
text \<open>Bachmair and Dershowitz 1986, Lemma 2. [Provided by Tjark Weber]\<close> |
| 60148 | 681 |
|
|
60493
866f41a869e6
New WF theorem by Tjark Weber. Replaced the proof of the subsequent theorem.
paulson <lp15@cam.ac.uk>
parents:
60148
diff
changeset
|
682 |
lemma qc_wf_relto_iff: |
| 61799 | 683 |
assumes "R O S \<subseteq> (R \<union> S)\<^sup>* O R" \<comment> \<open>R quasi-commutes over S\<close> |
| 63109 | 684 |
shows "wf (S\<^sup>* O R O S\<^sup>*) \<longleftrightarrow> wf R" |
| 63612 | 685 |
(is "wf ?S \<longleftrightarrow> _") |
|
60493
866f41a869e6
New WF theorem by Tjark Weber. Replaced the proof of the subsequent theorem.
paulson <lp15@cam.ac.uk>
parents:
60148
diff
changeset
|
686 |
proof |
| 63109 | 687 |
show "wf R" if "wf ?S" |
688 |
proof - |
|
689 |
have "R \<subseteq> ?S" by auto |
|
| 63612 | 690 |
with wf_subset [of ?S] that show "wf R" |
691 |
by auto |
|
| 63109 | 692 |
qed |
|
60493
866f41a869e6
New WF theorem by Tjark Weber. Replaced the proof of the subsequent theorem.
paulson <lp15@cam.ac.uk>
parents:
60148
diff
changeset
|
693 |
next |
| 63109 | 694 |
show "wf ?S" if "wf R" |
|
60493
866f41a869e6
New WF theorem by Tjark Weber. Replaced the proof of the subsequent theorem.
paulson <lp15@cam.ac.uk>
parents:
60148
diff
changeset
|
695 |
proof (rule wfI_pf) |
| 63109 | 696 |
fix A |
697 |
assume A: "A \<subseteq> ?S `` A" |
|
|
60493
866f41a869e6
New WF theorem by Tjark Weber. Replaced the proof of the subsequent theorem.
paulson <lp15@cam.ac.uk>
parents:
60148
diff
changeset
|
698 |
let ?X = "(R \<union> S)\<^sup>* `` A" |
|
866f41a869e6
New WF theorem by Tjark Weber. Replaced the proof of the subsequent theorem.
paulson <lp15@cam.ac.uk>
parents:
60148
diff
changeset
|
699 |
have *: "R O (R \<union> S)\<^sup>* \<subseteq> (R \<union> S)\<^sup>* O R" |
| 63109 | 700 |
proof - |
701 |
have "(x, z) \<in> (R \<union> S)\<^sup>* O R" if "(y, z) \<in> (R \<union> S)\<^sup>*" and "(x, y) \<in> R" for x y z |
|
702 |
using that |
|
703 |
proof (induct y z) |
|
704 |
case rtrancl_refl |
|
705 |
then show ?case by auto |
|
706 |
next |
|
707 |
case (rtrancl_into_rtrancl a b c) |
|
708 |
then have "(x, c) \<in> ((R \<union> S)\<^sup>* O (R \<union> S)\<^sup>*) O R" |
|
709 |
using assms by blast |
|
710 |
then show ?case by simp |
|
|
60493
866f41a869e6
New WF theorem by Tjark Weber. Replaced the proof of the subsequent theorem.
paulson <lp15@cam.ac.uk>
parents:
60148
diff
changeset
|
711 |
qed |
| 63109 | 712 |
then show ?thesis by auto |
713 |
qed |
|
714 |
then have "R O S\<^sup>* \<subseteq> (R \<union> S)\<^sup>* O R" |
|
715 |
using rtrancl_Un_subset by blast |
|
716 |
then have "?S \<subseteq> (R \<union> S)\<^sup>* O (R \<union> S)\<^sup>* O R" |
|
717 |
by (simp add: relcomp_mono rtrancl_mono) |
|
718 |
also have "\<dots> = (R \<union> S)\<^sup>* O R" |
|
719 |
by (simp add: O_assoc[symmetric]) |
|
720 |
finally have "?S O (R \<union> S)\<^sup>* \<subseteq> (R \<union> S)\<^sup>* O R O (R \<union> S)\<^sup>*" |
|
721 |
by (simp add: O_assoc[symmetric] relcomp_mono) |
|
722 |
also have "\<dots> \<subseteq> (R \<union> S)\<^sup>* O (R \<union> S)\<^sup>* O R" |
|
723 |
using * by (simp add: relcomp_mono) |
|
724 |
finally have "?S O (R \<union> S)\<^sup>* \<subseteq> (R \<union> S)\<^sup>* O R" |
|
725 |
by (simp add: O_assoc[symmetric]) |
|
726 |
then have "(?S O (R \<union> S)\<^sup>*) `` A \<subseteq> ((R \<union> S)\<^sup>* O R) `` A" |
|
727 |
by (simp add: Image_mono) |
|
728 |
moreover have "?X \<subseteq> (?S O (R \<union> S)\<^sup>*) `` A" |
|
729 |
using A by (auto simp: relcomp_Image) |
|
730 |
ultimately have "?X \<subseteq> R `` ?X" |
|
731 |
by (auto simp: relcomp_Image) |
|
732 |
then have "?X = {}"
|
|
733 |
using \<open>wf R\<close> by (simp add: wfE_pf) |
|
|
60493
866f41a869e6
New WF theorem by Tjark Weber. Replaced the proof of the subsequent theorem.
paulson <lp15@cam.ac.uk>
parents:
60148
diff
changeset
|
734 |
moreover have "A \<subseteq> ?X" by auto |
|
866f41a869e6
New WF theorem by Tjark Weber. Replaced the proof of the subsequent theorem.
paulson <lp15@cam.ac.uk>
parents:
60148
diff
changeset
|
735 |
ultimately show "A = {}" by simp
|
|
866f41a869e6
New WF theorem by Tjark Weber. Replaced the proof of the subsequent theorem.
paulson <lp15@cam.ac.uk>
parents:
60148
diff
changeset
|
736 |
qed |
|
866f41a869e6
New WF theorem by Tjark Weber. Replaced the proof of the subsequent theorem.
paulson <lp15@cam.ac.uk>
parents:
60148
diff
changeset
|
737 |
qed |
|
866f41a869e6
New WF theorem by Tjark Weber. Replaced the proof of the subsequent theorem.
paulson <lp15@cam.ac.uk>
parents:
60148
diff
changeset
|
738 |
|
|
866f41a869e6
New WF theorem by Tjark Weber. Replaced the proof of the subsequent theorem.
paulson <lp15@cam.ac.uk>
parents:
60148
diff
changeset
|
739 |
corollary wf_relcomp_compatible: |
| 60148 | 740 |
assumes "wf R" and "R O S \<subseteq> S O R" |
741 |
shows "wf (S O R)" |
|
|
60493
866f41a869e6
New WF theorem by Tjark Weber. Replaced the proof of the subsequent theorem.
paulson <lp15@cam.ac.uk>
parents:
60148
diff
changeset
|
742 |
proof - |
|
866f41a869e6
New WF theorem by Tjark Weber. Replaced the proof of the subsequent theorem.
paulson <lp15@cam.ac.uk>
parents:
60148
diff
changeset
|
743 |
have "R O S \<subseteq> (R \<union> S)\<^sup>* O R" |
|
866f41a869e6
New WF theorem by Tjark Weber. Replaced the proof of the subsequent theorem.
paulson <lp15@cam.ac.uk>
parents:
60148
diff
changeset
|
744 |
using assms by blast |
|
866f41a869e6
New WF theorem by Tjark Weber. Replaced the proof of the subsequent theorem.
paulson <lp15@cam.ac.uk>
parents:
60148
diff
changeset
|
745 |
then have "wf (S\<^sup>* O R O S\<^sup>*)" |
|
866f41a869e6
New WF theorem by Tjark Weber. Replaced the proof of the subsequent theorem.
paulson <lp15@cam.ac.uk>
parents:
60148
diff
changeset
|
746 |
by (simp add: assms qc_wf_relto_iff) |
|
866f41a869e6
New WF theorem by Tjark Weber. Replaced the proof of the subsequent theorem.
paulson <lp15@cam.ac.uk>
parents:
60148
diff
changeset
|
747 |
then show ?thesis |
|
866f41a869e6
New WF theorem by Tjark Weber. Replaced the proof of the subsequent theorem.
paulson <lp15@cam.ac.uk>
parents:
60148
diff
changeset
|
748 |
by (rule Wellfounded.wf_subset) blast |
| 60148 | 749 |
qed |
750 |
||
751 |
||
| 60758 | 752 |
subsection \<open>Acyclic relations\<close> |
| 33217 | 753 |
|
| 63108 | 754 |
lemma wf_acyclic: "wf r \<Longrightarrow> acyclic r" |
| 63572 | 755 |
by (simp add: acyclic_def) (blast elim: wf_trancl [THEN wf_irrefl]) |
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
756 |
|
| 80322 | 757 |
lemmas wfp_acyclicP = wf_acyclic [to_pred] |
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
758 |
|
| 63108 | 759 |
|
760 |
subsubsection \<open>Wellfoundedness of finite acyclic relations\<close> |
|
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
761 |
|
| 68646 | 762 |
lemma finite_acyclic_wf: |
763 |
assumes "finite r" "acyclic r" shows "wf r" |
|
764 |
using assms |
|
765 |
proof (induction r rule: finite_induct) |
|
766 |
case (insert x r) |
|
767 |
then show ?case |
|
768 |
by (cases x) simp |
|
769 |
qed simp |
|
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
770 |
|
| 63108 | 771 |
lemma finite_acyclic_wf_converse: "finite r \<Longrightarrow> acyclic r \<Longrightarrow> wf (r\<inverse>)" |
| 63572 | 772 |
apply (erule finite_converse [THEN iffD2, THEN finite_acyclic_wf]) |
773 |
apply (erule acyclic_converse [THEN iffD2]) |
|
774 |
done |
|
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
775 |
|
|
63088
f2177f5d2aed
a quasi-recursive characterization of the multiset order (by Christian Sternagel)
haftmann
parents:
61952
diff
changeset
|
776 |
text \<open> |
|
f2177f5d2aed
a quasi-recursive characterization of the multiset order (by Christian Sternagel)
haftmann
parents:
61952
diff
changeset
|
777 |
Observe that the converse of an irreflexive, transitive, |
|
f2177f5d2aed
a quasi-recursive characterization of the multiset order (by Christian Sternagel)
haftmann
parents:
61952
diff
changeset
|
778 |
and finite relation is again well-founded. Thus, we may |
|
f2177f5d2aed
a quasi-recursive characterization of the multiset order (by Christian Sternagel)
haftmann
parents:
61952
diff
changeset
|
779 |
employ it for well-founded induction. |
|
f2177f5d2aed
a quasi-recursive characterization of the multiset order (by Christian Sternagel)
haftmann
parents:
61952
diff
changeset
|
780 |
\<close> |
|
f2177f5d2aed
a quasi-recursive characterization of the multiset order (by Christian Sternagel)
haftmann
parents:
61952
diff
changeset
|
781 |
lemma wf_converse: |
|
f2177f5d2aed
a quasi-recursive characterization of the multiset order (by Christian Sternagel)
haftmann
parents:
61952
diff
changeset
|
782 |
assumes "irrefl r" and "trans r" and "finite r" |
|
f2177f5d2aed
a quasi-recursive characterization of the multiset order (by Christian Sternagel)
haftmann
parents:
61952
diff
changeset
|
783 |
shows "wf (r\<inverse>)" |
|
f2177f5d2aed
a quasi-recursive characterization of the multiset order (by Christian Sternagel)
haftmann
parents:
61952
diff
changeset
|
784 |
proof - |
|
f2177f5d2aed
a quasi-recursive characterization of the multiset order (by Christian Sternagel)
haftmann
parents:
61952
diff
changeset
|
785 |
have "acyclic r" |
| 63572 | 786 |
using \<open>irrefl r\<close> and \<open>trans r\<close> |
787 |
by (simp add: irrefl_def acyclic_irrefl) |
|
788 |
with \<open>finite r\<close> show ?thesis |
|
789 |
by (rule finite_acyclic_wf_converse) |
|
|
63088
f2177f5d2aed
a quasi-recursive characterization of the multiset order (by Christian Sternagel)
haftmann
parents:
61952
diff
changeset
|
790 |
qed |
|
f2177f5d2aed
a quasi-recursive characterization of the multiset order (by Christian Sternagel)
haftmann
parents:
61952
diff
changeset
|
791 |
|
| 63108 | 792 |
lemma wf_iff_acyclic_if_finite: "finite r \<Longrightarrow> wf r = acyclic r" |
| 63572 | 793 |
by (blast intro: finite_acyclic_wf wf_acyclic) |
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
794 |
|
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
795 |
|
| 69593 | 796 |
subsection \<open>\<^typ>\<open>nat\<close> is well-founded\<close> |
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
797 |
|
| 67399 | 798 |
lemma less_nat_rel: "(<) = (\<lambda>m n. n = Suc m)\<^sup>+\<^sup>+" |
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
799 |
proof (rule ext, rule ext, rule iffI) |
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
800 |
fix n m :: nat |
| 63108 | 801 |
show "(\<lambda>m n. n = Suc m)\<^sup>+\<^sup>+ m n" if "m < n" |
802 |
using that |
|
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
803 |
proof (induct n) |
| 63108 | 804 |
case 0 |
805 |
then show ?case by auto |
|
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
806 |
next |
| 63108 | 807 |
case (Suc n) |
808 |
then show ?case |
|
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
809 |
by (auto simp add: less_Suc_eq_le le_less intro: tranclp.trancl_into_trancl) |
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
810 |
qed |
| 63108 | 811 |
show "m < n" if "(\<lambda>m n. n = Suc m)\<^sup>+\<^sup>+ m n" |
812 |
using that by (induct n) (simp_all add: less_Suc_eq_le reflexive le_less) |
|
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
813 |
qed |
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
814 |
|
| 63108 | 815 |
definition pred_nat :: "(nat \<times> nat) set" |
816 |
where "pred_nat = {(m, n). n = Suc m}"
|
|
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
817 |
|
| 63108 | 818 |
definition less_than :: "(nat \<times> nat) set" |
819 |
where "less_than = pred_nat\<^sup>+" |
|
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
820 |
|
| 63108 | 821 |
lemma less_eq: "(m, n) \<in> pred_nat\<^sup>+ \<longleftrightarrow> m < n" |
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
822 |
unfolding less_nat_rel pred_nat_def trancl_def by simp |
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
823 |
|
| 63108 | 824 |
lemma pred_nat_trancl_eq_le: "(m, n) \<in> pred_nat\<^sup>* \<longleftrightarrow> m \<le> n" |
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
825 |
unfolding less_eq rtrancl_eq_or_trancl by auto |
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
826 |
|
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
827 |
lemma wf_pred_nat: "wf pred_nat" |
|
75669
43f5dfb7fa35
tuned (some HOL lints, by Yecine Megdiche);
Fabian Huch <huch@in.tum.de>
parents:
74971
diff
changeset
|
828 |
unfolding wf_def |
|
43f5dfb7fa35
tuned (some HOL lints, by Yecine Megdiche);
Fabian Huch <huch@in.tum.de>
parents:
74971
diff
changeset
|
829 |
proof clarify |
|
43f5dfb7fa35
tuned (some HOL lints, by Yecine Megdiche);
Fabian Huch <huch@in.tum.de>
parents:
74971
diff
changeset
|
830 |
fix P x |
|
43f5dfb7fa35
tuned (some HOL lints, by Yecine Megdiche);
Fabian Huch <huch@in.tum.de>
parents:
74971
diff
changeset
|
831 |
assume "\<forall>x'. (\<forall>y. (y, x') \<in> pred_nat \<longrightarrow> P y) \<longrightarrow> P x'" |
|
43f5dfb7fa35
tuned (some HOL lints, by Yecine Megdiche);
Fabian Huch <huch@in.tum.de>
parents:
74971
diff
changeset
|
832 |
then show "P x" |
|
43f5dfb7fa35
tuned (some HOL lints, by Yecine Megdiche);
Fabian Huch <huch@in.tum.de>
parents:
74971
diff
changeset
|
833 |
unfolding pred_nat_def by (induction x) blast+ |
|
43f5dfb7fa35
tuned (some HOL lints, by Yecine Megdiche);
Fabian Huch <huch@in.tum.de>
parents:
74971
diff
changeset
|
834 |
qed |
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
835 |
|
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
836 |
lemma wf_less_than [iff]: "wf less_than" |
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
837 |
by (simp add: less_than_def wf_pred_nat [THEN wf_trancl]) |
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
838 |
|
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
839 |
lemma trans_less_than [iff]: "trans less_than" |
| 35216 | 840 |
by (simp add: less_than_def) |
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
841 |
|
| 63108 | 842 |
lemma less_than_iff [iff]: "((x,y) \<in> less_than) = (x<y)" |
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
843 |
by (simp add: less_than_def less_eq) |
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
844 |
|
| 71827 | 845 |
lemma irrefl_less_than: "irrefl less_than" |
846 |
using irrefl_def by blast |
|
847 |
||
|
71935
82b00b8f1871
fixed the utterly weird definitions of asym / asymp, and added many asym lemmas
paulson <lp15@cam.ac.uk>
parents:
71827
diff
changeset
|
848 |
lemma asym_less_than: "asym less_than" |
|
76682
e260dabc88e6
added predicates asym_on and asymp_on and redefined asym and asymp to be abbreviations
desharna
parents:
76588
diff
changeset
|
849 |
by (rule asymI) simp |
|
71935
82b00b8f1871
fixed the utterly weird definitions of asym / asymp, and added many asym lemmas
paulson <lp15@cam.ac.uk>
parents:
71827
diff
changeset
|
850 |
|
|
71766
1249b998e377
New theory Library/List_Lenlexorder.thy, a type class instantiation for well-ordering lists
paulson <lp15@cam.ac.uk>
parents:
71544
diff
changeset
|
851 |
lemma total_less_than: "total less_than" and total_on_less_than [simp]: "total_on A less_than" |
|
1249b998e377
New theory Library/List_Lenlexorder.thy, a type class instantiation for well-ordering lists
paulson <lp15@cam.ac.uk>
parents:
71544
diff
changeset
|
852 |
using total_on_def by force+ |
|
71404
f2b783abfbe7
A few lemmas connected with orderings
paulson <lp15@cam.ac.uk>
parents:
69593
diff
changeset
|
853 |
|
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
854 |
lemma wf_less: "wf {(x, y::nat). x < y}"
|
|
60493
866f41a869e6
New WF theorem by Tjark Weber. Replaced the proof of the subsequent theorem.
paulson <lp15@cam.ac.uk>
parents:
60148
diff
changeset
|
855 |
by (rule Wellfounded.wellorder_class.wf) |
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
856 |
|
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
857 |
|
| 60758 | 858 |
subsection \<open>Accessible Part\<close> |
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
859 |
|
| 60758 | 860 |
text \<open> |
| 63108 | 861 |
Inductive definition of the accessible part \<open>acc r\<close> of a |
| 77172 | 862 |
relation; see also \<^cite>\<open>"paulin-tlca"\<close>. |
| 60758 | 863 |
\<close> |
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
864 |
|
| 63108 | 865 |
inductive_set acc :: "('a \<times> 'a) set \<Rightarrow> 'a set" for r :: "('a \<times> 'a) set"
|
866 |
where accI: "(\<And>y. (y, x) \<in> r \<Longrightarrow> y \<in> acc r) \<Longrightarrow> x \<in> acc r" |
|
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
867 |
|
| 63108 | 868 |
abbreviation termip :: "('a \<Rightarrow> 'a \<Rightarrow> bool) \<Rightarrow> 'a \<Rightarrow> bool"
|
869 |
where "termip r \<equiv> accp (r\<inverse>\<inverse>)" |
|
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
870 |
|
| 63108 | 871 |
abbreviation termi :: "('a \<times> 'a) set \<Rightarrow> 'a set"
|
872 |
where "termi r \<equiv> acc (r\<inverse>)" |
|
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
873 |
|
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
874 |
lemmas accpI = accp.accI |
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
875 |
|
| 63108 | 876 |
lemma accp_eq_acc [code]: "accp r = (\<lambda>x. x \<in> Wellfounded.acc {(x, y). r x y})"
|
| 54295 | 877 |
by (simp add: acc_def) |
878 |
||
879 |
||
| 60758 | 880 |
text \<open>Induction rules\<close> |
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
881 |
|
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
882 |
theorem accp_induct: |
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
883 |
assumes major: "accp r a" |
| 63108 | 884 |
assumes hyp: "\<And>x. accp r x \<Longrightarrow> \<forall>y. r y x \<longrightarrow> P y \<Longrightarrow> P x" |
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
885 |
shows "P a" |
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
886 |
apply (rule major [THEN accp.induct]) |
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
887 |
apply (rule hyp) |
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
888 |
apply (rule accp.accI) |
| 68646 | 889 |
apply auto |
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
890 |
done |
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
891 |
|
| 61337 | 892 |
lemmas accp_induct_rule = accp_induct [rule_format, induct set: accp] |
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
893 |
|
| 63108 | 894 |
theorem accp_downward: "accp r b \<Longrightarrow> r a b \<Longrightarrow> accp r a" |
| 63572 | 895 |
by (cases rule: accp.cases) |
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
896 |
|
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
897 |
lemma not_accp_down: |
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
898 |
assumes na: "\<not> accp R x" |
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
899 |
obtains z where "R z x" and "\<not> accp R z" |
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
900 |
proof - |
| 63572 | 901 |
assume a: "\<And>z. R z x \<Longrightarrow> \<not> accp R z \<Longrightarrow> thesis" |
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
902 |
show thesis |
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
903 |
proof (cases "\<forall>z. R z x \<longrightarrow> accp R z") |
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
904 |
case True |
| 63108 | 905 |
then have "\<And>z. R z x \<Longrightarrow> accp R z" by auto |
906 |
then have "accp R x" by (rule accp.accI) |
|
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
907 |
with na show thesis .. |
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
908 |
next |
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
909 |
case False then obtain z where "R z x" and "\<not> accp R z" |
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
910 |
by auto |
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
911 |
with a show thesis . |
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
912 |
qed |
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
913 |
qed |
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
914 |
|
| 63108 | 915 |
lemma accp_downwards_aux: "r\<^sup>*\<^sup>* b a \<Longrightarrow> accp r a \<longrightarrow> accp r b" |
| 63612 | 916 |
by (erule rtranclp_induct) (blast dest: accp_downward)+ |
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
917 |
|
| 63108 | 918 |
theorem accp_downwards: "accp r a \<Longrightarrow> r\<^sup>*\<^sup>* b a \<Longrightarrow> accp r b" |
| 63572 | 919 |
by (blast dest: accp_downwards_aux) |
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
920 |
|
| 80321 | 921 |
theorem accp_wfpI: "\<forall>x. accp r x \<Longrightarrow> wfp r" |
| 80322 | 922 |
proof (rule wfpUNIVI) |
|
75669
43f5dfb7fa35
tuned (some HOL lints, by Yecine Megdiche);
Fabian Huch <huch@in.tum.de>
parents:
74971
diff
changeset
|
923 |
fix P x |
|
43f5dfb7fa35
tuned (some HOL lints, by Yecine Megdiche);
Fabian Huch <huch@in.tum.de>
parents:
74971
diff
changeset
|
924 |
assume "\<forall>x. accp r x" "\<forall>x. (\<forall>y. r y x \<longrightarrow> P y) \<longrightarrow> P x" |
|
43f5dfb7fa35
tuned (some HOL lints, by Yecine Megdiche);
Fabian Huch <huch@in.tum.de>
parents:
74971
diff
changeset
|
925 |
then show "P x" |
|
43f5dfb7fa35
tuned (some HOL lints, by Yecine Megdiche);
Fabian Huch <huch@in.tum.de>
parents:
74971
diff
changeset
|
926 |
using accp_induct[where P = P] by blast |
|
43f5dfb7fa35
tuned (some HOL lints, by Yecine Megdiche);
Fabian Huch <huch@in.tum.de>
parents:
74971
diff
changeset
|
927 |
qed |
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
928 |
|
| 80321 | 929 |
theorem accp_wfpD: "wfp r \<Longrightarrow> accp r x" |
| 80322 | 930 |
apply (erule wfp_induct_rule) |
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
931 |
apply (rule accp.accI) |
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
932 |
apply blast |
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
933 |
done |
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
934 |
|
| 80316 | 935 |
theorem wfp_iff_accp: "wfp r = (\<forall>x. accp r x)" |
| 80321 | 936 |
by (blast intro: accp_wfpI dest: accp_wfpD) |
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
937 |
|
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
938 |
|
| 60758 | 939 |
text \<open>Smaller relations have bigger accessible parts:\<close> |
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
940 |
|
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
941 |
lemma accp_subset: |
| 63572 | 942 |
assumes "R1 \<le> R2" |
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
943 |
shows "accp R2 \<le> accp R1" |
|
26803
0af0f674845d
- Explicitely passed pred_subset_eq and pred_equals_eq as an argument to the
berghofe
parents:
26748
diff
changeset
|
944 |
proof (rule predicate1I) |
| 63572 | 945 |
fix x |
946 |
assume "accp R2 x" |
|
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
947 |
then show "accp R1 x" |
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
948 |
proof (induct x) |
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
949 |
fix x |
| 63572 | 950 |
assume "\<And>y. R2 y x \<Longrightarrow> accp R1 y" |
951 |
with assms show "accp R1 x" |
|
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
952 |
by (blast intro: accp.accI) |
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
953 |
qed |
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
954 |
qed |
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
955 |
|
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
956 |
|
| 60758 | 957 |
text \<open>This is a generalized induction theorem that works on |
958 |
subsets of the accessible part.\<close> |
|
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
959 |
|
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
960 |
lemma accp_subset_induct: |
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
961 |
assumes subset: "D \<le> accp R" |
| 63572 | 962 |
and dcl: "\<And>x z. D x \<Longrightarrow> R z x \<Longrightarrow> D z" |
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
963 |
and "D x" |
| 63572 | 964 |
and istep: "\<And>x. D x \<Longrightarrow> (\<And>z. R z x \<Longrightarrow> P z) \<Longrightarrow> P x" |
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
965 |
shows "P x" |
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
966 |
proof - |
| 60758 | 967 |
from subset and \<open>D x\<close> |
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
968 |
have "accp R x" .. |
| 60758 | 969 |
then show "P x" using \<open>D x\<close> |
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
970 |
proof (induct x) |
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
971 |
fix x |
| 63572 | 972 |
assume "D x" and "\<And>y. R y x \<Longrightarrow> D y \<Longrightarrow> P y" |
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
973 |
with dcl and istep show "P x" by blast |
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
974 |
qed |
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
975 |
qed |
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
976 |
|
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
977 |
|
| 60758 | 978 |
text \<open>Set versions of the above theorems\<close> |
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
979 |
|
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
980 |
lemmas acc_induct = accp_induct [to_set] |
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
981 |
lemmas acc_induct_rule = acc_induct [rule_format, induct set: acc] |
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
982 |
lemmas acc_downward = accp_downward [to_set] |
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
983 |
lemmas not_acc_down = not_accp_down [to_set] |
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
984 |
lemmas acc_downwards_aux = accp_downwards_aux [to_set] |
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
985 |
lemmas acc_downwards = accp_downwards [to_set] |
| 80321 | 986 |
lemmas acc_wfI = accp_wfpI [to_set] |
987 |
lemmas acc_wfD = accp_wfpD [to_set] |
|
| 80316 | 988 |
lemmas wf_iff_acc = wfp_iff_accp [to_set] |
|
46177
adac34829e10
pred_subset_eq and SUP_UN_eq2 are now standard pred_set_conv rules
berghofe
parents:
45970
diff
changeset
|
989 |
lemmas acc_subset = accp_subset [to_set] |
|
adac34829e10
pred_subset_eq and SUP_UN_eq2 are now standard pred_set_conv rules
berghofe
parents:
45970
diff
changeset
|
990 |
lemmas acc_subset_induct = accp_subset_induct [to_set] |
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
991 |
|
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
992 |
|
| 60758 | 993 |
subsection \<open>Tools for building wellfounded relations\<close> |
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
994 |
|
| 60758 | 995 |
text \<open>Inverse Image\<close> |
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
996 |
|
| 71544 | 997 |
lemma wf_inv_image [simp,intro!]: |
998 |
fixes f :: "'a \<Rightarrow> 'b" |
|
999 |
assumes "wf r" |
|
1000 |
shows "wf (inv_image r f)" |
|
|
75669
43f5dfb7fa35
tuned (some HOL lints, by Yecine Megdiche);
Fabian Huch <huch@in.tum.de>
parents:
74971
diff
changeset
|
1001 |
proof - |
|
43f5dfb7fa35
tuned (some HOL lints, by Yecine Megdiche);
Fabian Huch <huch@in.tum.de>
parents:
74971
diff
changeset
|
1002 |
have "\<And>x P. x \<in> P \<Longrightarrow> \<exists>z\<in>P. \<forall>y. (f y, f z) \<in> r \<longrightarrow> y \<notin> P" |
|
43f5dfb7fa35
tuned (some HOL lints, by Yecine Megdiche);
Fabian Huch <huch@in.tum.de>
parents:
74971
diff
changeset
|
1003 |
proof - |
|
43f5dfb7fa35
tuned (some HOL lints, by Yecine Megdiche);
Fabian Huch <huch@in.tum.de>
parents:
74971
diff
changeset
|
1004 |
fix P and x::'a |
|
43f5dfb7fa35
tuned (some HOL lints, by Yecine Megdiche);
Fabian Huch <huch@in.tum.de>
parents:
74971
diff
changeset
|
1005 |
assume "x \<in> P" |
|
43f5dfb7fa35
tuned (some HOL lints, by Yecine Megdiche);
Fabian Huch <huch@in.tum.de>
parents:
74971
diff
changeset
|
1006 |
then obtain w where w: "w \<in> {w. \<exists>x::'a. x \<in> P \<and> f x = w}"
|
|
43f5dfb7fa35
tuned (some HOL lints, by Yecine Megdiche);
Fabian Huch <huch@in.tum.de>
parents:
74971
diff
changeset
|
1007 |
by auto |
|
43f5dfb7fa35
tuned (some HOL lints, by Yecine Megdiche);
Fabian Huch <huch@in.tum.de>
parents:
74971
diff
changeset
|
1008 |
have *: "\<And>Q u. u \<in> Q \<Longrightarrow> \<exists>z\<in>Q. \<forall>y. (y, z) \<in> r \<longrightarrow> y \<notin> Q" |
|
43f5dfb7fa35
tuned (some HOL lints, by Yecine Megdiche);
Fabian Huch <huch@in.tum.de>
parents:
74971
diff
changeset
|
1009 |
using assms by (auto simp add: wf_eq_minimal) |
|
43f5dfb7fa35
tuned (some HOL lints, by Yecine Megdiche);
Fabian Huch <huch@in.tum.de>
parents:
74971
diff
changeset
|
1010 |
show "\<exists>z\<in>P. \<forall>y. (f y, f z) \<in> r \<longrightarrow> y \<notin> P" |
|
43f5dfb7fa35
tuned (some HOL lints, by Yecine Megdiche);
Fabian Huch <huch@in.tum.de>
parents:
74971
diff
changeset
|
1011 |
using * [OF w] by auto |
|
43f5dfb7fa35
tuned (some HOL lints, by Yecine Megdiche);
Fabian Huch <huch@in.tum.de>
parents:
74971
diff
changeset
|
1012 |
qed |
|
43f5dfb7fa35
tuned (some HOL lints, by Yecine Megdiche);
Fabian Huch <huch@in.tum.de>
parents:
74971
diff
changeset
|
1013 |
then show ?thesis |
|
43f5dfb7fa35
tuned (some HOL lints, by Yecine Megdiche);
Fabian Huch <huch@in.tum.de>
parents:
74971
diff
changeset
|
1014 |
by (clarsimp simp: inv_image_def wf_eq_minimal) |
| 71544 | 1015 |
qed |
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
1016 |
|
|
79999
dca9c237d108
added lemmas wfp_on_inv_imagep, wfp_on_if_convertible_to_wfp_on, and wf_on_if_convertible_to_wf_on
desharna
parents:
79997
diff
changeset
|
1017 |
lemma wfp_on_inv_imagep: |
|
dca9c237d108
added lemmas wfp_on_inv_imagep, wfp_on_if_convertible_to_wfp_on, and wf_on_if_convertible_to_wf_on
desharna
parents:
79997
diff
changeset
|
1018 |
assumes wf: "wfp_on (f ` A) R" |
|
dca9c237d108
added lemmas wfp_on_inv_imagep, wfp_on_if_convertible_to_wfp_on, and wf_on_if_convertible_to_wf_on
desharna
parents:
79997
diff
changeset
|
1019 |
shows "wfp_on A (inv_imagep R f)" |
|
dca9c237d108
added lemmas wfp_on_inv_imagep, wfp_on_if_convertible_to_wfp_on, and wf_on_if_convertible_to_wf_on
desharna
parents:
79997
diff
changeset
|
1020 |
unfolding wfp_on_iff_ex_minimal |
|
dca9c237d108
added lemmas wfp_on_inv_imagep, wfp_on_if_convertible_to_wfp_on, and wf_on_if_convertible_to_wf_on
desharna
parents:
79997
diff
changeset
|
1021 |
proof (intro allI impI) |
|
dca9c237d108
added lemmas wfp_on_inv_imagep, wfp_on_if_convertible_to_wfp_on, and wf_on_if_convertible_to_wf_on
desharna
parents:
79997
diff
changeset
|
1022 |
fix B assume "B \<subseteq> A" and "B \<noteq> {}"
|
|
dca9c237d108
added lemmas wfp_on_inv_imagep, wfp_on_if_convertible_to_wfp_on, and wf_on_if_convertible_to_wf_on
desharna
parents:
79997
diff
changeset
|
1023 |
hence "\<exists>z\<in>f ` B. \<forall>y. R y z \<longrightarrow> y \<notin> f ` B" |
|
dca9c237d108
added lemmas wfp_on_inv_imagep, wfp_on_if_convertible_to_wfp_on, and wf_on_if_convertible_to_wf_on
desharna
parents:
79997
diff
changeset
|
1024 |
using wf[unfolded wfp_on_iff_ex_minimal, rule_format, of "f ` B"] by blast |
|
dca9c237d108
added lemmas wfp_on_inv_imagep, wfp_on_if_convertible_to_wfp_on, and wf_on_if_convertible_to_wf_on
desharna
parents:
79997
diff
changeset
|
1025 |
thus "\<exists>z\<in>B. \<forall>y. inv_imagep R f y z \<longrightarrow> y \<notin> B" |
|
dca9c237d108
added lemmas wfp_on_inv_imagep, wfp_on_if_convertible_to_wfp_on, and wf_on_if_convertible_to_wf_on
desharna
parents:
79997
diff
changeset
|
1026 |
unfolding inv_imagep_def |
|
dca9c237d108
added lemmas wfp_on_inv_imagep, wfp_on_if_convertible_to_wfp_on, and wf_on_if_convertible_to_wf_on
desharna
parents:
79997
diff
changeset
|
1027 |
by auto |
|
dca9c237d108
added lemmas wfp_on_inv_imagep, wfp_on_if_convertible_to_wfp_on, and wf_on_if_convertible_to_wf_on
desharna
parents:
79997
diff
changeset
|
1028 |
qed |
|
dca9c237d108
added lemmas wfp_on_inv_imagep, wfp_on_if_convertible_to_wfp_on, and wf_on_if_convertible_to_wf_on
desharna
parents:
79997
diff
changeset
|
1029 |
|
|
76267
5ea1f8bfb795
added lemmas wf_if_convertible_to_wf, wfP_if_convertible_to_wfP, and wfP_if_convertible_to_nat
desharna
parents:
75669
diff
changeset
|
1030 |
|
|
5ea1f8bfb795
added lemmas wf_if_convertible_to_wf, wfP_if_convertible_to_wfP, and wfP_if_convertible_to_nat
desharna
parents:
75669
diff
changeset
|
1031 |
subsubsection \<open>Conversion to a known well-founded relation\<close> |
|
5ea1f8bfb795
added lemmas wf_if_convertible_to_wf, wfP_if_convertible_to_wfP, and wfP_if_convertible_to_nat
desharna
parents:
75669
diff
changeset
|
1032 |
|
|
79999
dca9c237d108
added lemmas wfp_on_inv_imagep, wfp_on_if_convertible_to_wfp_on, and wf_on_if_convertible_to_wf_on
desharna
parents:
79997
diff
changeset
|
1033 |
lemma wfp_on_if_convertible_to_wfp_on: |
|
dca9c237d108
added lemmas wfp_on_inv_imagep, wfp_on_if_convertible_to_wfp_on, and wf_on_if_convertible_to_wf_on
desharna
parents:
79997
diff
changeset
|
1034 |
assumes |
|
dca9c237d108
added lemmas wfp_on_inv_imagep, wfp_on_if_convertible_to_wfp_on, and wf_on_if_convertible_to_wf_on
desharna
parents:
79997
diff
changeset
|
1035 |
wf: "wfp_on (f ` A) Q" and |
|
dca9c237d108
added lemmas wfp_on_inv_imagep, wfp_on_if_convertible_to_wfp_on, and wf_on_if_convertible_to_wf_on
desharna
parents:
79997
diff
changeset
|
1036 |
convertible: "(\<And>x y. x \<in> A \<Longrightarrow> y \<in> A \<Longrightarrow> R x y \<Longrightarrow> Q (f x) (f y))" |
|
dca9c237d108
added lemmas wfp_on_inv_imagep, wfp_on_if_convertible_to_wfp_on, and wf_on_if_convertible_to_wf_on
desharna
parents:
79997
diff
changeset
|
1037 |
shows "wfp_on A R" |
|
dca9c237d108
added lemmas wfp_on_inv_imagep, wfp_on_if_convertible_to_wfp_on, and wf_on_if_convertible_to_wf_on
desharna
parents:
79997
diff
changeset
|
1038 |
unfolding wfp_on_iff_ex_minimal |
|
dca9c237d108
added lemmas wfp_on_inv_imagep, wfp_on_if_convertible_to_wfp_on, and wf_on_if_convertible_to_wf_on
desharna
parents:
79997
diff
changeset
|
1039 |
proof (intro allI impI) |
|
dca9c237d108
added lemmas wfp_on_inv_imagep, wfp_on_if_convertible_to_wfp_on, and wf_on_if_convertible_to_wf_on
desharna
parents:
79997
diff
changeset
|
1040 |
fix B assume "B \<subseteq> A" and "B \<noteq> {}"
|
|
dca9c237d108
added lemmas wfp_on_inv_imagep, wfp_on_if_convertible_to_wfp_on, and wf_on_if_convertible_to_wf_on
desharna
parents:
79997
diff
changeset
|
1041 |
moreover from wf have "wfp_on A (inv_imagep Q f)" |
|
dca9c237d108
added lemmas wfp_on_inv_imagep, wfp_on_if_convertible_to_wfp_on, and wf_on_if_convertible_to_wf_on
desharna
parents:
79997
diff
changeset
|
1042 |
by (rule wfp_on_inv_imagep) |
|
dca9c237d108
added lemmas wfp_on_inv_imagep, wfp_on_if_convertible_to_wfp_on, and wf_on_if_convertible_to_wf_on
desharna
parents:
79997
diff
changeset
|
1043 |
ultimately obtain y where "y \<in> B" and "\<And>z. Q (f z) (f y) \<Longrightarrow> z \<notin> B" |
|
dca9c237d108
added lemmas wfp_on_inv_imagep, wfp_on_if_convertible_to_wfp_on, and wf_on_if_convertible_to_wf_on
desharna
parents:
79997
diff
changeset
|
1044 |
unfolding wfp_on_iff_ex_minimal in_inv_imagep |
|
dca9c237d108
added lemmas wfp_on_inv_imagep, wfp_on_if_convertible_to_wfp_on, and wf_on_if_convertible_to_wf_on
desharna
parents:
79997
diff
changeset
|
1045 |
by blast |
|
dca9c237d108
added lemmas wfp_on_inv_imagep, wfp_on_if_convertible_to_wfp_on, and wf_on_if_convertible_to_wf_on
desharna
parents:
79997
diff
changeset
|
1046 |
thus "\<exists>z \<in> B. \<forall>y. R y z \<longrightarrow> y \<notin> B" |
|
dca9c237d108
added lemmas wfp_on_inv_imagep, wfp_on_if_convertible_to_wfp_on, and wf_on_if_convertible_to_wf_on
desharna
parents:
79997
diff
changeset
|
1047 |
using \<open>B \<subseteq> A\<close> convertible by blast |
|
dca9c237d108
added lemmas wfp_on_inv_imagep, wfp_on_if_convertible_to_wfp_on, and wf_on_if_convertible_to_wf_on
desharna
parents:
79997
diff
changeset
|
1048 |
qed |
|
dca9c237d108
added lemmas wfp_on_inv_imagep, wfp_on_if_convertible_to_wfp_on, and wf_on_if_convertible_to_wf_on
desharna
parents:
79997
diff
changeset
|
1049 |
|
|
dca9c237d108
added lemmas wfp_on_inv_imagep, wfp_on_if_convertible_to_wfp_on, and wf_on_if_convertible_to_wf_on
desharna
parents:
79997
diff
changeset
|
1050 |
lemma wf_on_if_convertible_to_wf_on: "wf_on (f ` A) Q \<Longrightarrow> (\<And>x y. x \<in> A \<Longrightarrow> y \<in> A \<Longrightarrow> (x, y) \<in> R \<Longrightarrow> (f x, f y) \<in> Q) \<Longrightarrow> wf_on A R" |
|
dca9c237d108
added lemmas wfp_on_inv_imagep, wfp_on_if_convertible_to_wfp_on, and wf_on_if_convertible_to_wf_on
desharna
parents:
79997
diff
changeset
|
1051 |
using wfp_on_if_convertible_to_wfp_on[to_set] . |
|
dca9c237d108
added lemmas wfp_on_inv_imagep, wfp_on_if_convertible_to_wfp_on, and wf_on_if_convertible_to_wf_on
desharna
parents:
79997
diff
changeset
|
1052 |
|
|
76267
5ea1f8bfb795
added lemmas wf_if_convertible_to_wf, wfP_if_convertible_to_wfP, and wfP_if_convertible_to_nat
desharna
parents:
75669
diff
changeset
|
1053 |
lemma wf_if_convertible_to_wf: |
|
5ea1f8bfb795
added lemmas wf_if_convertible_to_wf, wfP_if_convertible_to_wfP, and wfP_if_convertible_to_nat
desharna
parents:
75669
diff
changeset
|
1054 |
fixes r :: "'a rel" and s :: "'b rel" and f :: "'a \<Rightarrow> 'b" |
|
5ea1f8bfb795
added lemmas wf_if_convertible_to_wf, wfP_if_convertible_to_wfP, and wfP_if_convertible_to_nat
desharna
parents:
75669
diff
changeset
|
1055 |
assumes "wf s" and convertible: "\<And>x y. (x, y) \<in> r \<Longrightarrow> (f x, f y) \<in> s" |
|
5ea1f8bfb795
added lemmas wf_if_convertible_to_wf, wfP_if_convertible_to_wfP, and wfP_if_convertible_to_nat
desharna
parents:
75669
diff
changeset
|
1056 |
shows "wf r" |
|
79999
dca9c237d108
added lemmas wfp_on_inv_imagep, wfp_on_if_convertible_to_wfp_on, and wf_on_if_convertible_to_wf_on
desharna
parents:
79997
diff
changeset
|
1057 |
proof (rule wf_on_if_convertible_to_wf_on) |
|
dca9c237d108
added lemmas wfp_on_inv_imagep, wfp_on_if_convertible_to_wfp_on, and wf_on_if_convertible_to_wf_on
desharna
parents:
79997
diff
changeset
|
1058 |
show "wf_on (range f) s" |
|
dca9c237d108
added lemmas wfp_on_inv_imagep, wfp_on_if_convertible_to_wfp_on, and wf_on_if_convertible_to_wf_on
desharna
parents:
79997
diff
changeset
|
1059 |
using wf_on_subset[OF \<open>wf s\<close> subset_UNIV] . |
|
dca9c237d108
added lemmas wfp_on_inv_imagep, wfp_on_if_convertible_to_wfp_on, and wf_on_if_convertible_to_wf_on
desharna
parents:
79997
diff
changeset
|
1060 |
next |
|
dca9c237d108
added lemmas wfp_on_inv_imagep, wfp_on_if_convertible_to_wfp_on, and wf_on_if_convertible_to_wf_on
desharna
parents:
79997
diff
changeset
|
1061 |
show "\<And>x y. (x, y) \<in> r \<Longrightarrow> (f x, f y) \<in> s" |
|
dca9c237d108
added lemmas wfp_on_inv_imagep, wfp_on_if_convertible_to_wfp_on, and wf_on_if_convertible_to_wf_on
desharna
parents:
79997
diff
changeset
|
1062 |
using convertible . |
|
76267
5ea1f8bfb795
added lemmas wf_if_convertible_to_wf, wfP_if_convertible_to_wfP, and wfP_if_convertible_to_nat
desharna
parents:
75669
diff
changeset
|
1063 |
qed |
|
5ea1f8bfb795
added lemmas wf_if_convertible_to_wf, wfP_if_convertible_to_wfP, and wfP_if_convertible_to_nat
desharna
parents:
75669
diff
changeset
|
1064 |
|
| 80317 | 1065 |
lemma wfp_if_convertible_to_wfp: "wfp S \<Longrightarrow> (\<And>x y. R x y \<Longrightarrow> S (f x) (f y)) \<Longrightarrow> wfp R" |
|
76267
5ea1f8bfb795
added lemmas wf_if_convertible_to_wf, wfP_if_convertible_to_wfP, and wfP_if_convertible_to_nat
desharna
parents:
75669
diff
changeset
|
1066 |
using wf_if_convertible_to_wf[to_pred, of S R f] by simp |
|
5ea1f8bfb795
added lemmas wf_if_convertible_to_wf, wfP_if_convertible_to_wfP, and wfP_if_convertible_to_nat
desharna
parents:
75669
diff
changeset
|
1067 |
|
|
5ea1f8bfb795
added lemmas wf_if_convertible_to_wf, wfP_if_convertible_to_wfP, and wfP_if_convertible_to_nat
desharna
parents:
75669
diff
changeset
|
1068 |
text \<open>Converting to @{typ nat} is a very common special case that might be found more easily by
|
|
5ea1f8bfb795
added lemmas wf_if_convertible_to_wf, wfP_if_convertible_to_wfP, and wfP_if_convertible_to_nat
desharna
parents:
75669
diff
changeset
|
1069 |
Sledgehammer.\<close> |
|
5ea1f8bfb795
added lemmas wf_if_convertible_to_wf, wfP_if_convertible_to_wfP, and wfP_if_convertible_to_nat
desharna
parents:
75669
diff
changeset
|
1070 |
|
| 80285 | 1071 |
lemma wfp_if_convertible_to_nat: |
|
76267
5ea1f8bfb795
added lemmas wf_if_convertible_to_wf, wfP_if_convertible_to_wfP, and wfP_if_convertible_to_nat
desharna
parents:
75669
diff
changeset
|
1072 |
fixes f :: "_ \<Rightarrow> nat" |
| 80317 | 1073 |
shows "(\<And>x y. R x y \<Longrightarrow> f x < f y) \<Longrightarrow> wfp R" |
| 80285 | 1074 |
by (rule wfp_if_convertible_to_wfp[of "(<) :: nat \<Rightarrow> nat \<Rightarrow> bool", simplified]) |
|
76267
5ea1f8bfb795
added lemmas wf_if_convertible_to_wf, wfP_if_convertible_to_wfP, and wfP_if_convertible_to_nat
desharna
parents:
75669
diff
changeset
|
1075 |
|
|
5ea1f8bfb795
added lemmas wf_if_convertible_to_wf, wfP_if_convertible_to_wfP, and wfP_if_convertible_to_nat
desharna
parents:
75669
diff
changeset
|
1076 |
|
|
5ea1f8bfb795
added lemmas wf_if_convertible_to_wf, wfP_if_convertible_to_wfP, and wfP_if_convertible_to_nat
desharna
parents:
75669
diff
changeset
|
1077 |
subsubsection \<open>Measure functions into \<^typ>\<open>nat\<close>\<close> |
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
1078 |
|
| 63108 | 1079 |
definition measure :: "('a \<Rightarrow> nat) \<Rightarrow> ('a \<times> 'a) set"
|
1080 |
where "measure = inv_image less_than" |
|
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
1081 |
|
| 63108 | 1082 |
lemma in_measure[simp, code_unfold]: "(x, y) \<in> measure f \<longleftrightarrow> f x < f y" |
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
1083 |
by (simp add:measure_def) |
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
1084 |
|
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
1085 |
lemma wf_measure [iff]: "wf (measure f)" |
| 63572 | 1086 |
unfolding measure_def by (rule wf_less_than [THEN wf_inv_image]) |
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
1087 |
|
| 63108 | 1088 |
lemma wf_if_measure: "(\<And>x. P x \<Longrightarrow> f(g x) < f x) \<Longrightarrow> wf {(y,x). P x \<and> y = g x}"
|
1089 |
for f :: "'a \<Rightarrow> nat" |
|
| 68646 | 1090 |
using wf_measure[of f] unfolding measure_def inv_image_def less_than_def less_eq |
1091 |
by (rule wf_subset) auto |
|
| 41720 | 1092 |
|
1093 |
||
| 63108 | 1094 |
subsubsection \<open>Lexicographic combinations\<close> |
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
1095 |
|
| 63108 | 1096 |
definition lex_prod :: "('a \<times>'a) set \<Rightarrow> ('b \<times> 'b) set \<Rightarrow> (('a \<times> 'b) \<times> ('a \<times> 'b)) set"
|
1097 |
(infixr "<*lex*>" 80) |
|
| 72184 | 1098 |
where "ra <*lex*> rb = {((a, b), (a', b')). (a, a') \<in> ra \<or> a = a' \<and> (b, b') \<in> rb}"
|
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
1099 |
|
| 72184 | 1100 |
lemma in_lex_prod[simp]: "((a, b), (a', b')) \<in> r <*lex*> s \<longleftrightarrow> (a, a') \<in> r \<or> a = a' \<and> (b, b') \<in> s" |
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
1101 |
by (auto simp:lex_prod_def) |
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
1102 |
|
| 71410 | 1103 |
lemma wf_lex_prod [intro!]: |
1104 |
assumes "wf ra" "wf rb" |
|
1105 |
shows "wf (ra <*lex*> rb)" |
|
1106 |
proof (rule wfI) |
|
1107 |
fix z :: "'a \<times> 'b" and P |
|
1108 |
assume * [rule_format]: "\<forall>u. (\<forall>v. (v, u) \<in> ra <*lex*> rb \<longrightarrow> P v) \<longrightarrow> P u" |
|
1109 |
obtain x y where zeq: "z = (x,y)" |
|
1110 |
by fastforce |
|
1111 |
have "P(x,y)" using \<open>wf ra\<close> |
|
1112 |
proof (induction x arbitrary: y rule: wf_induct_rule) |
|
1113 |
case (less x) |
|
1114 |
note lessx = less |
|
1115 |
show ?case using \<open>wf rb\<close> less |
|
1116 |
proof (induction y rule: wf_induct_rule) |
|
1117 |
case (less y) |
|
1118 |
show ?case |
|
1119 |
by (force intro: * less.IH lessx) |
|
1120 |
qed |
|
1121 |
qed |
|
1122 |
then show "P z" |
|
1123 |
by (simp add: zeq) |
|
1124 |
qed auto |
|
1125 |
||
| 76698 | 1126 |
lemma refl_lex_prod[simp]: "refl r\<^sub>B \<Longrightarrow> refl (r\<^sub>A <*lex*> r\<^sub>B)" |
1127 |
by (auto intro!: reflI dest: refl_onD) |
|
1128 |
||
|
76694
2f8219460ac9
added lemmas irrefl_on_lex_prod[simp] and irrefl_lex_prod[simp]
desharna
parents:
76682
diff
changeset
|
1129 |
lemma irrefl_on_lex_prod[simp]: |
|
2f8219460ac9
added lemmas irrefl_on_lex_prod[simp] and irrefl_lex_prod[simp]
desharna
parents:
76682
diff
changeset
|
1130 |
"irrefl_on A r\<^sub>A \<Longrightarrow> irrefl_on B r\<^sub>B \<Longrightarrow> irrefl_on (A \<times> B) (r\<^sub>A <*lex*> r\<^sub>B)" |
|
2f8219460ac9
added lemmas irrefl_on_lex_prod[simp] and irrefl_lex_prod[simp]
desharna
parents:
76682
diff
changeset
|
1131 |
by (auto intro!: irrefl_onI dest: irrefl_onD) |
|
2f8219460ac9
added lemmas irrefl_on_lex_prod[simp] and irrefl_lex_prod[simp]
desharna
parents:
76682
diff
changeset
|
1132 |
|
|
2f8219460ac9
added lemmas irrefl_on_lex_prod[simp] and irrefl_lex_prod[simp]
desharna
parents:
76682
diff
changeset
|
1133 |
lemma irrefl_lex_prod[simp]: "irrefl r\<^sub>A \<Longrightarrow> irrefl r\<^sub>B \<Longrightarrow> irrefl (r\<^sub>A <*lex*> r\<^sub>B)" |
|
2f8219460ac9
added lemmas irrefl_on_lex_prod[simp] and irrefl_lex_prod[simp]
desharna
parents:
76682
diff
changeset
|
1134 |
by (rule irrefl_on_lex_prod[of UNIV _ UNIV, unfolded UNIV_Times_UNIV]) |
|
2f8219460ac9
added lemmas irrefl_on_lex_prod[simp] and irrefl_lex_prod[simp]
desharna
parents:
76682
diff
changeset
|
1135 |
|
|
76695
e321569ec7a1
added lemmas sym_on_lex_prod[simp] and sym_lex_prod[simp]
desharna
parents:
76694
diff
changeset
|
1136 |
lemma sym_on_lex_prod[simp]: |
|
e321569ec7a1
added lemmas sym_on_lex_prod[simp] and sym_lex_prod[simp]
desharna
parents:
76694
diff
changeset
|
1137 |
"sym_on A r\<^sub>A \<Longrightarrow> sym_on B r\<^sub>B \<Longrightarrow> sym_on (A \<times> B) (r\<^sub>A <*lex*> r\<^sub>B)" |
|
e321569ec7a1
added lemmas sym_on_lex_prod[simp] and sym_lex_prod[simp]
desharna
parents:
76694
diff
changeset
|
1138 |
by (auto intro!: sym_onI dest: sym_onD) |
|
e321569ec7a1
added lemmas sym_on_lex_prod[simp] and sym_lex_prod[simp]
desharna
parents:
76694
diff
changeset
|
1139 |
|
|
e321569ec7a1
added lemmas sym_on_lex_prod[simp] and sym_lex_prod[simp]
desharna
parents:
76694
diff
changeset
|
1140 |
lemma sym_lex_prod[simp]: |
|
e321569ec7a1
added lemmas sym_on_lex_prod[simp] and sym_lex_prod[simp]
desharna
parents:
76694
diff
changeset
|
1141 |
"sym r\<^sub>A \<Longrightarrow> sym r\<^sub>B \<Longrightarrow> sym (r\<^sub>A <*lex*> r\<^sub>B)" |
|
e321569ec7a1
added lemmas sym_on_lex_prod[simp] and sym_lex_prod[simp]
desharna
parents:
76694
diff
changeset
|
1142 |
by (rule sym_on_lex_prod[of UNIV _ UNIV, unfolded UNIV_Times_UNIV]) |
|
e321569ec7a1
added lemmas sym_on_lex_prod[simp] and sym_lex_prod[simp]
desharna
parents:
76694
diff
changeset
|
1143 |
|
|
76696
b6b7f3caa74a
added lemmas asym_on_lex_prod[simp] and asym_lex_prod[simp]
desharna
parents:
76695
diff
changeset
|
1144 |
lemma asym_on_lex_prod[simp]: |
|
b6b7f3caa74a
added lemmas asym_on_lex_prod[simp] and asym_lex_prod[simp]
desharna
parents:
76695
diff
changeset
|
1145 |
"asym_on A r\<^sub>A \<Longrightarrow> asym_on B r\<^sub>B \<Longrightarrow> asym_on (A \<times> B) (r\<^sub>A <*lex*> r\<^sub>B)" |
|
b6b7f3caa74a
added lemmas asym_on_lex_prod[simp] and asym_lex_prod[simp]
desharna
parents:
76695
diff
changeset
|
1146 |
by (auto intro!: asym_onI dest: asym_onD) |
|
b6b7f3caa74a
added lemmas asym_on_lex_prod[simp] and asym_lex_prod[simp]
desharna
parents:
76695
diff
changeset
|
1147 |
|
|
b6b7f3caa74a
added lemmas asym_on_lex_prod[simp] and asym_lex_prod[simp]
desharna
parents:
76695
diff
changeset
|
1148 |
lemma asym_lex_prod[simp]: |
|
b6b7f3caa74a
added lemmas asym_on_lex_prod[simp] and asym_lex_prod[simp]
desharna
parents:
76695
diff
changeset
|
1149 |
"asym r\<^sub>A \<Longrightarrow> asym r\<^sub>B \<Longrightarrow> asym (r\<^sub>A <*lex*> r\<^sub>B)" |
|
b6b7f3caa74a
added lemmas asym_on_lex_prod[simp] and asym_lex_prod[simp]
desharna
parents:
76695
diff
changeset
|
1150 |
by (rule asym_on_lex_prod[of UNIV _ UNIV, unfolded UNIV_Times_UNIV]) |
|
b6b7f3caa74a
added lemmas asym_on_lex_prod[simp] and asym_lex_prod[simp]
desharna
parents:
76695
diff
changeset
|
1151 |
|
| 76753 | 1152 |
lemma trans_on_lex_prod[simp]: |
1153 |
assumes "trans_on A r\<^sub>A" and "trans_on B r\<^sub>B" |
|
1154 |
shows "trans_on (A \<times> B) (r\<^sub>A <*lex*> r\<^sub>B)" |
|
1155 |
proof (rule trans_onI) |
|
1156 |
fix x y z |
|
1157 |
show "x \<in> A \<times> B \<Longrightarrow> y \<in> A \<times> B \<Longrightarrow> z \<in> A \<times> B \<Longrightarrow> |
|
1158 |
(x, y) \<in> r\<^sub>A <*lex*> r\<^sub>B \<Longrightarrow> (y, z) \<in> r\<^sub>A <*lex*> r\<^sub>B \<Longrightarrow> (x, z) \<in> r\<^sub>A <*lex*> r\<^sub>B" |
|
1159 |
using trans_onD[OF \<open>trans_on A r\<^sub>A\<close>, of "fst x" "fst y" "fst z"] |
|
1160 |
using trans_onD[OF \<open>trans_on B r\<^sub>B\<close>, of "snd x" "snd y" "snd z"] |
|
1161 |
by auto |
|
1162 |
qed |
|
1163 |
||
1164 |
lemma trans_lex_prod [simp,intro!]: "trans r\<^sub>A \<Longrightarrow> trans r\<^sub>B \<Longrightarrow> trans (r\<^sub>A <*lex*> r\<^sub>B)" |
|
1165 |
by (rule trans_on_lex_prod[of UNIV _ UNIV, unfolded UNIV_Times_UNIV]) |
|
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
1166 |
|
|
76694
2f8219460ac9
added lemmas irrefl_on_lex_prod[simp] and irrefl_lex_prod[simp]
desharna
parents:
76682
diff
changeset
|
1167 |
lemma total_on_lex_prod[simp]: |
|
2f8219460ac9
added lemmas irrefl_on_lex_prod[simp] and irrefl_lex_prod[simp]
desharna
parents:
76682
diff
changeset
|
1168 |
"total_on A r\<^sub>A \<Longrightarrow> total_on B r\<^sub>B \<Longrightarrow> total_on (A \<times> B) (r\<^sub>A <*lex*> r\<^sub>B)" |
|
71404
f2b783abfbe7
A few lemmas connected with orderings
paulson <lp15@cam.ac.uk>
parents:
69593
diff
changeset
|
1169 |
by (auto simp: total_on_def) |
|
f2b783abfbe7
A few lemmas connected with orderings
paulson <lp15@cam.ac.uk>
parents:
69593
diff
changeset
|
1170 |
|
|
76694
2f8219460ac9
added lemmas irrefl_on_lex_prod[simp] and irrefl_lex_prod[simp]
desharna
parents:
76682
diff
changeset
|
1171 |
lemma total_lex_prod[simp]: "total r\<^sub>A \<Longrightarrow> total r\<^sub>B \<Longrightarrow> total (r\<^sub>A <*lex*> r\<^sub>B)" |
|
2f8219460ac9
added lemmas irrefl_on_lex_prod[simp] and irrefl_lex_prod[simp]
desharna
parents:
76682
diff
changeset
|
1172 |
by (rule total_on_lex_prod[of UNIV _ UNIV, unfolded UNIV_Times_UNIV]) |
|
2f8219460ac9
added lemmas irrefl_on_lex_prod[simp] and irrefl_lex_prod[simp]
desharna
parents:
76682
diff
changeset
|
1173 |
|
| 60758 | 1174 |
text \<open>lexicographic combinations with measure functions\<close> |
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
1175 |
|
| 63108 | 1176 |
definition mlex_prod :: "('a \<Rightarrow> nat) \<Rightarrow> ('a \<times> 'a) set \<Rightarrow> ('a \<times> 'a) set" (infixr "<*mlex*>" 80)
|
1177 |
where "f <*mlex*> R = inv_image (less_than <*lex*> R) (\<lambda>x. (f x, x))" |
|
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
1178 |
|
| 66952 | 1179 |
lemma |
1180 |
wf_mlex: "wf R \<Longrightarrow> wf (f <*mlex*> R)" and |
|
1181 |
mlex_less: "f x < f y \<Longrightarrow> (x, y) \<in> f <*mlex*> R" and |
|
1182 |
mlex_leq: "f x \<le> f y \<Longrightarrow> (x, y) \<in> R \<Longrightarrow> (x, y) \<in> f <*mlex*> R" and |
|
1183 |
mlex_iff: "(x, y) \<in> f <*mlex*> R \<longleftrightarrow> f x < f y \<or> f x = f y \<and> (x, y) \<in> R" |
|
| 63572 | 1184 |
by (auto simp: mlex_prod_def) |
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
1185 |
|
| 63572 | 1186 |
text \<open>Proper subset relation on finite sets.\<close> |
| 63108 | 1187 |
definition finite_psubset :: "('a set \<times> 'a set) set"
|
| 63572 | 1188 |
where "finite_psubset = {(A, B). A \<subset> B \<and> finite B}"
|
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
1189 |
|
| 63108 | 1190 |
lemma wf_finite_psubset[simp]: "wf finite_psubset" |
1191 |
apply (unfold finite_psubset_def) |
|
1192 |
apply (rule wf_measure [THEN wf_subset]) |
|
1193 |
apply (simp add: measure_def inv_image_def less_than_def less_eq) |
|
1194 |
apply (fast elim!: psubset_card_mono) |
|
1195 |
done |
|
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
1196 |
|
|
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
1197 |
lemma trans_finite_psubset: "trans finite_psubset" |
| 63612 | 1198 |
by (auto simp: finite_psubset_def less_le trans_def) |
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
1199 |
|
| 63572 | 1200 |
lemma in_finite_psubset[simp]: "(A, B) \<in> finite_psubset \<longleftrightarrow> A \<subset> B \<and> finite B" |
| 63108 | 1201 |
unfolding finite_psubset_def by auto |
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
1202 |
|
| 60758 | 1203 |
text \<open>max- and min-extension of order to finite sets\<close> |
|
28735
bed31381e6b6
min_ext/max_ext lifting wellfounded relations on finite sets. Preserves wf
krauss
parents:
28562
diff
changeset
|
1204 |
|
| 63108 | 1205 |
inductive_set max_ext :: "('a \<times> 'a) set \<Rightarrow> ('a set \<times> 'a set) set"
|
1206 |
for R :: "('a \<times> 'a) set"
|
|
| 63572 | 1207 |
where max_extI[intro]: |
1208 |
"finite X \<Longrightarrow> finite Y \<Longrightarrow> Y \<noteq> {} \<Longrightarrow> (\<And>x. x \<in> X \<Longrightarrow> \<exists>y\<in>Y. (x, y) \<in> R) \<Longrightarrow> (X, Y) \<in> max_ext R"
|
|
|
28735
bed31381e6b6
min_ext/max_ext lifting wellfounded relations on finite sets. Preserves wf
krauss
parents:
28562
diff
changeset
|
1209 |
|
|
bed31381e6b6
min_ext/max_ext lifting wellfounded relations on finite sets. Preserves wf
krauss
parents:
28562
diff
changeset
|
1210 |
lemma max_ext_wf: |
|
bed31381e6b6
min_ext/max_ext lifting wellfounded relations on finite sets. Preserves wf
krauss
parents:
28562
diff
changeset
|
1211 |
assumes wf: "wf r" |
|
bed31381e6b6
min_ext/max_ext lifting wellfounded relations on finite sets. Preserves wf
krauss
parents:
28562
diff
changeset
|
1212 |
shows "wf (max_ext r)" |
|
bed31381e6b6
min_ext/max_ext lifting wellfounded relations on finite sets. Preserves wf
krauss
parents:
28562
diff
changeset
|
1213 |
proof (rule acc_wfI, intro allI) |
| 63915 | 1214 |
show "M \<in> acc (max_ext r)" (is "_ \<in> ?W") for M |
1215 |
proof (induct M rule: infinite_finite_induct) |
|
1216 |
case empty |
|
1217 |
show ?case |
|
1218 |
by (rule accI) (auto elim: max_ext.cases) |
|
1219 |
next |
|
1220 |
case (insert a M) |
|
1221 |
from wf \<open>M \<in> ?W\<close> \<open>finite M\<close> show "insert a M \<in> ?W" |
|
1222 |
proof (induct arbitrary: M) |
|
1223 |
fix M a |
|
1224 |
assume "M \<in> ?W" |
|
1225 |
assume [intro]: "finite M" |
|
1226 |
assume hyp: "\<And>b M. (b, a) \<in> r \<Longrightarrow> M \<in> ?W \<Longrightarrow> finite M \<Longrightarrow> insert b M \<in> ?W" |
|
1227 |
have add_less: "M \<in> ?W \<Longrightarrow> (\<And>y. y \<in> N \<Longrightarrow> (y, a) \<in> r) \<Longrightarrow> N \<union> M \<in> ?W" |
|
1228 |
if "finite N" "finite M" for N M :: "'a set" |
|
1229 |
using that by (induct N arbitrary: M) (auto simp: hyp) |
|
1230 |
show "insert a M \<in> ?W" |
|
1231 |
proof (rule accI) |
|
1232 |
fix N |
|
1233 |
assume Nless: "(N, insert a M) \<in> max_ext r" |
|
1234 |
then have *: "\<And>x. x \<in> N \<Longrightarrow> (x, a) \<in> r \<or> (\<exists>y \<in> M. (x, y) \<in> r)" |
|
1235 |
by (auto elim!: max_ext.cases) |
|
|
28735
bed31381e6b6
min_ext/max_ext lifting wellfounded relations on finite sets. Preserves wf
krauss
parents:
28562
diff
changeset
|
1236 |
|
| 63915 | 1237 |
let ?N1 = "{n \<in> N. (n, a) \<in> r}"
|
1238 |
let ?N2 = "{n \<in> N. (n, a) \<notin> r}"
|
|
1239 |
have N: "?N1 \<union> ?N2 = N" by (rule set_eqI) auto |
|
1240 |
from Nless have "finite N" by (auto elim: max_ext.cases) |
|
1241 |
then have finites: "finite ?N1" "finite ?N2" by auto |
|
| 63108 | 1242 |
|
| 63915 | 1243 |
have "?N2 \<in> ?W" |
1244 |
proof (cases "M = {}")
|
|
1245 |
case [simp]: True |
|
1246 |
have Mw: "{} \<in> ?W" by (rule accI) (auto elim: max_ext.cases)
|
|
1247 |
from * have "?N2 = {}" by auto
|
|
1248 |
with Mw show "?N2 \<in> ?W" by (simp only:) |
|
1249 |
next |
|
1250 |
case False |
|
1251 |
from * finites have N2: "(?N2, M) \<in> max_ext r" |
|
|
75669
43f5dfb7fa35
tuned (some HOL lints, by Yecine Megdiche);
Fabian Huch <huch@in.tum.de>
parents:
74971
diff
changeset
|
1252 |
using max_extI[OF _ _ \<open>M \<noteq> {}\<close>, where ?X = ?N2] by auto
|
| 63915 | 1253 |
with \<open>M \<in> ?W\<close> show "?N2 \<in> ?W" by (rule acc_downward) |
|
28735
bed31381e6b6
min_ext/max_ext lifting wellfounded relations on finite sets. Preserves wf
krauss
parents:
28562
diff
changeset
|
1254 |
qed |
| 63915 | 1255 |
with finites have "?N1 \<union> ?N2 \<in> ?W" |
1256 |
by (rule add_less) simp |
|
1257 |
then show "N \<in> ?W" by (simp only: N) |
|
|
28735
bed31381e6b6
min_ext/max_ext lifting wellfounded relations on finite sets. Preserves wf
krauss
parents:
28562
diff
changeset
|
1258 |
qed |
|
bed31381e6b6
min_ext/max_ext lifting wellfounded relations on finite sets. Preserves wf
krauss
parents:
28562
diff
changeset
|
1259 |
qed |
|
bed31381e6b6
min_ext/max_ext lifting wellfounded relations on finite sets. Preserves wf
krauss
parents:
28562
diff
changeset
|
1260 |
next |
| 63982 | 1261 |
case infinite |
1262 |
show ?case |
|
1263 |
by (rule accI) (auto elim: max_ext.cases simp: infinite) |
|
|
28735
bed31381e6b6
min_ext/max_ext lifting wellfounded relations on finite sets. Preserves wf
krauss
parents:
28562
diff
changeset
|
1264 |
qed |
|
bed31381e6b6
min_ext/max_ext lifting wellfounded relations on finite sets. Preserves wf
krauss
parents:
28562
diff
changeset
|
1265 |
qed |
|
bed31381e6b6
min_ext/max_ext lifting wellfounded relations on finite sets. Preserves wf
krauss
parents:
28562
diff
changeset
|
1266 |
|
| 63572 | 1267 |
lemma max_ext_additive: "(A, B) \<in> max_ext R \<Longrightarrow> (C, D) \<in> max_ext R \<Longrightarrow> (A \<union> C, B \<union> D) \<in> max_ext R" |
| 63108 | 1268 |
by (force elim!: max_ext.cases) |
|
29125
d41182a8135c
method "sizechange" proves termination of functions; added more infrastructure for termination proofs
krauss
parents:
28845
diff
changeset
|
1269 |
|
| 63108 | 1270 |
definition min_ext :: "('a \<times> 'a) set \<Rightarrow> ('a set \<times> 'a set) set"
|
1271 |
where "min_ext r = {(X, Y) | X Y. X \<noteq> {} \<and> (\<forall>y \<in> Y. (\<exists>x \<in> X. (x, y) \<in> r))}"
|
|
|
28735
bed31381e6b6
min_ext/max_ext lifting wellfounded relations on finite sets. Preserves wf
krauss
parents:
28562
diff
changeset
|
1272 |
|
|
bed31381e6b6
min_ext/max_ext lifting wellfounded relations on finite sets. Preserves wf
krauss
parents:
28562
diff
changeset
|
1273 |
lemma min_ext_wf: |
|
bed31381e6b6
min_ext/max_ext lifting wellfounded relations on finite sets. Preserves wf
krauss
parents:
28562
diff
changeset
|
1274 |
assumes "wf r" |
|
bed31381e6b6
min_ext/max_ext lifting wellfounded relations on finite sets. Preserves wf
krauss
parents:
28562
diff
changeset
|
1275 |
shows "wf (min_ext r)" |
|
bed31381e6b6
min_ext/max_ext lifting wellfounded relations on finite sets. Preserves wf
krauss
parents:
28562
diff
changeset
|
1276 |
proof (rule wfI_min) |
| 66952 | 1277 |
show "\<exists>m \<in> Q. (\<forall>n. (n, m) \<in> min_ext r \<longrightarrow> n \<notin> Q)" if nonempty: "x \<in> Q" |
| 63108 | 1278 |
for Q :: "'a set set" and x |
1279 |
proof (cases "Q = {{}}")
|
|
1280 |
case True |
|
1281 |
then show ?thesis by (simp add: min_ext_def) |
|
|
28735
bed31381e6b6
min_ext/max_ext lifting wellfounded relations on finite sets. Preserves wf
krauss
parents:
28562
diff
changeset
|
1282 |
next |
| 63108 | 1283 |
case False |
1284 |
with nonempty obtain e x where "x \<in> Q" "e \<in> x" by force |
|
|
28735
bed31381e6b6
min_ext/max_ext lifting wellfounded relations on finite sets. Preserves wf
krauss
parents:
28562
diff
changeset
|
1285 |
then have eU: "e \<in> \<Union>Q" by auto |
| 63108 | 1286 |
with \<open>wf r\<close> |
1287 |
obtain z where z: "z \<in> \<Union>Q" "\<And>y. (y, z) \<in> r \<Longrightarrow> y \<notin> \<Union>Q" |
|
|
28735
bed31381e6b6
min_ext/max_ext lifting wellfounded relations on finite sets. Preserves wf
krauss
parents:
28562
diff
changeset
|
1288 |
by (erule wfE_min) |
|
bed31381e6b6
min_ext/max_ext lifting wellfounded relations on finite sets. Preserves wf
krauss
parents:
28562
diff
changeset
|
1289 |
from z obtain m where "m \<in> Q" "z \<in> m" by auto |
| 63572 | 1290 |
from \<open>m \<in> Q\<close> show ?thesis |
1291 |
proof (intro rev_bexI allI impI) |
|
|
28735
bed31381e6b6
min_ext/max_ext lifting wellfounded relations on finite sets. Preserves wf
krauss
parents:
28562
diff
changeset
|
1292 |
fix n |
|
bed31381e6b6
min_ext/max_ext lifting wellfounded relations on finite sets. Preserves wf
krauss
parents:
28562
diff
changeset
|
1293 |
assume smaller: "(n, m) \<in> min_ext r" |
| 63572 | 1294 |
with \<open>z \<in> m\<close> obtain y where "y \<in> n" "(y, z) \<in> r" |
1295 |
by (auto simp: min_ext_def) |
|
1296 |
with z(2) show "n \<notin> Q" by auto |
|
| 63108 | 1297 |
qed |
|
28735
bed31381e6b6
min_ext/max_ext lifting wellfounded relations on finite sets. Preserves wf
krauss
parents:
28562
diff
changeset
|
1298 |
qed |
|
bed31381e6b6
min_ext/max_ext lifting wellfounded relations on finite sets. Preserves wf
krauss
parents:
28562
diff
changeset
|
1299 |
qed |
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
1300 |
|
| 63108 | 1301 |
|
1302 |
subsubsection \<open>Bounded increase must terminate\<close> |
|
| 43137 | 1303 |
|
1304 |
lemma wf_bounded_measure: |
|
| 63108 | 1305 |
fixes ub :: "'a \<Rightarrow> nat" |
1306 |
and f :: "'a \<Rightarrow> nat" |
|
1307 |
assumes "\<And>a b. (b, a) \<in> r \<Longrightarrow> ub b \<le> ub a \<and> ub a \<ge> f b \<and> f b > f a" |
|
1308 |
shows "wf r" |
|
| 63572 | 1309 |
by (rule wf_subset[OF wf_measure[of "\<lambda>a. ub a - f a"]]) (auto dest: assms) |
| 43137 | 1310 |
|
1311 |
lemma wf_bounded_set: |
|
| 63108 | 1312 |
fixes ub :: "'a \<Rightarrow> 'b set" |
1313 |
and f :: "'a \<Rightarrow> 'b set" |
|
1314 |
assumes "\<And>a b. (b,a) \<in> r \<Longrightarrow> finite (ub a) \<and> ub b \<subseteq> ub a \<and> ub a \<supseteq> f b \<and> f b \<supset> f a" |
|
1315 |
shows "wf r" |
|
| 63572 | 1316 |
apply (rule wf_bounded_measure[of r "\<lambda>a. card (ub a)" "\<lambda>a. card (f a)"]) |
1317 |
apply (drule assms) |
|
| 63108 | 1318 |
apply (blast intro: card_mono finite_subset psubset_card_mono dest: psubset_eq[THEN iffD2]) |
1319 |
done |
|
| 43137 | 1320 |
|
|
63099
af0e964aad7b
Moved material from AFP/Randomised_Social_Choice to distribution
eberlm
parents:
63088
diff
changeset
|
1321 |
lemma finite_subset_wf: |
|
af0e964aad7b
Moved material from AFP/Randomised_Social_Choice to distribution
eberlm
parents:
63088
diff
changeset
|
1322 |
assumes "finite A" |
| 66952 | 1323 |
shows "wf {(X, Y). X \<subset> Y \<and> Y \<subseteq> A}"
|
1324 |
by (rule wf_subset[OF wf_finite_psubset[unfolded finite_psubset_def]]) |
|
1325 |
(auto intro: finite_subset[OF _ assms]) |
|
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
1326 |
|
| 54295 | 1327 |
hide_const (open) acc accp |
1328 |
||
|
79971
033f90dc441d
redefined wf as an abbreviation for "wf_on UNIV"
desharna
parents:
79965
diff
changeset
|
1329 |
|
|
033f90dc441d
redefined wf as an abbreviation for "wf_on UNIV"
desharna
parents:
79965
diff
changeset
|
1330 |
subsection \<open>Code Generation Setup\<close> |
|
033f90dc441d
redefined wf as an abbreviation for "wf_on UNIV"
desharna
parents:
79965
diff
changeset
|
1331 |
|
|
033f90dc441d
redefined wf as an abbreviation for "wf_on UNIV"
desharna
parents:
79965
diff
changeset
|
1332 |
text \<open>Code equations with \<^const>\<open>wf\<close> or \<^const>\<open>wfp\<close> on the left-hand side are not supported by the |
|
033f90dc441d
redefined wf as an abbreviation for "wf_on UNIV"
desharna
parents:
79965
diff
changeset
|
1333 |
code generation module because of the \<^const>\<open>UNIV\<close> hidden behind the abbreviations. To sidestep this |
|
033f90dc441d
redefined wf as an abbreviation for "wf_on UNIV"
desharna
parents:
79965
diff
changeset
|
1334 |
problem, we provide the following wrapper definitions and use @{attribute code_abbrev} to register
|
|
033f90dc441d
redefined wf as an abbreviation for "wf_on UNIV"
desharna
parents:
79965
diff
changeset
|
1335 |
the definitions with the pre- and post-processors of the code generator.\<close> |
|
033f90dc441d
redefined wf as an abbreviation for "wf_on UNIV"
desharna
parents:
79965
diff
changeset
|
1336 |
|
|
033f90dc441d
redefined wf as an abbreviation for "wf_on UNIV"
desharna
parents:
79965
diff
changeset
|
1337 |
definition wf_code :: "('a \<times> 'a) set \<Rightarrow> bool" where
|
|
033f90dc441d
redefined wf as an abbreviation for "wf_on UNIV"
desharna
parents:
79965
diff
changeset
|
1338 |
[code_abbrev]: "wf_code r \<longleftrightarrow> wf r" |
|
033f90dc441d
redefined wf as an abbreviation for "wf_on UNIV"
desharna
parents:
79965
diff
changeset
|
1339 |
|
|
033f90dc441d
redefined wf as an abbreviation for "wf_on UNIV"
desharna
parents:
79965
diff
changeset
|
1340 |
definition wfp_code :: "('a \<Rightarrow> 'a \<Rightarrow> bool) \<Rightarrow> bool" where
|
|
033f90dc441d
redefined wf as an abbreviation for "wf_on UNIV"
desharna
parents:
79965
diff
changeset
|
1341 |
[code_abbrev]: "wfp_code R \<longleftrightarrow> wfp R" |
|
033f90dc441d
redefined wf as an abbreviation for "wf_on UNIV"
desharna
parents:
79965
diff
changeset
|
1342 |
|
|
26748
4d51ddd6aa5c
Merged theories about wellfoundedness into one: Wellfounded.thy
krauss
parents:
diff
changeset
|
1343 |
end |