Skip to content

Commit

Permalink
Merge pull request #96 from coq-community/rm_deprecations
Browse files Browse the repository at this point in the history
Address some deprecation warnings
  • Loading branch information
proux01 authored Dec 8, 2024
2 parents 1f014ff + f82ed75 commit d9ff01f
Show file tree
Hide file tree
Showing 25 changed files with 61 additions and 54 deletions.
6 changes: 3 additions & 3 deletions BigN/BigN.v
Original file line number Diff line number Diff line change
Expand Up @@ -10,8 +10,8 @@

(** Initial Author: Arnaud Spiwack *)

Require Import Lia CyclicAxioms Ring63 NSig NSigNAxioms NMake
NProperties GenericMinMax.
From Stdlib Require Import Lia CyclicAxioms Ring63 NProperties GenericMinMax.
Require Import NSig NSigNAxioms NMake.
Import Cyclic63.

(** The following [BigN] module regroups both the operations and
Expand Down Expand Up @@ -44,7 +44,7 @@ Notation bigN := BigN.t.
Bind Scope bigN_scope with bigN.
Bind Scope bigN_scope with BigN.t.
Bind Scope bigN_scope with BigN.t'.
Arguments BigN.N0 _%int63.
Arguments BigN.N0 _%_int63.
Local Notation "0" := BigN.zero : bigN_scope. (* temporary notation *)
Local Notation "1" := BigN.one : bigN_scope. (* temporary notation *)
Local Notation "2" := BigN.two : bigN_scope. (* temporary notation *)
Expand Down
5 changes: 3 additions & 2 deletions BigN/NMake.v
Original file line number Diff line number Diff line change
Expand Up @@ -16,8 +16,9 @@
representation. The representation-dependent (and macro-generated) part
is now in [NMake_gen]. *)

Require Import Bool BigNumPrelude ZArith Lia Nnat CyclicAxioms DoubleType
Nbasic Wf_nat StreamMemo NSig NMake_gen.
From Stdlib Require Import Bool ZArith Lia Nnat CyclicAxioms DoubleType.
From Stdlib Require Import Wf_nat StreamMemo.
Require Import BigNumPrelude Nbasic NSig NMake_gen.

Module Make (W0:CyclicType) <: NType.

Expand Down
6 changes: 3 additions & 3 deletions BigN/Nbasic.v
Original file line number Diff line number Diff line change
Expand Up @@ -8,11 +8,11 @@
(* Benjamin Gregoire, Laurent Thery, INRIA, 2007 *)
(************************************************************************)

Require Import ZArith Lia.
From Stdlib Require Import ZArith Lia.
From Stdlib Require Import DoubleType.
From Stdlib Require Import CyclicAxioms.
Require Import BigNumPrelude.
Require Import DoubleType.
Require Import DoubleBase.
Require Import CyclicAxioms.
Require Import DoubleCyclic.

Arguments mk_zn2z_ops [t] ops.
Expand Down
6 changes: 3 additions & 3 deletions BigN/gen/NMake_gen.ml
Original file line number Diff line number Diff line change
Expand Up @@ -49,9 +49,9 @@ pr
(** Remark: File automatically generated by NMake_gen.ml, DO NOT EDIT ! *)
Require Import BigNumPrelude ZArith Lia CyclicAxioms
DoubleType DoubleMul DoubleDivn1 DoubleBase DoubleCyclic Nbasic
Wf_nat StreamMemo.
From Stdlib Require Import ZArith Lia CyclicAxioms DoubleType Wf_nat StreamMemo.
Require Import BigNumPrelude.
Require Import DoubleMul DoubleDivn1 DoubleBase DoubleCyclic Nbasic.
Local Close Scope Z.
Expand Down
16 changes: 8 additions & 8 deletions BigNumPrelude.v
Original file line number Diff line number Diff line change
Expand Up @@ -14,14 +14,14 @@
numbers. *)


