aboutsummaryrefslogtreecommitdiff
path: root/src/ModularArithmetic
diff options
context:
space:
mode:
authorGravatar jadep <jade.philipoom@gmail.com>2016-07-11 11:42:31 -0400
committerGravatar jadep <jade.philipoom@gmail.com>2016-07-11 11:42:31 -0400
commit9a7c5b2a18ce47dbfc2bc3513f36856001499d98 (patch)
tree5571f72198a7a0f3e8d2f0d74f9e28eb83281697 /src/ModularArithmetic
parentab70b1b36bb2dca5356392cefd2c5770f2d3ebb1 (diff)
ported Specific files to use ModularBaseSystemInterface
Diffstat (limited to 'src/ModularArithmetic')
-rw-r--r--src/ModularArithmetic/ModularBaseSystemInterface.v13
1 files changed, 0 insertions, 13 deletions
diff --git a/src/ModularArithmetic/ModularBaseSystemInterface.v b/src/ModularArithmetic/ModularBaseSystemInterface.v
index 2affd9793..e4192428e 100644
--- a/src/ModularArithmetic/ModularBaseSystemInterface.v
+++ b/src/ModularArithmetic/ModularBaseSystemInterface.v
@@ -51,7 +51,6 @@ Section s.
Definition opp (x : fe) : fe := phi_inv (ModularArithmetic.opp (phi x)).
-
Lemma add_correct : forall a b,
to_list (add a b) = BaseSystem.add (to_list a) (to_list b).
Proof.
@@ -68,18 +67,6 @@ Section s.
apply ModularBaseSystemProofs.add_rep; auto using decode_rep, length_to_list.
Qed.
- Lemma optimized_group : @group fe eq add zero opp.
- Proof.
- eapply @isomorphism_to_subgroup_group; cbv [opp zero eq]; intros;
- eauto; rewrite ?phi_inv_spec; try reflexivity.
- + econstructor; eauto. admit.
- + apply (eq_dec _ _).
- + admit.
- + admit.
- + admit.
- + apply add_phi.
- Qed.
-
Lemma mul_correct : forall a b,
to_list (mul a b) = carry_mul (to_list a) (to_list b).
Proof.