Skip to content

Commit

Permalink
chore(data/real/ennreal): add a few lemmas (#5071)
Browse files Browse the repository at this point in the history
Also swap LHS with RHS in `to_real_mul_to_real` and rename it to `to_real_mul`.
  • Loading branch information
urkud committed Nov 22, 2020
1 parent f627d76 commit 2044451
Show file tree
Hide file tree
Showing 3 changed files with 134 additions and 99 deletions.
2 changes: 1 addition & 1 deletion src/analysis/normed_space/enorm.lean
Expand Up @@ -184,6 +184,6 @@ lemma finite_norm_eq (x : e.finite_subspace) : ∥x∥ = (e x).to_real := rfl

/-- Normed space instance on `e.finite_subspace`. -/
instance : normed_space 𝕜 e.finite_subspace :=
{ norm_smul_le := λ c x, le_of_eq $ by simp [finite_norm_eq, ennreal.to_real_mul_to_real] }
{ norm_smul_le := λ c x, le_of_eq $ by simp [finite_norm_eq, ennreal.to_real_mul] }

end enorm

0 comments on commit 2044451

Please sign in to comment.