Loogle!
Result
Found 46 declarations mentioning intervalIntegral and Filter.Tendsto.
- intervalIntegral.tendsto_integral_filter_of_dominated_convergence ๐ Mathlib.MeasureTheory.Integral.DominatedConvergence
{E : Type u_2} [NormedAddCommGroup E] [NormedSpace โ E] {a b : โ} {f : โ โ E} {ฮผ : MeasureTheory.Measure โ} {ฮน : Type u_3} {l : Filter ฮน} [l.IsCountablyGenerated] {F : ฮน โ โ โ E} (bound : โ โ โ) (hF_meas : โแถ (n : ฮน) in l, MeasureTheory.AEStronglyMeasurable (F n) (ฮผ.restrict (Set.uIoc a b))) (h_bound : โแถ (n : ฮน) in l, โแต (x : โ) โฮผ, x โ Set.uIoc a b โ โF n xโ โค bound x) (bound_integrable : IntervalIntegrable bound ฮผ a b) (h_lim : โแต (x : โ) โฮผ, x โ Set.uIoc a b โ Filter.Tendsto (fun n => F n x) l (nhds (f x))) : Filter.Tendsto (fun n => โซ (x : โ) in a..b, F n x โฮผ) l (nhds (โซ (x : โ) in a..b, f x โฮผ)) - intervalIntegral.deriv_integral_of_tendsto_ae_right ๐ Mathlib.MeasureTheory.Integral.IntervalIntegral.FundThmCalculus
{E : Type u_3} [NormedAddCommGroup E] [NormedSpace โ E] [CompleteSpace E] {f : โ โ E} {c : E} {a b : โ} (hf : IntervalIntegrable f MeasureTheory.volume a b) (hmeas : StronglyMeasurableAtFilter f (nhds b) MeasureTheory.volume) (hb : Filter.Tendsto f (nhds b โ MeasureTheory.ae MeasureTheory.volume) (nhds c)) : deriv (fun u => โซ (x : โ) in a..u, f x) b = c - intervalIntegral.deriv_integral_of_tendsto_ae_left ๐ Mathlib.MeasureTheory.Integral.IntervalIntegral.FundThmCalculus
{E : Type u_3} [NormedAddCommGroup E] [NormedSpace โ E] [CompleteSpace E] {f : โ โ E} {c : E} {a b : โ} (hf : IntervalIntegrable f MeasureTheory.volume a b) (hmeas : StronglyMeasurableAtFilter f (nhds a) MeasureTheory.volume) (hb : Filter.Tendsto f (nhds a โ MeasureTheory.ae MeasureTheory.volume) (nhds c)) : deriv (fun u => โซ (x : โ) in u..b, f x) a = -c - intervalIntegral.measure_integral_sub_linear_isLittleO_of_tendsto_ae ๐ Mathlib.MeasureTheory.Integral.IntervalIntegral.FundThmCalculus
{ฮน : Type u_1} {E : Type u_3} [NormedAddCommGroup E] [NormedSpace โ E] {f : โ โ E} {a : โ} {c : E} {l l' : Filter โ} {lt : Filter ฮน} {ฮผ : MeasureTheory.Measure โ} {u v : ฮน โ โ} [MeasureTheory.IsLocallyFiniteMeasure ฮผ] [intervalIntegral.FTCFilter a l l'] (hfm : StronglyMeasurableAtFilter f l' ฮผ) (hf : Filter.Tendsto f (l' โ MeasureTheory.ae ฮผ) (nhds c)) (hu : Filter.Tendsto u lt l) (hv : Filter.Tendsto v lt l) : (fun t => โซ (x : โ) in u t..v t, f x โฮผ - โซ (x : โ) in u t..v t, c โฮผ) =o[lt] fun t => โซ (x : โ) in u t..v t, 1 โฮผ - intervalIntegral.measure_integral_sub_linear_isLittleO_of_tendsto_ae' ๐ Mathlib.MeasureTheory.Integral.IntervalIntegral.FundThmCalculus
{ฮน : Type u_1} {E : Type u_3} [NormedAddCommGroup E] [NormedSpace โ E] {f : โ โ E} {c : E} {l l' : Filter โ} {lt : Filter ฮน} {ฮผ : MeasureTheory.Measure โ} {u v : ฮน โ โ} [l'.IsMeasurablyGenerated] [Filter.TendstoIxxClass Set.Ioc l l'] (hfm : StronglyMeasurableAtFilter f l' ฮผ) (hf : Filter.Tendsto f (l' โ MeasureTheory.ae ฮผ) (nhds c)) (hl : ฮผ.FiniteAtFilter l') (hu : Filter.Tendsto u lt l) (hv : Filter.Tendsto v lt l) : (fun t => โซ (x : โ) in u t..v t, f x โฮผ - โซ (x : โ) in u t..v t, c โฮผ) =o[lt] fun t => โซ (x : โ) in u t..v t, 1 โฮผ - intervalIntegral.measure_integral_sub_integral_sub_linear_isLittleO_of_tendsto_ae_right ๐ Mathlib.MeasureTheory.Integral.IntervalIntegral.FundThmCalculus
{ฮน : Type u_1} {E : Type u_3} [NormedAddCommGroup E] [NormedSpace โ E] {f : โ โ E} {a b : โ} {c : E} {lb lb' : Filter โ} {lt : Filter ฮน} {ฮผ : MeasureTheory.Measure โ} {u v : ฮน โ โ} [MeasureTheory.IsLocallyFiniteMeasure ฮผ] [intervalIntegral.FTCFilter b lb lb'] (hab : IntervalIntegrable f ฮผ a b) (hmeas : StronglyMeasurableAtFilter f lb' ฮผ) (hf : Filter.Tendsto f (lb' โ MeasureTheory.ae ฮผ) (nhds c)) (hu : Filter.Tendsto u lt lb) (hv : Filter.Tendsto v lt lb) : (fun t => โซ (x : โ) in a..v t, f x โฮผ - โซ (x : โ) in a..u t, f x โฮผ - โซ (x : โ) in u t..v t, c โฮผ) =o[lt] fun t => โซ (x : โ) in u t..v t, 1 โฮผ - intervalIntegral.measure_integral_sub_integral_sub_linear_isLittleO_of_tendsto_ae_left ๐ Mathlib.MeasureTheory.Integral.IntervalIntegral.FundThmCalculus
{ฮน : Type u_1} {E : Type u_3} [NormedAddCommGroup E] [NormedSpace โ E] {f : โ โ E} {a b : โ} {c : E} {la la' : Filter โ} {lt : Filter ฮน} {ฮผ : MeasureTheory.Measure โ} {u v : ฮน โ โ} [MeasureTheory.IsLocallyFiniteMeasure ฮผ] [intervalIntegral.FTCFilter a la la'] (hab : IntervalIntegrable f ฮผ a b) (hmeas : StronglyMeasurableAtFilter f la' ฮผ) (hf : Filter.Tendsto f (la' โ MeasureTheory.ae ฮผ) (nhds c)) (hu : Filter.Tendsto u lt la) (hv : Filter.Tendsto v lt la) : (fun t => โซ (x : โ) in v t..b, f x โฮผ - โซ (x : โ) in u t..b, f x โฮผ + โซ (x : โ) in u t..v t, c โฮผ) =o[lt] fun t => โซ (x : โ) in u t..v t, 1 โฮผ - intervalIntegral.derivWithin_integral_of_tendsto_ae_right ๐ Mathlib.MeasureTheory.Integral.IntervalIntegral.FundThmCalculus
{E : Type u_3} [NormedAddCommGroup E] [NormedSpace โ E] [CompleteSpace E] {f : โ โ E} {c : E} {a b : โ} (hf : IntervalIntegrable f MeasureTheory.volume a b) {s t : Set โ} [intervalIntegral.FTCFilter b (nhdsWithin b s) (nhdsWithin b t)] (hmeas : StronglyMeasurableAtFilter f (nhdsWithin b t) MeasureTheory.volume) (hb : Filter.Tendsto f (nhdsWithin b t โ MeasureTheory.ae MeasureTheory.volume) (nhds c)) (hs : UniqueDiffWithinAt โ s b := by uniqueDiffWithinAt_Ici_Iic_univ) : derivWithin (fun u => โซ (x : โ) in a..u, f x) s b = c - intervalIntegral.derivWithin_integral_of_tendsto_ae_left ๐ Mathlib.MeasureTheory.Integral.IntervalIntegral.FundThmCalculus
{E : Type u_3} [NormedAddCommGroup E] [NormedSpace โ E] [CompleteSpace E] {f : โ โ E} {c : E} {a b : โ} (hf : IntervalIntegrable f MeasureTheory.volume a b) {s t : Set โ} [intervalIntegral.FTCFilter a (nhdsWithin a s) (nhdsWithin a t)] (hmeas : StronglyMeasurableAtFilter f (nhdsWithin a t) MeasureTheory.volume) (ha : Filter.Tendsto f (nhdsWithin a t โ MeasureTheory.ae MeasureTheory.volume) (nhds c)) (hs : UniqueDiffWithinAt โ s a := by uniqueDiffWithinAt_Ici_Iic_univ) : derivWithin (fun u => โซ (x : โ) in u..b, f x) s a = -c - intervalIntegral.integral_hasDerivAt_of_tendsto_ae_right ๐ Mathlib.MeasureTheory.Integral.IntervalIntegral.FundThmCalculus
{E : Type u_3} [NormedAddCommGroup E] [NormedSpace โ E] [CompleteSpace E] {f : โ โ E} {c : E} {a b : โ} (hf : IntervalIntegrable f MeasureTheory.volume a b) (hmeas : StronglyMeasurableAtFilter f (nhds b) MeasureTheory.volume) (hb : Filter.Tendsto f (nhds b โ MeasureTheory.ae MeasureTheory.volume) (nhds c)) : HasDerivAt (fun u => โซ (x : โ) in a..u, f x) c b - intervalIntegral.integral_hasStrictDerivAt_of_tendsto_ae_right ๐ Mathlib.MeasureTheory.Integral.IntervalIntegral.FundThmCalculus
{E : Type u_3} [NormedAddCommGroup E] [NormedSpace โ E] [CompleteSpace E] {f : โ โ E} {c : E} {a b : โ} (hf : IntervalIntegrable f MeasureTheory.volume a b) (hmeas : StronglyMeasurableAtFilter f (nhds b) MeasureTheory.volume) (hb : Filter.Tendsto f (nhds b โ MeasureTheory.ae MeasureTheory.volume) (nhds c)) : HasStrictDerivAt (fun u => โซ (x : โ) in a..u, f x) c b - intervalIntegral.integral_hasDerivAt_of_tendsto_ae_left ๐ Mathlib.MeasureTheory.Integral.IntervalIntegral.FundThmCalculus
{E : Type u_3} [NormedAddCommGroup E] [NormedSpace โ E] [CompleteSpace E] {f : โ โ E} {c : E} {a b : โ} (hf : IntervalIntegrable f MeasureTheory.volume a b) (hmeas : StronglyMeasurableAtFilter f (nhds a) MeasureTheory.volume) (ha : Filter.Tendsto f (nhds a โ MeasureTheory.ae MeasureTheory.volume) (nhds c)) : HasDerivAt (fun u => โซ (x : โ) in u..b, f x) (-c) a - intervalIntegral.integral_hasStrictDerivAt_of_tendsto_ae_left ๐ Mathlib.MeasureTheory.Integral.IntervalIntegral.FundThmCalculus
{E : Type u_3} [NormedAddCommGroup E] [NormedSpace โ E] [CompleteSpace E] {f : โ โ E} {c : E} {a b : โ} (hf : IntervalIntegrable f MeasureTheory.volume a b) (hmeas : StronglyMeasurableAtFilter f (nhds a) MeasureTheory.volume) (ha : Filter.Tendsto f (nhds a โ MeasureTheory.ae MeasureTheory.volume) (nhds c)) : HasStrictDerivAt (fun u => โซ (x : โ) in u..b, f x) (-c) a - intervalIntegral.integral_sub_linear_isLittleO_of_tendsto_ae ๐ Mathlib.MeasureTheory.Integral.IntervalIntegral.FundThmCalculus
{ฮน : Type u_1} {E : Type u_3} [NormedAddCommGroup E] [NormedSpace โ E] [CompleteSpace E] {f : โ โ E} {c : E} {l l' : Filter โ} {lt : Filter ฮน} {a : โ} [intervalIntegral.FTCFilter a l l'] (hfm : StronglyMeasurableAtFilter f l' MeasureTheory.volume) (hf : Filter.Tendsto f (l' โ MeasureTheory.ae MeasureTheory.volume) (nhds c)) {u v : ฮน โ โ} (hu : Filter.Tendsto u lt l) (hv : Filter.Tendsto v lt l) : (fun t => (โซ (x : โ) in u t..v t, f x) - (v t - u t) โข c) =o[lt] (v - u) - intervalIntegral.measure_integral_sub_linear_isLittleO_of_tendsto_ae_of_le ๐ Mathlib.MeasureTheory.Integral.IntervalIntegral.FundThmCalculus
{ฮน : Type u_1} {E : Type u_3} [NormedAddCommGroup E] [NormedSpace โ E] {f : โ โ E} {a : โ} {c : E} {l l' : Filter โ} {lt : Filter ฮน} {ฮผ : MeasureTheory.Measure โ} {u v : ฮน โ โ} [MeasureTheory.IsLocallyFiniteMeasure ฮผ] [CompleteSpace E] [intervalIntegral.FTCFilter a l l'] (hfm : StronglyMeasurableAtFilter f l' ฮผ) (hf : Filter.Tendsto f (l' โ MeasureTheory.ae ฮผ) (nhds c)) (hu : Filter.Tendsto u lt l) (hv : Filter.Tendsto v lt l) (huv : u โคแถ [lt] v) : (fun t => โซ (x : โ) in u t..v t, f x โฮผ - ฮผ.real (Set.Ioc (u t) (v t)) โข c) =o[lt] fun t => ฮผ.real (Set.Ioc (u t) (v t)) - intervalIntegral.measure_integral_sub_linear_isLittleO_of_tendsto_ae_of_le' ๐ Mathlib.MeasureTheory.Integral.IntervalIntegral.FundThmCalculus
{ฮน : Type u_1} {E : Type u_3} [NormedAddCommGroup E] [NormedSpace โ E] {f : โ โ E} {c : E} {l l' : Filter โ} {lt : Filter ฮน} {ฮผ : MeasureTheory.Measure โ} {u v : ฮน โ โ} [CompleteSpace E] [l'.IsMeasurablyGenerated] [Filter.TendstoIxxClass Set.Ioc l l'] (hfm : StronglyMeasurableAtFilter f l' ฮผ) (hf : Filter.Tendsto f (l' โ MeasureTheory.ae ฮผ) (nhds c)) (hl : ฮผ.FiniteAtFilter l') (hu : Filter.Tendsto u lt l) (hv : Filter.Tendsto v lt l) (huv : u โคแถ [lt] v) : (fun t => โซ (x : โ) in u t..v t, f x โฮผ - ฮผ.real (Set.Ioc (u t) (v t)) โข c) =o[lt] fun t => ฮผ.real (Set.Ioc (u t) (v t)) - intervalIntegral.integral_eq_sub_of_hasDerivAt_of_tendsto ๐ Mathlib.MeasureTheory.Integral.IntervalIntegral.FundThmCalculus
{E : Type u_3} [NormedAddCommGroup E] [NormedSpace โ E] {a b : โ} [CompleteSpace E] {f f' : โ โ E} (hab : a < b) {fa fb : E} (hderiv : โ x โ Set.Ioo a b, HasDerivAt f (f' x) x) (hint : IntervalIntegrable f' MeasureTheory.volume a b) (ha : Filter.Tendsto f (nhdsWithin a (Set.Ioi a)) (nhds fa)) (hb : Filter.Tendsto f (nhdsWithin b (Set.Iio b)) (nhds fb)) : โซ (y : โ) in a..b, f' y = fb - fa - intervalIntegral.integral_hasDerivWithinAt_of_tendsto_ae_right ๐ Mathlib.MeasureTheory.Integral.IntervalIntegral.FundThmCalculus
{E : Type u_3} [NormedAddCommGroup E] [NormedSpace โ E] [CompleteSpace E] {f : โ โ E} {c : E} {a b : โ} (hf : IntervalIntegrable f MeasureTheory.volume a b) {s t : Set โ} [intervalIntegral.FTCFilter b (nhdsWithin b s) (nhdsWithin b t)] (hmeas : StronglyMeasurableAtFilter f (nhdsWithin b t) MeasureTheory.volume) (hb : Filter.Tendsto f (nhdsWithin b t โ MeasureTheory.ae MeasureTheory.volume) (nhds c)) : HasDerivWithinAt (fun u => โซ (x : โ) in a..u, f x) c s b - intervalIntegral.measure_integral_sub_linear_isLittleO_of_tendsto_ae_of_ge ๐ Mathlib.MeasureTheory.Integral.IntervalIntegral.FundThmCalculus
{ฮน : Type u_1} {E : Type u_3} [NormedAddCommGroup E] [NormedSpace โ E] {f : โ โ E} {a : โ} {c : E} {l l' : Filter โ} {lt : Filter ฮน} {ฮผ : MeasureTheory.Measure โ} {u v : ฮน โ โ} [MeasureTheory.IsLocallyFiniteMeasure ฮผ] [CompleteSpace E] [intervalIntegral.FTCFilter a l l'] (hfm : StronglyMeasurableAtFilter f l' ฮผ) (hf : Filter.Tendsto f (l' โ MeasureTheory.ae ฮผ) (nhds c)) (hu : Filter.Tendsto u lt l) (hv : Filter.Tendsto v lt l) (huv : v โคแถ [lt] u) : (fun t => โซ (x : โ) in u t..v t, f x โฮผ + ฮผ.real (Set.Ioc (v t) (u t)) โข c) =o[lt] fun t => ฮผ.real (Set.Ioc (v t) (u t)) - intervalIntegral.measure_integral_sub_linear_isLittleO_of_tendsto_ae_of_ge' ๐ Mathlib.MeasureTheory.Integral.IntervalIntegral.FundThmCalculus
{ฮน : Type u_1} {E : Type u_3} [NormedAddCommGroup E] [NormedSpace โ E] {f : โ โ E} {c : E} {l l' : Filter โ} {lt : Filter ฮน} {ฮผ : MeasureTheory.Measure โ} {u v : ฮน โ โ} [CompleteSpace E] [l'.IsMeasurablyGenerated] [Filter.TendstoIxxClass Set.Ioc l l'] (hfm : StronglyMeasurableAtFilter f l' ฮผ) (hf : Filter.Tendsto f (l' โ MeasureTheory.ae ฮผ) (nhds c)) (hl : ฮผ.FiniteAtFilter l') (hu : Filter.Tendsto u lt l) (hv : Filter.Tendsto v lt l) (huv : v โคแถ [lt] u) : (fun t => โซ (x : โ) in u t..v t, f x โฮผ + ฮผ.real (Set.Ioc (v t) (u t)) โข c) =o[lt] fun t => ฮผ.real (Set.Ioc (v t) (u t)) - intervalIntegral.integral_hasDerivWithinAt_of_tendsto_ae_left ๐ Mathlib.MeasureTheory.Integral.IntervalIntegral.FundThmCalculus
{E : Type u_3} [NormedAddCommGroup E] [NormedSpace โ E] [CompleteSpace E] {f : โ โ E} {c : E} {a b : โ} (hf : IntervalIntegrable f MeasureTheory.volume a b) {s t : Set โ} [intervalIntegral.FTCFilter a (nhdsWithin a s) (nhdsWithin a t)] (hmeas : StronglyMeasurableAtFilter f (nhdsWithin a t) MeasureTheory.volume) (ha : Filter.Tendsto f (nhdsWithin a t โ MeasureTheory.ae MeasureTheory.volume) (nhds c)) : HasDerivWithinAt (fun u => โซ (x : โ) in u..b, f x) (-c) s a - intervalIntegral.integral_sub_integral_sub_linear_isLittleO_of_tendsto_ae_right ๐ Mathlib.MeasureTheory.Integral.IntervalIntegral.FundThmCalculus
{ฮน : Type u_1} {E : Type u_3} [NormedAddCommGroup E] [NormedSpace โ E] [CompleteSpace E] {f : โ โ E} {c : E} {lb lb' : Filter โ} {lt : Filter ฮน} {a b : โ} {u v : ฮน โ โ} [intervalIntegral.FTCFilter b lb lb'] (hab : IntervalIntegrable f MeasureTheory.volume a b) (hmeas : StronglyMeasurableAtFilter f lb' MeasureTheory.volume) (hf : Filter.Tendsto f (lb' โ MeasureTheory.ae MeasureTheory.volume) (nhds c)) (hu : Filter.Tendsto u lt lb) (hv : Filter.Tendsto v lt lb) : (fun t => ((โซ (x : โ) in a..v t, f x) - โซ (x : โ) in a..u t, f x) - (v t - u t) โข c) =o[lt] (v - u) - intervalIntegral.integral_sub_integral_sub_linear_isLittleO_of_tendsto_ae_left ๐ Mathlib.MeasureTheory.Integral.IntervalIntegral.FundThmCalculus
{ฮน : Type u_1} {E : Type u_3} [NormedAddCommGroup E] [NormedSpace โ E] [CompleteSpace E] {f : โ โ E} {c : E} {la la' : Filter โ} {lt : Filter ฮน} {a b : โ} {u v : ฮน โ โ} [intervalIntegral.FTCFilter a la la'] (hab : IntervalIntegrable f MeasureTheory.volume a b) (hmeas : StronglyMeasurableAtFilter f la' MeasureTheory.volume) (hf : Filter.Tendsto f (la' โ MeasureTheory.ae MeasureTheory.volume) (nhds c)) (hu : Filter.Tendsto u lt la) (hv : Filter.Tendsto v lt la) : (fun t => ((โซ (x : โ) in v t..b, f x) - โซ (x : โ) in u t..b, f x) + (v t - u t) โข c) =o[lt] (v - u) - intervalIntegral.measure_integral_sub_integral_sub_linear_isLittleO_of_tendsto_ae ๐ Mathlib.MeasureTheory.Integral.IntervalIntegral.FundThmCalculus
{ฮน : Type u_1} {E : Type u_3} [NormedAddCommGroup E] [NormedSpace โ E] {f : โ โ E} {a b : โ} {ca cb : E} {la la' lb lb' : Filter โ} {lt : Filter ฮน} {ฮผ : MeasureTheory.Measure โ} {ua va ub vb : ฮน โ โ} [MeasureTheory.IsLocallyFiniteMeasure ฮผ] [intervalIntegral.FTCFilter a la la'] [intervalIntegral.FTCFilter b lb lb'] (hab : IntervalIntegrable f ฮผ a b) (hmeas_a : StronglyMeasurableAtFilter f la' ฮผ) (hmeas_b : StronglyMeasurableAtFilter f lb' ฮผ) (ha_lim : Filter.Tendsto f (la' โ MeasureTheory.ae ฮผ) (nhds ca)) (hb_lim : Filter.Tendsto f (lb' โ MeasureTheory.ae ฮผ) (nhds cb)) (hua : Filter.Tendsto ua lt la) (hva : Filter.Tendsto va lt la) (hub : Filter.Tendsto ub lt lb) (hvb : Filter.Tendsto vb lt lb) : (fun t => โซ (x : โ) in va t..vb t, f x โฮผ - โซ (x : โ) in ua t..ub t, f x โฮผ - (โซ (x : โ) in ub t..vb t, cb โฮผ - โซ (x : โ) in ua t..va t, ca โฮผ)) =o[lt] fun t => โโซ (x : โ) in ua t..va t, 1 โฮผโ + โโซ (x : โ) in ub t..vb t, 1 โฮผโ - intervalIntegral.integral_sub_integral_sub_linear_isLittleO_of_tendsto_ae ๐ Mathlib.MeasureTheory.Integral.IntervalIntegral.FundThmCalculus
{ฮน : Type u_1} {E : Type u_3} [NormedAddCommGroup E] [NormedSpace โ E] [CompleteSpace E] {f : โ โ E} {ca cb : E} {la la' lb lb' : Filter โ} {lt : Filter ฮน} {a b : โ} {ua ub va vb : ฮน โ โ} [intervalIntegral.FTCFilter a la la'] [intervalIntegral.FTCFilter b lb lb'] (hab : IntervalIntegrable f MeasureTheory.volume a b) (hmeas_a : StronglyMeasurableAtFilter f la' MeasureTheory.volume) (hmeas_b : StronglyMeasurableAtFilter f lb' MeasureTheory.volume) (ha_lim : Filter.Tendsto f (la' โ MeasureTheory.ae MeasureTheory.volume) (nhds ca)) (hb_lim : Filter.Tendsto f (lb' โ MeasureTheory.ae MeasureTheory.volume) (nhds cb)) (hua : Filter.Tendsto ua lt la) (hva : Filter.Tendsto va lt la) (hub : Filter.Tendsto ub lt lb) (hvb : Filter.Tendsto vb lt lb) : (fun t => ((โซ (x : โ) in va t..vb t, f x) - โซ (x : โ) in ua t..ub t, f x) - ((vb t - ub t) โข cb - (va t - ua t) โข ca)) =o[lt] fun t => โva t - ua tโ + โvb t - ub tโ - intervalIntegral.integral_hasFDerivWithinAt ๐ Mathlib.MeasureTheory.Integral.IntervalIntegral.FundThmCalculus
{E : Type u_3} [NormedAddCommGroup E] [NormedSpace โ E] [CompleteSpace E] {f : โ โ E} {la lb : Filter โ} {a b : โ} (hf : IntervalIntegrable f MeasureTheory.volume a b) (hmeas_a : StronglyMeasurableAtFilter f la MeasureTheory.volume) (hmeas_b : StronglyMeasurableAtFilter f lb MeasureTheory.volume) {s t : Set โ} [intervalIntegral.FTCFilter a (nhdsWithin a s) la] [intervalIntegral.FTCFilter b (nhdsWithin b t) lb] (ha : Filter.Tendsto f la (nhds (f a))) (hb : Filter.Tendsto f lb (nhds (f b))) : HasFDerivWithinAt (fun p => โซ (x : โ) in p.1 ..p.2, f x) ((ContinuousLinearMap.snd โ โ โ).smulRight (f b) - (ContinuousLinearMap.fst โ โ โ).smulRight (f a)) (s รหข t) (a, b) - intervalIntegral.integral_hasFDerivAt_of_tendsto_ae ๐ Mathlib.MeasureTheory.Integral.IntervalIntegral.FundThmCalculus
{E : Type u_3} [NormedAddCommGroup E] [NormedSpace โ E] [CompleteSpace E] {f : โ โ E} {ca cb : E} {a b : โ} (hf : IntervalIntegrable f MeasureTheory.volume a b) (hmeas_a : StronglyMeasurableAtFilter f (nhds a) MeasureTheory.volume) (hmeas_b : StronglyMeasurableAtFilter f (nhds b) MeasureTheory.volume) (ha : Filter.Tendsto f (nhds a โ MeasureTheory.ae MeasureTheory.volume) (nhds ca)) (hb : Filter.Tendsto f (nhds b โ MeasureTheory.ae MeasureTheory.volume) (nhds cb)) : HasFDerivAt (fun p => โซ (x : โ) in p.1 ..p.2, f x) ((ContinuousLinearMap.snd โ โ โ).smulRight cb - (ContinuousLinearMap.fst โ โ โ).smulRight ca) (a, b) - intervalIntegral.integral_hasStrictFDerivAt_of_tendsto_ae ๐ Mathlib.MeasureTheory.Integral.IntervalIntegral.FundThmCalculus
{E : Type u_3} [NormedAddCommGroup E] [NormedSpace โ E] [CompleteSpace E] {f : โ โ E} {ca cb : E} {a b : โ} (hf : IntervalIntegrable f MeasureTheory.volume a b) (hmeas_a : StronglyMeasurableAtFilter f (nhds a) MeasureTheory.volume) (hmeas_b : StronglyMeasurableAtFilter f (nhds b) MeasureTheory.volume) (ha : Filter.Tendsto f (nhds a โ MeasureTheory.ae MeasureTheory.volume) (nhds ca)) (hb : Filter.Tendsto f (nhds b โ MeasureTheory.ae MeasureTheory.volume) (nhds cb)) : HasStrictFDerivAt (fun p => โซ (x : โ) in p.1 ..p.2, f x) ((ContinuousLinearMap.snd โ โ โ).smulRight cb - (ContinuousLinearMap.fst โ โ โ).smulRight ca) (a, b) - intervalIntegral.integral_hasFDerivWithinAt_of_tendsto_ae ๐ Mathlib.MeasureTheory.Integral.IntervalIntegral.FundThmCalculus
{E : Type u_3} [NormedAddCommGroup E] [NormedSpace โ E] [CompleteSpace E] {f : โ โ E} {ca cb : E} {la lb : Filter โ} {a b : โ} (hf : IntervalIntegrable f MeasureTheory.volume a b) {s t : Set โ} [intervalIntegral.FTCFilter a (nhdsWithin a s) la] [intervalIntegral.FTCFilter b (nhdsWithin b t) lb] (hmeas_a : StronglyMeasurableAtFilter f la MeasureTheory.volume) (hmeas_b : StronglyMeasurableAtFilter f lb MeasureTheory.volume) (ha : Filter.Tendsto f (la โ MeasureTheory.ae MeasureTheory.volume) (nhds ca)) (hb : Filter.Tendsto f (lb โ MeasureTheory.ae MeasureTheory.volume) (nhds cb)) : HasFDerivWithinAt (fun p => โซ (x : โ) in p.1 ..p.2, f x) ((ContinuousLinearMap.snd โ โ โ).smulRight cb - (ContinuousLinearMap.fst โ โ โ).smulRight ca) (s รหข t) (a, b) - intervalIntegral.fderiv_integral_of_tendsto_ae ๐ Mathlib.MeasureTheory.Integral.IntervalIntegral.FundThmCalculus
{E : Type u_3} [NormedAddCommGroup E] [NormedSpace โ E] [CompleteSpace E] {f : โ โ E} {ca cb : E} {a b : โ} (hf : IntervalIntegrable f MeasureTheory.volume a b) (hmeas_a : StronglyMeasurableAtFilter f (nhds a) MeasureTheory.volume) (hmeas_b : StronglyMeasurableAtFilter f (nhds b) MeasureTheory.volume) (ha : Filter.Tendsto f (nhds a โ MeasureTheory.ae MeasureTheory.volume) (nhds ca)) (hb : Filter.Tendsto f (nhds b โ MeasureTheory.ae MeasureTheory.volume) (nhds cb)) : fderiv โ (fun p => โซ (x : โ) in p.1 ..p.2, f x) (a, b) = (ContinuousLinearMap.snd โ โ โ).smulRight cb - (ContinuousLinearMap.fst โ โ โ).smulRight ca - intervalIntegral.fderivWithin_integral_of_tendsto_ae ๐ Mathlib.MeasureTheory.Integral.IntervalIntegral.FundThmCalculus
{E : Type u_3} [NormedAddCommGroup E] [NormedSpace โ E] [CompleteSpace E] {f : โ โ E} {ca cb : E} {la lb : Filter โ} {a b : โ} (hf : IntervalIntegrable f MeasureTheory.volume a b) (hmeas_a : StronglyMeasurableAtFilter f la MeasureTheory.volume) (hmeas_b : StronglyMeasurableAtFilter f lb MeasureTheory.volume) {s t : Set โ} [intervalIntegral.FTCFilter a (nhdsWithin a s) la] [intervalIntegral.FTCFilter b (nhdsWithin b t) lb] (ha : Filter.Tendsto f (la โ MeasureTheory.ae MeasureTheory.volume) (nhds ca)) (hb : Filter.Tendsto f (lb โ MeasureTheory.ae MeasureTheory.volume) (nhds cb)) (hs : UniqueDiffWithinAt โ s a := by uniqueDiffWithinAt_Ici_Iic_univ) (ht : UniqueDiffWithinAt โ t b := by uniqueDiffWithinAt_Ici_Iic_univ) : fderivWithin โ (fun p => โซ (x : โ) in p.1 ..p.2, f x) (s รหข t) (a, b) = (ContinuousLinearMap.snd โ โ โ).smulRight cb - (ContinuousLinearMap.fst โ โ โ).smulRight ca - MeasureTheory.intervalIntegral_tendsto_integral ๐ Mathlib.MeasureTheory.Integral.IntegralEqImproper
{ฮน : Type u_1} {E : Type u_2} {ฮผ : MeasureTheory.Measure โ} {l : Filter ฮน} [l.IsCountablyGenerated] [NormedAddCommGroup E] [NormedSpace โ E] {a b : ฮน โ โ} {f : โ โ E} (hfi : MeasureTheory.Integrable f ฮผ) (ha : Filter.Tendsto a l Filter.atBot) (hb : Filter.Tendsto b l Filter.atTop) : Filter.Tendsto (fun i => โซ (x : โ) in a i..b i, f x โฮผ) l (nhds (โซ (x : โ), f x โฮผ)) - MeasureTheory.intervalIntegral_tendsto_integral_Iic ๐ Mathlib.MeasureTheory.Integral.IntegralEqImproper
{ฮน : Type u_1} {E : Type u_2} {ฮผ : MeasureTheory.Measure โ} {l : Filter ฮน} [l.IsCountablyGenerated] [NormedAddCommGroup E] [NormedSpace โ E] {a : ฮน โ โ} {f : โ โ E} (b : โ) (hfi : MeasureTheory.IntegrableOn f (Set.Iic b) ฮผ) (ha : Filter.Tendsto a l Filter.atBot) : Filter.Tendsto (fun i => โซ (x : โ) in a i..b, f x โฮผ) l (nhds (โซ (x : โ) in Set.Iic b, f x โฮผ)) - MeasureTheory.intervalIntegral_tendsto_integral_Ioi ๐ Mathlib.MeasureTheory.Integral.IntegralEqImproper
{ฮน : Type u_1} {E : Type u_2} {ฮผ : MeasureTheory.Measure โ} {l : Filter ฮน} [l.IsCountablyGenerated] [NormedAddCommGroup E] [NormedSpace โ E] {b : ฮน โ โ} {f : โ โ E} (a : โ) (hfi : MeasureTheory.IntegrableOn f (Set.Ioi a) ฮผ) (hb : Filter.Tendsto b l Filter.atTop) : Filter.Tendsto (fun i => โซ (x : โ) in a..b i, f x โฮผ) l (nhds (โซ (x : โ) in Set.Ioi a, f x โฮผ)) - MeasureTheory.integrableOn_Iic_of_intervalIntegral_norm_bounded ๐ Mathlib.MeasureTheory.Integral.IntegralEqImproper
{ฮน : Type u_1} {E : Type u_2} {ฮผ : MeasureTheory.Measure โ} {l : Filter ฮน} [l.NeBot] [l.IsCountablyGenerated] [NormedAddCommGroup E] {a : ฮน โ โ} {f : โ โ E} (I b : โ) (hfi : โ (i : ฮน), MeasureTheory.IntegrableOn f (Set.Ioc (a i) b) ฮผ) (ha : Filter.Tendsto a l Filter.atBot) (h : โแถ (i : ฮน) in l, โซ (x : โ) in a i..b, โf xโ โฮผ โค I) : MeasureTheory.IntegrableOn f (Set.Iic b) ฮผ - MeasureTheory.integrableOn_Ioi_of_intervalIntegral_norm_bounded ๐ Mathlib.MeasureTheory.Integral.IntegralEqImproper
{ฮน : Type u_1} {E : Type u_2} {ฮผ : MeasureTheory.Measure โ} {l : Filter ฮน} [l.NeBot] [l.IsCountablyGenerated] [NormedAddCommGroup E] {b : ฮน โ โ} {f : โ โ E} (I a : โ) (hfi : โ (i : ฮน), MeasureTheory.IntegrableOn f (Set.Ioc a (b i)) ฮผ) (hb : Filter.Tendsto b l Filter.atTop) (h : โแถ (i : ฮน) in l, โซ (x : โ) in a..b i, โf xโ โฮผ โค I) : MeasureTheory.IntegrableOn f (Set.Ioi a) ฮผ - MeasureTheory.integrableOn_Iic_of_intervalIntegral_norm_tendsto ๐ Mathlib.MeasureTheory.Integral.IntegralEqImproper
{ฮน : Type u_1} {E : Type u_2} {ฮผ : MeasureTheory.Measure โ} {l : Filter ฮน} [l.NeBot] [l.IsCountablyGenerated] [NormedAddCommGroup E] {a : ฮน โ โ} {f : โ โ E} (I b : โ) (hfi : โ (i : ฮน), MeasureTheory.IntegrableOn f (Set.Ioc (a i) b) ฮผ) (ha : Filter.Tendsto a l Filter.atBot) (h : Filter.Tendsto (fun i => โซ (x : โ) in a i..b, โf xโ โฮผ) l (nhds I)) : MeasureTheory.IntegrableOn f (Set.Iic b) ฮผ - MeasureTheory.integrableOn_Ioi_of_intervalIntegral_norm_tendsto ๐ Mathlib.MeasureTheory.Integral.IntegralEqImproper
{ฮน : Type u_1} {E : Type u_2} {ฮผ : MeasureTheory.Measure โ} {l : Filter ฮน} [l.NeBot] [l.IsCountablyGenerated] [NormedAddCommGroup E] {b : ฮน โ โ} {f : โ โ E} (I a : โ) (hfi : โ (i : ฮน), MeasureTheory.IntegrableOn f (Set.Ioc a (b i)) ฮผ) (hb : Filter.Tendsto b l Filter.atTop) (h : Filter.Tendsto (fun i => โซ (x : โ) in a..b i, โf xโ โฮผ) l (nhds I)) : MeasureTheory.IntegrableOn f (Set.Ioi a) ฮผ - MeasureTheory.integrable_of_intervalIntegral_norm_bounded ๐ Mathlib.MeasureTheory.Integral.IntegralEqImproper
{ฮน : Type u_1} {E : Type u_2} {ฮผ : MeasureTheory.Measure โ} {l : Filter ฮน} [l.NeBot] [l.IsCountablyGenerated] [NormedAddCommGroup E] {a b : ฮน โ โ} {f : โ โ E} (I : โ) (hfi : โ (i : ฮน), MeasureTheory.IntegrableOn f (Set.Ioc (a i) (b i)) ฮผ) (ha : Filter.Tendsto a l Filter.atBot) (hb : Filter.Tendsto b l Filter.atTop) (h : โแถ (i : ฮน) in l, โซ (x : โ) in a i..b i, โf xโ โฮผ โค I) : MeasureTheory.Integrable f ฮผ - MeasureTheory.integrable_of_intervalIntegral_norm_tendsto ๐ Mathlib.MeasureTheory.Integral.IntegralEqImproper
{ฮน : Type u_1} {E : Type u_2} {ฮผ : MeasureTheory.Measure โ} {l : Filter ฮน} [l.NeBot] [l.IsCountablyGenerated] [NormedAddCommGroup E] {a b : ฮน โ โ} {f : โ โ E} (I : โ) (hfi : โ (i : ฮน), MeasureTheory.IntegrableOn f (Set.Ioc (a i) (b i)) ฮผ) (ha : Filter.Tendsto a l Filter.atBot) (hb : Filter.Tendsto b l Filter.atTop) (h : Filter.Tendsto (fun i => โซ (x : โ) in a i..b i, โf xโ โฮผ) l (nhds I)) : MeasureTheory.Integrable f ฮผ - Function.Periodic.tendsto_atBot_intervalIntegral_of_pos' ๐ Mathlib.MeasureTheory.Integral.IntervalIntegral.Periodic
{T : โ} {g : โ โ โ} (hg : Function.Periodic g T) (h_int : IntervalIntegrable g MeasureTheory.volume 0 T) (hโ : โ (x : โ), 0 < g x) (hT : 0 < T) : Filter.Tendsto (fun t => โซ (x : โ) in 0 ..t, g x) Filter.atBot Filter.atBot - Function.Periodic.tendsto_atTop_intervalIntegral_of_pos' ๐ Mathlib.MeasureTheory.Integral.IntervalIntegral.Periodic
{T : โ} {g : โ โ โ} (hg : Function.Periodic g T) (h_int : IntervalIntegrable g MeasureTheory.volume 0 T) (hโ : โ (x : โ), 0 < g x) (hT : 0 < T) : Filter.Tendsto (fun t => โซ (x : โ) in 0 ..t, g x) Filter.atTop Filter.atTop - Function.Periodic.tendsto_atBot_intervalIntegral_of_pos ๐ Mathlib.MeasureTheory.Integral.IntervalIntegral.Periodic
{T : โ} {g : โ โ โ} (hg : Function.Periodic g T) (hโ : 0 < โซ (x : โ) in 0 ..T, g x) (hT : 0 < T) : Filter.Tendsto (fun t => โซ (x : โ) in 0 ..t, g x) Filter.atBot Filter.atBot - Function.Periodic.tendsto_atTop_intervalIntegral_of_pos ๐ Mathlib.MeasureTheory.Integral.IntervalIntegral.Periodic
{T : โ} {g : โ โ โ} (hg : Function.Periodic g T) (hโ : 0 < โซ (x : โ) in 0 ..T, g x) (hT : 0 < T) : Filter.Tendsto (fun t => โซ (x : โ) in 0 ..t, g x) Filter.atTop Filter.atTop - EulerSine.tendsto_integral_cos_pow_mul_div ๐ Mathlib.Analysis.SpecialFunctions.Trigonometric.EulerSineProd
{f : โ โ โ} (hf : ContinuousOn f (Set.Icc 0 (Real.pi / 2))) : Filter.Tendsto (fun n => (โซ (x : โ) in 0 ..Real.pi / 2, โ(Real.cos x) ^ n * f x) / โ(โซ (x : โ) in 0 ..Real.pi / 2, Real.cos x ^ n)) Filter.atTop (nhds (f 0)) - Complex.approx_Gamma_integral_tendsto_Gamma_integral ๐ Mathlib.Analysis.SpecialFunctions.Gamma.Beta
{s : โ} (hs : 0 < s.re) : Filter.Tendsto (fun n => โซ (x : โ) in 0 ..โn, โ((1 - x / โn) ^ n) * โx ^ (s - 1)) Filter.atTop (nhds (Complex.Gamma s))
About
Loogle searches Lean and Mathlib definitions and theorems.
You can use Loogle from within the Lean4 VSCode language extension
using (by default) Ctrl-K Ctrl-S. You can also try the
#loogle
command from LeanSearchClient,
the CLI version, the Loogle
VS Code extension, the lean.nvim
integration or the Zulip bot.
Usage
Loogle finds definitions and lemmas in various ways:
By constant:
๐Real.sin
finds all lemmas whose statement somehow mentions the sine function.By lemma name substring:
๐"differ"
finds all lemmas that have"differ"
somewhere in their lemma name.By subexpression:
๐_ * (_ ^ _)
finds all lemmas whose statements somewhere include a product where the second argument is raised to some power.The pattern can also be non-linear, as in
๐Real.sqrt ?a * Real.sqrt ?a
If the pattern has parameters, they are matched in any order. Both of these will find
List.map
:
๐(?a -> ?b) -> List ?a -> List ?b
๐List ?a -> (?a -> ?b) -> List ?b
By main conclusion:
๐|- tsum _ = _ * tsum _
finds all lemmas where the conclusion (the subexpression to the right of allโ
andโ
) has the given shape.As before, if the pattern has parameters, they are matched against the hypotheses of the lemma in any order; for example,
๐|- _ < _ โ tsum _ < tsum _
will findtsum_lt_tsum
even though the hypothesisf i < g i
is not the last.
If you pass more than one such search filter, separated by commas
Loogle will return lemmas which match all of them. The
search
๐ Real.sin, "two", tsum, _ * _, _ ^ _, |- _ < _ โ _
would find all lemmas which mention the constants Real.sin
and tsum
, have "two"
as a substring of the
lemma name, include a product and a power somewhere in the type,
and have a hypothesis of the form _ < _
(if
there were any such lemmas). Metavariables (?a
) are
assigned independently in each filter.
The #lucky
button will directly send you to the
documentation of the first hit.
Source code
You can find the source code for this service at https://github.com/nomeata/loogle. The https://loogle.lean-lang.org/ service is provided by the Lean FRO.
This is Loogle revision 19971e9
serving mathlib revision c3b95a7