Zulip Chat Archive
Stream: Is there code for X?
Topic: Preimage of normed ball
Moritz Doll (Mar 30 2022 at 00:49):
Does this lemma already exist somewhere? I could not find it in normed_group
and neither could library_search
. If it does not exist what would be a good name?
import analysis.normed.group.basic
variables {π F : Type*}
variables [normed_group π]
variables (f : F β π)
lemma closed_ball_preimage (r : β) : {y : F | β₯f yβ₯ β€ r} =
f β»ΒΉ' (metric.closed_ball (0 : π) r) :=
by { ext y, simp }
Patrick Massot (Mar 30 2022 at 07:18):
It seems very specialized to me, do you really need this very often?
Eric Wieser (Mar 30 2022 at 07:43):
That's basically true by refl
besides the sub_zero
, right?
Eric Wieser (Mar 30 2022 at 07:45):
Which direction do you think you need the lemma in? Currently the name is for the opposite direction to the statement
Patrick Massot (Mar 30 2022 at 07:48):
You also need to use the fact that the distance is given by the norm.
Patrick Massot (Mar 30 2022 at 07:48):
A direct proof would be: unfold set.preimage, simp_rw mem_closed_ball_zero_iff
Moritz Doll (Mar 30 2022 at 08:27):
I only need it once (for now), so I have to problem with using it inline. To avoid an xy-problem: I want to prove that {y : F | β₯f yβ₯ β€ r}
is closed (for continuous f
).
Kevin Buzzard (Mar 30 2022 at 08:32):
This is just "closed balls are closed" plus "preimage of closed is closed"
Moritz Doll (Mar 30 2022 at 08:41):
Yes of course, but in Lean it needs some (trivial) rewrite first
Anatole Dedecker (Mar 30 2022 at 08:53):
I think you can avoid rewriting by using docs#continuous.norm and docs#is_closed_Iic, although itβs less mathematically satisfying
Floris van Doorn (Mar 30 2022 at 09:02):
Moritz Doll said:
I only need it once (for now), so I have to problem with using it inline. To avoid an xy-problem: I want to prove that
{y : F | β₯f yβ₯ β€ r}
is closed (for continuousf
).
If hf : continuous f
, then this is is_closed_le hf.norm continuous_const
.
Last updated: Dec 20 2023 at 11:08 UTC