Polar set #
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 #
LinearMap.polar
: The polar of a bilinear formB : E โโ[๐] F โโ[๐] ๐
.
Main statements #
LinearMap.polar_eq_iInter
: The polar as an intersection.LinearMap.subset_bipolar
: The polar is a subset of the bipolar.LinearMap.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
.
Instances For
The map B.polar : Set E โ Set F
forms an order-reversing Galois connection with
B.flip.polar : Set F โ Set E
. We use OrderDual.toDual
and OrderDual.ofDual
to express
that polar
is order-reversing.
The polar set is closed in the weak topology induced by B.flip
.
The polar of a set closed under scalar multiplication as a submodule
Equations
- B.polarSubmodule m = (โจ x โ m, LinearMap.ker (B x)).copy (B.polar โm) โฏ
Instances For
Alias of StrongDual.dualPairing_separatingLeft
.
Given a subset s
in a monoid M
(over a commutative ring R
), the polar polar R s
is the
subset of StrongDual R M
consisting of those functionals which evaluate to something of norm at
most one at all points z โ s
.
Equations
- StrongDual.polar R = (topDualPairing R M).flip.polar
Instances For
Alias of StrongDual.polar
.
Given a subset s
in a monoid M
(over a commutative ring R
), the polar polar R s
is the
subset of StrongDual R M
consisting of those functionals which evaluate to something of norm at
most one at all points z โ s
.
Equations
Instances For
Given a subset s
in a monoid M
(over a field ๐
) closed under scalar multiplication,
the polar polarSubmodule ๐ s
is the submodule of StrongDual ๐ M
consisting of those functionals
which evaluate to zero at all points z โ s
.
Equations
- StrongDual.polarSubmodule ๐ m = (topDualPairing ๐ M).flip.polarSubmodule m
Instances For
Alias of StrongDual.polarSubmodule
.
Given a subset s
in a monoid M
(over a field ๐
) closed under scalar multiplication,
the polar polarSubmodule ๐ s
is the submodule of StrongDual ๐ M
consisting of those functionals
which evaluate to zero at all points z โ s
.
Instances For
Alias of StrongDual.polarSubmodule_eq_polar
.
Alias of StrongDual.mem_polar_iff
.
Alias of StrongDual.polarSubmodule_eq_setOf
.
Alias of StrongDual.mem_polarSubmodule
.
Alias of StrongDual.zero_mem_polar
.
Alias of StrongDual.polar_nonempty
.
Alias of StrongDual.polar_empty
.
Alias of StrongDual.polar_singleton
.
Alias of StrongDual.mem_polar_singleton
.
Alias of StrongDual.polar_zero
.
Alias of StrongDual.polar_univ
.