Skip to content

Commit da217ff

Browse files
authored
Merge pull request #1664 from affeldt-aist/fixes_1616
fixes #1652
2 parents 8dd352a + bc815a3 commit da217ff

14 files changed

+86
-121
lines changed

CHANGELOG_UNRELEASED.md

Lines changed: 25 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -99,6 +99,9 @@
9999
- in `lebesgue_integral_fubini.v`:
100100
+ lemmas `integral21_prod_meas2`, `integral12_prod_meas2`
101101

102+
- in `lebesgue_integral_nonneg.v`:
103+
+ lemma `ge0_integral_ereal_sup` (was a `Let`)
104+
102105
### Changed
103106

104107
- in `convex.v`:
@@ -257,6 +260,12 @@
257260
+ `limZr` -> `limZl_tmp`
258261
+ `continuousZr` -> `continuousZl_tmp`
259262
+ `continuousZl` -> `continuousZr_tmp`
263+
- in `realfun.v`:
264+
+ `variationD` -> `variation_cat`
265+
266+
- in `lebesgue_integrable.v`:
267+
+ `integral_fune_lt_pinfty` -> `integrable_lty`
268+
+ `integral_fune_fin_num` -> `integrable_fin_num`
260269

261270
### Generalized
262271

@@ -294,6 +303,22 @@
294303
+ definition `almost_everywhere_notation`
295304
+ lemma `ess_sup_ge0`
296305

306+
- in `exp.v`:
307+
+ notation `expRMm` (deprecated since 1.1.0)
308+
309+
- in `constructive_ereal.v`:
310+
+ notations `lee_addl`, `lee_addr`, `lee_add2l`, `lee_add2r`, `lee_add`,
311+
`lee_sub`, `lee_add2lE`, `lee_oppl`, `lee_oppr`, `lte_oppl`, `lte_oppr`,
312+
`lte_add`, `lte_add2lE`, `lte_addl`, `lte_addr` (deprecated since 1.1.0)
313+
314+
- in `measure.v`:
315+
+ notations `sub_additive`, `sigma_sub_additive`, `content_sub_additive`,
316+
`ring_sigma_sub_additive`, `Content_SubSigmaAdditive_isMeasure.Build`,
317+
`measure_sigma_sub_additive`, `measure_sigma_sub_additive_tail`,
318+
`Measure_isSFinite_subdef.Build`, `sfinite_measure_subdef`,
319+
`@SigmaFinite_isFinite.Build`, `FiniteMeasure_isSubProbability.Build`
320+
(deprecated since 1.1.0)
321+
297322
### Infrastructure
298323

299324
### Misc

reals/constructive_ereal.v

Lines changed: 0 additions & 30 deletions
Original file line numberDiff line numberDiff line change
@@ -2859,36 +2859,6 @@ Arguments lee_sum_nneg_natl {R}.
28592859
Arguments lee_sum_npos_natl {R}.
28602860
#[global] Hint Extern 0 (is_true (0 <= `| _ |)%E) => solve [apply: abse_ge0] : core.
28612861

2862-
#[deprecated(since="mathcomp-analysis 1.1.0", note="Use leeDl instead.")]
2863-
Notation lee_addl := leeDl (only parsing).
2864-
#[deprecated(since="mathcomp-analysis 1.1.0", note="Use leeDr instead.")]
2865-
Notation lee_addr := leeDr (only parsing).
2866-
#[deprecated(since="mathcomp-analysis 1.1.0", note="Use leeD2l instead.")]
2867-
Notation lee_add2l := leeD2l (only parsing).
2868-
#[deprecated(since="mathcomp-analysis 1.1.0", note="Use leeD2r instead.")]
2869-
Notation lee_add2r := leeD2r (only parsing).
2870-
#[deprecated(since="mathcomp-analysis 1.1.0", note="Use leeD instead.")]
2871-
Notation lee_add := leeD (only parsing).
2872-
#[deprecated(since="mathcomp-analysis 1.1.0", note="Use leeB instead.")]
2873-
Notation lee_sub := leeB (only parsing).
2874-
#[deprecated(since="mathcomp-analysis 1.1.0", note="Use leeD2lE instead.")]
2875-
Notation lee_add2lE := leeD2lE (only parsing).
2876-
#[deprecated(since="mathcomp-analysis 1.1.0", note="Use leeNl instead.")]
2877-
Notation lee_oppl := leeNl (only parsing).
2878-
#[deprecated(since="mathcomp-analysis 1.1.0", note="Use leeNr instead.")]
2879-
Notation lee_oppr := leeNr (only parsing).
2880-
#[deprecated(since="mathcomp-analysis 1.1.0", note="Use lteNl instead.")]
2881-
Notation lte_oppl := lteNl (only parsing).
2882-
#[deprecated(since="mathcomp-analysis 1.1.0", note="Use lteNr instead.")]
2883-
Notation lte_oppr := lteNr (only parsing).
2884-
#[deprecated(since="mathcomp-analysis 1.1.0", note="Use lteD instead.")]
2885-
Notation lte_add := lteD (only parsing).
2886-
#[deprecated(since="mathcomp-analysis 1.1.0", note="Use lteD2lE instead.")]
2887-
Notation lte_add2lE := lteD2lE (only parsing).
2888-
#[deprecated(since="mathcomp-analysis 1.1.0", note="Use lteDl instead.")]
2889-
Notation lte_addl := lteDl (only parsing).
2890-
#[deprecated(since="mathcomp-analysis 1.1.0", note="Use lteDr instead.")]
2891-
Notation lte_addr := lteDr (only parsing).
28922862
#[deprecated(since="mathcomp-analysis 1.2.0", note="Use gee_pMl instead.")]
28932863
Notation gee_pmull := gee_pMl (only parsing).
28942864
#[deprecated(since="mathcomp-analysis 1.2.0", note="Use geeDl instead.")]

