Zulip Chat Archive
Stream: new members
Topic: Problem with mul_inv_eq_one
Luke Mantle (Feb 09 2023 at 21:34):
I'm using mul_inv_eq_one
in a larger proof but I can't seem to get it to work even in this very basic example:
import analysis.analytic.basic
open real
example (a : ℝ) : a * a⁻¹ = 1 :=
begin
apply mul_inv_eq_one.mpr,
end
Jireh Loreaux (Feb 09 2023 at 21:36):
you need docs#mul_inv_eq_one₀ because ℝ
isn't a group, it's a docs#group_with_zero.
Jireh Loreaux (Feb 09 2023 at 21:37):
And a hypothesis (ha : a ≠ 0)
.
Luke Mantle (Feb 10 2023 at 00:22):
Jireh Loreaux said:
you need docs#mul_inv_eq_one₀ because
ℝ
isn't a group, it's a docs#group_with_zero.
Ah, ok. Thanks!
Last updated: Dec 20 2023 at 11:08 UTC