aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Arith/Compare_dec.v
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2001-08-05 19:04:16 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2001-08-05 19:04:16 +0000
commit83c56744d7e232abeb5f23e6d0f23cd0abc14a9c (patch)
tree6d7d4c2ce3bb159b8f81a4193abde1e3573c28d4 /theories/Arith/Compare_dec.v
parentf7351ff222bad0cc906dbee3c06b20babf920100 (diff)
Expérimentation de NewDestruct et parfois NewInduction
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@1880 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Arith/Compare_dec.v')
-rwxr-xr-xtheories/Arith/Compare_dec.v14
1 files changed, 7 insertions, 7 deletions
diff --git a/theories/Arith/Compare_dec.v b/theories/Arith/Compare_dec.v
index 1397326b2..531e0a975 100755
--- a/theories/Arith/Compare_dec.v
+++ b/theories/Arith/Compare_dec.v
@@ -14,14 +14,14 @@ Require Gt.
Require Decidable.
Theorem zerop : (n:nat){n=O}+{lt O n}.
-Destruct n; Auto with arith.
+NewDestruct n; Auto with arith.
Save.
Theorem lt_eq_lt_dec : (n,m:nat){(lt n m)}+{n=m}+{(lt m n)}.
Proof.
-Induction n; Induction m; Auto with arith.
-Intros q H'; Elim (H q).
-Induction 1; Auto with arith.
+NewInduction n; NewInduction m; Auto with arith.
+Elim (IHn m).
+NewInduction 1; Auto with arith.
Auto with arith.
Qed.
@@ -30,11 +30,11 @@ Proof lt_eq_lt_dec.
Lemma le_lt_dec : (n,m:nat) {le n m} + {lt m n}.
Proof.
-Induction n.
+NewInduction n.
Auto with arith.
-Induction m.
+NewInduction m.
Auto with arith.
-Intros q H'; Elim (H q); Auto with arith.
+Elim (IHn m); Auto with arith.
Qed.
Lemma le_le_S_dec : (n,m:nat) {le n m} + {le (S m) n}.