File tree Expand file tree Collapse file tree 3 files changed +9
-10
lines changed
Expand file tree Collapse file tree 3 files changed +9
-10
lines changed Original file line number Diff line number Diff line change 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
Original file line number Diff line number Diff line change 1- (* mathcomp analysis (c) 2017 Inria and AIST. License: CeCILL-C. *)
1+ (* mathcomp analysis (c) 2025 Inria and AIST. License: CeCILL-C. *)
22From HB Require Import structures.
33From mathcomp Require Import all_ssreflect ssralg ssrnum interval.
44From mathcomp Require Import mathcomp_extra unstable boolp classical_sets.
@@ -120,12 +120,6 @@ move: b be zb => [[|]/= b|[|]//]; rewrite bnd_simp => be.
120120by move=> /le_lt_trans; exact.
121121Qed .
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-
129123Lemma set_itvoo x y : `]x, y[%classic = [set z | (x < z < y)%O].
130124Proof . by []. Qed .
131125
@@ -230,6 +224,8 @@ Notation set_itv_infty_c := set_itvNyc (only parsing).
230224Notation set_itv_pinfty_bnd := set_itv_ybnd (only parsing).
231225#[deprecated(since="mathcomp-analysis 1.10.0", note="renamed to `set_itv_bndNy`")]
232226Notation 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
234230Section set_itv_orderType.
235231Variables (d : Order.disp_t) (T : orderType d).
Original file line number Diff line number Diff line change @@ -463,7 +463,7 @@ rewrite le_eqVlt => /predU1P[<- _|ab intf].
463463apply/(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).
468468pose fab := f \_ `[a, b].
469469have /= 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.
634634have 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.
637637have cE : c = F a.
638638 apply/eqP; rewrite -(opprK c) eq_sym -addr_eq0 addrC.
639639 by have := cvg_unique _ GacFa Ga; rewrite Ga0 => ->.
You can’t perform that action at this time.
0 commit comments