|
1 | | -(* mathcomp analysis (c) 2022 Inria and AIST. License: CeCILL-C. *) |
| 1 | +(* mathcomp analysis (c) 2025 Inria and AIST. License: CeCILL-C. *) |
2 | 2 | From mathcomp Require Import all_ssreflect interval_inference. |
3 | 3 | From mathcomp Require Import ssralg poly ssrnum ssrint interval finmap. |
4 | 4 | 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' := |
678 | 678 | Lemma pairM (X Y : {RV P >-> T'}) : measurable_fun setT (pairRV X Y). |
679 | 679 | Proof. |
680 | 680 | rewrite /pairRV. |
681 | | -apply/prod_measurable_funP; split => //=. |
| 681 | +apply/measurable_fun_pairP; split => //=. |
682 | 682 | rewrite (_ : (fst \o (fun x : T * T => (X x.1, Y x.2))) = (fun x => X x.1))//. |
683 | 683 | by apply/measurableT_comp => //=. |
684 | 684 | 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 * |
808 | 808 | rewrite ge0_integral_distribution//=; last exact/measurable_EFinP. |
809 | 809 | rewrite ge0_integral_distribution//=; last exact/measurable_EFinP. |
810 | 810 | 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 => //. |
815 | 815 | by move/integrable_abse : iY => //. |
816 | 816 | Qed. |
817 | 817 |
|
@@ -1010,7 +1010,6 @@ apply: (@le_lt_trans _ _ 'E_P[(@normr _ _ \o X) * (@normr _ _ \o Y)]). |
1010 | 1010 | by move/Lfun1_integrable : iY => /measurable_int/measurable_EFinP. |
1011 | 1011 | apply: ge0_le_integral => //=. |
1012 | 1012 | - by apply/measurable_EFinP; exact/measurableT_comp. |
1013 | | - - by move=> x _; rewrite lee_fin/= mulr_ge0/=. |
1014 | 1013 | - by apply/measurable_EFinP; apply/measurable_funM; exact/measurableT_comp. |
1015 | 1014 | - by move=> t _; rewrite lee_fin/= normrM. |
1016 | 1015 | rewrite expectationM_ge0//=. |
|
0 commit comments