Skip to content

Commit 61acc8d

Browse files
authored
easy gen, rm deprecated (#1773)
1 parent 4f40788 commit 61acc8d

File tree

10 files changed

+52
-83
lines changed

10 files changed

+52
-83
lines changed

CHANGELOG_UNRELEASED.md

Lines changed: 36 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -17,15 +17,51 @@
1717

1818
### Renamed
1919

20+
- in `probability.v`:
21+
+ `derivable_oo_continuous_bnd_onemXnMr` -> `derivable_oo_LRcontinuous_onemXnMr`
22+
2023
### Generalized
2124

2225
- in `lebesgue_integral_under.v`:
2326
+ weaken an hypothesis of lemma `continuity_under_integral`
2427

28+
- in `lebesgue_integrable.v`:
29+
+ weaken an hypothesis of lemma `finite_measure_integrable_cst`
30+
2531
### Deprecated
2632

2733
### Removed
2834

35+
- in `lebesgue_stieltjes_measure.v`:
36+
+ notation `wlength_sigma_sub_additive` (deprecated since 1.1.0)
37+
38+
- in `constructive_ereal.v`:
39+
+ notations `gee_pmull`, `gee_addl`, `gee_addr`, `gte_addr`, `gte_addl`,
40+
`lte_subl_addr`, `lte_subl_addl`, `lte_subr_addr`, `lte_subr_addl`,
41+
`lee_subl_addr`, `lee_subl_addl`, `lee_subr_addr`, `lee_subr_addl`
42+
(deprecated since 1.2.0)
43+
44+
- in `signed.v`:
45+
+ notations `num_le_maxr`, `num_le_maxl`, `num_le_minr`, `num_le_minl`,
46+
`num_lt_maxr`, `num_lt_maxl`, `num_lt_minr`, `num_lt_minl`
47+
(deprecated since 1.2.0)
48+
49+
- in `measure_function.v`:
50+
+ notations `g_salgebra_measure_unique_trace`,
51+
`g_salgebra_measure_unique_cover`, `g_salgebra_measure_unique`
52+
(deprecated since 1.2.0)
53+
54+
- in `measurable_structure.v`:
55+
+ notations `monotone_class`, `monotone_class_g_salgebra`,
56+
`smallest_monotone_classE`, `monotone_class_subset`,
57+
`setI_closed_gdynkin_salgebra`, `dynkin_g_dynkin`, `dynkin_monotone`,
58+
`salgebraType`
59+
(deprecated since 1.2.0)
60+
61+
- in `sequences.v`:
62+
+ notation `eq_bigsetU_seqD`
63+
(deprecated since 1.2.0)
64+
2965
### Infrastructure
3066

3167
### Misc

reals/constructive_ereal.v

Lines changed: 0 additions & 26 deletions
Original file line numberDiff line numberDiff line change
@@ -2957,32 +2957,6 @@ Arguments lee_sum_nneg_natl {R}.
29572957
Arguments lee_sum_npos_natl {R}.
29582958
#[global] Hint Extern 0 (is_true (0 <= `| _ |)%E) => solve [apply: abse_ge0] : core.
29592959

2960-
#[deprecated(since="mathcomp-analysis 1.2.0", note="Use gee_pMl instead.")]
2961-
Notation gee_pmull := gee_pMl (only parsing).
2962-
#[deprecated(since="mathcomp-analysis 1.2.0", note="Use geeDl instead.")]
2963-
Notation gee_addl := geeDl (only parsing).
2964-
#[deprecated(since="mathcomp-analysis 1.2.0", note="Use geeDr instead.")]
2965-
Notation gee_addr := geeDr (only parsing).
2966-
#[deprecated(since="mathcomp-analysis 1.2.0", note="Use gteDr instead.")]
2967-
Notation gte_addr := gteDr (only parsing).
2968-
#[deprecated(since="mathcomp-analysis 1.2.0", note="Use gteDl instead.")]
2969-
Notation gte_addl := gteDl (only parsing).
2970-
#[deprecated(since="mathcomp-analysis 1.2.0", note="Use lteBlDr instead.")]
2971-
Notation lte_subl_addr := lteBlDr (only parsing).
2972-
#[deprecated(since="mathcomp-analysis 1.2.0", note="Use lteBlDl instead.")]
2973-
Notation lte_subl_addl := lteBlDl (only parsing).
2974-
#[deprecated(since="mathcomp-analysis 1.2.0", note="Use lteBrDr instead.")]
2975-
Notation lte_subr_addr := lteBrDr (only parsing).
2976-
#[deprecated(since="mathcomp-analysis 1.2.0", note="Use lteBrDl instead.")]
2977-
Notation lte_subr_addl := lteBrDl (only parsing).
2978-
#[deprecated(since="mathcomp-analysis 1.2.0", note="Use leeBlDr instead.")]
2979-
Notation lee_subl_addr := leeBlDr (only parsing).
2980-
#[deprecated(since="mathcomp-analysis 1.2.0", note="Use leeBlDl instead.")]
2981-
Notation lee_subl_addl := leeBlDl (only parsing).
2982-
#[deprecated(since="mathcomp-analysis 1.2.0", note="Use leeBrDr instead.")]
2983-
Notation lee_subr_addr := leeBrDr (only parsing).
2984-
#[deprecated(since="mathcomp-analysis 1.2.0", note="Use leeBrDl instead.")]
2985-
Notation lee_subr_addl := leeBrDl (only parsing).
29862960
#[deprecated(since="mathcomp-analysis 1.3.0", note="Use `lte_leD` instead.")]
29872961
Notation lte_le_add := lte_leD (only parsing).
29882962
#[deprecated(since="mathcomp-analysis 1.3.0", note="Use `lee_ltD` instead.")]

reals/signed.v

Lines changed: 0 additions & 16 deletions
Original file line numberDiff line numberDiff line change
@@ -1130,22 +1130,6 @@ Lemma num_gt_min a x y :
11301130
Proof. by rewrite -comparable_gt_min// real_comparable. Qed.
11311131

11321132
End MorphReal.
1133-
#[deprecated(since="mathcomp-analysis 1.2.0", note="renamed `num_le_max`")]
1134-
Notation num_le_maxr := num_le_max (only parsing).
1135-
#[deprecated(since="mathcomp-analysis 1.2.0", note="renamed `num_ge_max`")]
1136-
Notation num_le_maxl := num_ge_max (only parsing).
1137-
#[deprecated(since="mathcomp-analysis 1.2.0", note="renamed `num_le_min`")]
1138-
Notation num_le_minr := num_le_min (only parsing).
1139-
#[deprecated(since="mathcomp-analysis 1.2.0", note="renamed `num_ge_min`")]
1140-
Notation num_le_minl := num_ge_min (only parsing).
1141-
#[deprecated(since="mathcomp-analysis 1.2.0", note="renamed `num_lt_max`")]
1142-
Notation num_lt_maxr := num_lt_max (only parsing).
1143-
#[deprecated(since="mathcomp-analysis 1.2.0", note="renamed `num_gt_max`")]
1144-
Notation num_lt_maxl := num_gt_max (only parsing).
1145-
#[deprecated(since="mathcomp-analysis 1.2.0", note="renamed `num_lt_min`")]
1146-
Notation num_lt_minr := num_lt_min (only parsing).
1147-
#[deprecated(since="mathcomp-analysis 1.2.0", note="renamed `num_gt_min`")]
1148-
Notation num_lt_minl := num_gt_min (only parsing).
11491133

11501134
Section MorphGe0.
11511135
Context {R : numDomainType} {nz : nullity}.

theories/hoelder.v

Lines changed: 4 additions & 4 deletions
Original file line numberDiff line numberDiff line change
@@ -1183,11 +1183,11 @@ Variable mu : {finite_measure set T -> \bar R}.
11831183

11841184
Lemma Lfun_cst c r : cst c \in Lfun mu r%:E.
11851185
Proof.
1186-
rewrite inE; apply/andP; split; rewrite inE//= /finite_norm unlock/Lnorm poweR_lty//.
1186+
rewrite inE/=; apply/andP; split; rewrite inE//=.
1187+
rewrite /finite_norm unlock poweR_lty//.
11871188
under eq_integral => x _/= do rewrite (_ : `|c| `^ r = cst (`|c| `^ r) x)//.
1188-
have /integrableP[_/=] := finite_measure_integrable_cst mu (`|c| `^ r).
1189-
under eq_integral => x _ do rewrite ger0_norm ?powR_ge0//.
1190-
by [].
1189+
apply/integrable_lty => //.
1190+
exact: finite_measure_integrable_cst.
11911191
Qed.
11921192

11931193
End Lspace_finite_measure.

theories/lebesgue_integral_theory/lebesgue_integrable.v

Lines changed: 5 additions & 5 deletions
Original file line numberDiff line numberDiff line change
@@ -391,18 +391,18 @@ rewrite (@le_lt_trans _ _ (mu setT)) ?le_measure ?inE//.
391391
by rewrite ?ltry ?fin_num_fun_lty//; exact: fin_num_measure.
392392
Qed.
393393

394-
Lemma finite_measure_integrable_cst k : mu.-integrable [set: T] (EFin \o cst k).
394+
Lemma finite_measure_integrable_cst A k :
395+
measurable A -> mu.-integrable A (EFin \o cst k).
395396
Proof.
396-
apply/integrableP; split; first exact/measurable_EFinP.
397+
move=> mA; apply/integrableP; split; first exact/measurable_EFinP.
397398
have [k0|k0] := leP 0%R k.
398399
- under eq_integral do rewrite /= ger0_norm//.
399400
rewrite lebesgue_integral_nonneg.integral_cstr//= lte_mul_pinfty//.
400-
rewrite fin_num_fun_lty//.
401-
exact: fin_num_measure.
401+
by rewrite -ge0_fin_numE// fin_num_measure.
402402
- under eq_integral do rewrite /= ltr0_norm//.
403403
rewrite lebesgue_integral_nonneg.integral_cstr//= lte_mul_pinfty//.
404404
by rewrite lee_fin lerNr oppr0 ltW.
405-
by rewrite fin_num_fun_lty//; exact: fin_num_measure.
405+
by rewrite -ge0_fin_numE// fin_num_measure.
406406
Qed.
407407

408408
End integrable_finite_measure.

theories/lebesgue_stieltjes_measure.v

Lines changed: 0 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -506,9 +506,6 @@ HB.instance Definition _ (f : cumulative R R) :=
506506
End wlength_extension.
507507
Arguments lebesgue_stieltjes_measure {R}.
508508

509-
#[deprecated(since="mathcomp-analysis 1.1.0", note="renamed `wlength_sigma_subadditive`")]
510-
Notation wlength_sigma_sub_additive := wlength_sigma_subadditive (only parsing).
511-
512509
Definition measurableTypeR (R : realType) :=
513510
g_sigma_algebraType R.-ocitv.-measurable.
514511

theories/measure_theory/measurable_structure.v

Lines changed: 0 additions & 16 deletions
Original file line numberDiff line numberDiff line change
@@ -221,8 +221,6 @@ Definition lambda_system :=
221221
Definition monotone := ndseq_closed /\ niseq_closed.
222222

223223
End set_systems.
224-
#[deprecated(since="mathcomp-analysis 1.2.0", note="renamed `lambda_system`")]
225-
Notation monotone_class := lambda_system (only parsing).
226224
(*#[deprecated(since="mathcomp-analysis 1.3.0", note="renamed `setSD_closed`")]
227225
Notation setD_closed := setSD_closed (only parsing).*)
228226
#[deprecated(since="mathcomp-analysis 1.9.0", note="renamed `setD_closed`")]
@@ -430,8 +428,6 @@ Proof.
430428
move=> sDGD; have := smallest_sigma_algebra D G.
431429
by move=> /(sigma_algebraP sDGD) [sT sD snd sI]; split.
432430
Qed.
433-
#[deprecated(since="mathcomp-analysis 1.2.0", note="renamed `g_sigma_algebra_lambda_system`")]
434-
Notation monotone_class_g_salgebra := g_sigma_algebra_lambda_system (only parsing).
435431

436432
Lemma smallest_sigma_ring T (G : set (set T)) : sigma_ring <<sr G >>.
437433
Proof.
@@ -594,8 +590,6 @@ by move=> *; apply HHH_.
594590
Qed.
595591

596592
End smallest_lambda_system.
597-
#[deprecated(since="mathcomp-analysis 1.2.0", note="renamed `smallest_lambda_system`")]
598-
Notation smallest_monotone_classE := smallest_lambda_system (only parsing).
599593

600594
Section lambda_system_subset.
601595
Variables (T : Type) (G : set (set T)) (setIG : setI_closed G) (D : set T).
@@ -613,8 +607,6 @@ rewrite -(@smallest_lambda_system _ _ setIG D) //.
613607
Qed.
614608

615609
End lambda_system_subset.
616-
#[deprecated(since="mathcomp-analysis 1.2.0", note="renamed `lambda_system_subset`")]
617-
Notation monotone_class_subset := lambda_system_subset (only parsing).
618610

619611
Section dynkin.
620612
Variable T : Type.
@@ -740,12 +732,6 @@ exact: g_dynkin_dynkin.
740732
Qed.
741733

742734
End dynkin_lemmas.
743-
#[deprecated(since="mathcomp-analysis 1.2.0", note="renamed into `setI_closed_g_dynkin_g_sigma_algebra`")]
744-
Notation setI_closed_gdynkin_salgebra := setI_closed_g_dynkin_g_sigma_algebra (only parsing).
745-
#[deprecated(since="mathcomp-analysis 1.2.0", note="renamed into `g_dynkin_dynkin`")]
746-
Notation dynkin_g_dynkin := g_dynkin_dynkin (only parsing).
747-
#[deprecated(since="mathcomp-analysis 1.2.0", note="renamed into `dynkin_lambda_system`")]
748-
Notation dynkin_monotone := dynkin_lambda_system (only parsing).
749735

750736
Section trace.
751737
Variable (T : Type).
@@ -1270,8 +1256,6 @@ Definition sigma_display {T} : set (set T) -> measure_display.
12701256
Proof. exact. Qed.
12711257

12721258
Definition g_sigma_algebraType {T} (G : set (set T)) := T.
1273-
#[deprecated(since="mathcomp-analysis 1.2.0", note="renamed into `g_sigma_algebraType`")]
1274-
Notation salgebraType := g_sigma_algebraType (only parsing).
12751259

12761260
Section g_salgebra_instance.
12771261
Variables (T : pointedType) (G : set (set T)).

theories/measure_theory/measure_function.v

Lines changed: 0 additions & 6 deletions
Original file line numberDiff line numberDiff line change
@@ -1747,8 +1747,6 @@ Qed.
17471747

17481748
End g_sigma_algebra_measure_unique_trace.
17491749
Arguments g_sigma_algebra_measure_unique_trace {d R T} G D.
1750-
#[deprecated(since="mathcomp-analysis 1.2.0", note="renamed `g_sigma_algebra_measure_unique_trace`")]
1751-
Notation g_salgebra_measure_unique_trace := g_sigma_algebra_measure_unique_trace (only parsing).
17521750

17531751
Definition lim_sup_set T (F : (set T)^nat) := \bigcap_n \bigcup_(j >= n) F j.
17541752

@@ -1932,10 +1930,6 @@ Qed.
19321930

19331931
End g_sigma_algebra_measure_unique.
19341932
Arguments g_sigma_algebra_measure_unique {d R T} G.
1935-
#[deprecated(since="mathcomp-analysis 1.2.0", note="renamed `g_sigma_algebra_measure_unique_cover`")]
1936-
Notation g_salgebra_measure_unique_cover := g_sigma_algebra_measure_unique_cover (only parsing).
1937-
#[deprecated(since="mathcomp-analysis 1.2.0", note="renamed `g_sigma_algebra_measure_unique`")]
1938-
Notation g_salgebra_measure_unique := g_sigma_algebra_measure_unique (only parsing).
19391933

19401934
Section measure_unique.
19411935
Context d (R : realType) (T : measurableType d).

theories/probability.v

Lines changed: 7 additions & 5 deletions
Original file line numberDiff line numberDiff line change
@@ -2191,19 +2191,19 @@ have := @derivableX _ _ (@onem R) n x 1.
21912191
by rewrite fctE; apply; exact: derivableB.
21922192
Qed.
21932193

2194-
Lemma derivable_oo_continuous_bnd_onemXnMr n x :
2195-
derivable_oo_continuous_bnd (fun y => `1-y ^+ n * x) 0 1.
2194+
Lemma derivable_oo_LRcontinuous_onemXnMr n x :
2195+
derivable_oo_LRcontinuous (fun y => `1-y ^+ n * x) 0 1.
21962196
Proof.
21972197
split.
21982198
- by move=> y y01; apply: derivableM => //=; exact: onemXn_derivable.
21992199
- apply: cvgM; last exact: cvg_cst.
22002200
apply: cvg_at_right_filter.
2201-
apply: (@cvg_comp _ _ _ (fun x => `1-x) (fun x => x ^+ n)).
2201+
apply: (@cvg_comp _ _ _ onem (fun x => x ^+ n)).
22022202
by apply: cvgB; [exact: cvg_cst|exact: cvg_id].
22032203
exact: exprn_continuous.
22042204
- apply: cvg_at_left_filter.
22052205
apply: cvgM; last exact: cvg_cst.
2206-
apply: (@cvg_comp _ _ _ (fun x => `1-x) (fun x => x ^+ n)).
2206+
apply: (@cvg_comp _ _ _ onem (fun x => x ^+ n)).
22072207
by apply: cvgB; [exact: cvg_cst|exact: cvg_id].
22082208
exact: exprn_continuous.
22092209
Qed.
@@ -2225,12 +2225,14 @@ rewrite (@continuous_FTC2 _ _ (fun x => `1-x ^+ n.+1 / - n.+1%:R))//=.
22252225
- rewrite onem1 expr0n/= mul0r onem0 expr1n mul1r sub0r.
22262226
by rewrite -invrN -2!mulNrn opprK.
22272227
- by apply: continuous_in_subspaceT => x x01; exact: continuous_onemXn.
2228-
- exact: derivable_oo_continuous_bnd_onemXnMr.
2228+
- exact: derivable_oo_LRcontinuous_onemXnMr.
22292229
- move=> x x01; rewrite derive1Mr//; last exact: onemXn_derivable.
22302230
by rewrite derive_onemXn mulrAC divff// mul1r.
22312231
Qed.
22322232

22332233
End about_onemXn.
2234+
#[deprecated(since="mathcomp-analysis 1.15.0", note="renamed to `derivable_oo_LRcontinuous_onemXnMr`")]
2235+
Notation derivable_oo_continuous_bnd_onemXnMr := derivable_oo_LRcontinuous_onemXnMr (only parsing).
22342236

22352237
(**md about the function $x \mapsto x^a (1 - x)^b$ *)
22362238
Section XMonemX.

theories/sequences.v

Lines changed: 0 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -364,8 +364,6 @@ by exists i => //; rewrite big_ord_recr/=; right.
364364
Qed.
365365

366366
End seqD.
367-
#[deprecated(since="mathcomp-analysis 1.2.0", note="renamed to `nondecreasing_bigsetU_seqD`")]
368-
Notation eq_bigsetU_seqD := nondecreasing_bigsetU_seqD (only parsing).
369367

370368
Lemma seqDUE {R : realDomainType} n (r : R) :
371369
(seqDU (fun n => `]r, r + n%:R]) n = `]r + n.-1%:R, r + n%:R])%classic.

0 commit comments

Comments
 (0)