From d20594e78dd86d588f37dd2e0db58ec74d8fb382 Mon Sep 17 00:00:00 2001 From: letouzey Date: Sun, 28 Sep 2003 16:37:51 +0000 Subject: 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 --- theories/Arith/Compare_dec.v | 5 ++--- 1 file 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)}. -- cgit v1.2.3