Skip to content

Commit

Permalink
fix: Use notation3 for neighborhood notations (#8690)
Browse files Browse the repository at this point in the history
The point is to get delaborators for free. This was previously blocked on `notation3` not supporting `scoped`.
  • Loading branch information
PatrickMassot committed Nov 29, 2023
1 parent b9d519b commit bc29663
Showing 1 changed file with 5 additions and 5 deletions.
10 changes: 5 additions & 5 deletions Mathlib/Topology/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -848,19 +848,19 @@ scoped[Topology] notation "𝓝" => nhds
scoped[Topology] notation "𝓝[" s "] " x:100 => nhdsWithin x s

/-- Notation for the filter of punctured neighborhoods of a point. -/
scoped[Topology] notation "𝓝[β‰ ] " x:100 => nhdsWithin x (@singleton _ (Set _) instSingletonSet x)ᢜ
scoped[Topology] notation3 "𝓝[β‰ ] " x:100 => nhdsWithin x (@singleton _ (Set _) instSingletonSet x)ᢜ

/-- Notation for the filter of right neighborhoods of a point. -/
scoped[Topology] notation "𝓝[β‰₯] " x:100 => nhdsWithin x (Set.Ici x)
scoped[Topology] notation3 "𝓝[β‰₯] " x:100 => nhdsWithin x (Set.Ici x)

/-- Notation for the filter of left neighborhoods of a point. -/
scoped[Topology] notation "𝓝[≀] " x:100 => nhdsWithin x (Set.Iic x)
scoped[Topology] notation3 "𝓝[≀] " x:100 => nhdsWithin x (Set.Iic x)

/-- Notation for the filter of punctured right neighborhoods of a point. -/
scoped[Topology] notation "𝓝[>] " x:100 => nhdsWithin x (Set.Ioi x)
scoped[Topology] notation3 "𝓝[>] " x:100 => nhdsWithin x (Set.Ioi x)

/-- Notation for the filter of punctured left neighborhoods of a point. -/
scoped[Topology] notation "𝓝[<] " x:100 => nhdsWithin x (Set.Iio x)
scoped[Topology] notation3 "𝓝[<] " x:100 => nhdsWithin x (Set.Iio x)

end

Expand Down

0 comments on commit bc29663

Please sign in to comment.