Documentation

Mathlib.Algebra.Invertible.Ring

Theorems about invertible elements in rings #

def invertibleNeg {α : Type u} [Mul α] [One α] [HasDistribNeg α] (a : α) [Invertible a] :

-⅟a is the inverse of -a

Equations
Instances For
    @[simp]
    theorem invOf_neg {α : Type u} [Monoid α] [HasDistribNeg α] (a : α) [Invertible a] [Invertible (-a)] :
    (-a) = -a
    @[simp]
    theorem one_sub_invOf_two {α : Type u} [Ring α] [Invertible 2] :
    1 - 2 = 2
    @[simp]
    theorem pos_of_invertible_cast {α : Type u} [Semiring α] [Nontrivial α] (n : ) [Invertible n] :
    0 < n