Commit 2024-07-10 10:39 7bc13f8d
View on Github →feat(LinearAlgebra/LinearDisjoint): definition and properties of linearly disjoint of submodules (#12434)
This is part 1 of #9651.
We adapt the definitions in https://en.wikipedia.org/wiki/Linearly_disjoint.
Let R
be a commutative ring, S
be an R
-algebra (not necessarily commutative).
Two R
-submodules M
and N
in S
are linearly disjoint,
if the natural R
-linear map M ⊗[R] N →ₗ[R] S
(Submodule.mulMap M N
)
induced by the multiplication in S
is injective.
The following is the first equivalent characterization of linearly disjointness:
Submodule.LinearDisjoint.linearIndependent_left_of_flat
: ifM
andN
are linearly disjoint, ifN
is a flatR
-module, then for any family ofR
-linearly independent elements{ m_i }
ofM
, they are alsoN
-linearly independent, in the sense that theR
-linear map fromι →₀ N
toS
which maps{ n_i }
to the sum ofm_i * n_i
(Submodule.mulLeftMap N m
) is injective.Submodule.LinearDisjoint.of_basis_left
: conversely, if{ m_i }
is anR
-basis ofM
, which is alsoN
-linearly independent, thenM
andN
are linearly disjoint. Dually, we have:Submodule.LinearDisjoint.linearIndependent_right_of_flat
: ifM
andN
are linearly disjoint, ifM
is a flatR
-module, then for any family ofR
-linearly independent elements{ n_i }
ofN
, they are alsoM
-linearly independent, in the sense that theR
-linear map fromι →₀ M
toS
which maps{ m_i }
to the sum ofm_i * n_i
(Submodule.mulRightMap M n
) is injective.Submodule.LinearDisjoint.of_basis_right
: conversely, if{ n_i }
is anR
-basis ofN
, which is alsoM
-linearly independent, thenM
andN
are linearly disjoint. The following is the second equivalent characterization of linearly disjointness:Submodule.LinearDisjoint.linearIndependent_mul_of_flat
: ifM
andN
are linearly disjoint, if one ofM
andN
is flat, then for any family ofR
-linearly independent elements{ m_i }
ofM
, and any family ofR
-linearly independent elements{ n_j }
ofN
, the family{ m_i * n_j }
inS
is alsoR
-linearly independent.Submodule.LinearDisjoint.of_basis_mul
: conversely, if{ m_i }
is anR
-basis ofM
, if{ n_i }
is anR
-basis ofN
, such that the family{ m_i * n_j }
inS
isR
-linearly independent, thenM
andN
are linearly disjoint. Other results:Submodule.LinearDisjoint.symm_of_commute
,Submodule.linearDisjoint_symm_of_commute
: linearly disjoint is symmetric under some commutative conditions.Submodule.linearDisjoint_op
: linearly disjoint is preserved by taking multiplicative opposite.Submodule.LinearDisjoint.of_le_left_of_flat
,Submodule.LinearDisjoint.of_le_right_of_flat
,Submodule.LinearDisjoint.of_le_of_flat_left
,Submodule.LinearDisjoint.of_le_of_flat_right
: linearly disjoint is preserved by taking submodules under some flatness conditions.Submodule.LinearDisjoint.of_linearDisjoint_fg_left
,Submodule.LinearDisjoint.of_linearDisjoint_fg_right
,Submodule.LinearDisjoint.of_linearDisjoint_fg
: conversely, if any finitely generated submodules ofM
andN
are linearly disjoint, thenM
andN
themselves are linearly disjoint.Submodule.LinearDisjoint.bot_left
,Submodule.LinearDisjoint.bot_right
: the zero module is linearly disjoint with any other submodules.Submodule.LinearDisjoint.one_left
,Submodule.LinearDisjoint.one_right
: the image ofR
inS
is linearly disjoint with any other submodules.Submodule.LinearDisjoint.of_left_le_one_of_flat
,Submodule.LinearDisjoint.of_right_le_one_of_flat
: if a submodule is contained in the image ofR
inS
, then it is linearly disjoint with any other submodules, under some flatness conditions.Submodule.LinearDisjoint.not_linearIndependent_pair_of_commute_of_flat
,Submodule.LinearDisjoint.rank_inf_le_one_of_commute_of_flat
: ifM
andN
are linearly disjoint, if one ofM
andN
is flat, then any two commutative elements contained in the intersection ofM
andN
are notR
-linearly independent (namely, their span is notR ^ 2
). In particular, if any two elements in the intersection ofM
andN
are commutative, then the rank of the intersection ofM
andN
is at most one.Submodule.LinearDisjoint.rank_le_one_of_commute_of_flat_of_self
: ifM
and itself are linearly disjoint, ifM
is flat, if any two elements inM
are commutative, then the rank ofM
is at most one. The results with name containing "of_commute" also have corresponding specified versions assumingS
is commutative.