diff options
author | letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7> | 2003-09-28 16:37:51 +0000 |
---|---|---|
committer | letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7> | 2003-09-28 16:37:51 +0000 |
commit | d20594e78dd86d588f37dd2e0db58ec74d8fb382 (patch) | |
tree | 1d35bd98a75af3eabfe6729f31358fd8abf0f89f /theories/Arith | |
parent | 8e6d56704b9fd21a286d87c7e2871b052a15a98f (diff) |
une induction de moins dans lt_eq_lt_dec
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@4495 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Arith')
-rwxr-xr-x | theories/Arith/Compare_dec.v | 5 |
1 files changed, 2 insertions, 3 deletions
diff --git a/theories/Arith/Compare_dec.v b/theories/Arith/Compare_dec.v index 1518727e4..a7cb9bd92 100755 --- a/theories/Arith/Compare_dec.v +++ b/theories/Arith/Compare_dec.v @@ -24,10 +24,9 @@ Defined. Definition lt_eq_lt_dec : (n,m:nat){(lt n m)}+{n=m}+{(lt m n)}. Proof. -NewInduction n; NewInduction m; Auto with arith. -Elim (IHn m). +NewInduction n; Destruct m; Auto with arith. +Intros m0; Elim (IHn m0); Auto with arith. NewInduction 1; Auto with arith. -Auto with arith. Defined. Lemma gt_eq_gt_dec : (n,m:nat)({(gt m n)}+{n=m})+{(gt n m)}. |