Zulip Chat Archive
Stream: mathlib4
Topic: pushforwardObj claims unexpected notation
Eric Wieser (Jul 01 2024 at 16:51):
This is pretty surprising behavior:
import Mathlib.Tactic
example : 1 * 2 = 2 * 1 := by
show _*_ = _*_ -- works
norm_num
import Mathlib
example : 1 * 2 = 2 * 1 := by
show _*_ = _*_ -- fails
norm_num
Can we change docs#TopCat.Presheaf.pushforwardObj to use less intrusive notation?
Kyle Miller (Jul 01 2024 at 16:54):
It ought to be scoped at least!
Eric Wieser (Jul 01 2024 at 16:54):
Also, was there a better way for me to track this down than pruning imports until it worked?
Eric Wieser (Jul 01 2024 at 16:54):
Can I get Lean to tell me what it thinks the tokens are?
Damiano Testa (Jul 02 2024 at 13:10):
Eric, is this the list of tokens?
import Lean.Elab.Command
open Lean Parser in
run_cmd
logInfo m!"{(getTokenTable (← getEnv)).values}"
Last updated: May 02 2025 at 03:31 UTC