Skip to content

Commit 28b1e65

Browse files
committed
rebase, rm warnings
1 parent de38944 commit 28b1e65

File tree

2 files changed

+6
-8
lines changed

2 files changed

+6
-8
lines changed

theories/independence.v

Lines changed: 6 additions & 7 deletions
Original file line numberDiff line numberDiff line change
@@ -1,4 +1,4 @@
1-
(* mathcomp analysis (c) 2022 Inria and AIST. License: CeCILL-C. *)
1+
(* mathcomp analysis (c) 2025 Inria and AIST. License: CeCILL-C. *)
22
From mathcomp Require Import all_ssreflect interval_inference.
33
From mathcomp Require Import ssralg poly ssrnum ssrint interval finmap.
44
From mathcomp Require Import mathcomp_extra boolp classical_sets functions.
@@ -678,7 +678,7 @@ Definition pairRV (X Y : {RV P >-> T'}) : T * T -> T' * T' :=
678678
Lemma pairM (X Y : {RV P >-> T'}) : measurable_fun setT (pairRV X Y).
679679
Proof.
680680
rewrite /pairRV.
681-
apply/prod_measurable_funP; split => //=.
681+
apply/measurable_fun_pairP; split => //=.
682682
rewrite (_ : (fst \o (fun x : T * T => (X x.1, Y x.2))) = (fun x => X x.1))//.
683683
by apply/measurableT_comp => //=.
684684
rewrite (_ : (snd \o (fun x : T * T => (X x.1, Y x.2))) = (fun x => Y x.2))//.
@@ -808,10 +808,10 @@ rewrite [ltLHS](_ : _ = \int[distribution P X]_x `|x|%:E *
808808
rewrite ge0_integral_distribution//=; last exact/measurable_EFinP.
809809
rewrite ge0_integral_distribution//=; last exact/measurable_EFinP.
810810
rewrite lte_mul_pinfty//.
811-
by apply: integral_ge0 => //.
812-
apply: integral_fune_fin_num => //=.
813-
by move/integrable_abse : iX => //.
814-
apply: integral_fune_lt_pinfty => //.
811+
exact: integral_ge0.
812+
apply: integrable_fin_num => //=.
813+
by move/integrable_abse : iX.
814+
apply: integrable_lty => //.
815815
by move/integrable_abse : iY => //.
816816
Qed.
817817

@@ -1010,7 +1010,6 @@ apply: (@le_lt_trans _ _ 'E_P[(@normr _ _ \o X) * (@normr _ _ \o Y)]).
10101010
by move/Lfun1_integrable : iY => /measurable_int/measurable_EFinP.
10111011
apply: ge0_le_integral => //=.
10121012
- by apply/measurable_EFinP; exact/measurableT_comp.
1013-
- by move=> x _; rewrite lee_fin/= mulr_ge0/=.
10141013
- by apply/measurable_EFinP; apply/measurable_funM; exact/measurableT_comp.
10151014
- by move=> t _; rewrite lee_fin/= normrM.
10161015
rewrite expectationM_ge0//=.

theories/probability.v

Lines changed: 0 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -1490,7 +1490,6 @@ apply: (@le_lt_trans _ _ 'E_P[(@normr _ _ \o X) * (@normr _ _ \o Y)]).
14901490
by move/Lfun1_integrable : iY => /measurable_int.
14911491
apply: ge0_le_integral => //=.
14921492
- by apply/measurable_EFinP; exact/measurableT_comp.
1493-
- by move=> x _; rewrite lee_fin/= mulr_ge0/=.
14941493
- by apply/measurable_EFinP; apply/measurable_funM; exact/measurableT_comp.
14951494
- by move=> t _; rewrite lee_fin/= normrM.
14961495
rewrite expectationM_ge0//=.

0 commit comments

Comments
 (0)