aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/ZArith/ZArith_dec.v
diff options
context:
space:
mode:
authorGravatar notin <notin@85f007b7-540e-0410-9357-904b9bb8a0f7>2007-04-12 17:46:54 +0000
committerGravatar notin <notin@85f007b7-540e-0410-9357-904b9bb8a0f7>2007-04-12 17:46:54 +0000
commita914fb843800aefcc3833d93b0c1f260ab152d30 (patch)
treed0a148e4fcc61d8f6f7a59df4e9cc1b5ac2c1d89 /theories/ZArith/ZArith_dec.v
parent7aeb305493f1d297dfebf9d0430a17ad0b7c4822 (diff)
Transparency of Z_lt_le_dec
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@9759 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/ZArith/ZArith_dec.v')
-rw-r--r--theories/ZArith/ZArith_dec.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/theories/ZArith/ZArith_dec.v b/theories/ZArith/ZArith_dec.v
index 563b25ae4..d1f93d498 100644
--- a/theories/ZArith/ZArith_dec.v
+++ b/theories/ZArith/ZArith_dec.v
@@ -94,7 +94,7 @@ Section decidability.
elim Z_lt_ge_dec.
intros; left; assumption.
intros; right; apply Zge_le; assumption.
- Qed.
+ Defined.
Definition Z_le_gt_dec : {x <= y} + {x > y}.
Proof.