Skip to content

Commit

Permalink
Merge pull request #214 from coq-community/coq_19801
Browse files Browse the repository at this point in the history
Adapt to coq/coq#19801
  • Loading branch information
proux01 authored Jan 7, 2025
2 parents 736118d + 5aca257 commit a75b14f
Show file tree
Hide file tree
Showing 31 changed files with 121 additions and 104 deletions.
1 change: 1 addition & 0 deletions metric2/Compact.v
Original file line number Diff line number Diff line change
Expand Up @@ -18,6 +18,7 @@ COPYRIGHT HOLDERS BE LIABLE FOR ANY CLAIM, DAMAGES OR OTHER LIABILITY, WHETHER
IN AN ACTION OF CONTRACT, TORT OR OTHERWISE, ARISING FROM, OUT OF OR IN
CONNECTION WITH THE PROOF OR THE USE OR OTHER DEALINGS IN THE PROOF.
*)
From Coq Require Import ZArith.
Require Import CoRN.model.totalorder.QposMinMax.
Require Import CoRN.metric2.Limit.
Require Export CoRN.metric2.FinEnum.
Expand Down
1 change: 1 addition & 0 deletions metric2/FinEnum.v
Original file line number Diff line number Diff line change
Expand Up @@ -18,6 +18,7 @@ COPYRIGHT HOLDERS BE LIABLE FOR ANY CLAIM, DAMAGES OR OTHER LIABILITY, WHETHER
IN AN ACTION OF CONTRACT, TORT OR OTHERWISE, ARISING FROM, OUT OF OR IN
CONNECTION WITH THE PROOF OR THE USE OR OTHER DEALINGS IN THE PROOF.
*)
From Coq Require Import ZArith.
Require Import CoRN.model.totalorder.QposMinMax.
Require Export CoRN.metric2.Hausdorff.
Require Import CoRN.logic.Classic.
Expand Down
1 change: 1 addition & 0 deletions metric2/Limit.v
Original file line number Diff line number Diff line change
Expand Up @@ -19,6 +19,7 @@ IN AN ACTION OF CONTRACT, TORT OR OTHERWISE, ARISING FROM, OUT OF OR IN
CONNECTION WITH THE PROOF OR THE USE OR OTHER DEALINGS IN THE PROOF.
*)

From Coq Require Import ZArith.
Require Import CoRN.algebra.RSetoid.
Require Import CoRN.model.totalorder.QposMinMax.
From Coq Require Import QArith.
Expand Down
1 change: 1 addition & 0 deletions model/structures/QnonNeg.v
Original file line number Diff line number Diff line change
@@ -1,5 +1,6 @@
(* This module is designed to *not* be Import'ed, only Require'd. *)

From Coq Require Import ZArith.
Require Import CoRN.model.totalorder.QposMinMax.
From Coq Require Import Program.
Require Import CoRN.model.structures.QposInf.
Expand Down
1 change: 1 addition & 0 deletions reals/fast/CRAlternatingSum.v
Original file line number Diff line number Diff line change
Expand Up @@ -21,6 +21,7 @@ CONNECTION WITH THE PROOF OR THE USE OR OTHER DEALINGS IN THE PROOF.

From Coq Require Import ArithRing.
From Coq Require Import Bool.
From Coq Require Import ZArith.
From Coq Require Import Qpower Qabs.
Require Import CoRN.algebra.RSetoid.
Require Import CoRN.metric2.Metric.
Expand Down
2 changes: 1 addition & 1 deletion reals/fast/CRGeometricSum.v
Original file line number Diff line number Diff line change
Expand Up @@ -18,6 +18,7 @@ COPYRIGHT HOLDERS BE LIABLE FOR ANY CLAIM, DAMAGES OR OTHER LIABILITY, WHETHER
IN AN ACTION OF CONTRACT, TORT OR OTHERWISE, ARISING FROM, OUT OF OR IN
CONNECTION WITH THE PROOF OR THE USE OR OTHER DEALINGS IN THE PROOF.
*)
From Coq Require Import ZArith.
Require Import CoRN.metric2.Metric.
Require Import CoRN.metric2.UniformContinuity.
Require Import CoRN.reals.fast.CRAlternatingSum.
Expand Down Expand Up @@ -1119,4 +1120,3 @@ Proof.
intros. destruct (Qle_total a b).
apply H, q. symmetry. apply H, q.
Qed.

