The topological strong dual of a module #
Main definitions #
strongDualPairing
: The strong dual pairing as a bilinear form.StrongDual.polar
: Given a subsets
in a monoidM
(over a commutative ringR
), the polarpolar R s
is the subset ofStrongDual R M
consisting of those functionals which evaluate to something of norm at most one at all pointsz ∈ s
.StrongDual.polarSubmodule
: Given a subsets
in a monoidM
(over a field𝕜
) closed under scalar multiplication, the polarpolarSubmodule 𝕜 s
is the submodule ofStrongDual 𝕜 M
consisting of those functionals which evaluate to zero at all pointsz ∈ s
.
References #
Tags #
StrongDual, polar
The StrongDual pairing as a bilinear form.
Equations
Instances For
Alias of strongDualPairing
.
The StrongDual pairing as a bilinear form.
Instances For
Alias of StrongDual.dualPairing_apply
.
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 = (strongDualPairing 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 = (strongDualPairing 𝕜 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
.