aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Arith/Peano_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/Peano_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/Peano_dec.v')
-rw-r--r--theories/Arith/Peano_dec.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/theories/Arith/Peano_dec.v b/theories/Arith/Peano_dec.v
index 5a9e98073..42335f98b 100644
--- a/theories/Arith/Peano_dec.v
+++ b/theories/Arith/Peano_dec.v
@@ -23,7 +23,7 @@ Defined.
Theorem eq_nat_dec : forall n m, {n = m} + {n <> m}.
Proof.
- induction n; induction m; auto.
+ induction n; destruct m; auto.
elim (IHn m); auto.
Defined.