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

Commit 8cf7c4c

Browse files
jcommelinmergify[bot]
authored andcommitted
chore(topology/algebra/monoid): continuous_mul_left/right (#1065)
1 parent 593938c commit 8cf7c4c

File tree

1 file changed

+8
-0
lines changed

1 file changed

+8
-0
lines changed

src/topology/algebra/monoid.lean

Lines changed: 8 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -46,6 +46,14 @@ lemma continuous_mul [topological_space β] {f : β → α} {g : β → α}
4646
continuous (λx, f x * g x) :=
4747
continuous_mul'.comp (hf.prod_mk hg)
4848

49+
@[to_additive continuous_add_left]
50+
lemma continuous_mul_left (a : α) : continuous (λ b:α, a * b) :=
51+
continuous_mul continuous_const continuous_id
52+
53+
@[to_additive continuous_add_right]
54+
lemma continuous_mul_right (a : α) : continuous (λ b:α, b * a) :=
55+
continuous_mul continuous_id continuous_const
56+
4957
-- @[to_additive continuous_smul]
5058
lemma continuous_pow : ∀ n : ℕ, continuous (λ a : α, a ^ n)
5159
| 0 := by simpa using continuous_const

0 commit comments

Comments
 (0)