Exercise 2.14

Let P be a bounded polyhedron in n, let a be a vector in n, and let b be some scalar. We define

Q = {x Pax = b}.

Show that every extreme point of Q is either an extreme point of P or a convex combination of two adjacent extreme points of P.

Answers

By definition, we can write P as {x nAx = b} for some m × n matrix A and an m-dimensional vector b. Since Q is just P with one more additional hyperplane constraint, we can write Q as

Q = {x n [ A a a ]x = [ b b b ] }.

In other words, the resulting figure Q is another polyhedron inside P and since it always intersects the edges of P, its own extreme points will either be the extreme points of P or will strictly lie on the edges of P as demonstrated in the figure below. We formalize this intuition.

PIC

Figure 1: Intersecting a cube with hyperplane results in a polyhedron of lower dimension.

Proof. If Q is empty, the assertion is trivial. Else, let x be an arbitrary extreme point of Q. By Definition 2.9, n out of the active constraints in x are active. But x is also an element of P; We have two cases.

If the newly added condition ax = b is linearly dependent in x, then, even after excluding it, x still has n linearly independent active constraints in P as well; thus, x is an extreme point of P.

If, however, x P has n 1 linearly independent constraints after excluding the new condition ax = b, then all of the vectors ai, 1 i n 1, lie in a proper subspace of n and there exists a nonzero vector d n such that aid = 0, for every 1 i n 1. The scenario is similar to the setting of Theorem 2.6, yet the condition is stronger - P is bounded. We modify the proof a little. Let us consider the line consisting of all points of the form y = x± λd, where λ is an arbitrary positive scalar. For 1 i n 1, we have aiy = aix + λaid = aix = bi. Thus, those constraints that are active at x remain active at all points on the line. However, since the polyhedron P is assumed to be bounded, it follows that as we wary λ in two directions, some constraints will be eventually violated. At the points where some constraints are about to be violated, a new constraint must become active, and we conclude that there exits some λ+,an+ and some λ,an+ such that

an+(x + λ+d) = b i+,a n(x λd) = b i.

PIC
Figure 2: Moving from x (green point) to x + λ+d and x λd (red points).

The obtained columns an+ and an are linearly independent of the vectors ai, 1 i n 1. Indeed, we have anxbn± and an(x + λ±) = bn± (by the definition of λ+,λ). Thus, ajd0. On the other hand, and = 0 for every 1 i n 1 (by definition of d) and therefore, d is orthogonal to any linear combination of the vectors ai, 1 i n. Since d is not orthogonal to an+ and an, we conclude that aj is not a linear combination of the vectors ai, 1 i n. Thus, the points y+ := x + λ+d and y := x λd are two adjacent vertices of P and we have

x = λ λ + λ+y+ + λ+ λ + λ+y.

as desired. □

User profile picture
2021-12-11 15:51
Comments

Assume Q. Let A,d be a matrix and a vector such that P = {x nAx d}. Let x^ be an extreme point of Q, equivalently it is a basic feasible solution. Therefore ax^ = b and there are n linearly independent active constraints at x^ (possibly including ax^ = b in these n constraints).

If it is possible to find n linearly independent active constraints at x^ all in the collection Ax^ d, it implies that x^ is an extreme point of P too.

Otherwise there are only n 1 linearly independent active constraints in the set of constraints Ax^ d, which means that x^ lies on a face of dimension 1 of P. Let v n be the direction of the face on which x^ lies. Since P is bounded, there exist scalars μ1,μ2 such that x^ + μ1v and x^ + μ2v are the two vertices (extreme points) of the segment x^ is on. Therefore x^ is a convex combination of these two vectors.

User profile picture
2021-12-11 19:35
Comments
  • Hello, I didn't understand very well the part where it is mentioned that "Otherwise there are only $n-1$ linearly independent active constraints in the set of constraints $A\hat{x} \leq d$". It is not so clear to me why it is possible to ensure that proposition, could you please explain to me?
    BSupreme2024-04-17
  • To Nicolas: because $a^Tx=b$ is just one single extra constraint defining Q besides the constraints defining P.
    GT_Buzz2024-08-27