Zulip Chat Archive
Stream: Is there code for X?
Topic: Positive overlap
Vincent Beffara (Sep 13 2023 at 09:07):
Do we have this somewhere? (Possibly in much larger generality like a uniform space?)
import Mathlib
variable {K : Set ℝ} {S : Finset (Set ℝ)}
lemma bla (hK : IsCompact K) (hS : ∀ s ∈ S, IsOpen s) (hKS : K ⊆ ⋃ s ∈ S, s) :
∃ ε > 0, ∀ x ∈ K, ∃ s ∈ S, closedBall x ε ⊆ s := by
sorry
Sebastien Gouezel (Sep 13 2023 at 09:39):
Something like docs#lebesgue_number_lemma, maybe?
Vincent Beffara (Sep 13 2023 at 09:46):
Yes exactly! Thanks!
Sebastien Gouezel (Sep 13 2023 at 09:50):
There is now a very cool way to find the anwer to this kind of question: ask loogle to state all theorems mentioning all the stuff that should be in your statements.
Sebastien Gouezel (Sep 13 2023 at 09:51):
@loogle IsCompact, IsOpen, Set, (∃ _, _), (⋃ _, _)
loogle (Sep 13 2023 at 09:51):
:search: isCompact_iff_finite_subcover, isCompact_of_finite_subcover, and 12 more
Sebastien Gouezel (Sep 13 2023 at 09:52):
I've been pretty vague in my query since it wasn't clear if it would be in metric or uniformity terms, but for sure there would be an existential, a union, and IsCompact
, IsOpen
and Set
.
Sebastien Gouezel (Sep 13 2023 at 09:53):
And I notice in the suggestions by loogle a better answer to your question: docs#lebesgue_number_lemma_of_metric
Vincent Beffara (Sep 13 2023 at 09:57):
Yes I just saw it. It is just stated in terms of an indexed family instead of a set of sets, which I guess is why exact?
was not helping.
Vincent Beffara (Sep 13 2023 at 09:58):
It's kind of amazing that loogle works that well (I would have expected a much longer list of lemmas with that request ...)
Last updated: Dec 20 2023 at 11:08 UTC