Documentation

Mathlib.Analysis.Normed.Group.Lemmas

Further lemmas about normed groups #

This file contains further lemmas about normed groups, requiring heavier imports than Mathlib/Analysis/Normed/Group/Basic.lean.

TODO #

theorem eventually_nnnorm_sub_lt {E : Type u_1} [SeminormedAddCommGroup E] (x₀ : E) {ε : NNReal} (ε_pos : 0 < ε) :
∀ᶠ (x : E) in nhds x₀, x - x₀‖₊ < ε
theorem eventually_norm_sub_lt {E : Type u_1} [SeminormedAddCommGroup E] (x₀ : E) {ε : } (ε_pos : 0 < ε) :
∀ᶠ (x : E) in nhds x₀, x - x₀ < ε