aboutsummaryrefslogtreecommitdiff
path: root/theories/Sorting
diff options
context:
space:
mode:
authorJason Gross2020-03-23 15:53:26 -0400
committerJason Gross2020-03-23 15:55:40 -0400
commit528dd28a48dd7b1898212e2aae9b43bb19fb91cc (patch)
treec797790a1aa47c14286b92a4dca0526c0262fc35 /theories/Sorting
parentb079040702d34ab06a0b1da2893d739e04477b78 (diff)
Fix levels of `<=?` and `<?` in the stdlib
They were defined at level 70, no associativity in all but three places, where they were instead declared at level 35. Fixes #11890
Diffstat (limited to 'theories/Sorting')
-rw-r--r--theories/Sorting/Mergesort.v3
1 files changed, 1 insertions, 2 deletions
diff --git a/theories/Sorting/Mergesort.v b/theories/Sorting/Mergesort.v
index a761dba62d..e9171cfdb3 100644
--- a/theories/Sorting/Mergesort.v
+++ b/theories/Sorting/Mergesort.v
@@ -259,7 +259,7 @@ Module NatOrder <: TotalLeBool.
| _, 0 => false
| S x', S y' => leb x' y'
end.
- Infix "<=?" := leb (at level 35).
+ Infix "<=?" := leb (at level 70, no associativity).
Theorem leb_total : forall a1 a2, a1 <=? a2 \/ a2 <=? a1.
Proof.
induction a1; destruct a2; simpl; auto.
@@ -269,4 +269,3 @@ End NatOrder.
Module Import NatSort := Sort NatOrder.
Example SimpleMergeExample := Eval compute in sort [5;3;6;1;8;6;0].
-