Skip to content
This repository was archived by the owner on Jul 24, 2024. It is now read-only.

Commit e5c66a0

Browse files
committed
chore(topology/continuous_function/bounded): add comp_continuous (#10134)
1 parent e5acda4 commit e5c66a0

File tree

1 file changed

+10
-0
lines changed

1 file changed

+10
-0
lines changed

src/topology/continuous_function/bounded.lean

Lines changed: 10 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -238,6 +238,16 @@ begin
238238
exact λ N, (dist_le (b0 _)).2 (λx, fF_bdd x N) }
239239
end
240240

241+
/-- Composition of a bounded continuous function and a continuous function. -/
242+
@[simps { fully_applied := ff }]
243+
def comp_continuous {δ : Type*} [topological_space δ] (f : α →ᵇ β) (g : C(δ, α)) : δ →ᵇ β :=
244+
{ to_continuous_map := f.1.comp g,
245+
bounded' := f.bounded'.imp (λ C hC x y, hC _ _) }
246+
247+
/-- Restrict a bounded continuous function to a set. -/
248+
@[simps apply { fully_applied := ff }]
249+
def restrict (f : α →ᵇ β) (s : set α) : s →ᵇ β := f.comp_continuous (continuous_map.id.restrict s)
250+
241251
/-- Composition (in the target) of a bounded continuous function with a Lipschitz map again
242252
gives a bounded continuous function -/
243253
def comp (G : β → γ) {C : ℝ≥0} (H : lipschitz_with C G)

0 commit comments

Comments
 (0)