5 changes: 3 additions & 2 deletions reals/fast/CRpower.v
Original file line number Diff line number Diff line change
Expand Up @@ -19,6 +19,7 @@ COPYRIGHT HOLDERS BE LIABLE FOR ANY CLAIM, DAMAGES OR OTHER LIABILITY, WHETHER
IN AN ACTION OF CONTRACT, TORT OR OTHERWISE, ARISING FROM, OUT OF OR IN
CONNECTION WITH THE PROOF OR THE USE OR OTHER DEALINGS IN THE PROOF.
*)
From Coq Require Import ZArith.
Require Import CoRN.algebra.RSetoid.
Require Import CoRN.metric2.Metric.
Require Import CoRN.metric2.ProductMetric.
Expand All @@ -27,7 +28,7 @@ From Coq Require Import Qpower.
From Coq Require Import Qabs.
Require Import CoRN.model.metric2.Qmetric.
Require Import CoRN.model.totalorder.QMinMax.
Require Import CoRN.model.totalorder.QposMinMax.
Require Import CoRN.model.totalorder.QposMinMax.
Require Import MathClasses.interfaces.canonical_names.
Require Import MathClasses.interfaces.additional_operations.

Expand Down Expand Up @@ -581,4 +582,4 @@ Proof.
rewrite Nnat.nat_of_Nplus.
simpl.
rewrite CRpower_N_correct. reflexivity.
Qed.
Qed.
4 changes: 2 additions & 2 deletions reals/fast/CRstreams.v
Original file line number Diff line number Diff line change
Expand Up @@ -20,9 +20,10 @@ IN AN ACTION OF CONTRACT, TORT OR OTHERWISE, ARISING FROM, OUT OF OR IN
CONNECTION WITH THE PROOF OR THE USE OR OTHER DEALINGS IN THE PROOF.
*)

From Coq Require Import ZArith.
Require Import CoRN.algebra.RSetoid.
Require Import CoRN.model.totalorder.QposMinMax.
Require Import CoRN.model.metric2.Qmetric.
Require Import CoRN.model.metric2.Qmetric.
Require Import CoRN.metric2.Limit.
From Coq Require Import Qabs.
From Coq Require Import Arith.
Expand Down Expand Up @@ -817,4 +818,3 @@ Proof.
destruct q. unfold Qopp; simpl.
rewrite Z.opp_involutive. reflexivity.
Qed.

1 change: 1 addition & 0 deletions reals/fast/CRsum.v
Original file line number Diff line number Diff line change
Expand Up @@ -18,6 +18,7 @@ COPYRIGHT HOLDERS BE LIABLE FOR ANY CLAIM, DAMAGES OR OTHER LIABILITY, WHETHER
IN AN ACTION OF CONTRACT, TORT OR OTHERWISE, ARISING FROM, OUT OF OR IN
CONNECTION WITH THE PROOF OR THE USE OR OTHER DEALINGS IN THE PROOF.
*)
From Coq Require Import ZArith.
Require Import CoRN.metric2.Metric.
Require Import CoRN.metric2.UniformContinuity.
Require Import CoRN.model.totalorder.QposMinMax.
Expand Down
1 change: 1 addition & 0 deletions reals/fast/Compress.v
Original file line number Diff line number Diff line change
Expand Up @@ -19,6 +19,7 @@ IN AN ACTION OF CONTRACT, TORT OR OTHERWISE, ARISING FROM, OUT OF OR IN
CONNECTION WITH THE PROOF OR THE USE OR OTHER DEALINGS IN THE PROOF.
*)

