aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Structures
diff options
context:
space:
mode:
authorGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2011-06-21 21:18:47 +0000
committerGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2011-06-21 21:18:47 +0000
commitb03db7e43a67251406c4b27fa179f1d46c248906 (patch)
treea22d3a52c779149be1d7f7f3f982d12d5b51e923 /theories/Structures
parent6810929f652be3ebe40de86fe360665c6aded049 (diff)
Follow-up concerning eqb / ltb / leb comparisons
- All statement using reflect are made transparent. (Otherwise, since reflect isn't in Prop, extraction complains now about opaque Type definition). - remove two local Peqb_spec and Neqb_spec, now provided globally as Pos.eqb_spec and N.eqb_spec. git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@14232 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Structures')
-rw-r--r--theories/Structures/Equalities.v2
-rw-r--r--theories/Structures/OrdersFacts.v4
2 files changed, 3 insertions, 3 deletions
diff --git a/theories/Structures/Equalities.v b/theories/Structures/Equalities.v
index 933c4ea0e..eb5373859 100644
--- a/theories/Structures/Equalities.v
+++ b/theories/Structures/Equalities.v
@@ -196,7 +196,7 @@ Qed.
Lemma eqb_spec x y : reflect (x==y) (x =? y).
Proof.
apply iff_reflect. symmetry. apply eqb_eq.
-Qed.
+Defined.
(** Negated form of [eqb_eq] *)
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.