Zulip Chat Archive
Stream: mathlib4
Topic: Bad TopCat.Presheaf.pushforward notation
Eric Wieser (Sep 24 2024 at 15:29):
I'm sure I made this thread before, but now I can't find it. The following code works:
example : ∃ x, x = 2 * 3 := by
exact ⟨_*_, rfl⟩
but with import Mathlib
, it fails:
import Mathlib
example : ∃ x, x = 2 * 3 := by
exact ⟨_*_, rfl⟩ -- bizarre error message
-- the notation parses as this now!
#check _ _* _
Can we make this notation scoped, or pick something different?
Eric Wieser (Sep 24 2024 at 15:34):
Last updated: May 02 2025 at 03:31 UTC