Zulip Chat Archive
Stream: mathlib4
Topic: Aggressive notation, Y
Eric Wieser (Nov 20 2024 at 11:56):
In the following code, the letter Y
ends up as a syntax error
import Mathlib -- works fine with a smaller import
open Polynomial
theorem something_polynomial : X + 1 ≠ (0 : ℚ[X]) := sorry -- ok
theorem something_not_polynomial (X : Nat) : X + 1 ≠ 0 := sorry -- ok
theorem something_polynomial2 : Y + 1 ≠ (0 : ℚ[X][Y]) := sorry -- ok
theorem something_not_polynomial2 (Y : Nat) : X + 1 ≠ 0 := sorry -- syntax error
Should we replace docs#Polynomial.termY with an abbrev
instead?
Eric Wieser (Nov 20 2024 at 11:56):
cc @Junyan Xu
Eric Wieser (Nov 20 2024 at 12:42):
Another option would be to move it into the Polynomial.Bivariate
scope instead of Polynomial
Junyan Xu (Nov 20 2024 at 13:08):
Or PolynomialPolynomial
scope as was originally the case; see the poll here.
Eric Wieser (Nov 20 2024 at 14:23):
#19292 moves it to Polynomial.Bivariate
; feel free to push a different namespace to that PR, or switch it to abbrev
.
Last updated: May 02 2025 at 03:31 UTC