Documentation

Mathlib.LinearAlgebra.Matrix.ZPow

Integer powers of square matrices #

In this file, we define integer power of matrices, relying on the nonsingular inverse definition for negative powers.

Implementation details #

The main definition is a direct recursive call on the integer inductive type, as provided by the DivInvMonoid.Pow default implementation. The lemma names are taken from Algebra.GroupWithZero.Power.

Tags #

matrix inverse, matrix powers

noncomputable instance Matrix.instDivInvMonoidMatrix {n' : Type u_1} [DecidableEq n'] [Fintype n'] {R : Type u_2} [CommRing R] :
Equations
  • Matrix.instDivInvMonoidMatrix = let __src := let_fun this := inferInstance; this; let __src_1 := let_fun this := inferInstance; this; DivInvMonoid.mk zpowRec
@[simp]
theorem Matrix.inv_pow' {n' : Type u_1} [DecidableEq n'] [Fintype n'] {R : Type u_2} [CommRing R] (A : Matrix n' n' R) (n : ) :
A⁻¹ ^ n = (A ^ n)⁻¹
theorem Matrix.pow_sub' {n' : Type u_1} [DecidableEq n'] [Fintype n'] {R : Type u_2} [CommRing R] (A : Matrix n' n' R) {m : } {n : } (ha : IsUnit (Matrix.det A)) (h : n m) :
A ^ (m - n) = A ^ m * (A ^ n)⁻¹
theorem Matrix.pow_inv_comm' {n' : Type u_1} [DecidableEq n'] [Fintype n'] {R : Type u_2} [CommRing R] (A : Matrix n' n' R) (m : ) (n : ) :
A⁻¹ ^ m * A ^ n = A ^ n * A⁻¹ ^ m
@[simp]
theorem Matrix.one_zpow {n' : Type u_1} [DecidableEq n'] [Fintype n'] {R : Type u_2} [CommRing R] (n : ) :
1 ^ n = 1
theorem Matrix.zero_zpow {n' : Type u_1} [DecidableEq n'] [Fintype n'] {R : Type u_2} [CommRing R] (z : ) :
z 00 ^ z = 0
theorem Matrix.zero_zpow_eq {n' : Type u_1} [DecidableEq n'] [Fintype n'] {R : Type u_2} [CommRing R] (n : ) :
0 ^ n = if n = 0 then 1 else 0
theorem Matrix.inv_zpow {n' : Type u_1} [DecidableEq n'] [Fintype n'] {R : Type u_2} [CommRing R] (A : Matrix n' n' R) (n : ) :
A⁻¹ ^ n = (A ^ n)⁻¹
@[simp]
theorem Matrix.zpow_neg_one {n' : Type u_1} [DecidableEq n'] [Fintype n'] {R : Type u_2} [CommRing R] (A : Matrix n' n' R) :
A ^ (-1) = A⁻¹
@[simp]
theorem Matrix.zpow_neg_natCast {n' : Type u_1} [DecidableEq n'] [Fintype n'] {R : Type u_2} [CommRing R] (A : Matrix n' n' R) (n : ) :
A ^ (-n) = (A ^ n)⁻¹
@[deprecated Matrix.zpow_neg_natCast]
theorem Matrix.zpow_neg_coe_nat {n' : Type u_1} [DecidableEq n'] [Fintype n'] {R : Type u_2} [CommRing R] (A : Matrix n' n' R) (n : ) :
A ^ (-n) = (A ^ n)⁻¹

Alias of Matrix.zpow_neg_natCast.

theorem IsUnit.det_zpow {n' : Type u_1} [DecidableEq n'] [Fintype n'] {R : Type u_2} [CommRing R] {A : Matrix n' n' R} (h : IsUnit (Matrix.det A)) (n : ) :
theorem Matrix.isUnit_det_zpow_iff {n' : Type u_1} [DecidableEq n'] [Fintype n'] {R : Type u_2} [CommRing R] {A : Matrix n' n' R} {z : } :
theorem Matrix.zpow_neg {n' : Type u_1} [DecidableEq n'] [Fintype n'] {R : Type u_2} [CommRing R] {A : Matrix n' n' R} (h : IsUnit (Matrix.det A)) (n : ) :
A ^ (-n) = (A ^ n)⁻¹
theorem Matrix.inv_zpow' {n' : Type u_1} [DecidableEq n'] [Fintype n'] {R : Type u_2} [CommRing R] {A : Matrix n' n' R} (h : IsUnit (Matrix.det A)) (n : ) :
A⁻¹ ^ n = A ^ (-n)
theorem Matrix.zpow_add_one {n' : Type u_1} [DecidableEq n'] [Fintype n'] {R : Type u_2} [CommRing R] {A : Matrix n' n' R} (h : IsUnit (Matrix.det A)) (n : ) :
A ^ (n + 1) = A ^ n * A
theorem Matrix.zpow_sub_one {n' : Type u_1} [DecidableEq n'] [Fintype n'] {R : Type u_2} [CommRing R] {A : Matrix n' n' R} (h : IsUnit (Matrix.det A)) (n : ) :
A ^ (n - 1) = A ^ n * A⁻¹
theorem Matrix.zpow_add {n' : Type u_1} [DecidableEq n'] [Fintype n'] {R : Type u_2} [CommRing R] {A : Matrix n' n' R} (ha : IsUnit (Matrix.det A)) (m : ) (n : ) :
A ^ (m + n) = A ^ m * A ^ n
theorem Matrix.zpow_add_of_nonpos {n' : Type u_1} [DecidableEq n'] [Fintype n'] {R : Type u_2} [CommRing R] {A : Matrix n' n' R} {m : } {n : } (hm : m 0) (hn : n 0) :
A ^ (m + n) = A ^ m * A ^ n
theorem Matrix.zpow_add_of_nonneg {n' : Type u_1} [DecidableEq n'] [Fintype n'] {R : Type u_2} [CommRing R] {A : Matrix n' n' R} {m : } {n : } (hm : 0 m) (hn : 0 n) :
A ^ (m + n) = A ^ m * A ^ n
theorem Matrix.zpow_one_add {n' : Type u_1} [DecidableEq n'] [Fintype n'] {R : Type u_2} [CommRing R] {A : Matrix n' n' R} (h : IsUnit (Matrix.det A)) (i : ) :
A ^ (1 + i) = A * A ^ i
theorem Matrix.SemiconjBy.zpow_right {n' : Type u_1} [DecidableEq n'] [Fintype n'] {R : Type u_2} [CommRing R] {A : Matrix n' n' R} {X : Matrix n' n' R} {Y : Matrix n' n' R} (hx : IsUnit (Matrix.det X)) (hy : IsUnit (Matrix.det Y)) (h : SemiconjBy A X Y) (m : ) :
SemiconjBy A (X ^ m) (Y ^ m)
theorem Matrix.Commute.zpow_right {n' : Type u_1} [DecidableEq n'] [Fintype n'] {R : Type u_2} [CommRing R] {A : Matrix n' n' R} {B : Matrix n' n' R} (h : Commute A B) (m : ) :
Commute A (B ^ m)
theorem Matrix.Commute.zpow_left {n' : Type u_1} [DecidableEq n'] [Fintype n'] {R : Type u_2} [CommRing R] {A : Matrix n' n' R} {B : Matrix n' n' R} (h : Commute A B) (m : ) :
Commute (A ^ m) B
theorem Matrix.Commute.zpow_zpow {n' : Type u_1} [DecidableEq n'] [Fintype n'] {R : Type u_2} [CommRing R] {A : Matrix n' n' R} {B : Matrix n' n' R} (h : Commute A B) (m : ) (n : ) :
Commute (A ^ m) (B ^ n)
theorem Matrix.Commute.zpow_self {n' : Type u_1} [DecidableEq n'] [Fintype n'] {R : Type u_2} [CommRing R] (A : Matrix n' n' R) (n : ) :
Commute (A ^ n) A
theorem Matrix.Commute.self_zpow {n' : Type u_1} [DecidableEq n'] [Fintype n'] {R : Type u_2} [CommRing R] (A : Matrix n' n' R) (n : ) :
Commute A (A ^ n)
theorem Matrix.Commute.zpow_zpow_self {n' : Type u_1} [DecidableEq n'] [Fintype n'] {R : Type u_2} [CommRing R] (A : Matrix n' n' R) (m : ) (n : ) :
Commute (A ^ m) (A ^ n)
theorem Matrix.zpow_bit0 {n' : Type u_1} [DecidableEq n'] [Fintype n'] {R : Type u_2} [CommRing R] (A : Matrix n' n' R) (n : ) :
A ^ bit0 n = A ^ n * A ^ n
theorem Matrix.zpow_add_one_of_ne_neg_one {n' : Type u_1} [DecidableEq n'] [Fintype n'] {R : Type u_2} [CommRing R] {A : Matrix n' n' R} (n : ) :
n -1A ^ (n + 1) = A ^ n * A
theorem Matrix.zpow_bit1 {n' : Type u_1} [DecidableEq n'] [Fintype n'] {R : Type u_2} [CommRing R] (A : Matrix n' n' R) (n : ) :
A ^ bit1 n = A ^ n * A ^ n * A
theorem Matrix.zpow_mul {n' : Type u_1} [DecidableEq n'] [Fintype n'] {R : Type u_2} [CommRing R] (A : Matrix n' n' R) (h : IsUnit (Matrix.det A)) (m : ) (n : ) :
A ^ (m * n) = (A ^ m) ^ n
theorem Matrix.zpow_mul' {n' : Type u_1} [DecidableEq n'] [Fintype n'] {R : Type u_2} [CommRing R] (A : Matrix n' n' R) (h : IsUnit (Matrix.det A)) (m : ) (n : ) :
A ^ (m * n) = (A ^ n) ^ m
@[simp]
theorem Matrix.coe_units_zpow {n' : Type u_1} [DecidableEq n'] [Fintype n'] {R : Type u_2} [CommRing R] (u : (Matrix n' n' R)ˣ) (n : ) :
(u ^ n) = u ^ n
theorem Matrix.zpow_ne_zero_of_isUnit_det {n' : Type u_1} [DecidableEq n'] [Fintype n'] {R : Type u_2} [CommRing R] [Nonempty n'] [Nontrivial R] {A : Matrix n' n' R} (ha : IsUnit (Matrix.det A)) (z : ) :
A ^ z 0
theorem Matrix.zpow_sub {n' : Type u_1} [DecidableEq n'] [Fintype n'] {R : Type u_2} [CommRing R] {A : Matrix n' n' R} (ha : IsUnit (Matrix.det A)) (z1 : ) (z2 : ) :
A ^ (z1 - z2) = A ^ z1 / A ^ z2
theorem Matrix.Commute.mul_zpow {n' : Type u_1} [DecidableEq n'] [Fintype n'] {R : Type u_2} [CommRing R] {A : Matrix n' n' R} {B : Matrix n' n' R} (h : Commute A B) (i : ) :
(A * B) ^ i = A ^ i * B ^ i
theorem Matrix.zpow_bit0' {n' : Type u_1} [DecidableEq n'] [Fintype n'] {R : Type u_2} [CommRing R] (A : Matrix n' n' R) (n : ) :
A ^ bit0 n = (A * A) ^ n
theorem Matrix.zpow_bit1' {n' : Type u_1} [DecidableEq n'] [Fintype n'] {R : Type u_2} [CommRing R] (A : Matrix n' n' R) (n : ) :
A ^ bit1 n = (A * A) ^ n * A
theorem Matrix.zpow_neg_mul_zpow_self {n' : Type u_1} [DecidableEq n'] [Fintype n'] {R : Type u_2} [CommRing R] (n : ) {A : Matrix n' n' R} (h : IsUnit (Matrix.det A)) :
A ^ (-n) * A ^ n = 1
theorem Matrix.one_div_pow {n' : Type u_1} [DecidableEq n'] [Fintype n'] {R : Type u_2} [CommRing R] {A : Matrix n' n' R} (n : ) :
(1 / A) ^ n = 1 / A ^ n
theorem Matrix.one_div_zpow {n' : Type u_1} [DecidableEq n'] [Fintype n'] {R : Type u_2} [CommRing R] {A : Matrix n' n' R} (n : ) :
(1 / A) ^ n = 1 / A ^ n
@[simp]
theorem Matrix.transpose_zpow {n' : Type u_1} [DecidableEq n'] [Fintype n'] {R : Type u_2} [CommRing R] (A : Matrix n' n' R) (n : ) :
@[simp]
theorem Matrix.conjTranspose_zpow {n' : Type u_1} [DecidableEq n'] [Fintype n'] {R : Type u_2} [CommRing R] [StarRing R] (A : Matrix n' n' R) (n : ) :
theorem Matrix.IsSymm.zpow {n' : Type u_1} [DecidableEq n'] [Fintype n'] {R : Type u_2} [CommRing R] {A : Matrix n' n' R} (h : Matrix.IsSymm A) (k : ) :