Skip to content

Commit fe37644

Browse files
authored
fixes #1790 (#1799)
1 parent d4e376f commit fe37644

File tree

3 files changed

+9
-10
lines changed

3 files changed

+9
-10
lines changed

CHANGELOG_UNRELEASED.md

Lines changed: 3 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -196,6 +196,9 @@
196196
- in `charge.v`:
197197
+ lemma `dominates_charge_variation` (use `charge_null_dominatesP` instead)
198198

199+
- in `set_interval.v`:
200+
+ lemma `interval_set1` (use `set_itv1` instead)
201+
199202
### Infrastructure
200203

201204
### Misc

classical/set_interval.v

Lines changed: 3 additions & 7 deletions
Original file line numberDiff line numberDiff line change
@@ -1,4 +1,4 @@
1-
(* mathcomp analysis (c) 2017 Inria and AIST. License: CeCILL-C. *)
1+
(* mathcomp analysis (c) 2025 Inria and AIST. License: CeCILL-C. *)
22
From HB Require Import structures.
33
From mathcomp Require Import all_ssreflect ssralg ssrnum interval.
44
From mathcomp Require Import mathcomp_extra unstable boolp classical_sets.
@@ -120,12 +120,6 @@ move: b be zb => [[|]/= b|[|]//]; rewrite bnd_simp => be.
120120
by move=> /le_lt_trans; exact.
121121
Qed.
122122

123-
Lemma interval_set1 x : `[x, x]%classic = [set x] :> set T.
124-
Proof.
125-
apply/seteqP; split => [y/=|y <-]; last by rewrite /= in_itv/= lexx.
126-
by rewrite in_itv/= => /andP[yx xy]; apply/eqP; rewrite eq_le yx xy.
127-
Qed.
128-
129123
Lemma set_itvoo x y : `]x, y[%classic = [set z | (x < z < y)%O].
130124
Proof. by []. Qed.
131125

@@ -230,6 +224,8 @@ Notation set_itv_infty_c := set_itvNyc (only parsing).
230224
Notation set_itv_pinfty_bnd := set_itv_ybnd (only parsing).
231225
#[deprecated(since="mathcomp-analysis 1.10.0", note="renamed to `set_itv_bndNy`")]
232226
Notation set_itv_bnd_ninfty := set_itv_bndNy (only parsing).
227+
#[deprecated(since="mathcomp-analysis 1.15.0", note="use `set_itv1` instead")]
228+
Notation interval_set1 := set_itv1 (only parsing).
233229

234230
Section set_itv_orderType.
235231
Variables (d : Order.disp_t) (T : orderType d).

theories/ftc.v

Lines changed: 3 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -463,7 +463,7 @@ rewrite le_eqVlt => /predU1P[<- _|ab intf].
463463
apply/(continuous_within_itvP _ ab); split; first last.
464464
exact: parameterized_integral_cvg_at_left.
465465
apply/cvg_at_right_filter.
466-
rewrite {2}/int /parameterized_integral interval_set1 Rintegral_set1.
466+
rewrite {2}/int /parameterized_integral set_itv1 Rintegral_set1.
467467
exact: (parameterized_integral_cvg_left ab).
468468
pose fab := f \_ `[a, b].
469469
have /= int_normr_cont : forall e : R, 0 < e ->
@@ -630,10 +630,10 @@ have Ga : G x @[x --> a^'+] --> G a.
630630
have := parameterized_integral_cvg_left ab iabfab.
631631
rewrite (_ : 0 = G a)%R.
632632
by move=> /left_right_continuousP[].
633-
by rewrite /G interval_set1 Rintegral_set1.
633+
by rewrite /G set_itv1 Rintegral_set1.
634634
have Gb : G x @[x --> b^'-] --> G b.
635635
exact: (parameterized_integral_cvg_at_left ab iabfab).
636-
have Ga0 : G a = 0%R by rewrite /G interval_set1// Rintegral_set1.
636+
have Ga0 : G a = 0%R by rewrite /G set_itv1// Rintegral_set1.
637637
have cE : c = F a.
638638
apply/eqP; rewrite -(opprK c) eq_sym -addr_eq0 addrC.
639639
by have := cvg_unique _ GacFa Ga; rewrite Ga0 => ->.

0 commit comments

Comments
 (0)