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

Commit fa2e399

Browse files
sgouezeldigama0
authored andcommitted
feat(topology/bounded_continuous_function): constructor in normed groups (#607)
1 parent 3fcba7d commit fa2e399

File tree

1 file changed

+16
-0
lines changed

1 file changed

+16
-0
lines changed

src/topology/bounded_continuous_function.lean

Lines changed: 16 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -440,5 +440,21 @@ by rw normed_group.dist_eq; exact @norm_coe_le_norm _ _ _ _ (f-g) x
440440
lemma coe_le_coe_add_dist {f g : α →ᵇ ℝ} : f x ≤ g x + dist f g :=
441441
sub_le_iff_le_add'.1 $ (abs_le.1 $ @dist_coe_le_dist _ _ _ _ f g x).2
442442

443+
/-- Constructing a bounded continuous function from a uniformly bounded continuous
444+
function taking values in a normed group. -/
445+
def of_normed_group {α : Type u} {β : Type v} [topological_space α] [normed_group β]
446+
(f : α → β) (C : ℝ) (H : ∀x, norm (f x) ≤ C) (Hf : continuous f) : α →ᵇ β :=
447+
⟨λn, f n, ⟨Hf, ⟨C + C, λ m n,
448+
calc dist (f m) (f n) ≤ dist (f m) 0 + dist (f n) 0 : dist_triangle_right _ _ _
449+
... = norm (f m) + norm (f n) : by simp
450+
... ≤ C + C : add_le_add (H m) (H n)⟩⟩⟩
451+
452+
/-- Constructing a bounded continuous function from a uniformly bounded
453+
function on a discrete space, taking values in a normed group -/
454+
def of_normed_group_discrete {α : Type u} {β : Type v}
455+
[topological_space α] [discrete_topology α] [normed_group β]
456+
(f : α → β) (C : ℝ) (H : ∀x, norm (f x) ≤ C) : α →ᵇ β :=
457+
of_normed_group f C H continuous_of_discrete_topology
458+
443459
end normed_group
444460
end bounded_continuous_function

0 commit comments

Comments
 (0)