Skip to content

Commit

Permalink
add deprecation warnings for Int31
Browse files Browse the repository at this point in the history
  • Loading branch information
andres-erbsen committed Jun 15, 2023
1 parent ba574c6 commit ebbdb41
Show file tree
Hide file tree
Showing 5 changed files with 257 additions and 1 deletion.
6 changes: 6 additions & 0 deletions doc/changelog/11-standard-library/17734-warn-Int31.rst
@@ -0,0 +1,6 @@
- **Deprecated:** :g: Deprecation warnings are now generated for
:g:`Numbers.Cyclic.Int31.Cyclic31`, :g:`NNumbers.Cyclic.Int31.Int31`, and
:g:`NNumbers.Cyclic.Int31.Ring31`. These modules have been deprecated since
Coq 8.10. The modules under :g:`Numbers.Cyclic.Int63` remain available
(`#17734 <https://github.com/coq/coq/pull/17734>`_,
by Andres Erbsen).
2 changes: 1 addition & 1 deletion test-suite/output/Int31NumberSyntax.v
@@ -1,5 +1,5 @@
Require Import Int31 Cyclic31.

Local Set Warnings "-deprecated".
Open Scope int31_scope.
Check I31. (* Would be nice to have I31 : digits->digits->...->int31
For the moment, I31 : digits31 int31, which is better
Expand Down

0 comments on commit ebbdb41

Please sign in to comment.