Math Problem Statement

The following lemma (called Farkas’ Lemma) is a useful consequence of the separating hyperplane theorem. Lemma 1. Let A ∈ RM×N and b ∈ RM. Exactly one of the following is true: (a) there exists a vector x ∈ R N + such that Ax = b. (b) there exists λ ∈ RM such that AT λ ≤ 0, and λ T · b > 0.Prove the lemma (for arbitrary A).

Solution

To prove this version of Farkas' Lemma using the separating hyperplane theorem, let's restate the lemma clearly:

Farkas' Lemma:

Let ARM×NA \in \mathbb{R}^{M \times N} and bRMb \in \mathbb{R}^M. Exactly one of the following two statements is true:

  1. There exists a vector xR+Nx \in \mathbb{R}^N_+ (meaning x0x \geq 0 component-wise) such that Ax=bAx = b.
  2. There exists a vector λRM\lambda \in \mathbb{R}^M such that ATλ0A^T \lambda \leq 0 (component-wise), and λTb>0\lambda^T b > 0.

Proof:

  1. Assume (1) is true:

    • There exists x0x \geq 0 such that Ax=bAx = b.
    • Now, assume for contradiction that (2) also holds.
    • This means there exists λRM\lambda \in \mathbb{R}^M such that ATλ0A^T \lambda \leq 0 and λTb>0\lambda^T b > 0.
    • Consider the expression λTb=λTAx\lambda^T b = \lambda^T A x.
    • Since λTA0\lambda^T A \leq 0 and x0x \geq 0, it follows that λTAx0\lambda^T A x \leq 0.
    • However, we assumed that λTb>0\lambda^T b > 0, which contradicts λTb=λTAx0\lambda^T b = \lambda^T A x \leq 0.
    • Therefore, if (1) is true, (2) cannot be true.
  2. Assume (1) is false:

    • This means there is no x0x \geq 0 such that Ax=bAx = b.
    • Let C={Ax:x0}RMC = \{Ax : x \geq 0\} \subset \mathbb{R}^M. This set CC is a convex cone.
    • Since bCb \notin C, by the separating hyperplane theorem, there exists a nonzero vector λRM\lambda \in \mathbb{R}^M and a scalar γ\gamma such that: λTyγfor all yC,\lambda^T y \leq \gamma \quad \text{for all } y \in C, λTb>γ.\lambda^T b > \gamma.
    • Since CC is a cone (closed under non-negative scalar multiplication), the inequality for all yCy \in C implies γ\gamma must be non-positive (i.e., γ0\gamma \leq 0).
    • If γ<0\gamma < 0, then for any x0x \geq 0, we would have λTAxγ<0\lambda^T A x \leq \gamma < 0, contradicting the existence of any x0x \geq 0 such that Ax=bAx = b.
    • Hence, γ=0\gamma = 0 and thus λTAx0\lambda^T A x \leq 0 for all x0x \geq 0. This means ATλ0A^T \lambda \leq 0.
    • Moreover, since λTb>γ=0\lambda^T b > \gamma = 0, it follows that λTb>0\lambda^T b > 0.
    • Therefore, (2) must hold if (1) does not.

This completes the proof of Farkas' Lemma: either (1) or (2) holds, but not both simultaneously.

Would you like to delve into any aspect of this proof further or have any questions?

Related Questions

  1. How does the separating hyperplane theorem apply to the proof of Farkas' Lemma?
  2. Can you provide an example illustrating Farkas' Lemma in practice?
  3. What is the significance of the condition λTb>0\lambda^T b > 0 in the lemma?
  4. How is Farkas' Lemma used in duality theory in linear programming?
  5. What are some practical applications of Farkas' Lemma in optimization problems?

Tip:

In understanding the role of the separating hyperplane theorem in Farkas' Lemma, it’s helpful to think about the geometric implications of the cone generated by AxAx and how it relates to the vector bb.

Ask a new question for Free

By Image

Drop file here or Click Here to upload

Math Problem Analysis

Mathematical Concepts

Linear Algebra
Convex Sets
Separating Hyperplane Theorem

Formulas

-

Theorems

Farkas' Lemma

Suitable Grade Level

Advanced Undergraduate