| author | wenzelm |
| Thu, 28 Jul 2016 20:39:46 +0200 | |
| changeset 63558 | 0aa33085c8b1 |
| parent 63516 | 76492eaf3dc1 |
| child 63649 | e690d6f2185b |
| permissions | -rw-r--r-- |
| 36648 | 1 |
(* Title: HOL/Library/Convex.thy |
2 |
Author: Armin Heller, TU Muenchen |
|
3 |
Author: Johannes Hoelzl, TU Muenchen |
|
4 |
*) |
|
5 |
||
| 60423 | 6 |
section \<open>Convexity in real vector spaces\<close> |
| 36648 | 7 |
|
| 36623 | 8 |
theory Convex |
| 63485 | 9 |
imports Product_Vector |
| 36623 | 10 |
begin |
11 |
||
| 60423 | 12 |
subsection \<open>Convexity\<close> |
| 36623 | 13 |
|
| 49609 | 14 |
definition convex :: "'a::real_vector set \<Rightarrow> bool" |
15 |
where "convex s \<longleftrightarrow> (\<forall>x\<in>s. \<forall>y\<in>s. \<forall>u\<ge>0. \<forall>v\<ge>0. u + v = 1 \<longrightarrow> u *\<^sub>R x + v *\<^sub>R y \<in> s)" |
|
| 36623 | 16 |
|
| 53676 | 17 |
lemma convexI: |
18 |
assumes "\<And>x y u v. x \<in> s \<Longrightarrow> y \<in> s \<Longrightarrow> 0 \<le> u \<Longrightarrow> 0 \<le> v \<Longrightarrow> u + v = 1 \<Longrightarrow> u *\<^sub>R x + v *\<^sub>R y \<in> s" |
|
19 |
shows "convex s" |
|
20 |
using assms unfolding convex_def by fast |
|
21 |
||
22 |
lemma convexD: |
|
23 |
assumes "convex s" and "x \<in> s" and "y \<in> s" and "0 \<le> u" and "0 \<le> v" and "u + v = 1" |
|
24 |
shows "u *\<^sub>R x + v *\<^sub>R y \<in> s" |
|
25 |
using assms unfolding convex_def by fast |
|
26 |
||
| 63485 | 27 |
lemma convex_alt: "convex s \<longleftrightarrow> (\<forall>x\<in>s. \<forall>y\<in>s. \<forall>u. 0 \<le> u \<and> u \<le> 1 \<longrightarrow> ((1 - u) *\<^sub>R x + u *\<^sub>R y) \<in> s)" |
| 36623 | 28 |
(is "_ \<longleftrightarrow> ?alt") |
29 |
proof |
|
| 63485 | 30 |
show "convex s" if alt: ?alt |
31 |
proof - |
|
32 |
{
|
|
33 |
fix x y and u v :: real |
|
34 |
assume mem: "x \<in> s" "y \<in> s" |
|
35 |
assume "0 \<le> u" "0 \<le> v" |
|
36 |
moreover |
|
37 |
assume "u + v = 1" |
|
38 |
then have "u = 1 - v" by auto |
|
39 |
ultimately have "u *\<^sub>R x + v *\<^sub>R y \<in> s" |
|
40 |
using alt [rule_format, OF mem] by auto |
|
41 |
} |
|
42 |
then show ?thesis |
|
43 |
unfolding convex_def by auto |
|
44 |
qed |
|
45 |
show ?alt if "convex s" |
|
46 |
using that by (auto simp: convex_def) |
|
47 |
qed |
|
| 36623 | 48 |
|
|
61426
d53db136e8fd
new material on path_component_sets, inside, outside, etc. And more default simprules
paulson <lp15@cam.ac.uk>
parents:
61070
diff
changeset
|
49 |
lemma convexD_alt: |
| 36623 | 50 |
assumes "convex s" "a \<in> s" "b \<in> s" "0 \<le> u" "u \<le> 1" |
51 |
shows "((1 - u) *\<^sub>R a + u *\<^sub>R b) \<in> s" |
|
52 |
using assms unfolding convex_alt by auto |
|
53 |
||
|
61520
8f85bb443d33
Cauchy's integral formula, required lemmas, and a bit of reorganisation
paulson <lp15@cam.ac.uk>
parents:
61518
diff
changeset
|
54 |
lemma mem_convex_alt: |
|
8f85bb443d33
Cauchy's integral formula, required lemmas, and a bit of reorganisation
paulson <lp15@cam.ac.uk>
parents:
61518
diff
changeset
|
55 |
assumes "convex S" "x \<in> S" "y \<in> S" "u \<ge> 0" "v \<ge> 0" "u + v > 0" |
|
8f85bb443d33
Cauchy's integral formula, required lemmas, and a bit of reorganisation
paulson <lp15@cam.ac.uk>
parents:
61518
diff
changeset
|
56 |
shows "((u/(u+v)) *\<^sub>R x + (v/(u+v)) *\<^sub>R y) \<in> S" |
|
8f85bb443d33
Cauchy's integral formula, required lemmas, and a bit of reorganisation
paulson <lp15@cam.ac.uk>
parents:
61518
diff
changeset
|
57 |
apply (rule convexD) |
|
8f85bb443d33
Cauchy's integral formula, required lemmas, and a bit of reorganisation
paulson <lp15@cam.ac.uk>
parents:
61518
diff
changeset
|
58 |
using assms |
| 63485 | 59 |
apply (simp_all add: zero_le_divide_iff add_divide_distrib [symmetric]) |
|
61520
8f85bb443d33
Cauchy's integral formula, required lemmas, and a bit of reorganisation
paulson <lp15@cam.ac.uk>
parents:
61518
diff
changeset
|
60 |
done |
|
8f85bb443d33
Cauchy's integral formula, required lemmas, and a bit of reorganisation
paulson <lp15@cam.ac.uk>
parents:
61518
diff
changeset
|
61 |
|
| 60303 | 62 |
lemma convex_empty[intro,simp]: "convex {}"
|
| 36623 | 63 |
unfolding convex_def by simp |
64 |
||
| 60303 | 65 |
lemma convex_singleton[intro,simp]: "convex {a}"
|
| 36623 | 66 |
unfolding convex_def by (auto simp: scaleR_left_distrib[symmetric]) |
67 |
||
| 60303 | 68 |
lemma convex_UNIV[intro,simp]: "convex UNIV" |
| 36623 | 69 |
unfolding convex_def by auto |
70 |
||
|
63007
aa894a49f77d
new theorems about convex hulls, etc.; also, renamed some theorems
paulson <lp15@cam.ac.uk>
parents:
62418
diff
changeset
|
71 |
lemma convex_Inter: "(\<And>s. s\<in>f \<Longrightarrow> convex s) \<Longrightarrow> convex(\<Inter>f)" |
| 36623 | 72 |
unfolding convex_def by auto |
73 |
||
74 |
lemma convex_Int: "convex s \<Longrightarrow> convex t \<Longrightarrow> convex (s \<inter> t)" |
|
75 |
unfolding convex_def by auto |
|
76 |
||
|
63007
aa894a49f77d
new theorems about convex hulls, etc.; also, renamed some theorems
paulson <lp15@cam.ac.uk>
parents:
62418
diff
changeset
|
77 |
lemma convex_INT: "(\<And>i. i \<in> A \<Longrightarrow> convex (B i)) \<Longrightarrow> convex (\<Inter>i\<in>A. B i)" |
| 53596 | 78 |
unfolding convex_def by auto |
79 |
||
80 |
lemma convex_Times: "convex s \<Longrightarrow> convex t \<Longrightarrow> convex (s \<times> t)" |
|
81 |
unfolding convex_def by auto |
|
82 |
||
| 36623 | 83 |
lemma convex_halfspace_le: "convex {x. inner a x \<le> b}"
|
84 |
unfolding convex_def |
|
| 44142 | 85 |
by (auto simp: inner_add intro!: convex_bound_le) |
| 36623 | 86 |
|
87 |
lemma convex_halfspace_ge: "convex {x. inner a x \<ge> b}"
|
|
88 |
proof - |
|
| 56796 | 89 |
have *: "{x. inner a x \<ge> b} = {x. inner (-a) x \<le> -b}"
|
90 |
by auto |
|
91 |
show ?thesis |
|
92 |
unfolding * using convex_halfspace_le[of "-a" "-b"] by auto |
|
| 36623 | 93 |
qed |
94 |
||
95 |
lemma convex_hyperplane: "convex {x. inner a x = b}"
|
|
| 49609 | 96 |
proof - |
| 56796 | 97 |
have *: "{x. inner a x = b} = {x. inner a x \<le> b} \<inter> {x. inner a x \<ge> b}"
|
98 |
by auto |
|
| 36623 | 99 |
show ?thesis using convex_halfspace_le convex_halfspace_ge |
100 |
by (auto intro!: convex_Int simp: *) |
|
101 |
qed |
|
102 |
||
103 |
lemma convex_halfspace_lt: "convex {x. inner a x < b}"
|
|
104 |
unfolding convex_def |
|
105 |
by (auto simp: convex_bound_lt inner_add) |
|
106 |
||
107 |
lemma convex_halfspace_gt: "convex {x. inner a x > b}"
|
|
108 |
using convex_halfspace_lt[of "-a" "-b"] by auto |
|
109 |
||
|
61518
ff12606337e9
new lemmas about topology, etc., for Cauchy integral formula
paulson
parents:
61426
diff
changeset
|
110 |
lemma convex_real_interval [iff]: |
| 36623 | 111 |
fixes a b :: "real" |
112 |
shows "convex {a..}" and "convex {..b}"
|
|
| 49609 | 113 |
and "convex {a<..}" and "convex {..<b}"
|
114 |
and "convex {a..b}" and "convex {a<..b}"
|
|
115 |
and "convex {a..<b}" and "convex {a<..<b}"
|
|
| 36623 | 116 |
proof - |
| 60423 | 117 |
have "{a..} = {x. a \<le> inner 1 x}"
|
118 |
by auto |
|
119 |
then show 1: "convex {a..}"
|
|
120 |
by (simp only: convex_halfspace_ge) |
|
121 |
have "{..b} = {x. inner 1 x \<le> b}"
|
|
122 |
by auto |
|
123 |
then show 2: "convex {..b}"
|
|
124 |
by (simp only: convex_halfspace_le) |
|
125 |
have "{a<..} = {x. a < inner 1 x}"
|
|
126 |
by auto |
|
127 |
then show 3: "convex {a<..}"
|
|
128 |
by (simp only: convex_halfspace_gt) |
|
129 |
have "{..<b} = {x. inner 1 x < b}"
|
|
130 |
by auto |
|
131 |
then show 4: "convex {..<b}"
|
|
132 |
by (simp only: convex_halfspace_lt) |
|
133 |
have "{a..b} = {a..} \<inter> {..b}"
|
|
134 |
by auto |
|
135 |
then show "convex {a..b}"
|
|
136 |
by (simp only: convex_Int 1 2) |
|
137 |
have "{a<..b} = {a<..} \<inter> {..b}"
|
|
138 |
by auto |
|
139 |
then show "convex {a<..b}"
|
|
140 |
by (simp only: convex_Int 3 2) |
|
141 |
have "{a..<b} = {a..} \<inter> {..<b}"
|
|
142 |
by auto |
|
143 |
then show "convex {a..<b}"
|
|
144 |
by (simp only: convex_Int 1 4) |
|
145 |
have "{a<..<b} = {a<..} \<inter> {..<b}"
|
|
146 |
by auto |
|
147 |
then show "convex {a<..<b}"
|
|
148 |
by (simp only: convex_Int 3 4) |
|
| 36623 | 149 |
qed |
150 |
||
| 61070 | 151 |
lemma convex_Reals: "convex \<real>" |
| 59862 | 152 |
by (simp add: convex_def scaleR_conv_of_real) |
| 60423 | 153 |
|
154 |
||
155 |
subsection \<open>Explicit expressions for convexity in terms of arbitrary sums\<close> |
|
| 36623 | 156 |
|
157 |
lemma convex_setsum: |
|
158 |
fixes C :: "'a::real_vector set" |
|
| 56796 | 159 |
assumes "finite s" |
160 |
and "convex C" |
|
161 |
and "(\<Sum> i \<in> s. a i) = 1" |
|
162 |
assumes "\<And>i. i \<in> s \<Longrightarrow> a i \<ge> 0" |
|
163 |
and "\<And>i. i \<in> s \<Longrightarrow> y i \<in> C" |
|
| 36623 | 164 |
shows "(\<Sum> j \<in> s. a j *\<^sub>R y j) \<in> C" |
| 55909 | 165 |
using assms(1,3,4,5) |
166 |
proof (induct arbitrary: a set: finite) |
|
| 49609 | 167 |
case empty |
| 55909 | 168 |
then show ?case by simp |
| 36623 | 169 |
next |
| 55909 | 170 |
case (insert i s) note IH = this(3) |
| 56796 | 171 |
have "a i + setsum a s = 1" |
172 |
and "0 \<le> a i" |
|
173 |
and "\<forall>j\<in>s. 0 \<le> a j" |
|
174 |
and "y i \<in> C" |
|
175 |
and "\<forall>j\<in>s. y j \<in> C" |
|
| 55909 | 176 |
using insert.hyps(1,2) insert.prems by simp_all |
| 56796 | 177 |
then have "0 \<le> setsum a s" |
178 |
by (simp add: setsum_nonneg) |
|
| 55909 | 179 |
have "a i *\<^sub>R y i + (\<Sum>j\<in>s. a j *\<^sub>R y j) \<in> C" |
| 63516 | 180 |
proof (cases "setsum a s = 0") |
181 |
case True |
|
| 60423 | 182 |
with \<open>a i + setsum a s = 1\<close> have "a i = 1" |
| 56796 | 183 |
by simp |
| 63516 | 184 |
from setsum_nonneg_0 [OF \<open>finite s\<close> _ True] \<open>\<forall>j\<in>s. 0 \<le> a j\<close> have "\<forall>j\<in>s. a j = 0" |
| 56796 | 185 |
by simp |
| 60423 | 186 |
show ?thesis using \<open>a i = 1\<close> and \<open>\<forall>j\<in>s. a j = 0\<close> and \<open>y i \<in> C\<close> |
| 56796 | 187 |
by simp |
| 55909 | 188 |
next |
| 63516 | 189 |
case False |
| 60423 | 190 |
with \<open>0 \<le> setsum a s\<close> have "0 < setsum a s" |
| 56796 | 191 |
by simp |
| 55909 | 192 |
then have "(\<Sum>j\<in>s. (a j / setsum a s) *\<^sub>R y j) \<in> C" |
| 60423 | 193 |
using \<open>\<forall>j\<in>s. 0 \<le> a j\<close> and \<open>\<forall>j\<in>s. y j \<in> C\<close> |
|
56571
f4635657d66f
added divide_nonneg_nonneg and co; made it a simp rule
hoelzl
parents:
56544
diff
changeset
|
194 |
by (simp add: IH setsum_divide_distrib [symmetric]) |
| 60423 | 195 |
from \<open>convex C\<close> and \<open>y i \<in> C\<close> and this and \<open>0 \<le> a i\<close> |
196 |
and \<open>0 \<le> setsum a s\<close> and \<open>a i + setsum a s = 1\<close> |
|
| 55909 | 197 |
have "a i *\<^sub>R y i + setsum a s *\<^sub>R (\<Sum>j\<in>s. (a j / setsum a s) *\<^sub>R y j) \<in> C" |
198 |
by (rule convexD) |
|
| 56796 | 199 |
then show ?thesis |
| 63516 | 200 |
by (simp add: scaleR_setsum_right False) |
| 55909 | 201 |
qed |
| 60423 | 202 |
then show ?case using \<open>finite s\<close> and \<open>i \<notin> s\<close> |
| 56796 | 203 |
by simp |
| 36623 | 204 |
qed |
205 |
||
206 |
lemma convex: |
|
| 49609 | 207 |
"convex s \<longleftrightarrow> (\<forall>(k::nat) u x. (\<forall>i. 1\<le>i \<and> i\<le>k \<longrightarrow> 0 \<le> u i \<and> x i \<in>s) \<and> (setsum u {1..k} = 1)
|
208 |
\<longrightarrow> setsum (\<lambda>i. u i *\<^sub>R x i) {1..k} \<in> s)"
|
|
| 36623 | 209 |
proof safe |
| 49609 | 210 |
fix k :: nat |
211 |
fix u :: "nat \<Rightarrow> real" |
|
212 |
fix x |
|
| 36623 | 213 |
assume "convex s" |
214 |
"\<forall>i. 1 \<le> i \<and> i \<le> k \<longrightarrow> 0 \<le> u i \<and> x i \<in> s" |
|
215 |
"setsum u {1..k} = 1"
|
|
| 60423 | 216 |
with convex_setsum[of "{1 .. k}" s] show "(\<Sum>j\<in>{1 .. k}. u j *\<^sub>R x j) \<in> s"
|
| 56796 | 217 |
by auto |
| 36623 | 218 |
next |
| 60423 | 219 |
assume *: "\<forall>k u x. (\<forall> i :: nat. 1 \<le> i \<and> i \<le> k \<longrightarrow> 0 \<le> u i \<and> x i \<in> s) \<and> setsum u {1..k} = 1
|
| 36623 | 220 |
\<longrightarrow> (\<Sum>i = 1..k. u i *\<^sub>R (x i :: 'a)) \<in> s" |
| 56796 | 221 |
{
|
222 |
fix \<mu> :: real |
|
| 49609 | 223 |
fix x y :: 'a |
224 |
assume xy: "x \<in> s" "y \<in> s" |
|
225 |
assume mu: "\<mu> \<ge> 0" "\<mu> \<le> 1" |
|
226 |
let ?u = "\<lambda>i. if (i :: nat) = 1 then \<mu> else 1 - \<mu>" |
|
227 |
let ?x = "\<lambda>i. if (i :: nat) = 1 then x else y" |
|
| 56796 | 228 |
have "{1 :: nat .. 2} \<inter> - {x. x = 1} = {2}"
|
229 |
by auto |
|
230 |
then have card: "card ({1 :: nat .. 2} \<inter> - {x. x = 1}) = 1"
|
|
231 |
by simp |
|
| 49609 | 232 |
then have "setsum ?u {1 .. 2} = 1"
|
| 57418 | 233 |
using setsum.If_cases[of "{(1 :: nat) .. 2}" "\<lambda> x. x = 1" "\<lambda> x. \<mu>" "\<lambda> x. 1 - \<mu>"]
|
| 36623 | 234 |
by auto |
| 60423 | 235 |
with *[rule_format, of "2" ?u ?x] have s: "(\<Sum>j \<in> {1..2}. ?u j *\<^sub>R ?x j) \<in> s"
|
| 36623 | 236 |
using mu xy by auto |
237 |
have grarr: "(\<Sum>j \<in> {Suc (Suc 0)..2}. ?u j *\<^sub>R ?x j) = (1 - \<mu>) *\<^sub>R y"
|
|
238 |
using setsum_head_Suc[of "Suc (Suc 0)" 2 "\<lambda> j. (1 - \<mu>) *\<^sub>R y"] by auto |
|
239 |
from setsum_head_Suc[of "Suc 0" 2 "\<lambda> j. ?u j *\<^sub>R ?x j", simplified this] |
|
| 56796 | 240 |
have "(\<Sum>j \<in> {1..2}. ?u j *\<^sub>R ?x j) = \<mu> *\<^sub>R x + (1 - \<mu>) *\<^sub>R y"
|
241 |
by auto |
|
242 |
then have "(1 - \<mu>) *\<^sub>R y + \<mu> *\<^sub>R x \<in> s" |
|
| 60423 | 243 |
using s by (auto simp: add.commute) |
| 49609 | 244 |
} |
| 56796 | 245 |
then show "convex s" |
246 |
unfolding convex_alt by auto |
|
| 36623 | 247 |
qed |
248 |
||
249 |
||
250 |
lemma convex_explicit: |
|
251 |
fixes s :: "'a::real_vector set" |
|
252 |
shows "convex s \<longleftrightarrow> |
|
| 49609 | 253 |
(\<forall>t u. finite t \<and> t \<subseteq> s \<and> (\<forall>x\<in>t. 0 \<le> u x) \<and> setsum u t = 1 \<longrightarrow> setsum (\<lambda>x. u x *\<^sub>R x) t \<in> s)" |
| 36623 | 254 |
proof safe |
| 49609 | 255 |
fix t |
256 |
fix u :: "'a \<Rightarrow> real" |
|
| 56796 | 257 |
assume "convex s" |
258 |
and "finite t" |
|
259 |
and "t \<subseteq> s" "\<forall>x\<in>t. 0 \<le> u x" "setsum u t = 1" |
|
| 49609 | 260 |
then show "(\<Sum>x\<in>t. u x *\<^sub>R x) \<in> s" |
| 36623 | 261 |
using convex_setsum[of t s u "\<lambda> x. x"] by auto |
262 |
next |
|
| 60423 | 263 |
assume *: "\<forall>t. \<forall> u. finite t \<and> t \<subseteq> s \<and> (\<forall>x\<in>t. 0 \<le> u x) \<and> |
| 56796 | 264 |
setsum u t = 1 \<longrightarrow> (\<Sum>x\<in>t. u x *\<^sub>R x) \<in> s" |
| 36623 | 265 |
show "convex s" |
266 |
unfolding convex_alt |
|
267 |
proof safe |
|
| 49609 | 268 |
fix x y |
269 |
fix \<mu> :: real |
|
| 60423 | 270 |
assume **: "x \<in> s" "y \<in> s" "0 \<le> \<mu>" "\<mu> \<le> 1" |
271 |
show "(1 - \<mu>) *\<^sub>R x + \<mu> *\<^sub>R y \<in> s" |
|
272 |
proof (cases "x = y") |
|
273 |
case False |
|
274 |
then show ?thesis |
|
275 |
using *[rule_format, of "{x, y}" "\<lambda> z. if z = x then 1 - \<mu> else \<mu>"] **
|
|
| 63485 | 276 |
by auto |
| 60423 | 277 |
next |
278 |
case True |
|
279 |
then show ?thesis |
|
280 |
using *[rule_format, of "{x, y}" "\<lambda> z. 1"] **
|
|
| 63485 | 281 |
by (auto simp: field_simps real_vector.scale_left_diff_distrib) |
| 60423 | 282 |
qed |
| 36623 | 283 |
qed |
284 |
qed |
|
285 |
||
| 49609 | 286 |
lemma convex_finite: |
287 |
assumes "finite s" |
|
| 56796 | 288 |
shows "convex s \<longleftrightarrow> (\<forall>u. (\<forall>x\<in>s. 0 \<le> u x) \<and> setsum u s = 1 \<longrightarrow> setsum (\<lambda>x. u x *\<^sub>R x) s \<in> s)" |
| 36623 | 289 |
unfolding convex_explicit |
| 49609 | 290 |
proof safe |
291 |
fix t u |
|
292 |
assume sum: "\<forall>u. (\<forall>x\<in>s. 0 \<le> u x) \<and> setsum u s = 1 \<longrightarrow> (\<Sum>x\<in>s. u x *\<^sub>R x) \<in> s" |
|
| 36623 | 293 |
and as: "finite t" "t \<subseteq> s" "\<forall>x\<in>t. 0 \<le> u x" "setsum u t = (1::real)" |
| 56796 | 294 |
have *: "s \<inter> t = t" |
295 |
using as(2) by auto |
|
| 49609 | 296 |
have if_distrib_arg: "\<And>P f g x. (if P then f else g) x = (if P then f x else g x)" |
297 |
by simp |
|
| 36623 | 298 |
show "(\<Sum>x\<in>t. u x *\<^sub>R x) \<in> s" |
| 63485 | 299 |
using sum[THEN spec[where x="\<lambda>x. if x\<in>t then u x else 0"]] as * |
300 |
by (auto simp: assms setsum.If_cases if_distrib if_distrib_arg) |
|
| 36623 | 301 |
qed (erule_tac x=s in allE, erule_tac x=u in allE, auto) |
302 |
||
| 56796 | 303 |
|
| 60423 | 304 |
subsection \<open>Functions that are convex on a set\<close> |
| 55909 | 305 |
|
| 49609 | 306 |
definition convex_on :: "'a::real_vector set \<Rightarrow> ('a \<Rightarrow> real) \<Rightarrow> bool"
|
307 |
where "convex_on s f \<longleftrightarrow> |
|
308 |
(\<forall>x\<in>s. \<forall>y\<in>s. \<forall>u\<ge>0. \<forall>v\<ge>0. u + v = 1 \<longrightarrow> f (u *\<^sub>R x + v *\<^sub>R y) \<le> u * f x + v * f y)" |
|
| 36623 | 309 |
|
|
61531
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
eberlm
parents:
61520
diff
changeset
|
310 |
lemma convex_onI [intro?]: |
|
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
eberlm
parents:
61520
diff
changeset
|
311 |
assumes "\<And>t x y. t > 0 \<Longrightarrow> t < 1 \<Longrightarrow> x \<in> A \<Longrightarrow> y \<in> A \<Longrightarrow> |
| 63485 | 312 |
f ((1 - t) *\<^sub>R x + t *\<^sub>R y) \<le> (1 - t) * f x + t * f y" |
313 |
shows "convex_on A f" |
|
|
61531
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
eberlm
parents:
61520
diff
changeset
|
314 |
unfolding convex_on_def |
|
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
eberlm
parents:
61520
diff
changeset
|
315 |
proof clarify |
| 63485 | 316 |
fix x y |
317 |
fix u v :: real |
|
318 |
assume A: "x \<in> A" "y \<in> A" "u \<ge> 0" "v \<ge> 0" "u + v = 1" |
|
319 |
from A(5) have [simp]: "v = 1 - u" |
|
320 |
by (simp add: algebra_simps) |
|
321 |
from A(1-4) show "f (u *\<^sub>R x + v *\<^sub>R y) \<le> u * f x + v * f y" |
|
322 |
using assms[of u y x] |
|
|
61531
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
eberlm
parents:
61520
diff
changeset
|
323 |
by (cases "u = 0 \<or> u = 1") (auto simp: algebra_simps) |
|
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
eberlm
parents:
61520
diff
changeset
|
324 |
qed |
|
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
eberlm
parents:
61520
diff
changeset
|
325 |
|
|
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
eberlm
parents:
61520
diff
changeset
|
326 |
lemma convex_on_linorderI [intro?]: |
|
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
eberlm
parents:
61520
diff
changeset
|
327 |
fixes A :: "('a::{linorder,real_vector}) set"
|
|
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
eberlm
parents:
61520
diff
changeset
|
328 |
assumes "\<And>t x y. t > 0 \<Longrightarrow> t < 1 \<Longrightarrow> x \<in> A \<Longrightarrow> y \<in> A \<Longrightarrow> x < y \<Longrightarrow> |
| 63485 | 329 |
f ((1 - t) *\<^sub>R x + t *\<^sub>R y) \<le> (1 - t) * f x + t * f y" |
330 |
shows "convex_on A f" |
|
|
61531
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
eberlm
parents:
61520
diff
changeset
|
331 |
proof |
| 63485 | 332 |
fix x y |
333 |
fix t :: real |
|
334 |
assume A: "x \<in> A" "y \<in> A" "t > 0" "t < 1" |
|
335 |
with assms [of t x y] assms [of "1 - t" y x] |
|
| 62418 | 336 |
show "f ((1 - t) *\<^sub>R x + t *\<^sub>R y) \<le> (1 - t) * f x + t * f y" |
337 |
by (cases x y rule: linorder_cases) (auto simp: algebra_simps) |
|
|
61531
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
eberlm
parents:
61520
diff
changeset
|
338 |
qed |
|
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
eberlm
parents:
61520
diff
changeset
|
339 |
|
|
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
eberlm
parents:
61520
diff
changeset
|
340 |
lemma convex_onD: |
|
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
eberlm
parents:
61520
diff
changeset
|
341 |
assumes "convex_on A f" |
| 63485 | 342 |
shows "\<And>t x y. t \<ge> 0 \<Longrightarrow> t \<le> 1 \<Longrightarrow> x \<in> A \<Longrightarrow> y \<in> A \<Longrightarrow> |
343 |
f ((1 - t) *\<^sub>R x + t *\<^sub>R y) \<le> (1 - t) * f x + t * f y" |
|
344 |
using assms by (auto simp: convex_on_def) |
|
|
61531
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
eberlm
parents:
61520
diff
changeset
|
345 |
|
|
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
eberlm
parents:
61520
diff
changeset
|
346 |
lemma convex_onD_Icc: |
|
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
eberlm
parents:
61520
diff
changeset
|
347 |
assumes "convex_on {x..y} f" "x \<le> (y :: _ :: {real_vector,preorder})"
|
| 63485 | 348 |
shows "\<And>t. t \<ge> 0 \<Longrightarrow> t \<le> 1 \<Longrightarrow> |
349 |
f ((1 - t) *\<^sub>R x + t *\<^sub>R y) \<le> (1 - t) * f x + t * f y" |
|
350 |
using assms(2) by (intro convex_onD [OF assms(1)]) simp_all |
|
|
61531
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
eberlm
parents:
61520
diff
changeset
|
351 |
|
| 36623 | 352 |
lemma convex_on_subset: "convex_on t f \<Longrightarrow> s \<subseteq> t \<Longrightarrow> convex_on s f" |
353 |
unfolding convex_on_def by auto |
|
354 |
||
|
53620
3c7f5e7926dc
generalized and simplified proofs of several theorems about convex sets
huffman
parents:
53596
diff
changeset
|
355 |
lemma convex_on_add [intro]: |
| 56796 | 356 |
assumes "convex_on s f" |
357 |
and "convex_on s g" |
|
| 36623 | 358 |
shows "convex_on s (\<lambda>x. f x + g x)" |
| 49609 | 359 |
proof - |
| 56796 | 360 |
{
|
361 |
fix x y |
|
362 |
assume "x \<in> s" "y \<in> s" |
|
| 49609 | 363 |
moreover |
364 |
fix u v :: real |
|
365 |
assume "0 \<le> u" "0 \<le> v" "u + v = 1" |
|
366 |
ultimately |
|
367 |
have "f (u *\<^sub>R x + v *\<^sub>R y) + g (u *\<^sub>R x + v *\<^sub>R y) \<le> (u * f x + v * f y) + (u * g x + v * g y)" |
|
| 60423 | 368 |
using assms unfolding convex_on_def by (auto simp: add_mono) |
| 49609 | 369 |
then have "f (u *\<^sub>R x + v *\<^sub>R y) + g (u *\<^sub>R x + v *\<^sub>R y) \<le> u * (f x + g x) + v * (f y + g y)" |
370 |
by (simp add: field_simps) |
|
371 |
} |
|
| 56796 | 372 |
then show ?thesis |
373 |
unfolding convex_on_def by auto |
|
| 36623 | 374 |
qed |
375 |
||
|
53620
3c7f5e7926dc
generalized and simplified proofs of several theorems about convex sets
huffman
parents:
53596
diff
changeset
|
376 |
lemma convex_on_cmul [intro]: |
| 56796 | 377 |
fixes c :: real |
378 |
assumes "0 \<le> c" |
|
379 |
and "convex_on s f" |
|
| 36623 | 380 |
shows "convex_on s (\<lambda>x. c * f x)" |
| 56796 | 381 |
proof - |
| 63485 | 382 |
have *: "u * (c * fx) + v * (c * fy) = c * (u * fx + v * fy)" |
383 |
for u c fx v fy :: real |
|
| 49609 | 384 |
by (simp add: field_simps) |
385 |
show ?thesis using assms(2) and mult_left_mono [OF _ assms(1)] |
|
386 |
unfolding convex_on_def and * by auto |
|
| 36623 | 387 |
qed |
388 |
||
389 |
lemma convex_lower: |
|
| 56796 | 390 |
assumes "convex_on s f" |
391 |
and "x \<in> s" |
|
392 |
and "y \<in> s" |
|
393 |
and "0 \<le> u" |
|
394 |
and "0 \<le> v" |
|
395 |
and "u + v = 1" |
|
| 36623 | 396 |
shows "f (u *\<^sub>R x + v *\<^sub>R y) \<le> max (f x) (f y)" |
| 56796 | 397 |
proof - |
| 36623 | 398 |
let ?m = "max (f x) (f y)" |
399 |
have "u * f x + v * f y \<le> u * max (f x) (f y) + v * max (f x) (f y)" |
|
| 60423 | 400 |
using assms(4,5) by (auto simp: mult_left_mono add_mono) |
| 56796 | 401 |
also have "\<dots> = max (f x) (f y)" |
| 60423 | 402 |
using assms(6) by (simp add: distrib_right [symmetric]) |
| 36623 | 403 |
finally show ?thesis |
|
44890
22f665a2e91c
new fastforce replacing fastsimp - less confusing name
nipkow
parents:
44282
diff
changeset
|
404 |
using assms unfolding convex_on_def by fastforce |
| 36623 | 405 |
qed |
406 |
||
|
53620
3c7f5e7926dc
generalized and simplified proofs of several theorems about convex sets
huffman
parents:
53596
diff
changeset
|
407 |
lemma convex_on_dist [intro]: |
| 36623 | 408 |
fixes s :: "'a::real_normed_vector set" |
409 |
shows "convex_on s (\<lambda>x. dist a x)" |
|
| 60423 | 410 |
proof (auto simp: convex_on_def dist_norm) |
| 49609 | 411 |
fix x y |
| 56796 | 412 |
assume "x \<in> s" "y \<in> s" |
| 49609 | 413 |
fix u v :: real |
| 56796 | 414 |
assume "0 \<le> u" |
415 |
assume "0 \<le> v" |
|
416 |
assume "u + v = 1" |
|
| 49609 | 417 |
have "a = u *\<^sub>R a + v *\<^sub>R a" |
| 60423 | 418 |
unfolding scaleR_left_distrib[symmetric] and \<open>u + v = 1\<close> by simp |
| 49609 | 419 |
then have *: "a - (u *\<^sub>R x + v *\<^sub>R y) = (u *\<^sub>R (a - x)) + (v *\<^sub>R (a - y))" |
| 60423 | 420 |
by (auto simp: algebra_simps) |
| 36623 | 421 |
show "norm (a - (u *\<^sub>R x + v *\<^sub>R y)) \<le> u * norm (a - x) + v * norm (a - y)" |
422 |
unfolding * using norm_triangle_ineq[of "u *\<^sub>R (a - x)" "v *\<^sub>R (a - y)"] |
|
| 60423 | 423 |
using \<open>0 \<le> u\<close> \<open>0 \<le> v\<close> by auto |
| 36623 | 424 |
qed |
425 |
||
| 49609 | 426 |
|
| 60423 | 427 |
subsection \<open>Arithmetic operations on sets preserve convexity\<close> |
| 49609 | 428 |
|
|
53620
3c7f5e7926dc
generalized and simplified proofs of several theorems about convex sets
huffman
parents:
53596
diff
changeset
|
429 |
lemma convex_linear_image: |
| 56796 | 430 |
assumes "linear f" |
431 |
and "convex s" |
|
432 |
shows "convex (f ` s)" |
|
|
53620
3c7f5e7926dc
generalized and simplified proofs of several theorems about convex sets
huffman
parents:
53596
diff
changeset
|
433 |
proof - |
|
3c7f5e7926dc
generalized and simplified proofs of several theorems about convex sets
huffman
parents:
53596
diff
changeset
|
434 |
interpret f: linear f by fact |
| 60423 | 435 |
from \<open>convex s\<close> show "convex (f ` s)" |
|
53620
3c7f5e7926dc
generalized and simplified proofs of several theorems about convex sets
huffman
parents:
53596
diff
changeset
|
436 |
by (simp add: convex_def f.scaleR [symmetric] f.add [symmetric]) |
| 36623 | 437 |
qed |
438 |
||
|
53620
3c7f5e7926dc
generalized and simplified proofs of several theorems about convex sets
huffman
parents:
53596
diff
changeset
|
439 |
lemma convex_linear_vimage: |
| 56796 | 440 |
assumes "linear f" |
441 |
and "convex s" |
|
442 |
shows "convex (f -` s)" |
|
|
53620
3c7f5e7926dc
generalized and simplified proofs of several theorems about convex sets
huffman
parents:
53596
diff
changeset
|
443 |
proof - |
|
3c7f5e7926dc
generalized and simplified proofs of several theorems about convex sets
huffman
parents:
53596
diff
changeset
|
444 |
interpret f: linear f by fact |
| 60423 | 445 |
from \<open>convex s\<close> show "convex (f -` s)" |
|
53620
3c7f5e7926dc
generalized and simplified proofs of several theorems about convex sets
huffman
parents:
53596
diff
changeset
|
446 |
by (simp add: convex_def f.add f.scaleR) |
|
3c7f5e7926dc
generalized and simplified proofs of several theorems about convex sets
huffman
parents:
53596
diff
changeset
|
447 |
qed |
|
3c7f5e7926dc
generalized and simplified proofs of several theorems about convex sets
huffman
parents:
53596
diff
changeset
|
448 |
|
|
3c7f5e7926dc
generalized and simplified proofs of several theorems about convex sets
huffman
parents:
53596
diff
changeset
|
449 |
lemma convex_scaling: |
| 56796 | 450 |
assumes "convex s" |
451 |
shows "convex ((\<lambda>x. c *\<^sub>R x) ` s)" |
|
|
53620
3c7f5e7926dc
generalized and simplified proofs of several theorems about convex sets
huffman
parents:
53596
diff
changeset
|
452 |
proof - |
| 56796 | 453 |
have "linear (\<lambda>x. c *\<^sub>R x)" |
454 |
by (simp add: linearI scaleR_add_right) |
|
455 |
then show ?thesis |
|
| 60423 | 456 |
using \<open>convex s\<close> by (rule convex_linear_image) |
|
53620
3c7f5e7926dc
generalized and simplified proofs of several theorems about convex sets
huffman
parents:
53596
diff
changeset
|
457 |
qed |
|
3c7f5e7926dc
generalized and simplified proofs of several theorems about convex sets
huffman
parents:
53596
diff
changeset
|
458 |
|
|
60178
f620c70f9e9b
generalized differentiable_bound; some further variations of differentiable_bound
immler
parents:
59862
diff
changeset
|
459 |
lemma convex_scaled: |
|
f620c70f9e9b
generalized differentiable_bound; some further variations of differentiable_bound
immler
parents:
59862
diff
changeset
|
460 |
assumes "convex s" |
|
f620c70f9e9b
generalized differentiable_bound; some further variations of differentiable_bound
immler
parents:
59862
diff
changeset
|
461 |
shows "convex ((\<lambda>x. x *\<^sub>R c) ` s)" |
|
f620c70f9e9b
generalized differentiable_bound; some further variations of differentiable_bound
immler
parents:
59862
diff
changeset
|
462 |
proof - |
|
f620c70f9e9b
generalized differentiable_bound; some further variations of differentiable_bound
immler
parents:
59862
diff
changeset
|
463 |
have "linear (\<lambda>x. x *\<^sub>R c)" |
|
f620c70f9e9b
generalized differentiable_bound; some further variations of differentiable_bound
immler
parents:
59862
diff
changeset
|
464 |
by (simp add: linearI scaleR_add_left) |
|
f620c70f9e9b
generalized differentiable_bound; some further variations of differentiable_bound
immler
parents:
59862
diff
changeset
|
465 |
then show ?thesis |
| 60423 | 466 |
using \<open>convex s\<close> by (rule convex_linear_image) |
|
60178
f620c70f9e9b
generalized differentiable_bound; some further variations of differentiable_bound
immler
parents:
59862
diff
changeset
|
467 |
qed |
|
f620c70f9e9b
generalized differentiable_bound; some further variations of differentiable_bound
immler
parents:
59862
diff
changeset
|
468 |
|
|
53620
3c7f5e7926dc
generalized and simplified proofs of several theorems about convex sets
huffman
parents:
53596
diff
changeset
|
469 |
lemma convex_negations: |
| 56796 | 470 |
assumes "convex s" |
471 |
shows "convex ((\<lambda>x. - x) ` s)" |
|
|
53620
3c7f5e7926dc
generalized and simplified proofs of several theorems about convex sets
huffman
parents:
53596
diff
changeset
|
472 |
proof - |
| 56796 | 473 |
have "linear (\<lambda>x. - x)" |
474 |
by (simp add: linearI) |
|
475 |
then show ?thesis |
|
| 60423 | 476 |
using \<open>convex s\<close> by (rule convex_linear_image) |
| 36623 | 477 |
qed |
478 |
||
479 |
lemma convex_sums: |
|
| 56796 | 480 |
assumes "convex s" |
481 |
and "convex t" |
|
| 36623 | 482 |
shows "convex {x + y| x y. x \<in> s \<and> y \<in> t}"
|
|
53620
3c7f5e7926dc
generalized and simplified proofs of several theorems about convex sets
huffman
parents:
53596
diff
changeset
|
483 |
proof - |
|
3c7f5e7926dc
generalized and simplified proofs of several theorems about convex sets
huffman
parents:
53596
diff
changeset
|
484 |
have "linear (\<lambda>(x, y). x + y)" |
| 60423 | 485 |
by (auto intro: linearI simp: scaleR_add_right) |
|
53620
3c7f5e7926dc
generalized and simplified proofs of several theorems about convex sets
huffman
parents:
53596
diff
changeset
|
486 |
with assms have "convex ((\<lambda>(x, y). x + y) ` (s \<times> t))" |
|
3c7f5e7926dc
generalized and simplified proofs of several theorems about convex sets
huffman
parents:
53596
diff
changeset
|
487 |
by (intro convex_linear_image convex_Times) |
|
3c7f5e7926dc
generalized and simplified proofs of several theorems about convex sets
huffman
parents:
53596
diff
changeset
|
488 |
also have "((\<lambda>(x, y). x + y) ` (s \<times> t)) = {x + y| x y. x \<in> s \<and> y \<in> t}"
|
|
3c7f5e7926dc
generalized and simplified proofs of several theorems about convex sets
huffman
parents:
53596
diff
changeset
|
489 |
by auto |
|
3c7f5e7926dc
generalized and simplified proofs of several theorems about convex sets
huffman
parents:
53596
diff
changeset
|
490 |
finally show ?thesis . |
| 36623 | 491 |
qed |
492 |
||
493 |
lemma convex_differences: |
|
494 |
assumes "convex s" "convex t" |
|
495 |
shows "convex {x - y| x y. x \<in> s \<and> y \<in> t}"
|
|
496 |
proof - |
|
497 |
have "{x - y| x y. x \<in> s \<and> y \<in> t} = {x + y |x y. x \<in> s \<and> y \<in> uminus ` t}"
|
|
| 60423 | 498 |
by (auto simp: diff_conv_add_uminus simp del: add_uminus_conv_diff) |
| 49609 | 499 |
then show ?thesis |
500 |
using convex_sums[OF assms(1) convex_negations[OF assms(2)]] by auto |
|
| 36623 | 501 |
qed |
502 |
||
| 49609 | 503 |
lemma convex_translation: |
504 |
assumes "convex s" |
|
505 |
shows "convex ((\<lambda>x. a + x) ` s)" |
|
506 |
proof - |
|
| 56796 | 507 |
have "{a + y |y. y \<in> s} = (\<lambda>x. a + x) ` s"
|
508 |
by auto |
|
| 49609 | 509 |
then show ?thesis |
510 |
using convex_sums[OF convex_singleton[of a] assms] by auto |
|
511 |
qed |
|
| 36623 | 512 |
|
| 49609 | 513 |
lemma convex_affinity: |
514 |
assumes "convex s" |
|
515 |
shows "convex ((\<lambda>x. a + c *\<^sub>R x) ` s)" |
|
516 |
proof - |
|
| 56796 | 517 |
have "(\<lambda>x. a + c *\<^sub>R x) ` s = op + a ` op *\<^sub>R c ` s" |
518 |
by auto |
|
| 49609 | 519 |
then show ?thesis |
520 |
using convex_translation[OF convex_scaling[OF assms], of a c] by auto |
|
521 |
qed |
|
| 36623 | 522 |
|
| 49609 | 523 |
lemma pos_is_convex: "convex {0 :: real <..}"
|
524 |
unfolding convex_alt |
|
| 36623 | 525 |
proof safe |
526 |
fix y x \<mu> :: real |
|
| 60423 | 527 |
assume *: "y > 0" "x > 0" "\<mu> \<ge> 0" "\<mu> \<le> 1" |
| 56796 | 528 |
{
|
529 |
assume "\<mu> = 0" |
|
| 63485 | 530 |
then have "\<mu> *\<^sub>R x + (1 - \<mu>) *\<^sub>R y = y" |
531 |
by simp |
|
532 |
then have "\<mu> *\<^sub>R x + (1 - \<mu>) *\<^sub>R y > 0" |
|
533 |
using * by simp |
|
| 56796 | 534 |
} |
| 36623 | 535 |
moreover |
| 56796 | 536 |
{
|
537 |
assume "\<mu> = 1" |
|
| 63485 | 538 |
then have "\<mu> *\<^sub>R x + (1 - \<mu>) *\<^sub>R y > 0" |
539 |
using * by simp |
|
| 56796 | 540 |
} |
| 36623 | 541 |
moreover |
| 56796 | 542 |
{
|
543 |
assume "\<mu> \<noteq> 1" "\<mu> \<noteq> 0" |
|
| 63485 | 544 |
then have "\<mu> > 0" "(1 - \<mu>) > 0" |
545 |
using * by auto |
|
546 |
then have "\<mu> *\<^sub>R x + (1 - \<mu>) *\<^sub>R y > 0" |
|
547 |
using * by (auto simp: add_pos_pos) |
|
| 56796 | 548 |
} |
549 |
ultimately show "(1 - \<mu>) *\<^sub>R y + \<mu> *\<^sub>R x > 0" |
|
| 63092 | 550 |
by fastforce |
| 36623 | 551 |
qed |
552 |
||
553 |
lemma convex_on_setsum: |
|
554 |
fixes a :: "'a \<Rightarrow> real" |
|
| 49609 | 555 |
and y :: "'a \<Rightarrow> 'b::real_vector" |
556 |
and f :: "'b \<Rightarrow> real" |
|
| 36623 | 557 |
assumes "finite s" "s \<noteq> {}"
|
| 49609 | 558 |
and "convex_on C f" |
559 |
and "convex C" |
|
560 |
and "(\<Sum> i \<in> s. a i) = 1" |
|
561 |
and "\<And>i. i \<in> s \<Longrightarrow> a i \<ge> 0" |
|
562 |
and "\<And>i. i \<in> s \<Longrightarrow> y i \<in> C" |
|
| 36623 | 563 |
shows "f (\<Sum> i \<in> s. a i *\<^sub>R y i) \<le> (\<Sum> i \<in> s. a i * f (y i))" |
| 49609 | 564 |
using assms |
565 |
proof (induct s arbitrary: a rule: finite_ne_induct) |
|
| 36623 | 566 |
case (singleton i) |
| 63485 | 567 |
then have ai: "a i = 1" |
568 |
by auto |
|
569 |
then show ?case |
|
570 |
by auto |
|
| 36623 | 571 |
next |
| 60423 | 572 |
case (insert i s) |
| 63485 | 573 |
then have "convex_on C f" |
574 |
by simp |
|
| 36623 | 575 |
from this[unfolded convex_on_def, rule_format] |
| 56796 | 576 |
have conv: "\<And>x y \<mu>. x \<in> C \<Longrightarrow> y \<in> C \<Longrightarrow> 0 \<le> \<mu> \<Longrightarrow> \<mu> \<le> 1 \<Longrightarrow> |
577 |
f (\<mu> *\<^sub>R x + (1 - \<mu>) *\<^sub>R y) \<le> \<mu> * f x + (1 - \<mu>) * f y" |
|
| 36623 | 578 |
by simp |
| 60423 | 579 |
show ?case |
580 |
proof (cases "a i = 1") |
|
581 |
case True |
|
| 49609 | 582 |
then have "(\<Sum> j \<in> s. a j) = 0" |
| 60423 | 583 |
using insert by auto |
| 49609 | 584 |
then have "\<And>j. j \<in> s \<Longrightarrow> a j = 0" |
|
62376
85f38d5f8807
Rename ordered_comm_monoid_add to ordered_cancel_comm_monoid_add. Introduce ordreed_comm_monoid_add, canonically_ordered_comm_monoid and dioid. Setup nat, entat and ennreal as dioids.
hoelzl
parents:
61694
diff
changeset
|
585 |
using insert by (fastforce simp: setsum_nonneg_eq_0_iff) |
| 60423 | 586 |
then show ?thesis |
587 |
using insert by auto |
|
588 |
next |
|
589 |
case False |
|
590 |
from insert have yai: "y i \<in> C" "a i \<ge> 0" |
|
591 |
by auto |
|
592 |
have fis: "finite (insert i s)" |
|
593 |
using insert by auto |
|
594 |
then have ai1: "a i \<le> 1" |
|
595 |
using setsum_nonneg_leq_bound[of "insert i s" a] insert by simp |
|
596 |
then have "a i < 1" |
|
597 |
using False by auto |
|
598 |
then have i0: "1 - a i > 0" |
|
599 |
by auto |
|
| 49609 | 600 |
let ?a = "\<lambda>j. a j / (1 - a i)" |
| 60423 | 601 |
have a_nonneg: "?a j \<ge> 0" if "j \<in> s" for j |
| 60449 | 602 |
using i0 insert that by fastforce |
| 60423 | 603 |
have "(\<Sum> j \<in> insert i s. a j) = 1" |
604 |
using insert by auto |
|
605 |
then have "(\<Sum> j \<in> s. a j) = 1 - a i" |
|
606 |
using setsum.insert insert by fastforce |
|
607 |
then have "(\<Sum> j \<in> s. a j) / (1 - a i) = 1" |
|
608 |
using i0 by auto |
|
609 |
then have a1: "(\<Sum> j \<in> s. ?a j) = 1" |
|
610 |
unfolding setsum_divide_distrib by simp |
|
611 |
have "convex C" using insert by auto |
|
| 49609 | 612 |
then have asum: "(\<Sum> j \<in> s. ?a j *\<^sub>R y j) \<in> C" |
| 63485 | 613 |
using insert convex_setsum [OF \<open>finite s\<close> \<open>convex C\<close> a1 a_nonneg] by auto |
| 36623 | 614 |
have asum_le: "f (\<Sum> j \<in> s. ?a j *\<^sub>R y j) \<le> (\<Sum> j \<in> s. ?a j * f (y j))" |
| 60423 | 615 |
using a_nonneg a1 insert by blast |
| 36623 | 616 |
have "f (\<Sum> j \<in> insert i s. a j *\<^sub>R y j) = f ((\<Sum> j \<in> s. a j *\<^sub>R y j) + a i *\<^sub>R y i)" |
| 60423 | 617 |
using setsum.insert[of s i "\<lambda> j. a j *\<^sub>R y j", OF \<open>finite s\<close> \<open>i \<notin> s\<close>] insert |
618 |
by (auto simp only: add.commute) |
|
| 36623 | 619 |
also have "\<dots> = f (((1 - a i) * inverse (1 - a i)) *\<^sub>R (\<Sum> j \<in> s. a j *\<^sub>R y j) + a i *\<^sub>R y i)" |
620 |
using i0 by auto |
|
621 |
also have "\<dots> = f ((1 - a i) *\<^sub>R (\<Sum> j \<in> s. (a j * inverse (1 - a i)) *\<^sub>R y j) + a i *\<^sub>R y i)" |
|
| 49609 | 622 |
using scaleR_right.setsum[of "inverse (1 - a i)" "\<lambda> j. a j *\<^sub>R y j" s, symmetric] |
| 60423 | 623 |
by (auto simp: algebra_simps) |
| 36623 | 624 |
also have "\<dots> = f ((1 - a i) *\<^sub>R (\<Sum> j \<in> s. ?a j *\<^sub>R y j) + a i *\<^sub>R y i)" |
|
36778
739a9379e29b
avoid using real-specific versions of generic lemmas
huffman
parents:
36648
diff
changeset
|
625 |
by (auto simp: divide_inverse) |
| 36623 | 626 |
also have "\<dots> \<le> (1 - a i) *\<^sub>R f ((\<Sum> j \<in> s. ?a j *\<^sub>R y j)) + a i * f (y i)" |
627 |
using conv[of "y i" "(\<Sum> j \<in> s. ?a j *\<^sub>R y j)" "a i", OF yai(1) asum yai(2) ai1] |
|
| 60423 | 628 |
by (auto simp: add.commute) |
| 36623 | 629 |
also have "\<dots> \<le> (1 - a i) * (\<Sum> j \<in> s. ?a j * f (y j)) + a i * f (y i)" |
| 63485 | 630 |
using add_right_mono [OF mult_left_mono [of _ _ "1 - a i", |
631 |
OF asum_le less_imp_le[OF i0]], of "a i * f (y i)"] |
|
632 |
by simp |
|
| 36623 | 633 |
also have "\<dots> = (\<Sum> j \<in> s. (1 - a i) * ?a j * f (y j)) + a i * f (y i)" |
| 63485 | 634 |
unfolding setsum_right_distrib[of "1 - a i" "\<lambda> j. ?a j * f (y j)"] |
635 |
using i0 by auto |
|
| 60423 | 636 |
also have "\<dots> = (\<Sum> j \<in> s. a j * f (y j)) + a i * f (y i)" |
637 |
using i0 by auto |
|
638 |
also have "\<dots> = (\<Sum> j \<in> insert i s. a j * f (y j))" |
|
639 |
using insert by auto |
|
640 |
finally show ?thesis |
|
| 56796 | 641 |
by simp |
| 60423 | 642 |
qed |
| 36623 | 643 |
qed |
644 |
||
645 |
lemma convex_on_alt: |
|
646 |
fixes C :: "'a::real_vector set" |
|
647 |
assumes "convex C" |
|
| 56796 | 648 |
shows "convex_on C f \<longleftrightarrow> |
649 |
(\<forall>x \<in> C. \<forall> y \<in> C. \<forall> \<mu> :: real. \<mu> \<ge> 0 \<and> \<mu> \<le> 1 \<longrightarrow> |
|
650 |
f (\<mu> *\<^sub>R x + (1 - \<mu>) *\<^sub>R y) \<le> \<mu> * f x + (1 - \<mu>) * f y)" |
|
| 36623 | 651 |
proof safe |
| 49609 | 652 |
fix x y |
653 |
fix \<mu> :: real |
|
| 60423 | 654 |
assume *: "convex_on C f" "x \<in> C" "y \<in> C" "0 \<le> \<mu>" "\<mu> \<le> 1" |
| 36623 | 655 |
from this[unfolded convex_on_def, rule_format] |
| 63485 | 656 |
have "0 \<le> u \<Longrightarrow> 0 \<le> v \<Longrightarrow> u + v = 1 \<Longrightarrow> f (u *\<^sub>R x + v *\<^sub>R y) \<le> u * f x + v * f y" for u v |
| 56796 | 657 |
by auto |
| 63485 | 658 |
from this [of "\<mu>" "1 - \<mu>", simplified] * |
| 56796 | 659 |
show "f (\<mu> *\<^sub>R x + (1 - \<mu>) *\<^sub>R y) \<le> \<mu> * f x + (1 - \<mu>) * f y" |
660 |
by auto |
|
| 36623 | 661 |
next |
| 60423 | 662 |
assume *: "\<forall>x\<in>C. \<forall>y\<in>C. \<forall>\<mu>. 0 \<le> \<mu> \<and> \<mu> \<le> 1 \<longrightarrow> |
| 56796 | 663 |
f (\<mu> *\<^sub>R x + (1 - \<mu>) *\<^sub>R y) \<le> \<mu> * f x + (1 - \<mu>) * f y" |
664 |
{
|
|
665 |
fix x y |
|
| 49609 | 666 |
fix u v :: real |
| 60423 | 667 |
assume **: "x \<in> C" "y \<in> C" "u \<ge> 0" "v \<ge> 0" "u + v = 1" |
| 49609 | 668 |
then have[simp]: "1 - u = v" by auto |
| 60423 | 669 |
from *[rule_format, of x y u] |
| 56796 | 670 |
have "f (u *\<^sub>R x + v *\<^sub>R y) \<le> u * f x + v * f y" |
| 60423 | 671 |
using ** by auto |
| 49609 | 672 |
} |
| 56796 | 673 |
then show "convex_on C f" |
674 |
unfolding convex_on_def by auto |
|
| 36623 | 675 |
qed |
676 |
||
| 43337 | 677 |
lemma convex_on_diff: |
678 |
fixes f :: "real \<Rightarrow> real" |
|
| 56796 | 679 |
assumes f: "convex_on I f" |
680 |
and I: "x \<in> I" "y \<in> I" |
|
681 |
and t: "x < t" "t < y" |
|
| 49609 | 682 |
shows "(f x - f t) / (x - t) \<le> (f x - f y) / (x - y)" |
| 56796 | 683 |
and "(f x - f y) / (x - y) \<le> (f t - f y) / (t - y)" |
| 43337 | 684 |
proof - |
| 63040 | 685 |
define a where "a \<equiv> (t - y) / (x - y)" |
| 56796 | 686 |
with t have "0 \<le> a" "0 \<le> 1 - a" |
687 |
by (auto simp: field_simps) |
|
| 60423 | 688 |
with f \<open>x \<in> I\<close> \<open>y \<in> I\<close> have cvx: "f (a * x + (1 - a) * y) \<le> a * f x + (1 - a) * f y" |
| 43337 | 689 |
by (auto simp: convex_on_def) |
| 56796 | 690 |
have "a * x + (1 - a) * y = a * (x - y) + y" |
691 |
by (simp add: field_simps) |
|
692 |
also have "\<dots> = t" |
|
| 60423 | 693 |
unfolding a_def using \<open>x < t\<close> \<open>t < y\<close> by simp |
| 56796 | 694 |
finally have "f t \<le> a * f x + (1 - a) * f y" |
695 |
using cvx by simp |
|
696 |
also have "\<dots> = a * (f x - f y) + f y" |
|
697 |
by (simp add: field_simps) |
|
698 |
finally have "f t - f y \<le> a * (f x - f y)" |
|
699 |
by simp |
|
| 43337 | 700 |
with t show "(f x - f t) / (x - t) \<le> (f x - f y) / (x - y)" |
| 44142 | 701 |
by (simp add: le_divide_eq divide_le_eq field_simps a_def) |
| 43337 | 702 |
with t show "(f x - f y) / (x - y) \<le> (f t - f y) / (t - y)" |
| 44142 | 703 |
by (simp add: le_divide_eq divide_le_eq field_simps) |
| 43337 | 704 |
qed |
| 36623 | 705 |
|
706 |
lemma pos_convex_function: |
|
707 |
fixes f :: "real \<Rightarrow> real" |
|
708 |
assumes "convex C" |
|
| 56796 | 709 |
and leq: "\<And>x y. x \<in> C \<Longrightarrow> y \<in> C \<Longrightarrow> f' x * (y - x) \<le> f y - f x" |
| 36623 | 710 |
shows "convex_on C f" |
| 49609 | 711 |
unfolding convex_on_alt[OF assms(1)] |
712 |
using assms |
|
| 36623 | 713 |
proof safe |
714 |
fix x y \<mu> :: real |
|
715 |
let ?x = "\<mu> *\<^sub>R x + (1 - \<mu>) *\<^sub>R y" |
|
| 60423 | 716 |
assume *: "convex C" "x \<in> C" "y \<in> C" "\<mu> \<ge> 0" "\<mu> \<le> 1" |
| 49609 | 717 |
then have "1 - \<mu> \<ge> 0" by auto |
| 56796 | 718 |
then have xpos: "?x \<in> C" |
| 60423 | 719 |
using * unfolding convex_alt by fastforce |
| 56796 | 720 |
have geq: "\<mu> * (f x - f ?x) + (1 - \<mu>) * (f y - f ?x) \<ge> |
721 |
\<mu> * f' ?x * (x - ?x) + (1 - \<mu>) * f' ?x * (y - ?x)" |
|
| 63485 | 722 |
using add_mono [OF mult_left_mono [OF leq [OF xpos *(2)] \<open>\<mu> \<ge> 0\<close>] |
723 |
mult_left_mono [OF leq [OF xpos *(3)] \<open>1 - \<mu> \<ge> 0\<close>]] |
|
| 56796 | 724 |
by auto |
| 49609 | 725 |
then have "\<mu> * f x + (1 - \<mu>) * f y - f ?x \<ge> 0" |
| 60423 | 726 |
by (auto simp: field_simps) |
| 49609 | 727 |
then show "f (\<mu> *\<^sub>R x + (1 - \<mu>) *\<^sub>R y) \<le> \<mu> * f x + (1 - \<mu>) * f y" |
| 36623 | 728 |
using convex_on_alt by auto |
729 |
qed |
|
730 |
||
731 |
lemma atMostAtLeast_subset_convex: |
|
732 |
fixes C :: "real set" |
|
733 |
assumes "convex C" |
|
| 49609 | 734 |
and "x \<in> C" "y \<in> C" "x < y" |
| 36623 | 735 |
shows "{x .. y} \<subseteq> C"
|
736 |
proof safe |
|
| 60423 | 737 |
fix z assume z: "z \<in> {x .. y}"
|
738 |
have less: "z \<in> C" if *: "x < z" "z < y" |
|
739 |
proof - |
|
| 49609 | 740 |
let ?\<mu> = "(y - z) / (y - x)" |
| 56796 | 741 |
have "0 \<le> ?\<mu>" "?\<mu> \<le> 1" |
| 60423 | 742 |
using assms * by (auto simp: field_simps) |
| 49609 | 743 |
then have comb: "?\<mu> * x + (1 - ?\<mu>) * y \<in> C" |
744 |
using assms iffD1[OF convex_alt, rule_format, of C y x ?\<mu>] |
|
745 |
by (simp add: algebra_simps) |
|
| 36623 | 746 |
have "?\<mu> * x + (1 - ?\<mu>) * y = (y - z) * x / (y - x) + (1 - (y - z) / (y - x)) * y" |
| 60423 | 747 |
by (auto simp: field_simps) |
| 36623 | 748 |
also have "\<dots> = ((y - z) * x + (y - x - (y - z)) * y) / (y - x)" |
| 63485 | 749 |
using assms by (simp only: add_divide_distrib) (auto simp: field_simps) |
| 36623 | 750 |
also have "\<dots> = z" |
| 49609 | 751 |
using assms by (auto simp: field_simps) |
| 60423 | 752 |
finally show ?thesis |
| 56796 | 753 |
using comb by auto |
| 60423 | 754 |
qed |
| 63485 | 755 |
show "z \<in> C" |
756 |
using z less assms by (auto simp: le_less) |
|
| 36623 | 757 |
qed |
758 |
||
759 |
lemma f''_imp_f': |
|
760 |
fixes f :: "real \<Rightarrow> real" |
|
761 |
assumes "convex C" |
|
| 49609 | 762 |
and f': "\<And>x. x \<in> C \<Longrightarrow> DERIV f x :> (f' x)" |
763 |
and f'': "\<And>x. x \<in> C \<Longrightarrow> DERIV f' x :> (f'' x)" |
|
764 |
and pos: "\<And>x. x \<in> C \<Longrightarrow> f'' x \<ge> 0" |
|
| 63485 | 765 |
and x: "x \<in> C" |
766 |
and y: "y \<in> C" |
|
| 36623 | 767 |
shows "f' x * (y - x) \<le> f y - f x" |
| 49609 | 768 |
using assms |
| 36623 | 769 |
proof - |
| 63485 | 770 |
have less_imp: "f y - f x \<ge> f' x * (y - x)" "f' y * (x - y) \<le> f x - f y" |
771 |
if *: "x \<in> C" "y \<in> C" "y > x" for x y :: real |
|
772 |
proof - |
|
773 |
from * have ge: "y - x > 0" "y - x \<ge> 0" |
|
| 60423 | 774 |
by auto |
775 |
from * have le: "x - y < 0" "x - y \<le> 0" |
|
776 |
by auto |
|
| 36623 | 777 |
then obtain z1 where z1: "z1 > x" "z1 < y" "f y - f x = (y - x) * f' z1" |
| 60423 | 778 |
using subsetD[OF atMostAtLeast_subset_convex[OF \<open>convex C\<close> \<open>x \<in> C\<close> \<open>y \<in> C\<close> \<open>x < y\<close>], |
| 63485 | 779 |
THEN f', THEN MVT2[OF \<open>x < y\<close>, rule_format, unfolded atLeastAtMost_iff[symmetric]]] |
| 36623 | 780 |
by auto |
| 60423 | 781 |
then have "z1 \<in> C" |
782 |
using atMostAtLeast_subset_convex \<open>convex C\<close> \<open>x \<in> C\<close> \<open>y \<in> C\<close> \<open>x < y\<close> |
|
783 |
by fastforce |
|
| 36623 | 784 |
from z1 have z1': "f x - f y = (x - y) * f' z1" |
| 60423 | 785 |
by (simp add: field_simps) |
| 36623 | 786 |
obtain z2 where z2: "z2 > x" "z2 < z1" "f' z1 - f' x = (z1 - x) * f'' z2" |
| 60423 | 787 |
using subsetD[OF atMostAtLeast_subset_convex[OF \<open>convex C\<close> \<open>x \<in> C\<close> \<open>z1 \<in> C\<close> \<open>x < z1\<close>], |
| 63485 | 788 |
THEN f'', THEN MVT2[OF \<open>x < z1\<close>, rule_format, unfolded atLeastAtMost_iff[symmetric]]] z1 |
| 36623 | 789 |
by auto |
790 |
obtain z3 where z3: "z3 > z1" "z3 < y" "f' y - f' z1 = (y - z1) * f'' z3" |
|
| 60423 | 791 |
using subsetD[OF atMostAtLeast_subset_convex[OF \<open>convex C\<close> \<open>z1 \<in> C\<close> \<open>y \<in> C\<close> \<open>z1 < y\<close>], |
| 63485 | 792 |
THEN f'', THEN MVT2[OF \<open>z1 < y\<close>, rule_format, unfolded atLeastAtMost_iff[symmetric]]] z1 |
| 36623 | 793 |
by auto |
794 |
have "f' y - (f x - f y) / (x - y) = f' y - f' z1" |
|
| 60423 | 795 |
using * z1' by auto |
796 |
also have "\<dots> = (y - z1) * f'' z3" |
|
797 |
using z3 by auto |
|
798 |
finally have cool': "f' y - (f x - f y) / (x - y) = (y - z1) * f'' z3" |
|
799 |
by simp |
|
800 |
have A': "y - z1 \<ge> 0" |
|
801 |
using z1 by auto |
|
802 |
have "z3 \<in> C" |
|
803 |
using z3 * atMostAtLeast_subset_convex \<open>convex C\<close> \<open>x \<in> C\<close> \<open>z1 \<in> C\<close> \<open>x < z1\<close> |
|
804 |
by fastforce |
|
805 |
then have B': "f'' z3 \<ge> 0" |
|
806 |
using assms by auto |
|
807 |
from A' B' have "(y - z1) * f'' z3 \<ge> 0" |
|
808 |
by auto |
|
809 |
from cool' this have "f' y - (f x - f y) / (x - y) \<ge> 0" |
|
810 |
by auto |
|
| 36623 | 811 |
from mult_right_mono_neg[OF this le(2)] |
812 |
have "f' y * (x - y) - (f x - f y) / (x - y) * (x - y) \<le> 0 * (x - y)" |
|
|
36778
739a9379e29b
avoid using real-specific versions of generic lemmas
huffman
parents:
36648
diff
changeset
|
813 |
by (simp add: algebra_simps) |
| 60423 | 814 |
then have "f' y * (x - y) - (f x - f y) \<le> 0" |
815 |
using le by auto |
|
816 |
then have res: "f' y * (x - y) \<le> f x - f y" |
|
817 |
by auto |
|
| 36623 | 818 |
have "(f y - f x) / (y - x) - f' x = f' z1 - f' x" |
| 60423 | 819 |
using * z1 by auto |
820 |
also have "\<dots> = (z1 - x) * f'' z2" |
|
821 |
using z2 by auto |
|
822 |
finally have cool: "(f y - f x) / (y - x) - f' x = (z1 - x) * f'' z2" |
|
823 |
by simp |
|
824 |
have A: "z1 - x \<ge> 0" |
|
825 |
using z1 by auto |
|
826 |
have "z2 \<in> C" |
|
827 |
using z2 z1 * atMostAtLeast_subset_convex \<open>convex C\<close> \<open>z1 \<in> C\<close> \<open>y \<in> C\<close> \<open>z1 < y\<close> |
|
828 |
by fastforce |
|
829 |
then have B: "f'' z2 \<ge> 0" |
|
830 |
using assms by auto |
|
831 |
from A B have "(z1 - x) * f'' z2 \<ge> 0" |
|
832 |
by auto |
|
833 |
with cool have "(f y - f x) / (y - x) - f' x \<ge> 0" |
|
834 |
by auto |
|
| 36623 | 835 |
from mult_right_mono[OF this ge(2)] |
836 |
have "(f y - f x) / (y - x) * (y - x) - f' x * (y - x) \<ge> 0 * (y - x)" |
|
|
36778
739a9379e29b
avoid using real-specific versions of generic lemmas
huffman
parents:
36648
diff
changeset
|
837 |
by (simp add: algebra_simps) |
| 60423 | 838 |
then have "f y - f x - f' x * (y - x) \<ge> 0" |
839 |
using ge by auto |
|
| 63485 | 840 |
then show "f y - f x \<ge> f' x * (y - x)" "f' y * (x - y) \<le> f x - f y" |
| 60423 | 841 |
using res by auto |
| 63485 | 842 |
qed |
843 |
show ?thesis |
|
844 |
proof (cases "x = y") |
|
845 |
case True |
|
846 |
with x y show ?thesis by auto |
|
847 |
next |
|
848 |
case False |
|
849 |
with less_imp x y show ?thesis |
|
850 |
by (auto simp: neq_iff) |
|
851 |
qed |
|
| 36623 | 852 |
qed |
853 |
||
854 |
lemma f''_ge0_imp_convex: |
|
855 |
fixes f :: "real \<Rightarrow> real" |
|
856 |
assumes conv: "convex C" |
|
| 49609 | 857 |
and f': "\<And>x. x \<in> C \<Longrightarrow> DERIV f x :> (f' x)" |
858 |
and f'': "\<And>x. x \<in> C \<Longrightarrow> DERIV f' x :> (f'' x)" |
|
859 |
and pos: "\<And>x. x \<in> C \<Longrightarrow> f'' x \<ge> 0" |
|
| 36623 | 860 |
shows "convex_on C f" |
| 56796 | 861 |
using f''_imp_f'[OF conv f' f'' pos] assms pos_convex_function |
862 |
by fastforce |
|
| 36623 | 863 |
|
864 |
lemma minus_log_convex: |
|
865 |
fixes b :: real |
|
866 |
assumes "b > 1" |
|
867 |
shows "convex_on {0 <..} (\<lambda> x. - log b x)"
|
|
868 |
proof - |
|
| 56796 | 869 |
have "\<And>z. z > 0 \<Longrightarrow> DERIV (log b) z :> 1 / (ln b * z)" |
870 |
using DERIV_log by auto |
|
| 49609 | 871 |
then have f': "\<And>z. z > 0 \<Longrightarrow> DERIV (\<lambda> z. - log b z) z :> - 1 / (ln b * z)" |
|
56479
91958d4b30f7
revert c1bbd3e22226, a14831ac3023, and 36489d77c484: divide_minus_left/right are again simp rules
hoelzl
parents:
56409
diff
changeset
|
872 |
by (auto simp: DERIV_minus) |
| 63485 | 873 |
have "\<And>z::real. z > 0 \<Longrightarrow> DERIV inverse z :> - (inverse z ^ Suc (Suc 0))" |
| 36623 | 874 |
using less_imp_neq[THEN not_sym, THEN DERIV_inverse] by auto |
875 |
from this[THEN DERIV_cmult, of _ "- 1 / ln b"] |
|
| 63485 | 876 |
have "\<And>z::real. z > 0 \<Longrightarrow> |
| 49609 | 877 |
DERIV (\<lambda> z. (- 1 / ln b) * inverse z) z :> (- 1 / ln b) * (- (inverse z ^ Suc (Suc 0)))" |
| 36623 | 878 |
by auto |
| 56796 | 879 |
then have f''0: "\<And>z::real. z > 0 \<Longrightarrow> |
880 |
DERIV (\<lambda> z. - 1 / (ln b * z)) z :> 1 / (ln b * z * z)" |
|
| 60423 | 881 |
unfolding inverse_eq_divide by (auto simp: mult.assoc) |
| 56796 | 882 |
have f''_ge0: "\<And>z::real. z > 0 \<Longrightarrow> 1 / (ln b * z * z) \<ge> 0" |
| 60423 | 883 |
using \<open>b > 1\<close> by (auto intro!: less_imp_le) |
| 63485 | 884 |
from f''_ge0_imp_convex[OF pos_is_convex, unfolded greaterThan_iff, OF f' f''0 f''_ge0] |
885 |
show ?thesis |
|
886 |
by auto |
|
| 36623 | 887 |
qed |
888 |
||
|
61531
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
eberlm
parents:
61520
diff
changeset
|
889 |
|
|
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
eberlm
parents:
61520
diff
changeset
|
890 |
subsection \<open>Convexity of real functions\<close> |
|
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
eberlm
parents:
61520
diff
changeset
|
891 |
|
|
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
eberlm
parents:
61520
diff
changeset
|
892 |
lemma convex_on_realI: |
|
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
eberlm
parents:
61520
diff
changeset
|
893 |
assumes "connected A" |
| 63485 | 894 |
and "\<And>x. x \<in> A \<Longrightarrow> (f has_real_derivative f' x) (at x)" |
895 |
and "\<And>x y. x \<in> A \<Longrightarrow> y \<in> A \<Longrightarrow> x \<le> y \<Longrightarrow> f' x \<le> f' y" |
|
896 |
shows "convex_on A f" |
|
|
61531
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
eberlm
parents:
61520
diff
changeset
|
897 |
proof (rule convex_on_linorderI) |
|
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
eberlm
parents:
61520
diff
changeset
|
898 |
fix t x y :: real |
| 63485 | 899 |
assume t: "t > 0" "t < 1" |
900 |
assume xy: "x \<in> A" "y \<in> A" "x < y" |
|
| 63040 | 901 |
define z where "z = (1 - t) * x + t * y" |
| 63485 | 902 |
with \<open>connected A\<close> and xy have ivl: "{x..y} \<subseteq> A"
|
903 |
using connected_contains_Icc by blast |
|
|
61694
6571c78c9667
Removed some legacy theorems; minor adjustments to simplification rules; new material on homotopic paths
paulson <lp15@cam.ac.uk>
parents:
61585
diff
changeset
|
904 |
|
| 63485 | 905 |
from xy t have xz: "z > x" |
906 |
by (simp add: z_def algebra_simps) |
|
907 |
have "y - z = (1 - t) * (y - x)" |
|
908 |
by (simp add: z_def algebra_simps) |
|
909 |
also from xy t have "\<dots> > 0" |
|
910 |
by (intro mult_pos_pos) simp_all |
|
911 |
finally have yz: "z < y" |
|
912 |
by simp |
|
|
61694
6571c78c9667
Removed some legacy theorems; minor adjustments to simplification rules; new material on homotopic paths
paulson <lp15@cam.ac.uk>
parents:
61585
diff
changeset
|
913 |
|
|
61531
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
eberlm
parents:
61520
diff
changeset
|
914 |
from assms xz yz ivl t have "\<exists>\<xi>. \<xi> > x \<and> \<xi> < z \<and> f z - f x = (z - x) * f' \<xi>" |
|
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
eberlm
parents:
61520
diff
changeset
|
915 |
by (intro MVT2) (auto intro!: assms(2)) |
| 63485 | 916 |
then obtain \<xi> where \<xi>: "\<xi> > x" "\<xi> < z" "f' \<xi> = (f z - f x) / (z - x)" |
917 |
by auto |
|
|
61531
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
eberlm
parents:
61520
diff
changeset
|
918 |
from assms xz yz ivl t have "\<exists>\<eta>. \<eta> > z \<and> \<eta> < y \<and> f y - f z = (y - z) * f' \<eta>" |
|
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
eberlm
parents:
61520
diff
changeset
|
919 |
by (intro MVT2) (auto intro!: assms(2)) |
| 63485 | 920 |
then obtain \<eta> where \<eta>: "\<eta> > z" "\<eta> < y" "f' \<eta> = (f y - f z) / (y - z)" |
921 |
by auto |
|
|
61694
6571c78c9667
Removed some legacy theorems; minor adjustments to simplification rules; new material on homotopic paths
paulson <lp15@cam.ac.uk>
parents:
61585
diff
changeset
|
922 |
|
|
61531
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
eberlm
parents:
61520
diff
changeset
|
923 |
from \<eta>(3) have "(f y - f z) / (y - z) = f' \<eta>" .. |
| 63485 | 924 |
also from \<xi> \<eta> ivl have "\<xi> \<in> A" "\<eta> \<in> A" |
925 |
by auto |
|
926 |
with \<xi> \<eta> have "f' \<eta> \<ge> f' \<xi>" |
|
927 |
by (intro assms(3)) auto |
|
|
61531
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
eberlm
parents:
61520
diff
changeset
|
928 |
also from \<xi>(3) have "f' \<xi> = (f z - f x) / (z - x)" . |
|
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
eberlm
parents:
61520
diff
changeset
|
929 |
finally have "(f y - f z) * (z - x) \<ge> (f z - f x) * (y - z)" |
|
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
eberlm
parents:
61520
diff
changeset
|
930 |
using xz yz by (simp add: field_simps) |
| 63485 | 931 |
also have "z - x = t * (y - x)" |
932 |
by (simp add: z_def algebra_simps) |
|
933 |
also have "y - z = (1 - t) * (y - x)" |
|
934 |
by (simp add: z_def algebra_simps) |
|
935 |
finally have "(f y - f z) * t \<ge> (f z - f x) * (1 - t)" |
|
936 |
using xy by simp |
|
937 |
then show "(1 - t) * f x + t * f y \<ge> f ((1 - t) *\<^sub>R x + t *\<^sub>R y)" |
|
|
61531
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
eberlm
parents:
61520
diff
changeset
|
938 |
by (simp add: z_def algebra_simps) |
|
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
eberlm
parents:
61520
diff
changeset
|
939 |
qed |
|
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
eberlm
parents:
61520
diff
changeset
|
940 |
|
|
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
eberlm
parents:
61520
diff
changeset
|
941 |
lemma convex_on_inverse: |
|
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
eberlm
parents:
61520
diff
changeset
|
942 |
assumes "A \<subseteq> {0<..}"
|
| 63485 | 943 |
shows "convex_on A (inverse :: real \<Rightarrow> real)" |
|
61531
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
eberlm
parents:
61520
diff
changeset
|
944 |
proof (rule convex_on_subset[OF _ assms], intro convex_on_realI[of _ _ "\<lambda>x. -inverse (x^2)"]) |
| 63485 | 945 |
fix u v :: real |
946 |
assume "u \<in> {0<..}" "v \<in> {0<..}" "u \<le> v"
|
|
|
61531
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
eberlm
parents:
61520
diff
changeset
|
947 |
with assms show "-inverse (u^2) \<le> -inverse (v^2)" |
|
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
eberlm
parents:
61520
diff
changeset
|
948 |
by (intro le_imp_neg_le le_imp_inverse_le power_mono) (simp_all) |
|
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
eberlm
parents:
61520
diff
changeset
|
949 |
qed (insert assms, auto intro!: derivative_eq_intros simp: divide_simps power2_eq_square) |
|
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
eberlm
parents:
61520
diff
changeset
|
950 |
|
|
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
eberlm
parents:
61520
diff
changeset
|
951 |
lemma convex_onD_Icc': |
|
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
eberlm
parents:
61520
diff
changeset
|
952 |
assumes "convex_on {x..y} f" "c \<in> {x..y}"
|
|
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
eberlm
parents:
61520
diff
changeset
|
953 |
defines "d \<equiv> y - x" |
| 63485 | 954 |
shows "f c \<le> (f y - f x) / d * (c - x) + f x" |
955 |
proof (cases x y rule: linorder_cases) |
|
956 |
case less |
|
957 |
then have d: "d > 0" |
|
958 |
by (simp add: d_def) |
|
|
61694
6571c78c9667
Removed some legacy theorems; minor adjustments to simplification rules; new material on homotopic paths
paulson <lp15@cam.ac.uk>
parents:
61585
diff
changeset
|
959 |
from assms(2) less have A: "0 \<le> (c - x) / d" "(c - x) / d \<le> 1" |
|
61531
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
eberlm
parents:
61520
diff
changeset
|
960 |
by (simp_all add: d_def divide_simps) |
| 63485 | 961 |
have "f c = f (x + (c - x) * 1)" |
962 |
by simp |
|
963 |
also from less have "1 = ((y - x) / d)" |
|
964 |
by (simp add: d_def) |
|
|
61694
6571c78c9667
Removed some legacy theorems; minor adjustments to simplification rules; new material on homotopic paths
paulson <lp15@cam.ac.uk>
parents:
61585
diff
changeset
|
965 |
also from d have "x + (c - x) * \<dots> = (1 - (c - x) / d) *\<^sub>R x + ((c - x) / d) *\<^sub>R y" |
|
61531
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
eberlm
parents:
61520
diff
changeset
|
966 |
by (simp add: field_simps) |
| 63485 | 967 |
also have "f \<dots> \<le> (1 - (c - x) / d) * f x + (c - x) / d * f y" |
968 |
using assms less by (intro convex_onD_Icc) simp_all |
|
969 |
also from d have "\<dots> = (f y - f x) / d * (c - x) + f x" |
|
970 |
by (simp add: field_simps) |
|
|
61531
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
eberlm
parents:
61520
diff
changeset
|
971 |
finally show ?thesis . |
|
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
eberlm
parents:
61520
diff
changeset
|
972 |
qed (insert assms(2), simp_all) |
|
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
eberlm
parents:
61520
diff
changeset
|
973 |
|
|
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
eberlm
parents:
61520
diff
changeset
|
974 |
lemma convex_onD_Icc'': |
|
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
eberlm
parents:
61520
diff
changeset
|
975 |
assumes "convex_on {x..y} f" "c \<in> {x..y}"
|
|
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
eberlm
parents:
61520
diff
changeset
|
976 |
defines "d \<equiv> y - x" |
| 63485 | 977 |
shows "f c \<le> (f x - f y) / d * (y - c) + f y" |
978 |
proof (cases x y rule: linorder_cases) |
|
979 |
case less |
|
980 |
then have d: "d > 0" |
|
981 |
by (simp add: d_def) |
|
|
61694
6571c78c9667
Removed some legacy theorems; minor adjustments to simplification rules; new material on homotopic paths
paulson <lp15@cam.ac.uk>
parents:
61585
diff
changeset
|
982 |
from assms(2) less have A: "0 \<le> (y - c) / d" "(y - c) / d \<le> 1" |
|
61531
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
eberlm
parents:
61520
diff
changeset
|
983 |
by (simp_all add: d_def divide_simps) |
| 63485 | 984 |
have "f c = f (y - (y - c) * 1)" |
985 |
by simp |
|
986 |
also from less have "1 = ((y - x) / d)" |
|
987 |
by (simp add: d_def) |
|
|
61694
6571c78c9667
Removed some legacy theorems; minor adjustments to simplification rules; new material on homotopic paths
paulson <lp15@cam.ac.uk>
parents:
61585
diff
changeset
|
988 |
also from d have "y - (y - c) * \<dots> = (1 - (1 - (y - c) / d)) *\<^sub>R x + (1 - (y - c) / d) *\<^sub>R y" |
|
61531
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
eberlm
parents:
61520
diff
changeset
|
989 |
by (simp add: field_simps) |
| 63485 | 990 |
also have "f \<dots> \<le> (1 - (1 - (y - c) / d)) * f x + (1 - (y - c) / d) * f y" |
991 |
using assms less by (intro convex_onD_Icc) (simp_all add: field_simps) |
|
992 |
also from d have "\<dots> = (f x - f y) / d * (y - c) + f y" |
|
993 |
by (simp add: field_simps) |
|
|
61531
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
eberlm
parents:
61520
diff
changeset
|
994 |
finally show ?thesis . |
|
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
eberlm
parents:
61520
diff
changeset
|
995 |
qed (insert assms(2), simp_all) |
|
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
eberlm
parents:
61520
diff
changeset
|
996 |
|
| 36623 | 997 |
end |