aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Structures/OrdersFacts.v
diff options
context:
space:
mode:
Diffstat (limited to 'theories/Structures/OrdersFacts.v')
-rw-r--r--theories/Structures/OrdersFacts.v4
1 files changed, 2 insertions, 2 deletions
diff --git a/theories/Structures/OrdersFacts.v b/theories/Structures/OrdersFacts.v
index a447e8fb5..2e9c0cf56 100644
--- a/theories/Structures/OrdersFacts.v
+++ b/theories/Structures/OrdersFacts.v
@@ -365,7 +365,7 @@ Include CompareBasedOrderFacts E C O.
Lemma leb_spec0 x y : reflect (x<=y) (x<=?y).
Proof.
apply iff_reflect. symmetry. apply leb_le.
-Qed.
+Defined.
Lemma leb_spec x y : BoolSpec (x<=y) (y<x) (x<=?y).
Proof.
@@ -376,7 +376,7 @@ Qed.
Lemma ltb_spec0 x y : reflect (x<y) (x<?y).
Proof.
apply iff_reflect. symmetry. apply ltb_lt.
-Qed.
+Defined.
Lemma ltb_spec x y : BoolSpec (x<y) (y<=x) (x<?y).
Proof.