aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Numbers/Natural/Peano/NPeano.v
diff options
context:
space:
mode:
Diffstat (limited to 'theories/Numbers/Natural/Peano/NPeano.v')
-rw-r--r--theories/Numbers/Natural/Peano/NPeano.v6
1 files changed, 3 insertions, 3 deletions
diff --git a/theories/Numbers/Natural/Peano/NPeano.v b/theories/Numbers/Natural/Peano/NPeano.v
index ce8e03a5a..60c59b323 100644
--- a/theories/Numbers/Natural/Peano/NPeano.v
+++ b/theories/Numbers/Natural/Peano/NPeano.v
@@ -127,9 +127,9 @@ Proof.
now rewrite <- mult_n_O, minus_diag, <- !plus_n_O in U.
Qed.
-Lemma mod_upper_bound : forall x y, y<>0 -> x mod y < y.
+Lemma mod_bound_pos : forall x y, 0<=x -> 0<y -> 0 <= x mod y < y.
Proof.
- intros x y Hy.
+ intros x y Hx Hy. split. auto with arith.
destruct y; [ now elim Hy | clear Hy ].
unfold modulo.
apply le_n_S, le_minus.
@@ -515,7 +515,7 @@ Definition modulo := modulo.
Program Instance div_wd : Proper (eq==>eq==>eq) div.
Program Instance mod_wd : Proper (eq==>eq==>eq) modulo.
Definition div_mod := div_mod.
-Definition mod_upper_bound := mod_upper_bound.
+Definition mod_bound_pos := mod_bound_pos.
Definition divide := divide.
Definition gcd := gcd.