Zulip Chat Archive
Stream: Is there code for X?
Topic: product of reciprocal fractions is one
Roman Bacik (Jun 16 2024 at 14:32):
I am new to lean4 and have trouble showing:
lemma mult_rec_is_one (m : ℕ)(n : ℕ)(hm : 0 < m)(hn : 0 < n) : (m/n)*(n/m) = 1 := by
sorry
Is there already a code for it?
Roman Bacik (Jun 16 2024 at 14:46):
Got it:
lemma mult_rec_is_one (m : ℕ)(n : ℕ)(hm : 0 < m)(hn : 0 < n) : (m/n : ℚ)*(n/m : ℚ) = 1 := by
field_simp
Richard Copley (Jun 16 2024 at 14:50):
(The tactic slim_check
will give you a counterexample for the lemma as originally stated.)
Roman Bacik (Jun 16 2024 at 14:54):
Thank you very much, this slim_check
seems to be very helpful.
Junyan Xu (Jun 16 2024 at 16:17):
@loogle (?a / ?b) * (?b / ?a) = 1
loogle (Jun 16 2024 at 16:17):
:shrug: nothing found
Last updated: May 02 2025 at 03:31 UTC