Skip to content

Commit b012cf4

Browse files
authored
Merge pull request #595 from math-comp/measure_20220311
fixes #566
2 parents c5437dd + 5a6daa7 commit b012cf4

File tree

4 files changed

+107
-99
lines changed

4 files changed

+107
-99
lines changed

CHANGELOG_UNRELEASED.md

Lines changed: 6 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -48,6 +48,12 @@
4848
+ `oinv_valLr` -> `oinv_valR`
4949
+ `valLr_inj_subproof` -> `valR_inj_subproof`
5050
+ `valLr_surj_subproof` -> `valR_surj_subproof`
51+
- in `measure.v`:
52+
+ `measurable_bigcup` -> `bigcupT_measurable`
53+
+ `measurable_bigcap` -> `bigcapT_measurable`
54+
+ `measurable_bigcup_rat` -> `bigcupT_measurable_rat`
55+
- in `lebesgue_measure.v`:
56+
+ `emeasurable_bigcup` -> `bigcupT_emeasurable`
5157

5258
### Removed
5359

theories/lebesgue_integral.v

Lines changed: 6 additions & 6 deletions
Original file line numberDiff line numberDiff line change
@@ -929,7 +929,7 @@ apply: ereal_cvgrM => //; rewrite [X in _ --> X](_ : _ =
929929
mu (\bigcup_n (f @^-1` [set r] `&` fleg c n))); last first.
930930
by rewrite -setI_bigcupr bigcup_fleg// setIT.
931931
have ? k i : measurable (f @^-1` [set k] `&` fleg c i) by exact: measurableI.
932-
apply: cvg_mu_inc => //; first exact: measurable_bigcup.
932+
apply: cvg_mu_inc => //; first exact: bigcupT_measurable.
933933
move=> n m nm; apply/subsetPset; apply: setIS.
934934
by move/(nd_fleg c) : nm => /subsetPset.
935935
Unshelve. all: by end_near. Qed.
@@ -2874,7 +2874,7 @@ move=> mf; split=> [iDf0|Df0].
28742874
apply/esym/cvg_lim => //; apply: cvg_mu_inc.
28752875
- move=> i; apply: emeasurable_fun_c_infty => //.
28762876
exact: measurable_fun_comp.
2877-
- apply: measurable_bigcup => i.
2877+
- apply: bigcupT_measurable => i.
28782878
by apply: emeasurable_fun_c_infty => //; exact: measurable_fun_comp.
28792879
- move=> m n mn; apply/subsetPset; apply: setIS => t /=.
28802880
by apply: le_trans; rewrite lee_fin lef_pinv // ?ler_nat // posrE.
@@ -3491,11 +3491,11 @@ Let B := [set A | measurable A /\ measurable_fun setT (phi A)].
34913491
Lemma xsection_ndseq_closed : ndseq_closed B.
34923492
Proof.
34933493
move=> F ndF; rewrite /B /= => BF; split.
3494-
by apply: measurable_bigcup => n; have [] := BF n.
3494+
by apply: bigcupT_measurable => n; have [] := BF n.
34953495
have phiF x : (fun i => phi (F i) x) --> phi (\bigcup_i F i) x.
34963496
rewrite /phi /= xsection_bigcup; apply: cvg_mu_inc => //.
34973497
- by move=> n; apply: measurable_xsection; case: (BF n).
3498-
- by apply: measurable_bigcup => i; apply: measurable_xsection; case: (BF i).
3498+
- by apply: bigcupT_measurable => i; apply: measurable_xsection; case: (BF i).
34993499
- move=> m n mn; apply/subsetPset => y; rewrite /xsection/= !inE.
35003500
by have /subsetPset FmFn := ndF _ _ mn; exact: FmFn.
35013501
apply: (emeasurable_fun_cvg (phi \o F)) => //.
@@ -3512,11 +3512,11 @@ Let B := [set A | measurable A /\ measurable_fun setT (psi A)].
35123512
Lemma ysection_ndseq_closed : ndseq_closed B.
35133513
Proof.
35143514
move=> F ndF; rewrite /B /= => BF; split.
3515-
by apply: measurable_bigcup => n; have [] := BF n.
3515+
by apply: bigcupT_measurable => n; have [] := BF n.
35163516
have psiF x : (fun i => psi (F i) x) --> psi (\bigcup_i F i) x.
35173517
rewrite /psi /= ysection_bigcup; apply: cvg_mu_inc => //.
35183518
- by move=> n; apply: measurable_ysection; case: (BF n).
3519-
- by apply: measurable_bigcup => i; apply: measurable_ysection; case: (BF i).
3519+
- by apply: bigcupT_measurable => i; apply: measurable_ysection; case: (BF i).
35203520
- move=> m n mn; apply/subsetPset => y; rewrite /ysection/= !inE.
35213521
by have /subsetPset FmFn := ndF _ _ mn; exact: FmFn.
35223522
apply: (emeasurable_fun_cvg (psi \o F)) => //.

0 commit comments

Comments
 (0)