Topological properties of matrices #
This file is a place to collect topological results about matrices.
Main definitions: #
Matrix.topologicalRing
: square matrices form a topological ring
Main results #
- Sets of matrices:
IsOpen.matrix
: the set of finite matrices with entries in an open set is itself an open set.IsCompact.matrix
: the set of matrices with entries in a compact set is itself a compact set.
- Continuity:
Continuous.matrix_det
: the determinant is continuous over a topological ring.Continuous.matrix_adjugate
: the adjugate is continuous over a topological ring.
- Infinite sums
Matrix.transpose_tsum
: transpose commutes with infinite sumsMatrix.diagonal_tsum
: diagonal commutes with infinite sumsMatrix.blockDiagonal_tsum
: block diagonal commutes with infinite sumsMatrix.blockDiagonal'_tsum
: non-uniform block diagonal commutes with infinite sums
The topology on finite matrices over a discrete space is discrete.
Lemmas about continuity of operations #
To show a function into matrices is continuous it suffices to show the coefficients of the resulting matrix are continuous
Alias of Continuous.matrix_replicateCol
.
Alias of Continuous.matrix_replicateRow
.
Alias of Continuous.dotProduct
.
For square matrices the usual continuous_mul
can be used.
When Ring.inverse
is continuous at the determinant (such as in a NormedRing
, or a
topological field), so is Matrix.inv
.
Lemmas about infinite sums #
Lemmas about matrix groups #
The determinant is continuous as a map from the general linear group to the units.
If R
is a commutative ring with the discrete topology, then SL(n, R)
has the discrete
topology.
The special linear group over a topological ring is a topological group.
The natural map from SL n A
to GL n A
is continuous.
The natural map from SL n A
to GL n A
is inducing, i.e. the topology on
SL n A
is the pullback of the topology from GL n A
.
The natural map from SL n A
in GL n A
is an embedding, i.e. it is an injection and
the topology on SL n A
coincides with the subspace topology from GL n A
.
The natural inclusion of SL n A
in GL n A
is a closed embedding.