aboutsummaryrefslogtreecommitdiff
path: root/theories/Sorting
diff options
context:
space:
mode:
authorHugo Herbelin2020-03-26 08:56:05 +0100
committerHugo Herbelin2020-03-26 08:56:05 +0100
commit63f2da5b3703a16c7722b91ce2f2c78617dec9a7 (patch)
tree621f684b05604d4ab76dd365542f2f5eecfc580f /theories/Sorting
parent84f6394f78baea5b1f261765164ae23cd245a357 (diff)
parentd1e00bb24abb5045aad35723722c2b0ae7a0a8aa (diff)
Merge PR #11885: Sorting: Swap the names of Sorted_sort and LocallySorted_sort
Reviewed-by: herbelin
Diffstat (limited to 'theories/Sorting')
-rw-r--r--theories/Sorting/Mergesort.v8
1 files changed, 4 insertions, 4 deletions
diff --git a/theories/Sorting/Mergesort.v b/theories/Sorting/Mergesort.v
index e9171cfdb3..f6a1efdd37 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.