Skip to content
This repository was archived by the owner on Jul 24, 2024. It is now read-only.

Commit fdc3136

Browse files
committed
feat(analysis/normed/group/basic): closure of {0} in a seminormed group (#17287)
1 parent 7e2084a commit fdc3136

File tree

1 file changed

+6
-0
lines changed

1 file changed

+6
-0
lines changed

src/analysis/normed/group/basic.lean

Lines changed: 6 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -748,6 +748,12 @@ lipschitz_with_one_norm'.uniform_continuous
748748
lemma uniform_continuous_nnnorm' : uniform_continuous (λ (a : E), ∥a∥₊) :=
749749
uniform_continuous_norm'.subtype_mk _
750750

751+
@[to_additive] lemma mem_closure_one_iff_norm {x : E} : x ∈ closure ({1} : set E) ↔ ∥x∥ = 0 :=
752+
by rw [←closed_ball_zero', mem_closed_ball_one_iff, (norm_nonneg' x).le_iff_eq]
753+
754+
@[to_additive] lemma closure_one_eq : closure ({1} : set E) = {x | ∥x∥ = 0} :=
755+
set.ext (λ x, mem_closure_one_iff_norm)
756+
751757
/-- A helper lemma used to prove that the (scalar or usual) product of a function that tends to one
752758
and a bounded function tends to one. This lemma is formulated for any binary operation
753759
`op : E → F → G` with an estimate `∥op x y∥ ≤ A * ∥x∥ * ∥y∥` for some constant A instead of

0 commit comments

Comments
 (0)