Require Import ArithRing.
Require Export ZArith.
Require Export Znumtheory.
Require Export Zpow_facts.
Require Uint63.
Require Import Lia.

Declare ML Module "bignums_syntax_plugin:coq-bignums.plugin".
From Stdlib Require Import ArithRing.
From Stdlib Require Export ZArith.
From Stdlib Require Export Znumtheory.
From Stdlib Require Export Zpow_facts.
From Stdlib Require Uint63.
From Stdlib Require Import Lia.

Declare ML Module "coq-bignums.plugin".

(* *** Nota Bene ***
All results that were general enough have been moved in ZArith.
Expand Down
3 changes: 2 additions & 1 deletion BigQ/BigQ.v
Original file line number Diff line number Diff line change
Expand Up @@ -10,8 +10,9 @@

(** Initial authors: Benjamin Gregoire, Laurent Thery, INRIA, 2007 *)

From Stdlib Require Import Field Qfield Orders GenericMinMax.
Require Export BigZ.
Require Import Field Qfield QSig QMake Orders GenericMinMax.
Require Import QSig QMake.

(** We choose for BigQ an implemention with
multiple representation of 0: 0, 1/0, 2/0 etc.
Expand Down
6 changes: 3 additions & 3 deletions BigQ/QMake.v
Original file line number Diff line number Diff line change
Expand Up @@ -10,9 +10,9 @@

(** Initial authors : Benjamin Gregoire, Laurent Thery, INRIA, 2007 *)

Require Import BigNumPrelude Lia.
Require Import QArith Qcanon Qpower Qminmax.
Require Import NSig ZSig QSig.
From Stdlib Require Import Lia.
From Stdlib Require Import QArith Qcanon Qpower Qminmax.
Require Import BigNumPrelude NSig ZSig QSig.

(** We will build rationals out of an implementation of integers [ZType]
for numerators and an implementation of natural numbers [NType] for
Expand Down
7 changes: 4 additions & 3 deletions BigZ/BigZ.v
Original file line number Diff line number Diff line change
Expand Up @@ -8,8 +8,9 @@
(* Benjamin Gregoire, Laurent Thery, INRIA, 2007 *)
(************************************************************************)

From Stdlib Require Import ZProperties ZDivFloor Ring Lia.
Require Export BigN.
Require Import ZProperties ZDivFloor ZSig ZSigZAxioms ZMake Ring Lia.
Require Import ZSig ZSigZAxioms ZMake.
Import Zpow_def Zdiv.

(** * [BigZ] : arbitrary large efficient integers.
Expand Down Expand Up @@ -45,8 +46,8 @@ Notation bigZ := BigZ.t.
Bind Scope bigZ_scope with bigZ.
Bind Scope bigZ_scope with BigZ.t.
Bind Scope bigZ_scope with BigZ.t_.
Arguments BigZ.Pos _%bigN.
Arguments BigZ.Neg _%bigN.
Arguments BigZ.Pos _%_bigN.
Arguments BigZ.Neg _%_bigN.
Local Notation "0" := BigZ.zero : bigZ_scope.
Local Notation "1" := BigZ.one : bigZ_scope.
Local Notation "2" := BigZ.two : bigZ_scope.
Expand Down
2 changes: 1 addition & 1 deletion BigZ/ZMake.v
Original file line number Diff line number Diff line change
Expand Up @@ -8,7 +8,7 @@
(* Benjamin Gregoire, Laurent Thery, INRIA, 2007 *)
(************************************************************************)

Require Import ZArith Lia.
From Stdlib Require Import ZArith Lia.
Require Import BigNumPrelude.
Require Import NSig.
Require Import ZSig.
Expand Down
4 changes: 2 additions & 2 deletions CyclicDouble/DoubleAdd.v
Original file line number Diff line number Diff line change
Expand Up @@ -10,9 +10,9 @@

Set Implicit Arguments.

Require Import ZArith Lia.
From Stdlib Require Import ZArith Lia.
From Stdlib Require Import DoubleType.
Require Import BigNumPrelude.
Require Import DoubleType.
Require Import DoubleBase.

Local Open Scope Z_scope.
Expand Down
5 changes: 2 additions & 3 deletions CyclicDouble/DoubleBase.v
Original file line number Diff line number Diff line change
Expand Up @@ -10,9 +10,9 @@

Set Implicit Arguments.

Require Import ZArith.
From Stdlib Require Import ZArith.
From Stdlib Require Import DoubleType.
Require Import BigNumPrelude.
Require Import DoubleType.

Local Open Scope Z_scope.

Expand Down Expand Up @@ -441,4 +441,3 @@ Section DoubleBase.
End DoubleProof.

End DoubleBase.

6 changes: 3 additions & 3 deletions CyclicDouble/DoubleCyclic.v
Original file line number Diff line number Diff line change
Expand Up @@ -10,9 +10,10 @@

Set Implicit Arguments.

Require Import ZArith Lia.
From Stdlib Require Import ZArith Lia.
From Stdlib Require Import DoubleType.
From Stdlib Require Import CyclicAxioms.
Require Import BigNumPrelude.
Require Import DoubleType.
Require Import DoubleBase.
Require Import DoubleAdd.
Require Import DoubleSub.
Expand All @@ -21,7 +22,6 @@ Require Import DoubleSqrt.
Require Import DoubleLift.
Require Import DoubleDivn1.
Require Import DoubleDiv.
Require Import CyclicAxioms.

Local Open Scope Z_scope.

Expand Down
4 changes: 2 additions & 2 deletions CyclicDouble/DoubleDiv.v
Original file line number Diff line number Diff line change
Expand Up @@ -10,9 +10,9 @@

Set Implicit Arguments.

Require Import ZArith Lia.
From Stdlib Require Import ZArith Lia.
From Stdlib Require Import DoubleType.
Require Import BigNumPrelude.
Require Import DoubleType.
Require Import DoubleBase.
Require Import DoubleDivn1.
Require Import DoubleAdd.
Expand Down
4 changes: 2 additions & 2 deletions CyclicDouble/DoubleDivn1.v
Original file line number Diff line number Diff line change
Expand Up @@ -10,9 +10,9 @@

Set Implicit Arguments.

Require Import ZArith Lia.
From Stdlib Require Import ZArith Lia.
From Stdlib Require Import DoubleType.
Require Import BigNumPrelude.
Require Import DoubleType.
Require Import DoubleBase.

Local Open Scope Z_scope.
Expand Down
4 changes: 2 additions & 2 deletions CyclicDouble/DoubleLift.v
Original file line number Diff line number Diff line change
Expand Up @@ -10,9 +10,9 @@

Set Implicit Arguments.

Require Import ZArith Lia.
From Stdlib Require Import ZArith Lia.
From Stdlib Require Import DoubleType.
Require Import BigNumPrelude.
Require Import DoubleType.
Require Import DoubleBase.

Local Open Scope Z_scope.
Expand Down
4 changes: 2 additions & 2 deletions CyclicDouble/DoubleMul.v
Original file line number Diff line number Diff line change
Expand Up @@ -10,9 +10,9 @@

Set Implicit Arguments.

Require Import ZArith Lia.
From Stdlib Require Import ZArith Lia.
From Stdlib Require Import DoubleType.
Require Import BigNumPrelude.
Require Import DoubleType.
Require Import DoubleBase.

Local Open Scope Z_scope.
Expand Down
4 changes: 2 additions & 2 deletions CyclicDouble/DoubleSqrt.v
Original file line number Diff line number Diff line change
Expand Up @@ -10,9 +10,9 @@

Set Implicit Arguments.

Require Import ZArith Lia.
From Stdlib Require Import ZArith Lia.
From Stdlib Require Import DoubleType.
Require Import BigNumPrelude.
Require Import DoubleType.
Require Import DoubleBase.

Local Open Scope Z_scope.
Expand Down
4 changes: 2 additions & 2 deletions CyclicDouble/DoubleSub.v
Original file line number Diff line number Diff line change
Expand Up @@ -11,9 +11,9 @@

Set Implicit Arguments.

Require Import ZArith Lia.
From Stdlib Require Import ZArith Lia.
From Stdlib Require Import DoubleType.
Require Import BigNumPrelude.
Require Import DoubleType.
Require Import DoubleBase.

Local Open Scope Z_scope.
Expand Down
3 changes: 2 additions & 1 deletion SpecViaQ/QSig.v
Original file line number Diff line number Diff line change
Expand Up @@ -6,7 +6,8 @@
(* * GNU Lesser General Public License Version 2.1 *)
(************************************************************************)

Require Import QArith Qpower Qminmax Orders RelationPairs GenericMinMax.
From Stdlib Require Import QArith Qpower Qminmax.
From Stdlib Require Import Orders RelationPairs GenericMinMax.

Open Scope Q_scope.

Expand Down
Binary file modified SpecViaZ/.lia.cache
Binary file not shown.
3 changes: 2 additions & 1 deletion SpecViaZ/NSig.v
Original file line number Diff line number Diff line change
Expand Up @@ -8,7 +8,8 @@
(* Benjamin Gregoire, Laurent Thery, INRIA, 2007 *)
(************************************************************************)

Require Import BinInt DoubleBase.
From Stdlib Require Import BinInt.
Require Import DoubleBase.

Open Scope Z_scope.

Expand Down
3 changes: 2 additions & 1 deletion SpecViaZ/NSigNAxioms.v
Original file line number Diff line number Diff line change
Expand Up @@ -6,7 +6,8 @@
(* * GNU Lesser General Public License Version 2.1 *)
(************************************************************************)

Require Import ZArith OrdersFacts Nnat NAxioms NSig Lia.
From Stdlib Require Import ZArith OrdersFacts Nnat NAxioms Lia.
Require Import NSig.

(** * The interface [NSig.NType] implies the interface [NAxiomsSig] *)

Expand Down
3 changes: 2 additions & 1 deletion SpecViaZ/ZSig.v
Original file line number Diff line number Diff line change
Expand Up @@ -8,7 +8,8 @@
(* Benjamin Gregoire, Laurent Thery, INRIA, 2007 *)
(************************************************************************)

Require Import BinInt DoubleBase.
From Stdlib Require Import BinInt.
Require Import DoubleBase.

Open Scope Z_scope.

Expand Down
3 changes: 2 additions & 1 deletion SpecViaZ/ZSigZAxioms.v
Original file line number Diff line number Diff line change
Expand Up @@ -6,7 +6,8 @@
(* * GNU Lesser General Public License Version 2.1 *)
(************************************************************************)

Require Import Bool ZArith OrdersFacts Nnat ZAxioms ZSig Lia.
From Stdlib Require Import Bool ZArith OrdersFacts Nnat ZAxioms Lia.
Require Import ZSig.

(** * The interface [ZSig.ZType] implies the interface [ZAxiomsSig] *)

Expand Down
4 changes: 2 additions & 2 deletions plugin/bignums_syntax.ml
Original file line number Diff line number Diff line change
Expand Up @@ -108,8 +108,8 @@ let word_of_pos_bigint ?loc hght n =
decomp hght n

let nat_of_int ?loc n =
let ref_O = DAst.make ?loc (GRef (Coqlib.lib_ref "num.nat.O", None)) in
let ref_S = DAst.make ?loc (GRef (Coqlib.lib_ref "num.nat.S", None)) in
let ref_O = DAst.make ?loc (GRef (Rocqlib.lib_ref "num.nat.O", None)) in
let ref_S = DAst.make ?loc (GRef (Rocqlib.lib_ref "num.nat.S", None)) in
let rec mk_nat acc n =
if Int.equal n 0 then acc
else
Expand Down

0 comments on commit d9ff01f

Please sign in to comment.