Skip to content

Commit

Permalink
fix(normed_space): fixed a typo from #4099 (#4147)
Browse files Browse the repository at this point in the history
This lemma was less general that it should be because migrating it to its
mathlib place messed up the typeclass assumptions.
  • Loading branch information
PatrickMassot committed Sep 14, 2020
1 parent 8877606 commit 6babb55
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion src/analysis/normed_space/basic.lean
Expand Up @@ -798,7 +798,7 @@ lemma nndist_smul [normed_space α β] (s : α) (x y : β) :
nndist (s • x) (s • y) = nnnorm s * nndist x y :=
nnreal.eq $ dist_smul s x y

lemma norm_smul_of_nonneg [normed_space ℝ α] {t : ℝ} (ht : 0 ≤ t) (x : α) : ∥t • x∥ = t * ∥x∥ :=
lemma norm_smul_of_nonneg [normed_space ℝ β] {t : ℝ} (ht : 0 ≤ t) (x : β) : ∥t • x∥ = t * ∥x∥ :=
by rw [norm_smul, real.norm_eq_abs, abs_of_nonneg ht]

variables {E : Type*} {F : Type*}
Expand Down

0 comments on commit 6babb55

Please sign in to comment.