Zulip Chat Archive
Stream: mathlib4
Topic: surprising abel_nf failures
Floris van Doorn (Mar 15 2024 at 14:11):
I don't know the exact scope of abel_nf
and I'm only using it through noncomm_ring
, but I expected the following to succeed (or at least, abel_nf
to make some kind of progress):
import Mathlib.Tactic.Abel
example {R} [Ring R] : (0 : R) + 1 = 1 := by abel_nf -- (abel does work)
example {R} [Ring R] : (0 : R) + 1 = 1 ∧ (1 : R) + 0 = 1 := by abel_nf
Last updated: May 02 2025 at 03:31 UTC