Skip to content

Commit 5bb7d0f

Browse files
committed
fix for compatibility with earlier versions
1 parent 897764e commit 5bb7d0f

File tree

1 file changed

+4
-2
lines changed

1 file changed

+4
-2
lines changed

theories/lebesgue_measure.v

Lines changed: 4 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -387,7 +387,9 @@ Qed.
387387
Definition lebesgue_measure := measure_extension [the measure _ _ of hlength].
388388
HB.instance Definition _ := Measure.on lebesgue_measure.
389389

390-
Let sigmaT_finite_lebesgue_measure : sigma_finite setT lebesgue_measure.
390+
(* TODO: this ought to be turned into a Let but older version of mathcomp/coq
391+
does not seem to allow, try to change asap *)
392+
Local Lemma sigmaT_finite_lebesgue_measure : sigma_finite setT lebesgue_measure.
391393
Proof. exact/measure_extension_sigma_finite/hlength_sigma_finite. Qed.
392394

393395
HB.instance Definition _ := @isSigmaFinite.Build _ _ _
@@ -2031,7 +2033,7 @@ Lemma lebesgue_regularity_inner_sup (D : set R) (eps : R) : measurable D ->
20312033
Proof.
20322034
move=> mD; have [?|] := ltP (mu D) +oo.
20332035
exact: lebesgue_regularity_innerE_bounded.
2034-
have /sigma_finiteP [/= F RFU [Fsub ffin]] := sigma_finiteT mu.
2036+
have /sigma_finiteP [/= F RFU [Fsub ffin]] := sigmaT_finite_lebesgue_measure R (*TODO: sigma_finiteT mu should be enough but does not seem to work with holder version of mathcomp/coq *).
20352037
rewrite leye_eq => /eqP /[dup] + ->.
20362038
have {1}-> : D = \bigcup_n (F n `&` D) by rewrite -setI_bigcupl -RFU setTI.
20372039
move=> FDp; apply/esym/eq_infty => M.

0 commit comments

Comments
 (0)