theories/charge.v

Lines changed: 3 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -1140,7 +1140,7 @@ Let nu0 : nu set0 = 0. Proof. by rewrite /nu integral_set0. Qed.
11401140

11411141
Let finnu A : measurable A -> nu A \is a fin_num.
11421142
Proof.
1143-
by move=> mA; apply: integral_fune_fin_num => //=; exact: integrableS intf.
1143+
by move=> mA; apply: integrable_fin_num => //=; exact: integrableS intf.
11441144
Qed.
11451145

11461146
Let snu : semi_sigma_additive nu.
@@ -1151,10 +1151,10 @@ rewrite (_ : SF = fun n =>
11511151
\sum_(0 <= i < n) (\int[mu]_(x in F i) f^\- x)); last first.
11521152
apply/funext => n; rewrite /SF; under eq_bigr do rewrite /nu integralE.
11531153
rewrite big_split/= sumeN//= => i j _ _.
1154-
rewrite fin_num_adde_defl// integral_fune_fin_num//= integrable_funeneg//=.
1154+
rewrite fin_num_adde_defl// integrable_fin_num//= integrable_funeneg//=.
11551155
exact: integrableS intf.
11561156
rewrite /nu integralE; apply: cvgeD.
1157-
- rewrite fin_num_adde_defr// integral_fune_fin_num//=.
1157+
- rewrite fin_num_adde_defr// integrable_fin_num//=.
11581158
by apply: integrable_funepos => //=; exact: integrableS intf.
11591159
- apply/semi_sigma_additive_nng_induced => //.
11601160
by apply: measurable_funepos; exact: (measurable_int mu).

theories/exp.v

Lines changed: 1 addition & 4 deletions
Original file line numberDiff line numberDiff line change
@@ -1,4 +1,4 @@
1-
(* mathcomp analysis (c) 2017 Inria and AIST. License: CeCILL-C. *)
1+
(* mathcomp analysis (c) 2025 Inria and AIST. License: CeCILL-C. *)
22
From mathcomp Require Import all_ssreflect ssralg ssrint ssrnum matrix.
33
From mathcomp Require Import interval rat.
44
From mathcomp Require Import boolp classical_sets functions mathcomp_extra.
@@ -605,9 +605,6 @@ Canonical expR_inum (i : Itv.t) (x : Itv.def (@Itv.num_sem R) i) :=
605605

606606
End expR.
607607

608-
#[deprecated(since="mathcomp-analysis 1.1.0", note="renamed `expRM_natl`")]
609-
Notation expRMm := expRM_natl (only parsing).
610-
611608
Section expeR.
612609
Context {R : realType}.
613610
Implicit Types (x y : \bar R) (r s : R).

theories/ftc.v

