Zulip Chat Archive

Stream: mathlib4

Topic: missing code action for `try this: ring_nf`


Asei Inoue (Apr 21 2024 at 14:39):

Why is there no code action to replace ring with ring_nf? I thought it should be implemented in mathlib.

import Mathlib.Tactic

example {n : Nat} (h : n = 2) : n * (3 + n) ^ 2 = n * (n ^ 2 + 10 * n + 1) := by
  /-
  Try this: ring_nf
  -/
  ring

Patrick Massot (Apr 21 2024 at 15:04):

Because nobody took time to do it. You could do it if this is important to you.

Asei Inoue (Apr 21 2024 at 15:24):

I'm relieved to know it's worth doing. Thanks.

Mario Carneiro (Apr 21 2024 at 15:39):

#12320


Last updated: May 02 2025 at 03:31 UTC