aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/ZArith/Zmax.v
diff options
context:
space:
mode:
authorGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2009-10-08 13:39:01 +0000
committerGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2009-10-08 13:39:01 +0000
commit93b74b4be215bd08ca7a123505177d6ec8ac7b4c (patch)
treecc5b80a8ba038a7c531afae977234f2afdc70699 /theories/ZArith/Zmax.v
parentbdec9fddcdaa13800e04e718ffa52f87bddc52d9 (diff)
Init/Tactics.v: tactic with nicer name 'exfalso' for 'elimtype False'
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@12380 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/ZArith/Zmax.v')
-rw-r--r--theories/ZArith/Zmax.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/theories/ZArith/Zmax.v b/theories/ZArith/Zmax.v
index 07eca7765..dd46e885d 100644
--- a/theories/ZArith/Zmax.v
+++ b/theories/ZArith/Zmax.v
@@ -180,7 +180,7 @@ Proof.
unfold Pminus; rewrite Pminus_mask_diag; auto.
intros; rewrite Pminus_Lt; auto.
destruct (Zmax_spec 1 (Zpos p - Zpos q)) as [(H1,H2)|(H1,H2)]; auto.
- elimtype False; clear H2.
+ exfalso; clear H2.
assert (H1':=Zlt_trans 0 1 _ Zlt_0_1 H1).
generalize (Zlt_0_minus_lt _ _ H1').
unfold Zlt; simpl.