aboutsummaryrefslogtreecommitdiff
path: root/src/ModularArithmetic/PseudoMersenneBaseParamProofs.v
diff options
context:
space:
mode:
authorGravatar jadep <jade.philipoom@gmail.com>2016-04-28 13:13:08 -0400
committerGravatar jadep <jade.philipoom@gmail.com>2016-04-28 13:13:08 -0400
commitcd07805915328fd5ee8d41b6cdd4d0340aa156aa (patch)
tree04a869de660aaa874fca7be13f9fefb86c12cafb /src/ModularArithmetic/PseudoMersenneBaseParamProofs.v
parent248282849e9b287fe817e64ccf53e09fa3991cbe (diff)
Cleanup: mostly moving lemmas to Util files, some moving lemmas to more general contexts.
Diffstat (limited to 'src/ModularArithmetic/PseudoMersenneBaseParamProofs.v')
-rw-r--r--src/ModularArithmetic/PseudoMersenneBaseParamProofs.v30
1 files changed, 0 insertions, 30 deletions
diff --git a/src/ModularArithmetic/PseudoMersenneBaseParamProofs.v b/src/ModularArithmetic/PseudoMersenneBaseParamProofs.v
index 0a58c81d2..1a7b3316e 100644
--- a/src/ModularArithmetic/PseudoMersenneBaseParamProofs.v
+++ b/src/ModularArithmetic/PseudoMersenneBaseParamProofs.v
@@ -89,26 +89,6 @@ Section PseudoMersenneBaseParamProofs.
- rewrite IHl by auto; ring.
Qed.
- (* TODO : move to LsitUtil *)
- Lemma fold_right_invariant : forall {A} P (f: A -> A -> A) l x,
- P x -> (forall y, In y l -> forall z, P z -> P (f y z)) ->
- P (fold_right f x l).
- Proof.
- induction l; intros ? ? step; auto.
- simpl.
- apply step; try apply in_eq.
- apply IHl; auto.
- intros y in_y_l.
- apply (in_cons a) in in_y_l.
- auto.
- Qed.
-
- (* TODO : move to ListUtil *)
- Lemma In_firstn : forall {T} n l (x : T), In x (firstn n l) -> In x l.
- Proof.
- induction n; destruct l; boring.
- Qed.
-
Lemma sum_firstn_limb_widths_nonneg : forall n, 0 <= sum_firstn limb_widths n.
Proof.
unfold sum_firstn; intros.
@@ -163,16 +143,6 @@ Section PseudoMersenneBaseParamProofs.
rewrite two_p_correct in nth_err_x.
congruence.
Qed.
-
-
- (* TODO : move to ZUtil *)
- Lemma mod_same_pow : forall a b c, 0 <= c <= b -> a ^ b mod a ^ c = 0.
- Proof.
- intros.
- replace b with (b - c + c) by ring.
- rewrite Z.pow_add_r by omega.
- apply Z_mod_mult.
- Qed.
Lemma base_matches_modulus: forall i j,
(i < length base)%nat ->