From Coq Require Import ZArith.
Require Import CoRN.algebra.RSetoid.
Require Import CoRN.metric2.Metric.
Require Import CoRN.metric2.UniformContinuity.
Expand Down
2 changes: 1 addition & 1 deletion reals/fast/Interval.v
Original file line number Diff line number Diff line change
Expand Up @@ -18,6 +18,7 @@ COPYRIGHT HOLDERS BE LIABLE FOR ANY CLAIM, DAMAGES OR OTHER LIABILITY, WHETHER
IN AN ACTION OF CONTRACT, TORT OR OTHERWISE, ARISING FROM, OUT OF OR IN
CONNECTION WITH THE PROOF OR THE USE OR OTHER DEALINGS IN THE PROOF.
*)
From Coq Require Import ZArith.
Require Import CoRN.algebra.RSetoid.
Require Import CoRN.metric2.Metric.
Require Import CoRN.metric2.UniformContinuity.
Expand Down Expand Up @@ -708,4 +709,3 @@ Proof.
apply (Qle_trans _ _ _ q).
apply Qlt_le_weak, ltde.
Qed.

2 changes: 1 addition & 1 deletion reals/fast/Plot.v
Original file line number Diff line number Diff line change
Expand Up @@ -18,7 +18,7 @@ COPYRIGHT HOLDERS BE LIABLE FOR ANY CLAIM, DAMAGES OR OTHER LIABILITY, WHETHER
IN AN ACTION OF CONTRACT, TORT OR OTHERWISE, ARISING FROM, OUT OF OR IN
CONNECTION WITH THE PROOF OR THE USE OR OTHER DEALINGS IN THE PROOF.
*)
From Coq Require Import Qround.
From Coq Require Import ZArith Qround.
Require Import CoRN.metric2.Metric.
Require Import CoRN.metric2.ProductMetric.
Require Import CoRN.metric2.UniformContinuity.
Expand Down
1 change: 1 addition & 0 deletions reals/fast/RasterQ.v
Original file line number Diff line number Diff line change
Expand Up @@ -18,6 +18,7 @@ COPYRIGHT HOLDERS BE LIABLE FOR ANY CLAIM, DAMAGES OR OTHER LIABILITY, WHETHER
IN AN ACTION OF CONTRACT, TORT OR OTHERWISE, ARISING FROM, OUT OF OR IN
CONNECTION WITH THE PROOF OR THE USE OR OTHER DEALINGS IN THE PROOF.
*)
From Coq Require Import ZArith.
Require Import CoRN.algebra.RSetoid.
Require Import CoRN.metric2.Metric.
Require Import CoRN.metric2.UniformContinuity.
Expand Down
1 change: 1 addition & 0 deletions reals/fast/RasterizeQ.v
Original file line number Diff line number Diff line change
Expand Up @@ -18,6 +18,7 @@ COPYRIGHT HOLDERS BE LIABLE FOR ANY CLAIM, DAMAGES OR OTHER LIABILITY, WHETHER
IN AN ACTION OF CONTRACT, TORT OR OTHERWISE, ARISING FROM, OUT OF OR IN
CONNECTION WITH THE PROOF OR THE USE OR OTHER DEALINGS IN THE PROOF.
*)
From Coq Require Import ZArith.
Require Import CoRN.algebra.RSetoid.
Require Import CoRN.metric2.Metric.
Require Import CoRN.metric2.UniformContinuity.
Expand Down
5 changes: 3 additions & 2 deletions reals/faster/ARexp.v
Original file line number Diff line number Diff line change
@@ -1,12 +1,13 @@
From Coq Require Import ZArith.
Require Import CoRN.algebra.RSetoid.
Require Import CoRN.metric2.Metric.
Require Import CoRN.metric2.UniformContinuity.
From Coq Require Import Program.
Require Import MathClasses.misc.workaround_tactics
CoRN.model.totalorder.QposMinMax
CoRN.model.totalorder.QposMinMax
CoRN.model.totalorder.QMinMax.
From Coq Require Import Qround Qabs.
Require Import CoRN.util.Qdlog CoRN.stdlib_omissions.Q
Require Import CoRN.util.Qdlog CoRN.stdlib_omissions.Q
CoRN.reals.fast.CRexp CoRN.reals.fast.CRstreams CoRN.reals.fast.CRAlternatingSum
CoRN.reals.fast.Compress CoRN.reals.fast.CRpower
CoRN.metric2.MetricMorphisms CoRN.reals.faster.ARAlternatingSum MathClasses.interfaces.abstract_algebra
Expand Down
7 changes: 3 additions & 4 deletions reals/faster/ARsin.v
Original file line number Diff line number Diff line change
@@ -1,5 +1,5 @@
From Coq Require Import Qround Qpower.
Require Import MathClasses.interfaces.abstract_algebra
From Coq Require Import ZArith Qround Qpower.
Require Import MathClasses.interfaces.abstract_algebra
MathClasses.theory.nat_pow
MathClasses.theory.int_pow
CoRN.algebra.RSetoid
Expand All @@ -8,7 +8,7 @@ Require Import MathClasses.interfaces.abstract_algebra
CoRN.metric2.UniformContinuity
CoRN.model.totalorder.QMinMax
CoRN.util.Qdlog
CoRN.stdlib_omissions.Q
CoRN.stdlib_omissions.Q
CoRN.reals.fast.CRsin
CoRN.reals.fast.CRstreams
CoRN.reals.fast.CRAlternatingSum
Expand Down Expand Up @@ -381,4 +381,3 @@ Lemma ARtoCR_preserves_sin x : ' ucFun ARsin x = ucFun sin_slow ('x).
Proof. apply preserves_unary_complete_fun. Qed.

