mathlib3 documentation

analysis.convex.cone.dual

Convex cones in inner product spaces #

THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.

We define set.inner_dual_cone to be the cone consisting of all points y such that for all points x in a given set 0 ≤ ⟪ x, y ⟫.

Main statements #

We prove the following theorems:

The dual cone #

The dual cone is the cone consisting of all points y such that for all points x in a given set 0 ≤ ⟪ x, y ⟫.

Equations
@[simp]
theorem mem_inner_dual_cone {H : Type u_5} [normed_add_comm_group H] [inner_product_space H] (y : H) (s : set H) :
@[simp]

Dual cone of the convex cone {0} is the total space.

@[simp]

Dual cone of the total space is the convex cone {0}.

The inner dual cone of a singleton is given by the preimage of the positive cone under the linear map λ y, ⟪x, y⟫.

theorem inner_dual_cone_Union {H : Type u_5} [normed_add_comm_group H] [inner_product_space H] {ι : Sort u_1} (f : ι set H) :
( (i : ι), f i).inner_dual_cone = (i : ι), (f i).inner_dual_cone

The dual cone of s equals the intersection of dual cones of the points in s.

This is a stronger version of the Hahn-Banach separation theorem for closed convex cones. This is also the geometric interpretation of Farkas' lemma.

The inner dual of inner dual of a non-empty, closed convex cone is itself.