Lines changed: 14 additions & 14 deletions
Original file line numberDiff line numberDiff line change
@@ -116,7 +116,7 @@ apply: cvg_at_right_left_dnbhs.
116116
- rewrite addeAC -[X in _ - X]integral_itv_bndo_bndc//=; last first.
117117
by case: locf => + _ _; exact: measurable_funS.
118118
rewrite subee ?add0e//.
119-
by apply: integral_fune_fin_num => //; exact: integrableS intf.
119+
by apply: integrable_fin_num => //; exact: integrableS intf.
120120
- by case: locf => + _ _; exact: measurable_funS.
121121
- apply/disj_setPRL => z/=.
122122
rewrite /E /= !in_itv/= => /andP[xz zxdn].
@@ -130,8 +130,8 @@ apply: cvg_at_right_left_dnbhs.
130130
fun n => (d n)^-1 *: fine (\int[mu]_(t in E x n) (f t)%:E)); last first.
131131
apply/funext => n; congr (_ *: _); rewrite -fineB/=.
132132
by rewrite /= (addrC (d n) x) ixdf.
133-
by apply: integral_fune_fin_num => //; exact: integrableS intf.
134-
by apply: integral_fune_fin_num => //; exact: integrableS intf.
133+
by apply: integrable_fin_num => //; exact: integrableS intf.
134+
by apply: integrable_fin_num => //; exact: integrableS intf.
135135
have := nice_lebesgue_differentiation nice_E locf fx.
136136
rewrite {ixdf} -/mu.
137137
rewrite [g in g n @[n --> _] --> _ -> _](_ : _ =
@@ -143,7 +143,7 @@ apply: cvg_at_right_left_dnbhs.
143143
suff : g = h by move=> <-.
144144
apply/funext => n.
145145
rewrite /g /h /= fineM//.
146-
apply: integral_fune_fin_num => //; first exact: (nice_E _).1.
146+
apply: integrable_fin_num => //; first exact: (nice_E _).1.
147147
by apply: integrableS intf => //; exact: (nice_E _).1.
148148
- apply/cvg_at_leftP => d [d_gt0 d0].
149149
have {}Nd_gt0 n : (0 < - d n)%R by rewrite ltrNr oppr0.
@@ -173,7 +173,7 @@ apply: cvg_at_right_left_dnbhs.
173173
rewrite -/mu -[LHS]oppeK; congr oppe.
174174
rewrite oppeB; last first.
175175
rewrite fin_num_adde_defl// fin_numN//.
176-
by apply: integral_fune_fin_num => //; exact: integrableS intf.
176+
by apply: integrable_fin_num => //; exact: integrableS intf.
177177
rewrite addeC.
178178
rewrite (_ : `]-oo, x] = `]-oo, (x + d n)%R] `|` E x n)%classic; last first.
179179
by rewrite -itv_bndbnd_setU//= bnd_simp ler_wnDr// ltW.
@@ -182,7 +182,7 @@ apply: cvg_at_right_left_dnbhs.
182182
rewrite -[X in X - _]integral_itv_bndo_bndc//; last first.
183183
by case: locf => + _ _; exact: measurable_funS.
184184
rewrite subee ?add0e//.
185-
by apply: integral_fune_fin_num => //; exact: integrableS intf.
185+
by apply: integrable_fin_num => //; exact: integrableS intf.
186186
- exact: (nice_E _).1.
187187
- by case: locf => + _ _; exact: measurable_funS.
188188
- apply/disj_setPLR => z/=.
@@ -198,7 +198,7 @@ apply: cvg_at_right_left_dnbhs.
198198
rewrite -/mu -[LHS]oppeK; congr oppe.
199199
rewrite oppeB; last first.
200200
rewrite fin_num_adde_defl// fin_numN//.
201-
by apply: integral_fune_fin_num => //; exact: integrableS intf.
201+
by apply: integrable_fin_num => //; exact: integrableS intf.
202202
rewrite addeC.
203203
rewrite (@itv_bndbnd_setU _ _ _ (BRight (x - - d n)%R))//; last 2 first.
204204
case: b in ax * => /=; rewrite bnd_simp.
@@ -211,7 +211,7 @@ apply: cvg_at_right_left_dnbhs.
211211
- rewrite addeAC -[X in X - _]integral_itv_bndo_bndc//; last first.
212212
by case: locf => + _ _; exact: measurable_funS.
213213
rewrite opprK subee ?add0e//.
214-
by apply: integral_fune_fin_num => //; exact: integrableS intf.
214+
by apply: integrable_fin_num => //; exact: integrableS intf.
215215
- by case: locf => + _ _; exact: measurable_funS.
216216
- apply/disj_setPLR => z/=.
217217
rewrite /E /= !in_itv/= => /andP[az zxdn].
@@ -220,16 +220,16 @@ apply: cvg_at_right_left_dnbhs.
220220
@[n --> \oo] --> f x.
221221
apply: cvg_trans; apply: near_eq_cvg; near=> n; congr (_ *: _).
222222
rewrite /F -fineN -fineB; last 2 first.
223-
by apply: integral_fune_fin_num => //; exact: integrableS intf.
224-
by apply: integral_fune_fin_num => //; exact: integrableS intf.
223+
by apply: integrable_fin_num => //; exact: integrableS intf.
224+
by apply: integrable_fin_num => //; exact: integrableS intf.
225225
by congr fine => /=; apply/esym; rewrite (addrC _ x); near: n.
226226
have := nice_lebesgue_differentiation nice_E locf fx.
227227
rewrite {ixdf} -/mu.
228228
move/fine_cvgP => [_ /=].
229229
set g := _ \o _ => gf.
230230
rewrite (@eq_cvg _ _ _ _ g)// => n.
231231
rewrite /g /= fineM//=; last first.
232-
apply: integral_fune_fin_num => //; first exact: (nice_E _).1.
232+
apply: integrable_fin_num => //; first exact: (nice_E _).1.
233233
by apply: integrableS intf => //; exact: (nice_E _).1.
234234
by rewrite muE inver oppr_eq0 lt_eqF.
235235
by rewrite muE/= inver oppr_eq0 lt_eqF// invrN mulNr -mulrN.
@@ -377,7 +377,7 @@ have acbc : `[a, c] `<=` `[a, b].
377377
apply: subset_itvl; rewrite bnd_simp; move: ac; near: c.
378378
exact: lt_nbhsl_le.
379379
rewrite -lee_fin fineK; last first.
380-
apply: integral_fune_fin_num => //=.
380+
apply: integrable_fin_num => //=.
381381
rewrite (_ : (fun _ => _) = abse \o ((EFin \o f) \_ `[a, b])); last first.
382382
by apply/funext => x /=; rewrite restrict_EFin.
383383
apply/integrable_abse/integrable_restrict => //=.
@@ -641,7 +641,7 @@ have GbFbc : G b = (F b - c)%R.
641641
rewrite -EFinB -cE -GbFbc /G /Rintegral/= fineK//.
642642
rewrite integralEpatch//=.
643643
by under eq_integral do rewrite restrict_EFin.
644-
exact: integral_fune_fin_num.
644+
exact: integrable_fin_num.
645645
Unshelve. all: by end_near. Qed.
646646

647647
Lemma ge0_continuous_FTC2y (f F : R -> R) a (l : R) :
@@ -826,7 +826,7 @@ have ? : mu.-integrable `[a, b] (fun x => ((f * G) x)%:E).
826826
+ have := derivable_oo_continuous_bnd_within Gab.
827827
by move/subspace_continuousP; exact.
828828
rewrite /= integralD//=.
829-
- by rewrite addeAC subee ?add0e// integral_fune_fin_num.
829+
- by rewrite addeAC subee ?add0e// integrable_fin_num.
830830
- apply: continuous_compact_integrable => //; first exact: segment_compact.
831831
apply/subspace_continuousP => x abx;apply: cvgM.
832832
+ have := derivable_oo_continuous_bnd_within Fab.

theories/gauss_integral.v

Lines changed: 3 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -262,7 +262,7 @@ under eq_integral do rewrite fctE/= EFinM.
262262
have ? : mu.-integrable `[0, 1] (fun y => (gauss_fun (y * x))%:E).
263263
apply: continuous_compact_integrable => //; first exact: segment_compact.
264264
by apply: continuous_subspaceT => z; exact: continuous_gaussM.
265-
rewrite integralZr//= fineM//=; last exact: integral_fune_fin_num.
265+
rewrite integralZr//= fineM//=; last exact: integrable_fin_num.
266266
by rewrite mulrC.
267267
Qed.
268268

@@ -288,10 +288,10 @@ have -> : gauss_fun x = \int[mu]_(t in `[0, 1]) cst (gauss_fun x) t.
288288
rewrite Rintegral_cst//.
289289
by rewrite /mu/= lebesgue_measure_itv//= lte01 oppr0 addr0 mulr1.
290290
rewrite fine_le//.
291-
- apply: integral_fune_fin_num => //=.
291+
- apply: integrable_fin_num => //=.
292292
apply: continuous_compact_integrable; first exact: segment_compact.
293293
by apply: continuous_in_subspaceT => z _; exact: continuous_u.
294-
- apply: integral_fune_fin_num => //=.
294+
- apply: integrable_fin_num => //=.
295295
apply: continuous_compact_integrable; first exact: segment_compact.
296296
by apply: continuous_subspaceT => z; exact: cvg_cst.
297297
apply: ge0_le_integral => //=.

theories/lebesgue_integral_theory/lebesgue_Rintegral.v

Lines changed: 3 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -92,7 +92,7 @@ Lemma RintegralZl D f r : measurable D -> mu.-integrable D (EFin \o f) ->
9292
\int[mu]_(x in D) (r * f x) = r * \int[mu]_(x in D) f x.
9393
Proof.
9494
move=> mD intf; rewrite (_ : r = fine r%:E)// -fineM//; last first.
95-
exact: integral_fune_fin_num.
95+
exact: integrable_fin_num.
9696
by congr fine; under eq_integral do rewrite EFinM; exact: integralZl.
9797
Qed.
9898

@@ -177,7 +177,7 @@ Lemma RintegralD D f1 f2 : measurable D ->
177177
\int[mu]_(x in D) f1 x + \int[mu]_(x in D) f2 x.
178178
Proof.
179179
move=> mD if1 if2.
180-
by rewrite /Rintegral integralD_EFin// fineD//; exact: integral_fune_fin_num.
180+
by rewrite /Rintegral integralD_EFin// fineD//; exact: integrable_fin_num.
181181
Qed.
182182

183183
Lemma RintegralB D f1 f2 : measurable D ->
@@ -186,7 +186,7 @@ Lemma RintegralB D f1 f2 : measurable D ->
186186
\int[mu]_(x in D) f1 x - \int[mu]_(x in D) f2 x.
187187
Proof.
188188
move=> mD if1 if2.
189-
by rewrite /Rintegral integralB_EFin// fineB//; exact: integral_fune_fin_num.
189+
by rewrite /Rintegral integralB_EFin// fineB//; exact: integrable_fin_num.
190190
Qed.
191191

192192
End Rintegral.

theories/lebesgue_integral_theory/lebesgue_integrable.v

Lines changed: 10 additions & 6 deletions
Original file line numberDiff line numberDiff line change
@@ -720,12 +720,12 @@ Qed.
720720

721721
End integralB.
722722

723-
Section integrable_fune.
723+
Section integrable_lty_fin_num.
724724
Context d (T : measurableType d) (R : realType).
725725
Variables (mu : {measure set T -> \bar R}) (D : set T) (mD : measurable D).
726726
Local Open Scope ereal_scope.
727727

728-
Lemma integral_fune_lt_pinfty (f : T -> \bar R) :
728+
Lemma integrable_lty (f : T -> \bar R) :
729729
mu.-integrable D f -> \int[mu]_(x in D) f x < +oo.
730730
Proof.
731731
move=> intf; rewrite (funeposneg f) integralB//;
@@ -734,15 +734,19 @@ rewrite lte_add_pinfty ?integral_funepos_lt_pinfty// lteNl ltNye_eq.
734734
by rewrite integrable_neg_fin_num.
735735
Qed.
736736

737-
Lemma integral_fune_fin_num (f : T -> \bar R) :
737+
Lemma integrable_fin_num (f : T -> \bar R) :
738738
mu.-integrable D f -> \int[mu]_(x in D) f x \is a fin_num.
739739
Proof.
740-
move=> h; apply/fin_numPlt; rewrite integral_fune_lt_pinfty// andbC/= -/(- +oo).
741-
rewrite lteNl -integralN; first exact/integral_fune_lt_pinfty/integrableN.
740+
move=> h; apply/fin_numPlt; rewrite integrable_lty// andbC/= -/(- +oo).
741+
rewrite lteNl -integralN; first exact/integrable_lty/integrableN.
742742
by rewrite fin_num_adde_defl// fin_numN integrable_neg_fin_num.
743743
Qed.
744744

745-
End integrable_fune.
745+
End integrable_lty_fin_num.
746+
#[deprecated(since="mathcomp-analysis 1.12.0", note="renamed to `integrable_lty`")]
747+
Notation integral_fune_lt_pinfty := integrable_lty (only parsing).
748+
#[deprecated(since="mathcomp-analysis 1.12.0", note="renamed to `integrable_fin_num`")]
749+
Notation integral_fune_fin_num := integrable_fin_num (only parsing).
746750

747751
Section transfer.
748752
Context d1 d2 (X : measurableType d1) (Y : measurableType d2) (R : realType).

theories/lebesgue_integral_theory/lebesgue_integral_differentiation.v

Lines changed: 7 additions & 7 deletions
Original file line numberDiff line numberDiff line change
@@ -115,7 +115,7 @@ have [g [gfe2 ig]] : exists g : {sfun R >-> rT},
115115
have [g_ [intG ?]] := approximation_sfun_integrable mE intf.
116116
move/fine_fcvg/cvg_ballP/(_ (eps%:num / 2)%R) => -[] // n _ Nb; exists (g_ n).
117117
have fg_fin_num : \int[mu]_(z in E) `|(f z - g_ n z)%:E| \is a fin_num.
118-
rewrite integral_fune_fin_num// integrable_abse//.
118+
rewrite integrable_fin_num// integrable_abse//.
119119
by under eq_fun do rewrite EFinB; apply: integrableB => //; exact: intG.
120120
split; last exact: intG.
121121
have /= := Nb _ (leqnn n); rewrite /ball/= sub0r normrN -fine_abse// -lte_fin.
@@ -228,9 +228,9 @@ have -> : f x = (r *+ 2)^-1 * \int[mu]_(z in `[x - r, x + r]) cst (f x) z.
228228
have intRf : mu.-integrable `[x - r, x + r] (EFin \o f).
229229
exact: (@integrableS _ _ _ mu _ _ _ _ _ xrA intf).
230230
rewrite /= -mulrBr -fineB; first last.
231-
- rewrite integral_fune_fin_num// continuous_compact_integrable// => ?.
231+
- rewrite integrable_fin_num// continuous_compact_integrable// => ?.
232232
exact: cvg_cst.
233-
- by rewrite integral_fune_fin_num.
233+
- by rewrite integrable_fin_num.
234234
rewrite -integralB_EFin //; first last.
235235
by apply: continuous_compact_integrable => // ?; exact: cvg_cst.
236236
under [fun _ => _ + _ ]eq_fun => ? do rewrite -EFinD.
@@ -239,17 +239,17 @@ have int_fx : mu.-integrable `[x - r, x + r] (fun z => (f z - f x)%:E).
239239
rewrite integrableB// continuous_compact_integrable// => ?.
240240
exact: cvg_cst.
241241
rewrite normrM ger0_norm // -fine_abse //; first last.
242-
by rewrite integral_fune_fin_num.
242+
by rewrite integrable_fin_num.
243243
suff : (\int[mu]_(z in `[(x - r)%R, (x + r)%R]) `|f z - f x|%:E <=
244244
(r *+ 2 * eps)%:E)%E.
245245
move=> intfeps; apply: le_trans.
246246
apply: (ler_pM r20 _ (le_refl _)); first exact: fine_ge0.
247247
apply: fine_le; last apply: le_abse_integral => //.
248-
- by rewrite abse_fin_num integral_fune_fin_num.
249-
- by rewrite integral_fune_fin_num// integrable_abse.
248+
- by rewrite abse_fin_num integrable_fin_num.
249+
- by rewrite integrable_fin_num// integrable_abse.
250250
- by case/integrableP : int_fx.
251251
rewrite ler_pdivrMl ?mulrn_wgt0 // -[_ * _]/(fine (_%:E)).
252-
by rewrite fine_le// integral_fune_fin_num// integrable_abse.
252+
by rewrite fine_le// integrable_fin_num// integrable_abse.
253253
apply: le_trans.
254254
- apply: (@integral_le_bound _ _ _ _ _ (fun z => (f z - f x)%:E) eps%:E) => //.
255255
+ by case/integrableP: int_fx.

theories/lebesgue_integral_theory/lebesgue_integral_dominated_convergence.v

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -328,8 +328,8 @@ have mfn : mu.-integrable E (fun z => `|f^\- z - (n_ n z)%:E|).
328328
rewrite -[X in (_ <= `|X|)%R]fineD // -integralD //.
329329
move: finfn finfp => _ _.
330330
rewrite !ger0_norm ?fine_ge0 ?integral_ge0 ?fine_le//.
331-
- by apply: integral_fune_fin_num => //; exact/integrable_abse/mfpn.
332-
- by apply: integral_fune_fin_num => //; exact: integrableD.
331+
- by apply: integrable_fin_num => //; exact/integrable_abse/mfpn.
332+
- by apply: integrable_fin_num => //; exact: integrableD.
333333
- apply: ge0_le_integral => //.
334334
+ by apply: measurableT_comp => //; case/integrableP: (mfpn n).
335335
+ by move=> x Ex; rewrite adde_ge0.

0 commit comments

Comments
 (0)