Skip to content

Commit

Permalink
chore(topology/algebra/monoid): continuous_mul_left/right (#1065)
Browse files Browse the repository at this point in the history
  • Loading branch information
jcommelin authored and mergify[bot] committed May 20, 2019
1 parent 593938c commit 8cf7c4c
Showing 1 changed file with 8 additions and 0 deletions.
8 changes: 8 additions & 0 deletions src/topology/algebra/monoid.lean
Expand Up @@ -46,6 +46,14 @@ lemma continuous_mul [topological_space β] {f : β → α} {g : β → α}
continuous (λx, f x * g x) :=
continuous_mul'.comp (hf.prod_mk hg)

@[to_additive continuous_add_left]
lemma continuous_mul_left (a : α) : continuous (λ b:α, a * b) :=
continuous_mul continuous_const continuous_id

@[to_additive continuous_add_right]
lemma continuous_mul_right (a : α) : continuous (λ b:α, b * a) :=
continuous_mul continuous_id continuous_const

-- @[to_additive continuous_smul]
lemma continuous_pow : ∀ n : ℕ, continuous (λ a : α, a ^ n)
| 0 := by simpa using continuous_const
Expand Down

0 comments on commit 8cf7c4c

Please sign in to comment.