Continuous alternating multilinear maps #
In this file we define bundled continuous alternating maps and develop basic API about these maps, by reusing API about continuous multilinear maps and alternating maps.
Notation #
M [Λ^ι]→L[R] N
: notation for R
-linear continuous alternating maps from M
to N
; the arguments
are indexed by i : ι
.
Keywords #
multilinear map, alternating map, continuous
- toFun : (ι → M) → N
- map_add' : ∀ [inst : DecidableEq ι] (m : ι → M) (i : ι) (x y : M), MultilinearMap.toFun s.toMultilinearMap (Function.update m i (x + y)) = MultilinearMap.toFun s.toMultilinearMap (Function.update m i x) + MultilinearMap.toFun s.toMultilinearMap (Function.update m i y)
- map_smul' : ∀ [inst : DecidableEq ι] (m : ι → M) (i : ι) (c : R) (x : M), MultilinearMap.toFun s.toMultilinearMap (Function.update m i (c • x)) = c • MultilinearMap.toFun s.toMultilinearMap (Function.update m i x)
- cont : Continuous s.toFun
- map_eq_zero_of_eq' : ∀ (v : ι → M) (i j : ι), v i = v j → i ≠ j → MultilinearMap.toFun s.toMultilinearMap v = 0
The map is alternating: if
v
has two equal coordinates, thenf v = 0
.
A continuous alternating map is a continuous map from ι → M
to N
that is
- multilinear :
f (update m i (c • x)) = c • f (update m i x)
andf (update m i (x + y)) = f (update m i x) + f (update m i y)
; - alternating :
f v = 0
wheneverv
has two equal coordinates.
Instances For
Projection to AlternatingMap
s.
Instances For
Restrict the codomain of a continuous alternating map to a submodule.
Instances For
Evaluation of a ContinuousAlternatingMap
at a vector as an AddMonoidHom
.
Instances For
Projection to ContinuousMultilinearMap
s as a bundled AddMonoidHom
.
Instances For
If f
is a continuous alternating map, then f.toContinuousLinearMap m i
is the continuous
linear map obtained by fixing all coordinates but i
equal to those of m
, and varying the
i
-th coordinate.
Instances For
The cartesian product of two continuous alternating maps, as a continuous alternating map.
Instances For
Combine a family of continuous alternating maps with the same domain and codomains M' i
into a
continuous alternating map taking values in the space of functions Π i, M' i
.
Instances For
The evaluation map from ι → M
to M
is alternating at a given i
when ι
is subsingleton.
Instances For
The constant map is alternating when ι
is empty.
Instances For
If g
is continuous alternating and f
is a continuous linear map, then g (f m₁, ..., f mₙ)
is again a continuous alternating map, that we call g.compContinuousLinearMap f
.
Instances For
Composing a continuous alternating map with a continuous linear map gives again a continuous alternating map.
Instances For
A continuous linear equivalence of domains defines an equivalence between continuous alternating maps.
Instances For
A continuous linear equivalence of codomains defines an equivalence between continuous alternating maps.
Instances For
Continuous linear equivalences between domains and codomains define an equivalence between the spaces of continuous alternating maps.
Instances For
ContinuousAlternatingMap.pi
as an Equiv
.
Instances For
In the specific case of continuous alternating maps on spaces indexed by Fin (n+1)
, where one
can build an element of Π(i : Fin (n+1)), M i
using cons
, one can express directly the
additivity of an alternating map along the first variable.
In the specific case of continuous alternating maps on spaces indexed by Fin (n+1)
, where one
can build an element of Π(i : Fin (n+1)), M i
using cons
, one can express directly the
additivity of an alternating map along the first variable.
In the specific case of continuous alternating maps on spaces indexed by Fin (n+1)
, where one
can build an element of Π(i : Fin (n+1)), M i
using cons
, one can express directly the
multiplicativity of an alternating map along the first variable.
In the specific case of continuous alternating maps on spaces indexed by Fin (n+1)
, where one
can build an element of Π(i : Fin (n+1)), M i
using cons
, one can express directly the
multiplicativity of an alternating map along the first variable.
Additivity of a continuous alternating map along all coordinates at the same time,
writing f (m + m')
as the sum of f (s.piecewise m m')
over all sets s
.
If f
is continuous alternating, then f (Σ_{j₁ ∈ A₁} g₁ j₁, ..., Σ_{jₙ ∈ Aₙ} gₙ jₙ)
is the
sum of f (g₁ (r 1), ..., gₙ (r n))
where r
ranges over all functions with r 1 ∈ A₁
, ...,
r n ∈ Aₙ
. This follows from multilinearity by expanding successively with respect to each
coordinate.
If f
is continuous alternating, then f (Σ_{j₁} g₁ j₁, ..., Σ_{jₙ} gₙ jₙ)
is the sum of
f (g₁ (r 1), ..., gₙ (r n))
where r
ranges over all functions r
. This follows from
multilinearity by expanding successively with respect to each coordinate.
Reinterpret a continuous A
-alternating map as a continuous R
-alternating map, if A
is an
algebra over R
and their actions on all involved modules agree with the action of R
on A
.
Instances For
Multiplicativity of a continuous alternating map along all coordinates at the same time,
writing f (λ i, c i • m i)
as (∏ i, c i) • f m
.
The space of continuous alternating maps over an algebra over R
is a module over R
, for the
pointwise addition and scalar multiplication.
Linear map version of the map toMultilinearMap
associating to a continuous alternating map
the corresponding multilinear map.
Instances For
ContinuousAlternatingMap.pi
as a LinearEquiv
.
Instances For
Given a continuous R
-alternating map f
taking values in R
, f.smulRight z
is the
continuous alternating map sending m
to f m • z
.
Instances For
ContinuousAlternatingMap.compContinuousLinearMap
as a bundled LinearMap
.
Instances For
ContinuousLinearMap.compContinuousAlternatingMap
as a bundled bilinear map.
Instances For
Alternatization of a continuous multilinear map.