Polar set #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
In this file we define the polar set. There are different notions of the polar, we will define the
absolute polar. The advantage over the real polar is that we can define the absolute polar for
any bilinear form B : E →ₗ[𝕜] F →ₗ[𝕜] 𝕜
, where 𝕜
is a normed commutative ring and
E
and F
are modules over 𝕜
.
Main definitions #
linear_map.polar
: The polar of a bilinear formB : E →ₗ[𝕜] F →ₗ[𝕜] 𝕜
.
Main statements #
linear_map.polar_eq_Inter
: The polar as an intersection.linear_map.subset_bipolar
: The polar is a subset of the bipolar.linear_map.polar_weak_closed
: The polar is closed in the weak topology induced byB.flip
.
References #
Tags #
polar
The (absolute) polar of s : set E
is given by the set of all y : F
such that ‖B x y‖ ≤ 1
for all x ∈ s
.
The map B.polar : set E → set F
forms an order-reversing Galois connection with
B.flip.polar : set F → set E
. We use order_dual.to_dual
and order_dual.of_dual
to express
that polar
is order-reversing.
The polar set is closed in the weak topology induced by B.flip
.