Exercise 1.2 (Sum of convex functions)

Suppose that f1,,fm are convex functions from n into and let f(x) = i=1mfi(x).

(a)
Show that if each fi is convex, so is f.
(b)
Show that if each fi is piecewise linear and convex, so is f.

Answers

(a)

Proof. Let x,y n and λ [0,1]. By convexity assumption on each of fi, we have

f (λx + (1 λ)y) = i=1mf i (λx + (1 λ)y) i=1mλf i (x) + (1 λ)fi (y) = λ i=1mf i (x) + (1 λ) i=1mf i (y) = λf (x) + (1 λ)f (y).
(b)

Proof. We induct on the number of functions m. The base case m = 1 is trivial. Now assume inductively that we have proven the theorem assertion for some m 𝔑. We then have

f (x) = i=1m+1f i (x) = i=1mf i (x) + fm+1 (x)

By definition, we can write fm+1(x) = max j=1, ,k (fjx + gj) for some vectors f1,,fk and scalars g1,,gk. At this point, we can employ the induction hypothesis and find some c1,,ck n and d1,,dk such that i=1mfi(x) = max i=1, ,k(cix + di). We then have

f (x) = max i=1, ,k (cix + d i) + max j=1, ,k (fjx + g j)

Using the fact that max iai + max jbj = max ijai + bj, we obtain

f (x) = max i=1, ,k;j=1, ,k (ci + f j)x + (d i + gj)

Enumerating all tuples (i,j) and renaming the (at most k k) vectors and scalars, we see that f is piecewise convex linear per definitionem. This closes the induction. □

User profile picture
2022-01-30 18:29
Comments
  • In part a, the second = should be $\ge$ by the definition of convexity, right?
    plodmatics2022-05-14
  • Correction added, thanks.
    eluthingol2022-05-17
  • how does summation of \(f(x)\) equals to piecewise linear convex function? \(\sum_{i=1}^{m} f_i(\mathbf{x}) = \max_{i=1,\ldots,k} (\mathbf{c}_i'\mathbf{x} + d_i)\)
    octocarl2022-10-08
  • @octocarl Summation of \(f(x)\) is not \(\sum_{i=1}^{m}f_i(\mathbf{x})\), it is \(\sum_{i=1}^{m+1}f_i(\mathbf{x})\). The fact that the latter is piecewise linear and convex follows by induction hypothesis, i.e., sum of any $m$ piecewise linear and convex functions is piecewise linear and convex. We then proceed to demonstrate that the same holds for \(m+1\), which is \(f(\mathbf{x})\).
    eluthingol2022-10-23
  • I'm also wondering how does the $\sum_{i=1}^m f_i(\mathbf{x})=\max _{i=1, \ldots, k}\left(\mathbf{c}_i^{\prime} \mathbf{x}+d_i\right)$? If $f_i$ is a piecewise linear convex function, doesn't that mean $f_i(\mathbf{x})=\max _{i=1, \ldots, k}\left(\mathbf{c}_i^{\prime} \mathbf{x}+d_i\right)$? Why the summation can be eliminated?
    johndst2023-09-28
  • The summation can be eliminated because \max_i a_i+\max_j b_j = \max_{i,j} {a_i+b_j}. Basically it means the summation of piecewise linear convex functions is still piecewise linear convex.
    Yulin2023-10-19