Proper cones #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
We define a proper cone as a nonempty, closed, convex cone. Proper cones are used in defining conic programs which generalize linear programs. A linear program is a conic program for the positive cone. We then prove Farkas' lemma for conic programs following the proof in the reference below. Farkas' lemma is equivalent to strong duality. So, once have the definitions of conic programs and linear programs, the results from this file can be used to prove duality theorems.
TODO #
The next steps are:
- Add convex_cone_class that extends set_like and replace the below instance
- Define the positive cone as a proper cone.
- Define primal and dual cone programs and prove weak duality.
- Prove regular and strong duality for cone programs using Farkas' lemma (see reference).
- Define linear programs and prove LP duality as a special case of cone duality.
- Find a better reference (textbook instead of lecture notes).
- Show submodules are (proper) cones.
References #
The closure of a convex cone inside a topological space as a convex cone. This construction is mainly used for defining maps between proper cones.
- to_convex_cone : convex_cone 𝕜 E
- nonempty' : self.to_convex_cone.carrier.nonempty
- is_closed' : is_closed self.to_convex_cone.carrier
A proper cone is a convex cone K
that is nonempty and closed. Proper cones have the nice
property that the dual of the dual of a proper cone is itself. This makes them useful for defining
cone programs and proving duality theorems.
Instances for proper_cone
- proper_cone.has_sizeof_inst
- proper_cone.convex_cone.has_coe
- proper_cone.set_like
- proper_cone.has_zero
- proper_cone.inhabited
Equations
- proper_cone.convex_cone.has_coe = {coe := λ (K : proper_cone 𝕜 E), K.to_convex_cone}
Equations
- proper_cone.set_like = {coe := λ (K : proper_cone 𝕜 E), K.to_convex_cone.carrier, coe_injective' := _}
Equations
- proper_cone.has_zero = {zero := {to_convex_cone := 0, nonempty' := _, is_closed' := _}}
Equations
- proper_cone.inhabited = {default := 0}
The closure of image of a proper cone under a continuous ℝ
-linear map is a proper cone. We
use continuous maps here so that the comap of f is also a map between proper cones.
Equations
- proper_cone.map f K = {to_convex_cone := (convex_cone.map ↑f ↑K).closure, nonempty' := _, is_closed' := _}
The inner dual cone of a proper cone is a proper cone.
Equations
- K.dual = {to_convex_cone := ↑K.inner_dual_cone, nonempty' := _, is_closed' := _}
The preimage of a proper cone under a continuous ℝ
-linear map is a proper cone.
Equations
- proper_cone.comap f S = {to_convex_cone := convex_cone.comap ↑f ↑S, nonempty' := _, is_closed' := _}
The dual of the dual of a proper cone is itself.
This is a relative version of
convex_cone.hyperplane_separation_of_nonempty_of_is_closed_of_nmem
, which we recover by setting
f
to be the identity map. This is a geometric interpretation of the Farkas' lemma
stated using proper cones.