Extra lemmas about invertible matrices #
A few of the Invertible lemmas generalize to multiplication of rectangular matrices.
For lemmas about the matrix inverse in terms of the determinant and adjugate, see Matrix.inv
in LinearAlgebra/Matrix/NonsingularInverse.lean.
Main results #
A copy of invOf_mul_cancel_left for rectangular matrices.
A copy of mul_invOf_cancel_left for rectangular matrices.
A copy of invOf_mul_cancel_right for rectangular matrices.
A copy of mul_invOf_cancel_right for rectangular matrices.
A copy oy of invOf_mul_eq_iff_eq_mul_left for rectangular matrices.
A copy oy of mul_left_eq_iff_eq_invOf_mul for rectangular matrices.
A copy oy of mul_invOf_eq_iff_eq_mul_right for rectangular matrices.
A copy oy of mul_right_eq_iff_eq_mul_invOf for rectangular matrices.
The conjugate transpose of an invertible matrix is invertible.
Equations
A matrix is invertible if the conjugate transpose is invertible.
Equations
Instances For
The transpose of an invertible matrix is invertible.
Aᵀ is invertible when A is.
Equations
Instances For
Together Matrix.invertibleTranspose and Matrix.invertibleOfInvertibleTranspose form an
equivalence, although both sides of the equiv are subsingleton anyway.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Like add_mul_mul_invOf_mul_eq_one, but with multiplication reversed.
If matrices A, C, and C⁻¹ + V * A⁻¹ * U are invertible, then so is A + U * C * V.
Equations
Instances For
The Woodbury Identity (⅟ version).
See Matrix.invOf_add_mul_mul' for the Binomial Inverse Theorem.
If matrices A and C + C * V * A⁻¹ * U * C are invertible, then so is A + U * C * V.
Equations
Instances For
The Binomial Inverse Theorem (⅟ version).
See Matrix.invOf_add_mul_mul for the Woodbury identity.