Theorems about invertible elements in a GroupWithZero
#
We intentionally keep imports minimal here as this file is used by Mathlib.Tactic.NormNum
.
theorem
Invertible.ne_zero
{α : Type u}
[MulZeroOneClass α]
(a : α)
[Nontrivial α]
[Invertible a]
:
a ≠ 0
@[deprecated Invertible.ne_zero]
theorem
nonzero_of_invertible
{α : Type u}
[MulZeroOneClass α]
(a : α)
[Nontrivial α]
[Invertible a]
:
a ≠ 0
Alias of Invertible.ne_zero
.
@[instance 100]
instance
Invertible.toNeZero
{α : Type u}
[MulZeroOneClass α]
[Nontrivial α]
(a : α)
[Invertible a]
:
NeZero a
Equations
- ⋯ = ⋯
@[simp]
theorem
Ring.inverse_invertible
{α : Type u}
[MonoidWithZero α]
(x : α)
[Invertible x]
:
Ring.inverse x = ⅟x
A variant of Ring.inverse_unit
.
a⁻¹
is an inverse of a
if a ≠ 0
Equations
- invertibleOfNonzero h = { invOf := a⁻¹, invOf_mul_self := ⋯, mul_invOf_self := ⋯ }
Instances For
@[simp]
@[simp]
a
is the inverse of a⁻¹
Equations
- invertibleInv = { invOf := a, invOf_mul_self := ⋯, mul_invOf_self := ⋯ }
Instances For
@[simp]
theorem
div_mul_cancel_of_invertible
{α : Type u}
[GroupWithZero α]
(a : α)
(b : α)
[Invertible b]
:
@[simp]
theorem
mul_div_cancel_of_invertible
{α : Type u}
[GroupWithZero α]
(a : α)
(b : α)
[Invertible b]
:
@[simp]
def
invertibleDiv
{α : Type u}
[GroupWithZero α]
(a : α)
(b : α)
[Invertible a]
[Invertible b]
:
Invertible (a / b)
b / a
is the inverse of a / b
Equations
- invertibleDiv a b = { invOf := b / a, invOf_mul_self := ⋯, mul_invOf_self := ⋯ }
Instances For
theorem
invOf_div
{α : Type u}
[GroupWithZero α]
(a : α)
(b : α)
[Invertible a]
[Invertible b]
[Invertible (a / b)]
: