Zulip Chat Archive
Stream: new members
Topic: Why does this theorem leads to contradiction?
Arshak Parsa (Aug 14 2024 at 15:06):
import Mathlib
open MeasureTheory Filter Set ProbabilityTheory Topology
lemma F_tendsto_atBot_inf {f : ℝ → ℝ} (hf : Integrable f) :
Tendsto (fun x ↦ ∫ (t : ℝ) in Iic x, f t) atBot (𝓝 0) := by
let s := fun i : ℝ => Iic (i)
have hmono : Monotone (⇑volume ∘ s) := by
unfold_let
rw [monotone_iff_forall_lt]
aesop
have h1 : Tendsto (⇑ℙ ∘ s) atBot (𝓝 (⨅ i, (⇑ℙ ∘ s) i)) := by
exact tendsto_atBot_iInf hmono
have hiInf : (⨅ i, (⇑ℙ ∘ s) i) = 0 := by
unfold_let
simp only [Function.comp_apply]
simp only [Real.volume_Iic]
rw [iInf]
simp
sorry
rw [hiInf] at h1
exact Integrable.tendsto_setIntegral_nhds_zero hf h1
After simp
my goal becomes False
.
btw could someone prove this theorem, it is too hard for me :/
Arshak Parsa (Aug 14 2024 at 15:09):
Is there a better notation for limit ?
like lim x → -∞ , (∫ (t : ℝ) in Iic x, f t) = 0
instead of Tendsto (fun x ↦ ∫ (t : ℝ) in Iic x, f t) atBot (𝓝 0)
Eric Wieser (Aug 14 2024 at 15:34):
hiInf
is false before the second simp only
because the goal is ⨅ i, ℙ (Iic i) = 0
, but in fact ⨅ i, ℙ (Iic i) = ∞
Eric Wieser (Aug 14 2024 at 15:35):
What's the math proof?
Arshak Parsa (Aug 14 2024 at 15:40):
Is f(x) = x
integrable ?
It is true only for integrable integrals.
(Actually, I am trying to prove that the limit of cumulative distribution function is 0 at -inf :grimacing:)
Arshak Parsa (Aug 14 2024 at 15:44):
Well, I guess it doesn't need a proof because when Iic x
goes to negative infinity, it is approaching the empty set, and the integral of empty set is zero.
(I am assuming that my integral is finite and positive)
Arshak Parsa (Aug 14 2024 at 15:47):
You are right, I think I need to add the f x > 0
to my hypothesis
Arshak Parsa (Aug 14 2024 at 15:52):
lemma F_tendsto_atBot_inf {f : ℝ → ℝ} (hf : Integrable f) (hpos : ∀x, f x ≥ 0):
Tendsto (fun x ↦ ∫ (t : ℝ) in Iic x, f t) atBot (𝓝 0) := by
sorry
this is my lemma
Etienne Marion (Aug 14 2024 at 16:46):
Hi! Here is a proof using dominated convergence theorem, you don't need nonnegativity assumption.
import Mathlib
open MeasureTheory Filter Set ProbabilityTheory Topology
lemma F_tendsto_atBot_inf {f : ℝ → ℝ} (hf : Integrable f) :
Tendsto (fun x ↦ ∫ (t : ℝ) in Iic x, f t) atBot (𝓝 0) := by
have this (x : ℝ) : ∫ t in Iic x, f t = ∫ t, (Iic x).indicator f t :=
(integral_indicator measurableSet_Iic).symm
simp_rw [this]
rw [← integral_zero]
apply tendsto_integral_filter_of_dominated_convergence (fun x ↦ ‖f x‖)
· exact eventually_of_forall fun x ↦ hf.aestronglyMeasurable.indicator measurableSet_Iic
· exact eventually_of_forall fun x ↦ eventually_of_forall fun y ↦ norm_indicator_le_norm_self _ _
· exact hf.norm
· refine eventually_of_forall fun x ↦ tendsto_const_nhds.congr' ?_
rw [EventuallyEq, eventually_atBot]
refine ⟨x - 1, fun y hy ↦ ?_⟩
simp [Set.indicator, (by linarith : ¬x ≤ y)]
Notification Bot (Aug 14 2024 at 19:23):
Arshak Parsa has marked this topic as resolved.
Notification Bot (Aug 14 2024 at 20:18):
Eric Wieser has marked this topic as unresolved.
Eric Wieser (Aug 14 2024 at 20:19):
I wonder if mathlib should have this result, and similarly for atTop?
Eric Wieser (Aug 14 2024 at 20:19):
Maybe an analyst can chime in (unresolving for visibility)
Arshak Parsa (Aug 14 2024 at 20:19):
Nice!
Arshak Parsa (Aug 14 2024 at 20:20):
I also need another theorem :grimacing:
Etienne Marion (Aug 15 2024 at 06:20):
Feel free to ask if you have any trouble!
Sébastien Gouëzel (Aug 15 2024 at 06:36):
Note that it should be possible to remove also the integrability assumption, as non-integrable functions have zero integral.
Last updated: May 02 2025 at 03:31 UTC