End ARsin.

11 changes: 6 additions & 5 deletions reals/stdlib/CMTDirac.v
Original file line number Diff line number Diff line change
Expand Up @@ -11,11 +11,12 @@ THE SOFTWARE IS PROVIDED "AS IS", WITHOUT WARRANTY OF ANY KIND, EXPRESS OR IMPLI

(** Dirac measure at zero. *)

Require Import QArith.
Require Import ConstructiveReals.
Require Import ConstructiveLimits.
Require Import ConstructiveAbs.
Require Import ConstructiveMinMax.
From Coq Require Import ZArith.
From Coq Require Import QArith.
From Coq Require Import ConstructiveReals.
From Coq Require Import ConstructiveLimits.
From Coq Require Import ConstructiveAbs.
From Coq Require Import ConstructiveMinMax.
Require Import ConstructivePartialFunctions.
Require Import CMTbase.

Expand Down
18 changes: 10 additions & 8 deletions reals/stdlib/CMTFullSets.v
Original file line number Diff line number Diff line change
Expand Up @@ -13,14 +13,16 @@ THE SOFTWARE IS PROVIDED "AS IS", WITHOUT WARRANTY OF ANY KIND, EXPRESS OR IMPLI
we now precisely define full sets, and prove that 2 functions equal on a
full set have the same integral. *)

Require Import QArith.
Require Import ConstructiveReals.
Require Import ConstructiveAbs.
Require Import ConstructiveMinMax.
Require Import ConstructiveCauchyAbs.
Require Import ConstructiveSum.
Require Import ConstructivePower.
Require Import ConstructiveLimits.
From Coq Require Import ZArith.
From Coq Require Import QArith.
From Coq Require Import ConstructiveReals.
From Coq Require Import ConstructiveAbs.
From Coq Require Import ConstructiveMinMax.
From Coq Require Import ConstructiveCauchyAbs.
From Coq Require Import ConstructiveSum.
From Coq Require Import ConstructivePower.
From Coq Require Import ConstructiveLimits.

Require Import ConstructiveDiagonal.
Require Import ConstructivePartialFunctions.

Expand Down
13 changes: 7 additions & 6 deletions reals/stdlib/CMTIntegrableFunctions.v
Original file line number Diff line number Diff line change
Expand Up @@ -18,12 +18,13 @@ THE SOFTWARE IS PROVIDED "AS IS", WITHOUT WARRANTY OF ANY KIND, EXPRESS OR IMPLI
IScomplete is complete, in the sense that its integrable functions are
already integrable functions of IS : no new functions are added. *)

