diff -r 9cde57cdd0e3 -r 8fa437809c67 src/HOL/Library/Convex.thy --- a/src/HOL/Library/Convex.thy Sun Aug 22 14:27:30 2010 +0200 +++ b/src/HOL/Library/Convex.thy Mon Aug 23 11:17:13 2010 +0200 @@ -244,7 +244,7 @@ shows "convex_on s (\x. c * f x)" proof- have *:"\u c fx v fy ::real. u * (c * fx) + v * (c * fy) = c * (u * fx + v * fy)" by (simp add: field_simps) - show ?thesis using assms(2) and mult_mono1[OF _ assms(1)] unfolding convex_on_def and * by auto + show ?thesis using assms(2) and mult_left_mono [OF _ assms(1)] unfolding convex_on_def and * by auto qed lemma convex_lower: @@ -253,7 +253,7 @@ proof- let ?m = "max (f x) (f y)" have "u * f x + v * f y \ u * max (f x) (f y) + v * max (f x) (f y)" - using assms(4,5) by(auto simp add: mult_mono1 add_mono) + using assms(4,5) by (auto simp add: mult_left_mono add_mono) also have "\ = max (f x) (f y)" using assms(6) unfolding distrib[THEN sym] by auto finally show ?thesis using assms unfolding convex_on_def by fastsimp @@ -481,8 +481,8 @@ hence xpos: "?x \ C" using asm unfolding convex_alt by fastsimp have geq: "\ * (f x - f ?x) + (1 - \) * (f y - f ?x) \ \ * f' ?x * (x - ?x) + (1 - \) * f' ?x * (y - ?x)" - using add_mono[OF mult_mono1[OF leq[OF xpos asm(2)] `\ \ 0`] - mult_mono1[OF leq[OF xpos asm(3)] `1 - \ \ 0`]] by auto + using add_mono[OF mult_left_mono[OF leq[OF xpos asm(2)] `\ \ 0`] + mult_left_mono[OF leq[OF xpos asm(3)] `1 - \ \ 0`]] by auto hence "\ * f x + (1 - \) * f y - f ?x \ 0" by (auto simp add:field_simps) thus "f (\ *\<^sub>R x + (1 - \) *\<^sub>R y) \ \ * f x + (1 - \) * f y"