aboutsummaryrefslogtreecommitdiff
path: root/src/Curves
diff options
context:
space:
mode:
authorGravatar Andres Erbsen <andreser@mit.edu>2017-07-06 22:52:02 -0400
committerGravatar Andres Erbsen <andreser@mit.edu>2017-07-06 22:52:02 -0400
commit3c713dfaf2122c5e179d7052ff8b4681dd37fabf (patch)
tree724b780902bb533600341a9531314a385560b13f /src/Curves
parent6e55d0f4ce8be20438c42aaac8852a0aa310b295 (diff)
Curves/Edwards/Affine: prove point compression admits
Diffstat (limited to 'src/Curves')
-rw-r--r--src/Curves/Edwards/AffineProofs.v30
1 files changed, 15 insertions, 15 deletions
diff --git a/src/Curves/Edwards/AffineProofs.v b/src/Curves/Edwards/AffineProofs.v
index ec67c25b2..8fd51e8a0 100644
--- a/src/Curves/Edwards/AffineProofs.v
+++ b/src/Curves/Edwards/AffineProofs.v
@@ -150,11 +150,11 @@ Module E.
| _ => progress Option.inversion_option
end.
destruct (dec (r = 0)).
- assert (s = 0); [|solve[setoid_subst_rel Feq; trivial] ].
- admit.
- progress rewrite parity_opp in * by assumption.
- destruct (parity r), p; cbv [negb] in *; congruence.
- Admitted.
+ { assert (s = 0) by Nsatz.nsatz_power 2%nat.
+ setoid_subst_rel Feq; trivial. }
+ { progress rewrite parity_opp in * by assumption.
+ destruct (parity r), p; cbv [negb] in *; congruence. }
+ Qed.
Local Ltac t_step :=
match goal with
@@ -199,16 +199,16 @@ Module E.
Proof.
cbv [compress decompress exist_option coordinates] in *; intros.
t.
- intro.
- match goal with
- | [ H0 : _ |- False ]
- => apply (H0 f); [|congruence]
- end.
- admit.
- intro. Prod.inversion_prod; subst.
- rewrite solve_correct in y.
- eapply H. eapply y.
- Admitted.
+ { intro.
+ match goal with
+ | [ H0 : _ |- False ]
+ => apply (H0 f); [t|congruence]; clear H0
+ end.
+ rewrite solve_correct in y; Nsatz.nsatz_power 2%nat. }
+ { intro. Prod.inversion_prod; subst.
+ rewrite solve_correct in y.
+ eapply H. eapply y. }
+ Qed.
End PointCompression.
End CompleteEdwardsCurveTheorems.
Section Homomorphism.