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

Commit a6f62a7

Browse files
committed
feat(topology/algebra/mul_action.lean): add smul_const (#7242)
add filter.tendsto.smul_const
1 parent 4d4b501 commit a6f62a7

File tree

1 file changed

+5
-0
lines changed

1 file changed

+5
-0
lines changed

src/topology/algebra/mul_action.lean

Lines changed: 5 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -58,6 +58,11 @@ lemma filter.tendsto.const_smul {f : β → α} {l : filter β} {a : α} (hf : t
5858
tendsto (λ x, c • f x) l (𝓝 (c • a)) :=
5959
tendsto_const_nhds.smul hf
6060

61+
lemma filter.tendsto.smul_const {f : β → M} {l : filter β} {c : M}
62+
(hf : tendsto f l (𝓝 c)) (a : α) :
63+
tendsto (λ x, (f x) • a) l (𝓝 (c • a)) :=
64+
hf.smul tendsto_const_nhds
65+
6166
variables [topological_space β] {f : β → M} {g : β → α} {b : β} {s : set β}
6267

6368
lemma continuous_within_at.smul (hf : continuous_within_at f s b)

0 commit comments

Comments
 (0)