Documentation

Mathlib.LinearAlgebra.PerfectPairing.Matrix

Perfect pairings and matrices #

The file contains results connecting perfect pairings and matrices.

Main definitions #

def Matrix.toPerfectPairing {R : Type u_1} {n : Type u_2} [CommRing R] [Fintype n] [DecidableEq n] (A : Matrix n n R) (h : Invertible A) :
PerfectPairing R (nR) (nR)

We may regard an invertible matrix as a perfect pairing.

Equations
Instances For
    @[simp]
    theorem Matrix.toPerfectPairing_apply_apply {R : Type u_1} {n : Type u_2} [CommRing R] [Fintype n] [DecidableEq n] (A : Matrix n n R) (h : Invertible A) (v w : nR) :
    ((A.toPerfectPairing h) v) w = A.mulVec v ⬝ᵥ w