aboutsummaryrefslogtreecommitdiff
diff options
context:
space:
mode:
authorThéo Zimmermann2020-01-22 19:11:35 +0100
committerThéo Zimmermann2020-01-22 19:11:35 +0100
commit8f836215f099ea5ec7f27fd67d7723743d2e42e0 (patch)
tree4d3988a4464fbd53fe270d8d9a6c62efd8c8616d
parent7161bca5659accd920c3c868ec561b143bb9212d (diff)
Add explicit types to changelog entries.
-rw-r--r--doc/changelog/03-notations/11113-remove-compat.rst2
-rw-r--r--doc/changelog/03-notations/11172-master+coercion-notation-interleaved-printing.rst3
-rw-r--r--doc/changelog/04-tactics/10760-more-rapply.rst3
-rw-r--r--doc/changelog/07-commands-and-options/11162-local-cs.rst4
-rw-r--r--doc/changelog/07-commands-and-options/11164-let-cs.rst4
5 files changed, 11 insertions, 5 deletions
diff --git a/doc/changelog/03-notations/11113-remove-compat.rst b/doc/changelog/03-notations/11113-remove-compat.rst
index 8c71d70cda..3bcdd3dd6f 100644
--- a/doc/changelog/03-notations/11113-remove-compat.rst
+++ b/doc/changelog/03-notations/11113-remove-compat.rst
@@ -1,4 +1,4 @@
-- Removed deprecated ``compat`` modifier of :cmd:`Notation`
+- **Removed:** deprecated ``compat`` modifier of :cmd:`Notation`
and :cmd:`Infix` commands
(`#11113 <https://github.com/coq/coq/pull/11113>`_,
by Théo Zimmermann, with help from Jason Gross).
diff --git a/doc/changelog/03-notations/11172-master+coercion-notation-interleaved-printing.rst b/doc/changelog/03-notations/11172-master+coercion-notation-interleaved-printing.rst
index a53fb7e970..f377b53ae2 100644
--- a/doc/changelog/03-notations/11172-master+coercion-notation-interleaved-printing.rst
+++ b/doc/changelog/03-notations/11172-master+coercion-notation-interleaved-printing.rst
@@ -1,2 +1,3 @@
-- The printing algorithm now interleaves search for notations and removal of coercions
+- **Changed:**
+ The printing algorithm now interleaves search for notations and removal of coercions
(`#11172 <https://github.com/coq/coq/pull/11172>`_, by Hugo Herbelin).
diff --git a/doc/changelog/04-tactics/10760-more-rapply.rst b/doc/changelog/04-tactics/10760-more-rapply.rst
index 2815f8af8a..eeae2ec519 100644
--- a/doc/changelog/04-tactics/10760-more-rapply.rst
+++ b/doc/changelog/04-tactics/10760-more-rapply.rst
@@ -1,4 +1,5 @@
-- The tactic :tacn:`rapply` in :g:`Coq.Program.Tactics` now handles
+- **Changed:**
+ The tactic :tacn:`rapply` in :g:`Coq.Program.Tactics` now handles
arbitrary numbers of underscores and takes in a :g:`uconstr`. In
rare cases where users were relying on :tacn:`rapply` inserting
exactly 15 underscores and no more, due to the lemma having a
diff --git a/doc/changelog/07-commands-and-options/11162-local-cs.rst b/doc/changelog/07-commands-and-options/11162-local-cs.rst
index 5a69a107cd..638222fbe1 100644
--- a/doc/changelog/07-commands-and-options/11162-local-cs.rst
+++ b/doc/changelog/07-commands-and-options/11162-local-cs.rst
@@ -1 +1,3 @@
-- Handle the ``#[local]`` attribute in :g:`Canonical Structure` declarations (`#11162 <https://github.com/coq/coq/pull/11162>`_, by Enrico Tassi).
+- **Added:** Handle the ``#[local]`` attribute in :g:`Canonical
+ Structure` declarations (`#11162
+ <https://github.com/coq/coq/pull/11162>`_, by Enrico Tassi).
diff --git a/doc/changelog/07-commands-and-options/11164-let-cs.rst b/doc/changelog/07-commands-and-options/11164-let-cs.rst
index b9ecd140e7..ec34c075ae 100644
--- a/doc/changelog/07-commands-and-options/11164-let-cs.rst
+++ b/doc/changelog/07-commands-and-options/11164-let-cs.rst
@@ -1 +1,3 @@
-- A section variable introduces with :g:`Let` can be declared as a :g:`Canonical Structure` (`#11164 <https://github.com/coq/coq/pull/11164>`_, by Enrico Tassi).
+- **Added:** A section variable introduces with :g:`Let` can be
+ declared as a :g:`Canonical Structure` (`#11164
+ <https://github.com/coq/coq/pull/11164>`_, by Enrico Tassi).