aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/NArith
diff options
context:
space:
mode:
authorGravatar emakarov <emakarov@85f007b7-540e-0410-9357-904b9bb8a0f7>2007-11-08 17:06:32 +0000
committerGravatar emakarov <emakarov@85f007b7-540e-0410-9357-904b9bb8a0f7>2007-11-08 17:06:32 +0000
commit8a51418e76da874843d6b58b6615dc12a82e2c0a (patch)
tree237cd1a934d3a24f1d954e7400e5a683476deb23 /theories/NArith
parentc08b8247aec05b34a908663aa160fdbd617b8220 (diff)
Moved several lemmas from theories/Numbers/NumPrelude to theories/Init/Logic.
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@10304 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/NArith')
-rw-r--r--theories/NArith/BinNat.v5
1 files changed, 2 insertions, 3 deletions
diff --git a/theories/NArith/BinNat.v b/theories/NArith/BinNat.v
index d2ea7617b..d0ed874dd 100644
--- a/theories/NArith/BinNat.v
+++ b/theories/NArith/BinNat.v
@@ -99,8 +99,7 @@ Notation Nplus_reg_l := (fun n m p : N => proj1 (plus_cancel_l m p n)) (only par
(** Properties of subtraction. *)
-Notation Nminus_N0_Nle :=
- (fun n m : N => (conj (proj2 (le_minus_0 n m)) (proj1 (le_minus_0 n m)))).
+Notation Nminus_N0_Nle := minus_0_le (only parsing).
Notation Nminus_0_r := minus_0_r (only parsing).
Notation Nminus_succ_r := minus_succ_r (only parsing).
@@ -117,7 +116,7 @@ Notation Nmult_comm := times_comm (only parsing).
Notation Nmult_assoc := times_assoc (only parsing).
Notation Nmult_plus_distr_r := times_plus_distr_r (only parsing).
Notation Nmult_reg_r :=
- (fun (n m p : N) (H : p <> N0) => proj1 (times_cancel_r n m p H)).
+ (fun (n m p : N) (H : p <> N0) => proj1 (times_cancel_r n m p H)) (only parsing).
(** Properties of comparison *)