Skip to content

Commit

Permalink
chore: rescope Ω notation for LoopSpace (#5714)
Browse files Browse the repository at this point in the history
  • Loading branch information
mattrobball committed Jul 5, 2023
1 parent d6a4516 commit abd65d5
Showing 1 changed file with 4 additions and 2 deletions.
6 changes: 4 additions & 2 deletions Mathlib/Topology/Homotopy/HomotopyGroup.lean
Expand Up @@ -94,7 +94,7 @@ def LoopSpace :=
#align loop_space LoopSpace

-- mathport name: exprΩ
scoped[Topology] notation "Ω" => LoopSpace
scoped[Topology.Homotopy] notation "Ω" => LoopSpace

instance LoopSpace.inhabited : Inhabited (Path x x) :=
⟨Path.refl x⟩
Expand All @@ -107,7 +107,9 @@ def GenLoop : Set C(I^N, X) :=
{p | ∀ y ∈ Cube.boundary N, p y = x}
#align gen_loop GenLoop

scoped[Topology] notation "Ω^" => GenLoop
scoped[Topology.Homotopy] notation "Ω^" => GenLoop

open Topology.Homotopy

variable {N X x}

Expand Down

0 comments on commit abd65d5

Please sign in to comment.