Require Import QArith.
Require Import ConstructiveReals.
Require Import ConstructiveAbs.
Require Import ConstructiveMinMax.
Require Import ConstructiveSum.
Require Import ConstructiveLimits.
From Coq Require Import ZArith.
From Coq Require Import QArith.
From Coq Require Import ConstructiveReals.
From Coq Require Import ConstructiveAbs.
From Coq Require Import ConstructiveMinMax.
From Coq Require Import ConstructiveSum.
From Coq Require Import ConstructiveLimits.
Require Import ConstructivePartialFunctions.
Require Import CMTbase.

Expand Down
1 change: 1 addition & 0 deletions reals/stdlib/CMTIntegrableSets.v
Original file line number Diff line number Diff line change
Expand Up @@ -27,6 +27,7 @@ THE SOFTWARE IS PROVIDED "AS IS", WITHOUT WARRANTY OF ANY KIND, EXPRESS OR IMPLI
*)

From Coq Require Import ConstructiveEpsilon.
From Coq Require Import ZArith.
From Coq Require Import QArith.
From Coq Require Import ConstructiveReals.
From Coq Require Import ConstructiveAbs.
Expand Down
14 changes: 7 additions & 7 deletions reals/stdlib/CMTMeasurableFunctions.v
Original file line number Diff line number Diff line change
Expand Up @@ -9,13 +9,13 @@ THE SOFTWARE IS PROVIDED "AS IS", WITHOUT WARRANTY OF ANY KIND, EXPRESS OR IMPLI
*)


Require Import QArith.
Require Import ConstructiveReals.
Require Import ConstructiveAbs.
Require Import ConstructiveMinMax.
Require Import ConstructiveSum.
Require Import ConstructivePower.
Require Import ConstructiveLimits.
From Coq Require Import ZArith QArith.
From Coq Require Import ConstructiveReals.
From Coq Require Import ConstructiveAbs.
From Coq Require Import ConstructiveMinMax.
From Coq Require Import ConstructiveSum.
From Coq Require Import ConstructivePower.
From Coq Require Import ConstructiveLimits.
Require Import ConstructivePartialFunctions.
Require Import CMTbase.
Require Import CMTIntegrableFunctions.
Expand Down
13 changes: 7 additions & 6 deletions reals/stdlib/CMTPositivity.v
Original file line number Diff line number Diff line change
Expand Up @@ -12,12 +12,13 @@ THE SOFTWARE IS PROVIDED "AS IS", WITHOUT WARRANTY OF ANY KIND, EXPRESS OR IMPLI
(* A lemma to simplify the proofs of Icontinuous in integration spaces.
It looks classical because it does not need to give a convergence modulus. *)

Require Import QArith.
Require Import ConstructiveReals.
Require Import ConstructiveAbs.
Require Import ConstructiveSum.
Require Import ConstructivePower.
Require Import ConstructiveLimits.
From Coq Require Import ZArith.
From Coq Require Import QArith.
From Coq Require Import ConstructiveReals.
From Coq Require Import ConstructiveAbs.
From Coq Require Import ConstructiveSum.
From Coq Require Import ConstructivePower.
From Coq Require Import ConstructiveLimits.
Require Import ConstructiveDiagonal.
Require Import ConstructivePartialFunctions.
Require Import CMTbase.
Expand Down
16 changes: 8 additions & 8 deletions reals/stdlib/CMTProductIntegral.v
Original file line number Diff line number Diff line change
Expand Up @@ -19,14 +19,14 @@ THE SOFTWARE IS PROVIDED "AS IS", WITHOUT WARRANTY OF ANY KIND, EXPRESS OR IMPLI
on disjoint rectangles. Then we can take the absolute of those
disjoint coefficients. *)

