aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Arith/Le.v
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2009-11-16 12:03:42 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2009-11-16 12:03:42 +0000
commit56c24c0c704119430ee5fde235cc8c76dc2746c3 (patch)
tree0b0b43e79cac6e0eb66f3d7d40e67f67a915d504 /theories/Arith/Le.v
parent9a5c74b8229f90b2ac1df5c41f7857cc1b0bf067 (diff)
Some lemmas about dependent choice + extensions of Compare_dec +
synonyms in Le.v, Lt.v, Gt.v. git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@12527 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Arith/Le.v')
-rw-r--r--theories/Arith/Le.v18
1 files changed, 12 insertions, 6 deletions
diff --git a/theories/Arith/Le.v b/theories/Arith/Le.v
index 1c00d7ec9..d85178dea 100644
--- a/theories/Arith/Le.v
+++ b/theories/Arith/Le.v
@@ -41,25 +41,25 @@ Hint Resolve le_trans: arith v62.
(** Comparison to 0 *)
-Theorem le_O_n : forall n, 0 <= n.
+Theorem le_0_n : forall n, 0 <= n.
Proof.
induction n; auto.
Qed.
-Theorem le_Sn_O : forall n, ~ S n <= 0.
+Theorem le_Sn_0 : forall n, ~ S n <= 0.
Proof.
red in |- *; intros n H.
change (IsSucc 0) in |- *; elim H; simpl in |- *; auto with arith.
Qed.
-Hint Resolve le_O_n le_Sn_O: arith v62.
+Hint Resolve le_0_n le_Sn_0: arith v62.
-Theorem le_n_O_eq : forall n, n <= 0 -> 0 = n.
+Theorem le_n_0_eq : forall n, n <= 0 -> 0 = n.
Proof.
induction n; auto with arith.
- intro; contradiction le_Sn_O with n.
+ intro; contradiction le_Sn_0 with n.
Qed.
-Hint Immediate le_n_O_eq: arith v62.
+Hint Immediate le_n_0_eq: arith v62.
(** [le] and successor *)
@@ -135,3 +135,9 @@ Proof.
intros m Le.
elim Le; auto with arith.
Qed.
+
+(* begin hide *)
+Notation le_O_n := le_0_n (only parsing).
+Notation le_Sn_O := le_Sn_0 (only parsing).
+Notation le_n_O_eq := le_n_0_eq (only parsing).
+(* end hide *)