aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Arith/Lt.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/Lt.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/Lt.v')
-rwxr-xr-xtheories/Arith/Lt.v24
1 files changed, 12 insertions, 12 deletions
diff --git a/theories/Arith/Lt.v b/theories/Arith/Lt.v
index 785685093..7b5e089c3 100755
--- a/theories/Arith/Lt.v
+++ b/theories/Arith/Lt.v
@@ -50,17 +50,17 @@ Hints Resolve lt_n_n : arith v62.
Lemma S_pred : (n,m:nat)(lt m n)->(n=(S (pred n))).
Proof.
-Induction 1; Auto with arith.
+NewInduction 1; Auto with arith.
Qed.
Lemma lt_pred : (n,p:nat)(lt (S n) p)->(lt n (pred p)).
Proof.
-Induction 1; Simpl; Auto with arith.
+NewInduction 1; Simpl; Auto with arith.
Qed.
Hints Immediate lt_pred : arith v62.
Lemma lt_pred_n_n : (n:nat)(lt O n)->(lt (pred n) n).
-Destruct 1; Simpl; Auto with arith.
+NewDestruct 1; Simpl; Auto with arith.
Save.
Hints Resolve lt_pred_n_n : arith v62.
@@ -92,14 +92,14 @@ Hints Immediate lt_le_weak : arith v62.
Theorem neq_O_lt : (n:nat)(~O=n)->(lt O n).
Proof.
-Induction n; Auto with arith.
+NewInduction n; Auto with arith.
Intros; Absurd O=O; Trivial with arith.
Qed.
Hints Immediate neq_O_lt : arith v62.
Theorem lt_O_neq : (n:nat)(lt O n)->(~O=n).
Proof.
-Induction 1; Auto with arith.
+NewInduction 1; Auto with arith.
Qed.
Hints Immediate lt_O_neq : arith v62.
@@ -107,35 +107,35 @@ Hints Immediate lt_O_neq : arith v62.
Theorem lt_trans : (n,m,p:nat)(lt n m)->(lt m p)->(lt n p).
Proof.
-Induction 2; Auto with arith.
+NewInduction 2; Auto with arith.
Qed.
Theorem lt_le_trans : (n,m,p:nat)(lt n m)->(le m p)->(lt n p).
Proof.
-Induction 2; Auto with arith.
+NewInduction 2; Auto with arith.
Qed.
Theorem le_lt_trans : (n,m,p:nat)(le n m)->(lt m p)->(lt n p).
Proof.
-Induction 2; Auto with arith.
+NewInduction 2; Auto with arith.
Qed.
Hints Resolve lt_trans lt_le_trans le_lt_trans : arith v62.
Theorem le_lt_or_eq : (n,m:nat)(le n m)->((lt n m) \/ n=m).
Proof.
-Induction 1; Auto with arith.
+NewInduction 1; Auto with arith.
Qed.
Theorem le_or_lt : (n,m:nat)((le n m)\/(lt m n)).
Proof.
Intros n m; Pattern n m; Apply nat_double_ind; Auto with arith.
-Induction 1; Auto with arith.
+NewInduction 1; Auto with arith.
Qed.
Theorem le_not_lt : (n,m:nat)(le n m) -> ~(lt m n).
Proof.
-Induction 1; Auto with arith.
+NewInduction 1; Auto with arith.
Qed.
Theorem lt_not_le : (n,m:nat)(lt n m) -> ~(le m n).
@@ -146,7 +146,7 @@ Hints Immediate le_not_lt lt_not_le : arith v62.
Theorem lt_not_sym : (n,m:nat)(lt n m) -> ~(lt m n).
Proof.
-Induction 1; Auto with arith.
+NewInduction 1; Auto with arith.
Qed.
Theorem nat_total_order: (m,n: nat) ~ m = n -> (lt m n) \/ (lt n m).