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

Commit e815675

Browse files
committed
chore(topology/algebra/module/basic): remove two duplicate lemmas (#12072)
`continuous_linear_map.continuous_nsmul` is nothing to do with `continuous_linear_map`s, and is the same as `continuous_nsmul`, but the latter doesn't require commutativity. There is no reason to keep the former. This lemma was added in #7084, but probably got missed due to how large that PR had to be. We can't remove `continuous_linear_map.continuous_zsmul` until #12055 is merged, as there is currently no `continuous_zsmul` in the root namespace.
1 parent a26d17f commit e815675

File tree

1 file changed

+0
-12
lines changed

1 file changed

+0
-12
lines changed

src/topology/algebra/module/basic.lean

Lines changed: 0 additions & 12 deletions
Original file line numberDiff line numberDiff line change
@@ -494,18 +494,6 @@ variables [has_continuous_add M₂]
494494
instance : has_add (M₁ →SL[σ₁₂] M₂) :=
495495
⟨λ f g, ⟨f + g, f.2.add g.2⟩⟩
496496

497-
lemma continuous_nsmul (n : ℕ) : continuous (λ (x : M₂), n • x) :=
498-
begin
499-
induction n with n ih,
500-
{ simp [continuous_const] },
501-
{ simp [nat.succ_eq_add_one, add_smul], exact ih.add continuous_id }
502-
end
503-
504-
@[continuity]
505-
lemma continuous.nsmul {α : Type*} [topological_space α] {n : ℕ} {f : α → M₂} (hf : continuous f) :
506-
continuous (λ (x : α), n • (f x)) :=
507-
(continuous_nsmul n).comp hf
508-
509497
@[simp] lemma add_apply : (f + g) x = f x + g x := rfl
510498
@[simp, norm_cast] lemma coe_add : (((f + g) : M₁ →SL[σ₁₂] M₂) : M₁ →ₛₗ[σ₁₂] M₂) = f + g := rfl
511499
@[norm_cast] lemma coe_add' : (((f + g) : M₁ →SL[σ₁₂] M₂) : M₁ → M₂) = (f : M₁ → M₂) + g := rfl

0 commit comments

Comments
 (0)