Skip to content

Commit

Permalink
feat(analysis/normed/group/basic): isometry.norm_map_of_map_zero (#…
Browse files Browse the repository at this point in the history
…14836)

Add the lemma that an isometry of `semi_normed_group`s that preserves
0 preserves the norm.
  • Loading branch information
jsm28 committed Jun 20, 2022
1 parent cf118ee commit 10a5275
Showing 1 changed file with 4 additions and 0 deletions.
4 changes: 4 additions & 0 deletions src/analysis/normed/group/basic.lean
Expand Up @@ -128,6 +128,10 @@ by rw [dist_eq_norm, sub_zero]
@[simp] lemma dist_zero_left : dist (0 : E) = norm :=
funext $ λ g, by rw [dist_comm, dist_zero_right]

lemma isometry.norm_map_of_map_zero {f : E → F} (hi : isometry f) (h0 : f 0 = 0) (x : E) :
∥f x∥ = ∥x∥ :=
by rw [←dist_zero_right, ←h0, hi.dist_eq, dist_zero_right]

lemma tendsto_norm_cocompact_at_top [proper_space E] :
tendsto norm (cocompact E) at_top :=
by simpa only [dist_zero_right] using tendsto_dist_right_cocompact_at_top (0 : E)
Expand Down

0 comments on commit 10a5275

Please sign in to comment.