Skip to content

Commit

Permalink
Update Mathlib/Topology/ContinuousMap/CompactlySupported.lean
Browse files Browse the repository at this point in the history
Co-authored-by: Yaël Dillies <[email protected]>
  • Loading branch information
yoh-tanimoto and YaelDillies authored Jan 31, 2025
1 parent b86d559 commit 8016324
Showing 1 changed file with 3 additions and 1 deletion.
4 changes: 3 additions & 1 deletion Mathlib/Topology/ContinuousMap/CompactlySupported.lean
Original file line number Diff line number Diff line change
Expand Up @@ -125,7 +125,9 @@ def ContinuousMap.liftCompactlySupported [CompactSpace α] : C(α, β) ≃ C_c(
right_inv _ := rfl

/-- Composition of a continuous function `f` with compact support with another continuous function
`g` from the left yields another continuous function `g ∘ f` with compact support. -/
`g` sending `0` to `0` from the left yields another continuous function `g ∘ f` with compact support.
If `g` doesn't send `0` to `0`, `f.compLeft g` defaults to `0`. -/
noncomputable def compLeft {γ : Type*} [TopologicalSpace γ] [Zero γ] (g : C(β, γ))
(f : C_c(α, β)) : C_c(α, γ) where
toContinuousMap := if g 0 = 0 then g.comp f else 0
Expand Down

0 comments on commit 8016324

Please sign in to comment.