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
A continuous alternating map from ι → M to N, denoted M [⋀^ι]→L[R] N,
is a continuous map 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 = 0whenevervhas two equal coordinates.
- toFun : (ι → M) → N
- map_update_add' [DecidableEq ι] (m : ι → M) (i : ι) (x y : M) : self.toFun (Function.update m i (x + y)) = self.toFun (Function.update m i x) + self.toFun (Function.update m i y)
- map_update_smul' [DecidableEq ι] (m : ι → M) (i : ι) (c : R) (x : M) : self.toFun (Function.update m i (c • x)) = c • self.toFun (Function.update m i x)
- cont : Continuous self.toFun
Instances For
A continuous alternating map from ι → M to N, denoted M [⋀^ι]→L[R] N,
is a continuous map 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 = 0whenevervhas two equal coordinates.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Restrict the codomain of a continuous alternating map to a submodule.
Equations
- f.codRestrict p h = { toContinuousMultilinearMap := f.codRestrict p h, map_eq_zero_of_eq' := ⋯ }
Instances For
Equations
- ContinuousAlternatingMap.instInhabited = { default := 0 }
Equations
- ContinuousAlternatingMap.instMulAction = { toSMul := ContinuousAlternatingMap.instSMul, one_smul := ⋯, mul_smul := ⋯ }
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
Evaluation of a ContinuousAlternatingMap at a vector as an AddMonoidHom.
Equations
Instances For
Projection to ContinuousMultilinearMaps as a bundled AddMonoidHom.
Equations
- ContinuousAlternatingMap.toMultilinearAddHom = { toFun := fun (f : M [⋀^ι]→L[R] N) => f.toContinuousMultilinearMap, map_zero' := ⋯, map_add' := ⋯ }
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.
Equations
- f.toContinuousLinearMap m i = f.toContinuousLinearMap m i
Instances For
The Cartesian product of two continuous alternating maps, as a continuous alternating map.
Equations
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.
Equations
- ContinuousAlternatingMap.pi f = { toContinuousMultilinearMap := ContinuousMultilinearMap.pi fun (i : ι') => (f i).toContinuousMultilinearMap, map_eq_zero_of_eq' := ⋯ }
Instances For
The natural equivalence between continuous linear maps from M to N
and continuous 1-multilinear alternating maps from M to N.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The constant map is alternating when ι is empty.
Equations
- ContinuousAlternatingMap.constOfIsEmpty R M ι m = { toContinuousMultilinearMap := ContinuousMultilinearMap.constOfIsEmpty R (fun (x : ι) => M) m, map_eq_zero_of_eq' := ⋯ }
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.
Equations
- g.compContinuousLinearMap f = { toContinuousMultilinearMap := g.compContinuousLinearMap fun (x : ι) => f, map_eq_zero_of_eq' := ⋯ }
Instances For
Composing a continuous alternating map with a continuous linear map gives again a continuous alternating map.
Equations
- g.compContinuousAlternatingMap f = { toContinuousMultilinearMap := g.compContinuousMultilinearMap f.toContinuousMultilinearMap, map_eq_zero_of_eq' := ⋯ }
Instances For
A continuous linear equivalence of domains defines an equivalence between continuous alternating maps.
This is available as a continuous linear isomorphism at
ContinuousLinearEquiv.continuousAlternatingMapCongrLeft.
This is ContinuousAlternatingMap.compContinuousLinearMap as an equivalence.
Equations
- One or more equations did not get rendered due to their size.
Instances For
A continuous linear equivalence of codomains defines an equivalence between continuous alternating maps.
Equations
- e.continuousAlternatingMapCongrRightEquiv = { toFun := (↑e).compContinuousAlternatingMap, invFun := (↑e.symm).compContinuousAlternatingMap, left_inv := ⋯, right_inv := ⋯ }
Instances For
Continuous linear equivalences between domains and codomains define an equivalence between the spaces of continuous alternating maps.
Equations
Instances For
ContinuousAlternatingMap.pi as an Equiv.
Equations
- One or more equations did not get rendered due to their size.
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.
Equations
- ContinuousAlternatingMap.restrictScalars R f = { toContinuousMultilinearMap := ContinuousMultilinearMap.restrictScalars R f.toContinuousMultilinearMap, map_eq_zero_of_eq' := ⋯ }
Instances For
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
Multiplicativity of a continuous alternating map along all coordinates at the same time,
writing f (fun i ↦ c i • m i) as (∏ i, c i) • f m.
If two continuous R-alternating maps from R are equal on 1, then they are equal.
This is the alternating version of ContinuousLinearMap.ext_ring.
The only continuous R-alternating map from two or more copies of R is the zero map.
Equations
- ContinuousAlternatingMap.uniqueOfCommRing = { toInhabited := ContinuousAlternatingMap.instInhabited, uniq := ⋯ }
Equations
- ContinuousAlternatingMap.instDistribMulAction = { toMulAction := ContinuousAlternatingMap.instMulAction, smul_zero := ⋯, smul_add := ⋯ }
The space of continuous alternating maps over an algebra over R is a module over R, for the
pointwise addition and scalar multiplication.
Equations
- ContinuousAlternatingMap.instModule = { toDistribMulAction := ContinuousAlternatingMap.instDistribMulAction, add_smul := ⋯, zero_smul := ⋯ }
Linear map version of the map toMultilinearMap associating to a continuous alternating map
the corresponding multilinear map.
Equations
- ContinuousAlternatingMap.toContinuousMultilinearMapLinear = { toFun := ContinuousAlternatingMap.toContinuousMultilinearMap, map_add' := ⋯, map_smul' := ⋯ }
Instances For
Linear map version of the map toAlternatingMap
associating to a continuous alternating map the corresponding alternating map.
Equations
- ContinuousAlternatingMap.toAlternatingMapLinear = { toFun := ContinuousAlternatingMap.toAlternatingMap, map_add' := ⋯, map_smul' := ⋯ }
Instances For
ContinuousAlternatingMap.pi as a LinearEquiv.
Equations
- One or more equations did not get rendered due to their size.
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.
Equations
- ContinuousAlternatingMap.compContinuousLinearMapₗ f = { toFun := fun (g : M' [⋀^ι]→L[R] N) => g.compContinuousLinearMap f, map_add' := ⋯, map_smul' := ⋯ }
Instances For
ContinuousLinearMap.compContinuousAlternatingMap as a bundled bilinear map.
Equations
Instances For
Alternatization of a continuous multilinear map.
Equations
- One or more equations did not get rendered due to their size.