aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/ZArith
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-06-13 09:29:56 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-06-13 09:29:56 +0000
commitfa0e44d143e0170958b834d669f75c2fb5b65c4c (patch)
tree507814b67788f8964051de33a9bc8aba70ac8a76 /theories/ZArith
parenta50ea4f8a88a438f38b41e744d00a5ee87b95793 (diff)
Deplacement d'un lemme sur nat de ZArith vers Arith
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@4146 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/ZArith')
-rw-r--r--theories/ZArith/fast_integer.v11
1 files changed, 0 insertions, 11 deletions
diff --git a/theories/ZArith/fast_integer.v b/theories/ZArith/fast_integer.v
index cb33104e4..4026ba222 100644
--- a/theories/ZArith/fast_integer.v
+++ b/theories/ZArith/fast_integer.v
@@ -1095,17 +1095,6 @@ Do 2 Rewrite convert_add; Do 2 Rewrite times_convert;
Do 3 Rewrite (mult_sym (convert x)); Apply mult_plus_distr.
Qed.
-Theorem lt_mult_left :
- (x,y,z:nat) (lt x y) -> (lt (mult (S z) x) (mult (S z) y)).
-Proof.
-Intros x y z H;Elim z; [
- Simpl; Do 2 Rewrite <- plus_n_O; Assumption
-| Simpl; Intros n H1; Apply lt_trans with m:=(plus y (plus x (mult n x))); [
- Rewrite (plus_sym x (plus x (mult n x)));
- Rewrite (plus_sym y (plus x (mult n x))); Apply lt_reg_l; Assumption
- | Apply lt_reg_l;Assumption ]].
-Qed.
-
Theorem times_true_sub_distr:
(x,y,z:positive) (compare y z EGAL) = SUPERIEUR ->
(times x (true_sub y z)) = (true_sub (times x y) (times x z)).