Zulip Chat Archive
Stream: mathlib4
Topic: Bug in push_neg
Yury G. Kudryashov (Feb 05 2023 at 21:31):
Here is an #mwe:
import Mathlib.Tactic.PushNeg
example {α} [Preorder α] (m n : α) (h : ¬(∃ k : ℕ, m ≤ n)) : m ≤ n := by
push_neg at h
While α
is not a LinearOrder
, push_neg
still tries to rewrite using [not_le]
and fails.
Yury G. Kudryashov (Feb 05 2023 at 21:32):
This used to work in Lean 3 (encountered for α = Filter β
in a file I'm porting).
Yury G. Kudryashov (Feb 05 2023 at 21:34):
@Frédéric Dupuis @Mario Carneiro you made most contributions to this file :up:
Frédéric Dupuis (Feb 06 2023 at 00:56):
I'll have a look right now. If I don't manage to fix it tonight, it might be a while before I have time again though.
Jireh Loreaux (Feb 06 2023 at 01:07):
@Frédéric Dupuis If you don't fix it tonight I'll take a look tomorrow
Frédéric Dupuis (Feb 06 2023 at 01:41):
Notification Bot (Feb 06 2023 at 02:02):
This topic was moved here from #lean4 > Bug in push_neg by Yury G. Kudryashov.
Last updated: Dec 20 2023 at 11:08 UTC