Zulip Chat Archive
Stream: mathlib4
Topic: Incompatible notations
Patrick Massot (Oct 26 2023 at 00:45):
In the next example, uncommenting the first line breaks everything.
-- import Mathlib
import Mathlib.Geometry.Manifold.ContMDiffMap
open scoped Manifold
variable {E : Type _} [NormedAddCommGroup E] [NormedSpace ℝ E] {H : Type _} [TopologicalSpace H]
(I : ModelWithCorners ℝ E H) (M : Type _) [TopologicalSpace M] [ChartedSpace H M]
[SmoothManifoldWithCorners I M] {E' : Type _} [NormedAddCommGroup E'] [NormedSpace ℝ E']
{H' : Type _} [TopologicalSpace H'] (I' : ModelWithCorners ℝ E' H') (M' : Type _)
[TopologicalSpace M'] [ChartedSpace H' M']
(n : ℕ)
#check C^n⟮I, M; I', M'⟯
Patrick Massot (Oct 26 2023 at 00:48):
import Mathlib.FieldTheory.Adjoin
is enough :angry:
Patrick Massot (Oct 26 2023 at 00:49):
Note the open scoped Manifold
says which notation is a good citizen.
Eric Wieser (Oct 26 2023 at 00:53):
In case you haven't already found it, the offending notation is here
Patrick Massot (Oct 26 2023 at 00:54):
I know, thanks.
Patrick Massot (Oct 26 2023 at 00:57):
The funny thing is that this notation also conflict with a third notation (that is already scoped) in elliptic curves (so this is not a story of algebra fighting geometry).
Patrick Massot (Oct 26 2023 at 01:14):
Fixed at #7938
Eric Rodriguez (Oct 26 2023 at 10:40):
Yeah, I ran into this whilst trying to fix an unrelated breakage before - thanks for fixing it!
Last updated: Dec 20 2023 at 11:08 UTC