Skip to content

Commit

Permalink
Deprecate obsolete files in NArith
Browse files Browse the repository at this point in the history
TODO: look at Ndec.v
  • Loading branch information
Villetaneuse committed Dec 12, 2023
1 parent d8f2ce5 commit 9ddd30f
Show file tree
Hide file tree
Showing 6 changed files with 7 additions and 0 deletions.
1 change: 1 addition & 0 deletions theories/NArith/Ndec.v
Original file line number Diff line number Diff line change
Expand Up @@ -19,6 +19,7 @@ Require Import Ndigits.

Local Open Scope N_scope.

Attributes deprecated(since="8.19", note="TODO").
(** Obsolete results about boolean comparisons over [N],
kept for compatibility with IntMap and SMC. *)

Expand Down
1 change: 1 addition & 0 deletions theories/NArith/Ndigits.v
Original file line number Diff line number Diff line change
Expand Up @@ -14,6 +14,7 @@ Require Import Bool Morphisms Setoid Bvector BinPos BinNat PeanoNat Pnat Nnat
Local Open Scope N_scope.
Local Open Scope program_scope.

Attributes deprecated(since="8.19", note="Use NArith.BinNat instead.").
(** This file is mostly obsolete, see directly [BinNat] now. *)
Local Set Warnings "-deprecated".

Expand Down
2 changes: 2 additions & 0 deletions theories/NArith/Ndist.v
Original file line number Diff line number Diff line change
Expand Up @@ -12,6 +12,8 @@ Require Import BinPos.
Require Import BinNat.
Require Import Ndigits.

Attributes deprecated(since="8.19", note="Please step up to maintain Ndist.v if you need it.").

Local Set Warnings "-deprecated".
(** An ultrametric distance over [N] numbers *)

Expand Down
1 change: 1 addition & 0 deletions theories/NArith/Ndiv_def.v
Original file line number Diff line number Diff line change
Expand Up @@ -11,6 +11,7 @@
Require Import BinNat.
Local Open Scope N_scope.

Attributes deprecated(since="8.19", note="Use NArith.BinNat instead.").
(** Obsolete file, see [BinNat] now,
only compatibility notations remain here. *)

Expand Down
1 change: 1 addition & 0 deletions theories/NArith/Ngcd_def.v
Original file line number Diff line number Diff line change
Expand Up @@ -11,6 +11,7 @@
Require Import BinPos BinNat.
Local Open Scope N_scope.

Attributes deprecated(since="8.19", note="Require BinNat instead.").
(** Obsolete file, see [BinNat] now,
only compatibility notations remain here. *)

Expand Down
1 change: 1 addition & 0 deletions theories/NArith/Nsqrt_def.v
Original file line number Diff line number Diff line change
Expand Up @@ -10,6 +10,7 @@

Require Import BinNat.

Attributes deprecated(since="8.19", note="Require BinNat instead.").
(** Obsolete file, see [BinNat] now,
only compatibility notations remain here. *)

Expand Down

0 comments on commit 9ddd30f

Please sign in to comment.