Zulip Chat Archive

Stream: new members

Topic: proving identity


Shi You (Aug 12 2021 at 07:14):

Hi. I am new to Lean. I found that by ring is a powerful tactic to check the correctness of an algebraic identity defined in a polynomial ring. However, I cannot find a tactic to prove identities in field of fractions.(something like x / y + y / x = (x^2 + y^2) / (x * y)). I don't know if there is a similar tool.

Eric Wieser (Aug 12 2021 at 07:22):

Have you tried proving it manually guys rewrites?

Rémy Degenne (Aug 12 2021 at 07:24):

the field_simp tactic could be useful. See https://leanprover-community.github.io/mathlib_docs/tactics.html#field_simp where the following example is given:

example (a b c d x y : ) (hx : x  0) (hy : y  0) :
  a + b / x + c / x^2 + d / x^3 = a + x⁻¹ * (y * b / y + (d / x + c) / x) :=
begin
  field_simp,
  ring
end

Last updated: Dec 20 2023 at 11:08 UTC