Basic lemmas about the general linear group $GL(n, R)$ #
This file lists various basic lemmas about the general linear group $GL(n, R)$. For the definitions,
see LinearAlgebra/Matrix/GeneralLinearGroup/Defs.lean
.
The matrix [a, -b; b, a] (inspired by multiplication by a complex number); it is an element of
$GL_2(R)$ if a ^ 2 + b ^ 2
is nonzero.
Equations
- Matrix.planeConformalMatrix a b hab = Matrix.GeneralLinearGroup.mkOfDetNeZero !![a, -b; b, a] ⋯
Instances For
theorem
Matrix.GeneralLinearGroup.mem_center_iff_val_eq_scalar
{R : Type u_1}
{n : Type u_2}
[Fintype n]
[DecidableEq n]
[CommRing R]
{g : GL n R}
:
The center of GL n R
consists of scalar matrices.
theorem
Matrix.GeneralLinearGroup.center_eq_range_units
{R : Type u_1}
{n : Type u_2}
[Fintype n]
[DecidableEq n]
[CommRing R]
:
The center of GL n R
is the image of Rˣ
.