Skip to content

Commit 5dcd49b

Browse files
committed
chore(Algebra): make invertibleInv an instance (#31916)
1 parent fe8d313 commit 5dcd49b

File tree

1 file changed

+1
-1
lines changed

1 file changed

+1
-1
lines changed

Mathlib/Algebra/GroupWithZero/Invertible.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -63,7 +63,7 @@ theorem mul_inv_cancel_of_invertible (a : α) [Invertible a] : a * a⁻¹ = 1 :=
6363
mul_inv_cancel₀ (Invertible.ne_zero a)
6464

6565
/-- `a` is the inverse of `a⁻¹` -/
66-
def invertibleInv {a : α} [Invertible a] : Invertible a⁻¹ :=
66+
instance invertibleInv {a : α} [Invertible a] : Invertible a⁻¹ :=
6767
⟨a, by simp, by simp⟩
6868

6969
@[simp]

0 commit comments

Comments
 (0)