Zulip Chat Archive
Stream: maths
Topic: measurable embedding
Yury G. Kudryashov (Oct 28 2021 at 17:50):
I'm going to introduce
structure measurable_embedding {α β : Type*} [measurable_space α] [measurable_space β] (f : α → β) :
Prop :=
(injective : injective f)
(measurable : measurable f)
(measurable_set_image' : ∀ ⦃s⦄, measurable_set s → measurable_set (f '' s))
Yury G. Kudryashov (Oct 28 2021 at 17:51):
Currently we have separate lemmas about closed_embedding
s and measurable_equiv
s.
Yury G. Kudryashov (Oct 28 2021 at 17:51):
With this definition we can generalize all these lemmas to measurable_embedding
s.
Yury G. Kudryashov (Oct 28 2021 at 17:52):
(an embedding
is a measurable_embedding
if it has a measurable range, so any closed embedding is a measurable embedding)
Yury G. Kudryashov (Oct 28 2021 at 17:52):
Any objections/comments?
Yakov Pechersky (Oct 28 2021 at 19:35):
Would it make sense to extend "embedding"?
Johan Commelin (Oct 28 2021 at 19:37):
That bundles the function, right?
Yakov Pechersky (Oct 28 2021 at 19:37):
Yes
Yakov Pechersky (Oct 28 2021 at 19:38):
I don't know the measure part of the library, how often one needs solely props or works with families of measurable functions.
Yury G. Kudryashov (Oct 28 2021 at 19:58):
An embedding
says something about topology, so I don't want to extend it.
Yury G. Kudryashov (Oct 28 2021 at 20:00):
I don't want to bundle the function because I'm not going to make statements about the space of all measurable embeddings (see also docs#embedding, docs#closed_embedding, docs#open_embedding).
Yury G. Kudryashov (Oct 28 2021 at 20:01):
With a predicate we can do rw [hf.some_lemma]
without moving to bundled functions first.
Yury G. Kudryashov (Oct 28 2021 at 20:24):
Right now I have theory about measurable_embedding
s up to
/-- If `g : α → β` is a measurable embedding and `f : β → ℝ≥0∞` is any function (not necessarily
measurable), then `∫⁻ a, f a ∂(map g μ) = ∫⁻ a, f (g a) ∂μ`. Compare with `lintegral_map` wich
applies to any measurable `g : α → β` but requires that `f` is measurable as well. -/
lemma lintegral_map_embedding [measurable_space β] (f : β → ℝ≥0∞) {g : α → β}
(hg : measurable_embedding g) :
∫⁻ a, f a ∂(map g μ) = ∫⁻ a, f (g a) ∂μ :=
Yakov Pechersky (Oct 28 2021 at 23:42):
Sorry I wasn't clear, I meant docs#function.embedding
Yaël Dillies (Oct 28 2021 at 23:43):
Also, should stuff in topology be disambiguated? There's docs#embedding, docs#locally_finite... I assume those names are historical artifacts because not much was here to concurrence them back when they got defined, right?
Yury G. Kudryashov (Oct 28 2021 at 23:56):
function.embedding
has bundled to_fun
, and I want to have a predicate like docs#embedding.
Last updated: Dec 20 2023 at 11:08 UTC