aboutsummaryrefslogtreecommitdiff
path: root/src/Experiments/SpecificCurve25519.v
blob: e1b86d22927ffc3bfe6050c3f910212fafb57ab3 (plain)
1
2
3
4
5
6
7
8
9
10
11
12
13
Require Import Crypto.Util.Notations Coq.ZArith.BinInt.
Require Import Crypto.Specific.GF25519.
Require Import Crypto.CompleteEdwardsCurve.ExtendedCoordinates.
Local Infix "<<" := Z.shiftr.
Local Infix "&" := Z.land.

Section Curve25519.
  Context {twice_d : fe25519}.

  Definition ge25519_add :=
    Eval cbv beta delta [Extended.add_coordinates fe25519 add mul sub ModularBaseSystemOpt.Let_In] in
      @Extended.add_coordinates fe25519 add sub mul twice_d.
End Curve25519.