src/HOL/Library/Convex.thy
changeset 63918 6bf55e6e0b75
parent 63649 e690d6f2185b
--- a/src/HOL/Library/Convex.thy	Mon Sep 19 12:53:30 2016 +0200
+++ b/src/HOL/Library/Convex.thy	Mon Sep 19 20:06:21 2016 +0200
@@ -633,7 +633,7 @@
             OF asum_le less_imp_le[OF i0]], of "a i * f (y i)"]
       by simp
     also have "\<dots> = (\<Sum> j \<in> s. (1 - a i) * ?a j * f (y j)) + a i * f (y i)"
-      unfolding setsum_right_distrib[of "1 - a i" "\<lambda> j. ?a j * f (y j)"]
+      unfolding setsum_distrib_left[of "1 - a i" "\<lambda> j. ?a j * f (y j)"]
       using i0 by auto
     also have "\<dots> = (\<Sum> j \<in> s. a j * f (y j)) + a i * f (y i)"
       using i0 by auto