aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Arith/Compare_dec.v
diff options
context:
space:
mode:
authorGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2007-03-12 17:11:32 +0000
committerGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2007-03-12 17:11:32 +0000
commit0b05b8de1bcb0716e1c6b19d265027da36b1c3cc (patch)
tree84f06b33a5b0d9c24b0092b77dc88a5bced78f7e /theories/Arith/Compare_dec.v
parentba7728cc8dce5034937d208ab13c847d1ec24db8 (diff)
Proof simplification for eq_nat_dec et le_lt_dec: induction over
2nd arg m can simply be a destruct. This helps (vm_)compute __a lot__. git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@9698 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Arith/Compare_dec.v')
-rw-r--r--theories/Arith/Compare_dec.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/theories/Arith/Compare_dec.v b/theories/Arith/Compare_dec.v
index ce54239f9..8b7e2c61d 100644
--- a/theories/Arith/Compare_dec.v
+++ b/theories/Arith/Compare_dec.v
@@ -34,7 +34,7 @@ Defined.
Definition le_lt_dec n m : {n <= m} + {m < n}.
induction n.
auto with arith.
- induction m.
+ destruct m.
auto with arith.
elim (IHn m); auto with arith.
Defined.