Skip to content

Commit 096ff50

Browse files
authored
Cleanup (#1763)
* Cleanup
1 parent 1d53f98 commit 096ff50

Some content is hidden

Large Commits have some content hidden by default. Use the searchbox below for content that may be hidden.

61 files changed

+393
-579
lines changed

CHANGELOG_UNRELEASED.md

Lines changed: 3 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -7,6 +7,9 @@
77
- in `cardinality.v`:
88
+ lemma `infinite_setD`
99

10+
- in `convex.v`:
11+
+ lemmas `convN`, `conv_le`
12+
1013
### Changed
1114

1215
### Renamed

analysis_stdlib/Rstruct_topology.v

Lines changed: 2 additions & 4 deletions
Original file line numberDiff line numberDiff line change
@@ -7,11 +7,9 @@
77
Require Import Rdefinitions Raxioms RIneq Rbasic_fun Zwf.
88
Require Import Epsilon FunctionalExtensionality Ranalysis1 Rsqrt_def.
99
Require Import Rtrigo1 Reals.
10-
From mathcomp Require Import all_ssreflect ssralg poly mxpoly ssrnum.
11-
From mathcomp Require Import archimedean.
1210
From HB Require Import structures.
13-
From mathcomp Require Import mathcomp_extra boolp classical_sets.
14-
From mathcomp Require Import reals interval_inference.
11+
From mathcomp Require Import all_ssreflect ssralg ssrnum archimedean.
12+
From mathcomp Require Import boolp classical_sets reals interval_inference.
1513
From mathcomp Require Export Rstruct.
1614
From mathcomp Require Import topology.
1715
(* The following line is for RexpE. *)

classical/filter.v

Lines changed: 1 addition & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -1,7 +1,6 @@
11
(* mathcomp analysis (c) 2017 Inria and AIST. License: CeCILL-C. *)
22
From HB Require Import structures.
3-
From mathcomp Require Import all_ssreflect all_algebra finmap generic_quotient.
4-
From mathcomp Require Import archimedean.
3+
From mathcomp Require Import all_ssreflect all_algebra finmap.
54
From mathcomp Require Import boolp classical_sets functions wochoice.
65
From mathcomp Require Import cardinality mathcomp_extra fsbigop set_interval.
76

classical/mathcomp_extra.v

Lines changed: 1 addition & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -1,6 +1,5 @@
11
(* mathcomp analysis (c) 2022 Inria and AIST. License: CeCILL-C. *)
2-
From mathcomp Require Import all_ssreflect finmap ssralg ssrnum ssrint.
3-
From mathcomp Require Import archimedean rat finset interval.
2+
From mathcomp Require Import all_ssreflect finmap ssralg ssrnum.
43

54
(**md**************************************************************************)
65
(* # MathComp extra *)

classical/set_interval.v

Lines changed: 2 additions & 5 deletions
Original file line numberDiff line numberDiff line change
@@ -569,13 +569,10 @@ Lemma line_path_id : line_path 0 1 = id.
569569
Proof. by apply/funext => t; rewrite /line_path mulr0 add0r mulr1. Qed.
570570

571571
Lemma line_pathEl a b t : line_path a b t = t * (b - a) + a.
572-
Proof. by rewrite /line_path mulrBl mul1r mulrBr addrAC [RHS]addrC addrA. Qed.
572+
Proof. by rewrite /line_path mulrBl addrAC -addrA -mulrBr mul1r addrC. Qed.
573573

574574
Lemma line_pathEr a b t : line_path a b t = (1 - t) * (a - b) + b.
575-
Proof.
576-
rewrite /line_path mulrBr -addrA; congr (_ + _).
577-
by rewrite mulrBl opprB mul1r addrNK.
578-
Qed.
575+
Proof. by rewrite mulrBl mul1r addrAC subrK -mulrN opprB addrC line_pathEl. Qed.
579576

580577
Lemma line_path10 t : line_path 1 0 t = 1 - t.
581578
Proof. by rewrite /line_path mulr0 addr0 mulr1. Qed.

classical/unstable.v

Lines changed: 4 additions & 7 deletions
Original file line numberDiff line numberDiff line change
@@ -1,6 +1,6 @@
11
(* mathcomp analysis (c) 2022 Inria and AIST. License: CeCILL-C. *)
2-
From mathcomp Require Import all_ssreflect finmap ssralg ssrnum ssrint rat.
3-
From mathcomp Require Import archimedean finset interval mathcomp_extra.
2+
From mathcomp Require Import all_ssreflect finmap ssralg ssrnum ssrint.
3+
From mathcomp Require Import archimedean interval mathcomp_extra.
44

55
(**md**************************************************************************)
66
(* # MathComp extra *)
@@ -277,16 +277,13 @@ Lemma onemK r : `1-(`1-r) = r. Proof. exact: subKr. Qed.
277277
Lemma add_onemK r : r + `1- r = 1. Proof. by rewrite /onem addrC subrK. Qed.
278278

279279
Lemma onemD r s : `1-(r + s) = `1-r - s.
280-
Proof. by rewrite /onem addrAC opprD addrA addrAC. Qed.
280+
Proof. by rewrite /onem opprD addrA. Qed.
281281

282282
Lemma onemMr r s : s * `1-r = s - s * r.
283283
Proof. by rewrite /onem mulrBr mulr1. Qed.
284284

285285
Lemma onemM r s : `1-(r * s) = `1-r + `1-s - `1-r * `1-s.
286-
Proof.
287-
rewrite /onem mulrBr mulr1 mulrBl mul1r opprB -addrA.
288-
by rewrite (addrC (1 - r)) !addrA subrK opprB addrA subrK addrK.
289-
Qed.
286+
Proof. by rewrite /onem mulrBl 2!mulrBr !mul1r mulr1 addrKA opprK subrKA. Qed.
290287

291288
End onem_ring.
292289

experimental_reals/distr.v

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -286,7 +286,7 @@ Local Lemma mrat_sup s : (0 < size s)%N ->
286286
Proof.
287287
move=> gt0_s; rewrite -mulr_suml -natr_sum.
288288
apply/(mulIf (x := (size s)%:R)); first by rewrite pnatr_eq0 -lt0n.
289-
rewrite mul1r -mulrA mulVf ?mulr1 ?pnatr_eq0 -?lt0n //; congr (_%:R).
289+
rewrite mul1r divfK ?pnatr_eq0 -?lt0n//; congr (_%:R).
290290
rewrite -sum1_size -[in RHS]big_undup_iterop_count/=; apply: eq_bigr => i _.
291291
by rewrite Monoid.iteropE iter_addn addn0 mul1n.
292292
Qed.

experimental_reals/realseq.v

Lines changed: 2 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -122,7 +122,7 @@ have gt0_e: 0 < e by rewrite subr_gt0.
122122
move=> x y; rewrite !inE/= /eclamp pmulr_rle0 // invr_le0.
123123
rewrite lern0 /= !ltr_distl => /andP[_ lt1] /andP[lt2 _].
124124
apply/(lt_trans lt1)/(le_lt_trans _ lt2).
125-
by rewrite lerBrDl addrCA -splitr /e addrC subrK.
125+
by rewrite lerBrDr -addrA -splitr subrKC.
126126
Qed.
127127

128128
Lemma separable {R : realType} (l1 l2 : \bar R) :
@@ -303,8 +303,7 @@ Lemma ncvgM u v lu lv : ncvg u lu%:E -> ncvg v lv%:E ->
303303
Proof.
304304
move=> cu cv; pose a := u \- lu%:S; pose b := v \- lv%:S.
305305
have eq: (u \* v) =1 (lu * lv)%:S \+ ((lu%:S \* b) \+ (a \* v)).
306-
move=> n; rewrite {}/a {}/b /=.
307-
by rewrite addrC mulrBr addrAC subrK addrC mulrBl subrK.
306+
by move=> n; rewrite /= addrA mulrBr mulrBl 2!subrKC.
308307
apply/(ncvg_eq eq); rewrite -[X in X%:E]addr0; apply/ncvgD.
309308
by apply/ncvgC. rewrite -[X in X%:E]addr0; apply/ncvgD.
310309
+ apply/ncvgMr; first rewrite -[X in X%:E](subrr lv).

experimental_reals/realsum.v

Lines changed: 1 addition & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -3,7 +3,7 @@
33
(* Copyright (c) - 2015--2018 - Inria *)
44
(* Copyright (c) - 2016--2018 - Polytechnique *)
55
(* -------------------------------------------------------------------- *)
6-
From mathcomp Require Import all_ssreflect all_algebra archimedean.
6+
From mathcomp Require Import all_ssreflect all_algebra.
77
From mathcomp.classical Require Import boolp.
88
From mathcomp Require Import xfinmap constructive_ereal reals discrete realseq.
99
From mathcomp.classical Require Import classical_sets functions.
@@ -14,7 +14,6 @@ Unset Printing Implicit Defensive.
1414
Unset SsrOldRewriteGoalsOrder.
1515

1616
Import Order.TTheory GRing.Theory Num.Theory.
17-
From mathcomp.classical Require Import mathcomp_extra.
1817

1918
Local Open Scope fset_scope.
2019
Local Open Scope ring_scope.

reals/real_interval.v

Lines changed: 2 additions & 4 deletions
Original file line numberDiff line numberDiff line change
@@ -1,9 +1,8 @@
11
(* mathcomp analysis (c) 2025 Inria and AIST. License: CeCILL-C. *)
2-
From mathcomp Require Import all_ssreflect ssralg ssrnum ssrint interval.
3-
From mathcomp Require Import fingroup perm rat archimedean finmap.
2+
From mathcomp Require Import all_ssreflect finmap ssralg ssrnum ssrint interval.
3+
From mathcomp Require Import archimedean.
44
From mathcomp Require Import boolp classical_sets functions.
55
From mathcomp Require Export set_interval.
6-
From HB Require Import structures.
76
From mathcomp Require Import reals interval_inference constructive_ereal.
87

98
(**md**************************************************************************)
@@ -14,7 +13,6 @@ Set Implicit Arguments.
1413
Unset Strict Implicit.
1514
Unset Printing Implicit Defensive.
1615
Import Order.TTheory GRing.Theory Num.Def Num.Theory.
17-
From mathcomp Require Import mathcomp_extra unstable.
1816

1917
Local Open Scope classical_set_scope.
2018
Local Open Scope ring_scope.

0 commit comments

Comments
 (0)