aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Arith/Le.v
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-11-12 19:20:11 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-11-12 19:20:11 +0000
commitce0730a894791ea19a2ac372a63c94a141102cf8 (patch)
tree3be1228b7d92f7be7e600f29aad3b2e33f0da37a /theories/Arith/Le.v
parentd56cb8c2382bc0c109e84d46bff9762275da38a5 (diff)
Cosmetique
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@4878 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Arith/Le.v')
-rwxr-xr-xtheories/Arith/Le.v9
1 files changed, 8 insertions, 1 deletions
diff --git a/theories/Arith/Le.v b/theories/Arith/Le.v
index 71b020e6a..c80689836 100755
--- a/theories/Arith/Le.v
+++ b/theories/Arith/Le.v
@@ -14,6 +14,13 @@ Open Local Scope nat_scope.
Implicit Variables Type m,n,p:nat.
+(** Reflexivity *)
+
+Theorem le_refl : (n:nat)(le n n).
+Proof.
+Exact le_n.
+Qed.
+
(** Transitivity *)
Theorem le_trans : (n,m,p:nat)(le n m)->(le m p)->(le n p).
@@ -60,7 +67,7 @@ Elim H ; Simpl ; Auto with arith.
Qed.
Hints Immediate le_S_n : arith v62.
-Lemma le_pred : (n,m:nat)(le n m)->(le (pred n) (pred m)).
+Theorem le_pred : (n,m:nat)(le n m)->(le (pred n) (pred m)).
Proof.
NewInduction n as [|n IHn]. Simpl. Auto with arith.
NewDestruct m as [|m]. Simpl. Intro H. Inversion H.