Skip to content

Commit 78426b9

Browse files
jjaassoonnkim-emRuben-VandeVeldeadomani
committed
feat: port Topology.Gluing (#3987)
Co-authored-by: Scott Morrison <scott@tqft.net> Co-authored-by: Ruben Van de Velde <65514131+Ruben-VandeVelde@users.noreply.github.com> Co-authored-by: adomani <adomani@gmail.com>
1 parent 817852e commit 78426b9

File tree

3 files changed

+543
-1
lines changed

3 files changed

+543
-1
lines changed

Mathlib.lean

Lines changed: 1 addition & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -2838,6 +2838,7 @@ import Mathlib.Topology.FiberBundle.IsHomeomorphicTrivialBundle
28382838
import Mathlib.Topology.FiberBundle.Trivialization
28392839
import Mathlib.Topology.Filter
28402840
import Mathlib.Topology.GDelta
2841+
import Mathlib.Topology.Gluing
28412842
import Mathlib.Topology.Hom.Open
28422843
import Mathlib.Topology.Homeomorph
28432844
import Mathlib.Topology.Homotopy.Basic

Mathlib/Topology/ContinuousFunction/Basic.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -83,7 +83,7 @@ namespace ContinuousMap
8383
variable {α β γ δ : Type _} [TopologicalSpace α] [TopologicalSpace β] [TopologicalSpace γ]
8484
[TopologicalSpace δ]
8585

86-
instance : ContinuousMapClass C(α, β) α β where
86+
instance toContinuousMapClass : ContinuousMapClass C(α, β) α β where
8787
coe := ContinuousMap.toFun
8888
coe_injective' f g h := by cases f; cases g; congr
8989
map_continuous := ContinuousMap.continuous_toFun

0 commit comments

Comments
 (0)