aboutsummaryrefslogtreecommitdiff
path: root/theories/Numbers/Cyclic/Int63/Cyclic63.v
diff options
context:
space:
mode:
Diffstat (limited to 'theories/Numbers/Cyclic/Int63/Cyclic63.v')
-rw-r--r--theories/Numbers/Cyclic/Int63/Cyclic63.v1
1 files changed, 0 insertions, 1 deletions
diff --git a/theories/Numbers/Cyclic/Int63/Cyclic63.v b/theories/Numbers/Cyclic/Int63/Cyclic63.v
index 2a26b6b12a..4bf971668d 100644
--- a/theories/Numbers/Cyclic/Int63/Cyclic63.v
+++ b/theories/Numbers/Cyclic/Int63/Cyclic63.v
@@ -218,7 +218,6 @@ Lemma div_lt : forall p x y, 0 <= x < y -> x / 2^p < y.
apply Zdiv_lt_upper_bound;auto with zarith.
apply Z.lt_le_trans with y;auto with zarith.
rewrite <- (Zmult_1_r y);apply Zmult_le_compat;auto with zarith.
- assert (0 < 2^p);auto with zarith.
replace (2^p) with 0.
destruct x;change (0<y);auto with zarith.
destruct p;trivial;discriminate.