We read every piece of feedback, and take your input very seriously.
To see all available qualifiers, see our documentation.
There was an error while loading. Please reload this page.
1 parent fe8d313 commit 5dcd49bCopy full SHA for 5dcd49b
Mathlib/Algebra/GroupWithZero/Invertible.lean
@@ -63,7 +63,7 @@ theorem mul_inv_cancel_of_invertible (a : α) [Invertible a] : a * a⁻¹ = 1 :=
63
mul_inv_cancel₀ (Invertible.ne_zero a)
64
65
/-- `a` is the inverse of `a⁻¹` -/
66
-def invertibleInv {a : α} [Invertible a] : Invertible a⁻¹ :=
+instance invertibleInv {a : α} [Invertible a] : Invertible a⁻¹ :=
67
⟨a, by simp, by simp⟩
68
69
@[simp]
0 commit comments