Require Import QArith_base.
Require Import List.
Require Import ConstructiveReals.
Require Import ConstructiveRealsMorphisms.
Require Import ConstructiveAbs.
Require Import ConstructiveSum.
Require Import ConstructiveMinMax.
Require Import ConstructiveLimits.
From Coq Require Import ZArith QArith_base.
From Coq Require Import List.
From Coq Require Import ConstructiveReals.
From Coq Require Import ConstructiveRealsMorphisms.
From Coq Require Import ConstructiveAbs.
From Coq Require Import ConstructiveSum.
From Coq Require Import ConstructiveMinMax.
From Coq Require Import ConstructiveLimits.
Require Import ConstructivePartialFunctions.
Require Import CMTbase.
Require Import CMTIntegrableFunctions.
Expand Down
16 changes: 8 additions & 8 deletions reals/stdlib/CMTReals.v
Original file line number Diff line number Diff line change
Expand Up @@ -29,14 +29,14 @@ THE SOFTWARE IS PROVIDED "AS IS", WITHOUT WARRANTY OF ANY KIND, EXPRESS OR IMPLI
of the values of the functions with zero.
*)

Require Import QArith Qminmax Qpower Qabs.

Require Import ConstructiveReals.
Require Import ConstructiveAbs.
Require Import ConstructiveMinMax.
Require Import ConstructiveSum.
Require Import ConstructivePower.
Require Import ConstructiveLimits.
From Coq Require Import ZArith QArith Qminmax Qpower Qabs.

From Coq Require Import ConstructiveReals.
From Coq Require Import ConstructiveAbs.
From Coq Require Import ConstructiveMinMax.
From Coq Require Import ConstructiveSum.
From Coq Require Import ConstructivePower.
From Coq Require Import ConstructiveLimits.
Require Import ConstructiveDiagonal.
Require Import ConstructivePartialFunctions.
Require Import ConstructiveUniformCont.
Expand Down
16 changes: 8 additions & 8 deletions reals/stdlib/CMTprofile.v
Original file line number Diff line number Diff line change
Expand Up @@ -25,13 +25,13 @@ THE SOFTWARE IS PROVIDED "AS IS", WITHOUT WARRANTY OF ANY KIND, EXPRESS OR IMPLI
prove that this non-increasing limit of integrals exists.
*)

Require Import QArith_base Qabs.
Require Import ConstructiveReals.
Require Import ConstructiveSum.
Require Import ConstructivePower.
Require Import ConstructiveAbs.
Require Import ConstructiveMinMax.
Require Import ConstructiveLimits.
From Coq Require Import ZArith QArith_base Qabs.
From Coq Require Import ConstructiveReals.
From Coq Require Import ConstructiveSum.
From Coq Require Import ConstructivePower.
From Coq Require Import ConstructiveAbs.
From Coq Require Import ConstructiveMinMax.
From Coq Require Import ConstructiveLimits.
Require Import ConstructiveUniformCont.
Require Import ConstructivePartialFunctions.
Require Import ConstructiveDiagonal.
Expand All @@ -40,7 +40,7 @@ Require Import CMTIntegrableFunctions.
Require Import CMTIntegrableSets.
Require Import CMTFullSets.
Require Import CMTReals.
Require Import Lia.
From Coq Require Import Lia.

Local Open Scope ConstructiveReals.

Expand Down
16 changes: 8 additions & 8 deletions reals/stdlib/ConstructiveCauchyIntegral.v
Original file line number Diff line number Diff line change
Expand Up @@ -21,14 +21,14 @@ THE SOFTWARE IS PROVIDED "AS IS", WITHOUT WARRANTY OF ANY KIND, EXPRESS OR IMPLI
functions.
*)

Require Import List Permutation Orders Sorted Mergesort.
Require Import QArith Qpower.
Require Import ConstructiveReals.
Require Import ConstructiveAbs.
Require Import ConstructiveMinMax.
Require Import ConstructiveSum.
Require Import ConstructiveLimits.
Require Import ConstructiveRcomplete.
From Coq Require Import List Permutation Orders Sorted Mergesort.
From Coq Require Import ZArith QArith Qpower.
From Coq Require Import ConstructiveReals.
From Coq Require Import ConstructiveAbs.
From Coq Require Import ConstructiveMinMax.
From Coq Require Import ConstructiveSum.
From Coq Require Import ConstructiveLimits.
From Coq Require Import ConstructiveRcomplete.
Require Import ConstructiveDiagonal.
Require Import ConstructiveUniformCont.

Expand Down
Loading

0 comments on commit a75b14f

Please sign in to comment.