aboutsummaryrefslogtreecommitdiff
diff options
context:
space:
mode:
authorLysxia2020-03-22 17:42:28 -0400
committerLysxia2020-03-23 13:38:22 -0400
commitd1e00bb24abb5045aad35723722c2b0ae7a0a8aa (patch)
tree7defd38e87533cfca8a0589bf7b3a3b6140adaae
parentb079040702d34ab06a0b1da2893d739e04477b78 (diff)
Sorting: Swap the names of Sorted_sort and LocallySorted_sort
-rw-r--r--doc/changelog/10-standard-library/1185-sort.rst5
-rw-r--r--theories/Sorting/Mergesort.v8
2 files changed, 9 insertions, 4 deletions
diff --git a/doc/changelog/10-standard-library/1185-sort.rst b/doc/changelog/10-standard-library/1185-sort.rst
new file mode 100644
index 0000000000..edb5ee3ac4
--- /dev/null
+++ b/doc/changelog/10-standard-library/1185-sort.rst
@@ -0,0 +1,5 @@
+- **Changed:**
+ The names of ``Sorted_sort`` and ``LocallySorted_sort`` in ``Coq.Sorting.MergeSort``
+ have been swapped to appropriately reflect their meanings
+ (`#1185 <https://github.com/coq/coq/pull/1185>`_,
+ by Lysxia).
diff --git a/theories/Sorting/Mergesort.v b/theories/Sorting/Mergesort.v
index a761dba62d..f629c7426b 100644
--- a/theories/Sorting/Mergesort.v
+++ b/theories/Sorting/Mergesort.v
@@ -230,13 +230,13 @@ Proof.
apply IHl.
Qed.
-Theorem Sorted_sort : forall l, Sorted (sort l).
+Theorem LocallySorted_sort : forall l, Sorted (sort l).
Proof.
intro; apply Sorted_iter_merge. constructor.
Qed.
-Corollary LocallySorted_sort : forall l, Sorted.Sorted leb (sort l).
-Proof. intro; eapply Sorted_LocallySorted_iff, Sorted_sort; auto. Qed.
+Corollary Sorted_sort : forall l, Sorted.Sorted leb (sort l).
+Proof. intro; eapply Sorted_LocallySorted_iff, LocallySorted_sort; auto. Qed.
Theorem Permuted_sort : forall l, Permutation l (sort l).
Proof.
@@ -245,7 +245,7 @@ Qed.
Corollary StronglySorted_sort : forall l,
Transitive leb -> StronglySorted leb (sort l).
-Proof. auto using Sorted_StronglySorted, LocallySorted_sort. Qed.
+Proof. auto using Sorted_StronglySorted, Sorted_sort. Qed.
End Sort.