Skip to content

Commit

Permalink
chore(CompHausLike): add constant morphisms (#17381)
Browse files Browse the repository at this point in the history
  • Loading branch information
dagurtomas committed Oct 4, 2024
1 parent 10237af commit 44f94cd
Showing 1 changed file with 9 additions and 0 deletions.
9 changes: 9 additions & 0 deletions Mathlib/Topology/Category/CompHausLike/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -255,4 +255,13 @@ def isoEquivHomeo {X Y : CompHausLike.{u} P} : (X ≅ Y) ≃ (X ≃ₜ Y) where
left_inv _ := rfl
right_inv _ := rfl

/-- A constant map as a morphism in `CompHausLike` -/
def const {P : TopCat.{u} → Prop}
(T : CompHausLike.{u} P) {S : CompHausLike.{u} P} (s : S) : T ⟶ S :=
ContinuousMap.const _ s

lemma const_comp {P : TopCat.{u} → Prop} {S T U : CompHausLike.{u} P}
(s : S) (g : S ⟶ U) : T.const s ≫ g = T.const (g s) :=
rfl

end CompHausLike

0 comments on commit 44f94cd

Please sign in to comment.