Zulip Chat Archive

Stream: mathlib4

Topic: Bug in `ring_nf`?


Heather Macbeth (Mar 06 2023 at 00:12):

The following fails on current master, with x + 0 failing to be normalized to x:

import Mathlib.Tactic.Ring

example {x : } (hn : 0 < x) : 0 < x + 0 := by
  ring_nf -- does nothing
  with_reducible assumption

Any thoughts on what the bug might be?

Mario Carneiro (Mar 06 2023 at 00:13):

Yes, this was reported earlier

Mario Carneiro (Mar 06 2023 at 00:13):

https://leanprover.zulipchat.com/#narrow/stream/287929-mathlib4/topic/ring_nf.20failing.20to.20fully.20normalize

Heather Macbeth (Mar 06 2023 at 00:15):

Is it wontfix then?

Mario Carneiro (Mar 06 2023 at 00:15):

the fix requires some substantial new code

Mario Carneiro (Mar 06 2023 at 00:16):

for now there is !4#2171

Heather Macbeth (Mar 06 2023 at 00:16):

huh

hrmacbeth added this to Teaching Features last month

Heather Macbeth (Mar 06 2023 at 00:18):

I must have forgotten about this issue! Can I motivate anyone to add it to their to-do list? I expect to start to use ring_nf heavily in teaching in about two weeks.


Last updated: Dec 20 2023 at 11:08 UTC