Skip to content

Commit

Permalink
chore(topology/algebra/infinite_sum): relax the requirements on `has_…
Browse files Browse the repository at this point in the history
…sum.smul` (#8312)
  • Loading branch information
eric-wieser committed Jul 16, 2021
1 parent 162221f commit 35a8d93
Showing 1 changed file with 2 additions and 2 deletions.
4 changes: 2 additions & 2 deletions src/topology/algebra/infinite_sum.lean
Expand Up @@ -735,9 +735,9 @@ end topological_semiring

section has_continuous_smul
variables {R : Type*}
[semiring R] [topological_space R]
[monoid R] [topological_space R]
[topological_space α] [add_comm_monoid α]
[module R α] [has_continuous_smul R α]
[distrib_mul_action R α] [has_continuous_smul R α]
{f : β → α}

lemma has_sum.smul {a : α} {r : R} (hf : has_sum f a) : has_sum (λ z, r • f z) (r • a) :=
Expand Down

0 comments on commit 35a8d93

Please sign in to comment.