Block Matrices from Rows and Columns #
This file provides the basic definitions of matrices composed from columns and rows.
The concatenation of two matrices with the same row indices can be expressed as
A = fromCols A₁ A₂
the concatenation of two matrices with the same column indices
can be expressed as B = fromRows B₁ B₂
.
We then provide a few lemmas that deal with the products of these with each other and with block matrices
Tags #
column matrices, row matrices, column row block matrices
Alias of Matrix.fromCols
.
Concatenate together two matrices B₁[m × n₁] and B₂[m × n₂] with the same rows (M) to get a bigger matrix indexed by [m × (n₁ ⊕ n₂)]
Equations
Instances For
Alias of Matrix.toCols₁
.
Given a column partitioned matrix extract the first column
Equations
Instances For
Alias of Matrix.toCols₂
.
Given a column partitioned matrix extract the second column
Equations
Instances For
Alias of Matrix.toCols₁_fromCols
.
Alias of Matrix.toCols₂_fromCols
.
Alias of Matrix.fromCols_toCols
.
Alias of Matrix.fromCols_inj
.
Alias of Matrix.fromCols_ext_iff
.
A column partitioned matrix when transposed gives a row partitioned matrix with columns of the initial matrix transposed to become rows.
Alias of Matrix.transpose_fromCols
.
A column partitioned matrix when transposed gives a row partitioned matrix with columns of the initial matrix transposed to become rows.
A row partitioned matrix when transposed gives a column partitioned matrix with rows of the initial matrix transposed to become columns.
Alias of Matrix.fromCols_neg
.
Negating a matrix partitioned by columns is equivalent to negating each of the columns.
Alias of Matrix.fromCols_fromRows_eq_fromBlocks
.
Alias of Matrix.fromRows_fromCols_eq_fromBlocks
.
Alias of Matrix.vecMul_fromCols
.
Alias of Matrix.fromCols_mulVec_sum_elim
.
Alias of Matrix.fromCols_zero
.
A row partitioned matrix multiplied by a column partitioned matrix gives a 2 by 2 block matrix.
Alias of Matrix.fromRows_mul_fromCols
.
A row partitioned matrix multiplied by a column partitioned matrix gives a 2 by 2 block matrix.
A column partitioned matrix multiplied by a row partitioned matrix gives the sum of the "outer" products of the block matrices.
Alias of Matrix.fromCols_mul_fromRows
.
A column partitioned matrix multiplied by a row partitioned matrix gives the sum of the "outer" products of the block matrices.
A column partitioned matrix multipiled by a block matrix results in a column partitioned matrix.
Alias of Matrix.fromCols_mul_fromBlocks
.
A column partitioned matrix multipiled by a block matrix results in a column partitioned matrix.
A block matrix multiplied by a row partitioned matrix gives a row partitioned matrix.
Multiplication of a matrix by its inverse is commutative.
This is the column and row partitioned matrix form of Matrix.mul_eq_one_comm
.
The condition e : n ≃ n₁ ⊕ n₂
states that fromCols A₁ A₂
and fromRows B₁ B₂
are "square".
Alias of Matrix.fromCols_mul_fromRows_eq_one_comm
.
Multiplication of a matrix by its inverse is commutative.
This is the column and row partitioned matrix form of Matrix.mul_eq_one_comm
.
The condition e : n ≃ n₁ ⊕ n₂
states that fromCols A₁ A₂
and fromRows B₁ B₂
are "square".
The lemma fromCols_mul_fromRows_eq_one_comm
specialized to the case where the index sets
n₁
and n₂
, are the result of subtyping by a predicate and its complement.
Alias of Matrix.equiv_compl_fromCols_mul_fromRows_eq_one_comm
.
The lemma fromCols_mul_fromRows_eq_one_comm
specialized to the case where the index sets
n₁
and n₂
, are the result of subtyping by a predicate and its complement.
A column partitioned matrix in a Star ring when conjugate transposed gives a row partitioned matrix with the columns of the initial matrix conjugate transposed to become rows.
Alias of Matrix.conjTranspose_fromCols_eq_fromRows_conjTranspose
.
A column partitioned matrix in a Star ring when conjugate transposed gives a row partitioned matrix with the columns of the initial matrix conjugate transposed to become rows.
A row partitioned matrix in a Star ring when conjugate transposed gives a column partitioned matrix with the rows of the initial matrix conjugate transposed to become columns.
Alias of Matrix.conjTranspose_fromRows_eq_fromCols_conjTranspose
.
A row partitioned matrix in a Star ring when conjugate transposed gives a column partitioned matrix with the rows of the initial matrix conjugate transposed to become columns.