Skip to content

Commit

Permalink
feat(analysis/normed_space/basic): add norm_algebra_map_nnreal (#16709
Browse files Browse the repository at this point in the history
)

This adds `simp` lemmas saying that `∥algebra_map ℝ≥0 𝕜 x∥ = x` and similarly for `∥⬝∥₊` whenever `𝕜` is a normed `ℝ`-algebra and satisfies `norm_one_class`. These are needed separately from `norm_algebra_map'` and `nnnorm_algebra_map'` because `𝕜` cannot be a normed `ℝ≥0`-algebra for the simple reason that `ℝ≥0` is not a normed field.
  • Loading branch information
j-loreaux committed Sep 30, 2022
1 parent 07e46bc commit 667f2a6
Showing 1 changed file with 12 additions and 0 deletions.
12 changes: 12 additions & 0 deletions src/analysis/normed_space/basic.lean
Expand Up @@ -446,6 +446,18 @@ by rw [norm_algebra_map, norm_one, mul_one]
@[simp] lemma nnnorm_algebra_map' [norm_one_class 𝕜'] (x : 𝕜) : ∥algebra_map 𝕜 𝕜' x∥₊ = ∥x∥₊ :=
subtype.ext $ norm_algebra_map' _ _

section nnreal

variables [norm_one_class 𝕜'] [normed_algebra ℝ 𝕜']

@[simp] lemma norm_algebra_map_nnreal (x : ℝ≥0) : ∥algebra_map ℝ≥0 𝕜' x∥ = x :=
(norm_algebra_map' 𝕜' (x : ℝ)).symm ▸ real.norm_of_nonneg x.prop

@[simp] lemma nnnorm_algebra_map_nnreal (x : ℝ≥0) : ∥algebra_map ℝ≥0 𝕜' x∥₊ = x :=
subtype.ext $ norm_algebra_map_nnreal 𝕜' x

end nnreal

variables (𝕜 𝕜')

/-- In a normed algebra, the inclusion of the base field in the extended field is an isometry. -/
Expand Down

0 comments on commit 667f2a6

Please sign in to comment.