aboutsummaryrefslogtreecommitdiff
path: root/src/Specific
diff options
context:
space:
mode:
authorGravatar Jason Gross <jgross@mit.edu>2017-06-18 21:58:12 -0400
committerGravatar Jason Gross <jgross@mit.edu>2017-06-18 21:58:12 -0400
commita9fa48664464295560be7e4727a7efc4ed06c4eb (patch)
tree1ab4e1b1e73eb7bac448405650db7aff4b377dbe /src/Specific
parent7673940e6896e358a6ebc543fd92be89bd1e6d20 (diff)
Don't unfold MulSplit
This closes #205
Diffstat (limited to 'src/Specific')
-rw-r--r--src/Specific/MontgomeryP256.v4
-rw-r--r--src/Specific/MontgomeryP256_128.v4
2 files changed, 0 insertions, 8 deletions
diff --git a/src/Specific/MontgomeryP256.v b/src/Specific/MontgomeryP256.v
index 61a7bbf90..6e33e9321 100644
--- a/src/Specific/MontgomeryP256.v
+++ b/src/Specific/MontgomeryP256.v
@@ -22,10 +22,6 @@ Proof.
eapply (lift2_sig (fun A B c => c = (redc (r:=r)(R_numlimbs:=sz) p256 A B 1)
)); eexists.
cbv -[Definitions.Z.add_get_carry Definitions.Z.mul_split_at_bitwidth runtime_add runtime_mul Let_In].
- (* TODO: is there a better way to do this? Maybe make runtime_mul_split_at_bitwidth? *)
- cbv [Definitions.Z.mul_split_at_bitwidth].
- change Z.mul with runtime_mul; change Z.shiftr with runtime_shr; change Z.land with runtime_and.
- cbv -[Definitions.Z.add_get_carry runtime_add runtime_mul runtime_and runtime_shr Let_In]. (* unfold Z.ones *)
(*
cbv [
r wt sz p256
diff --git a/src/Specific/MontgomeryP256_128.v b/src/Specific/MontgomeryP256_128.v
index 03520302a..7699d660b 100644
--- a/src/Specific/MontgomeryP256_128.v
+++ b/src/Specific/MontgomeryP256_128.v
@@ -22,10 +22,6 @@ Proof.
eapply (lift2_sig (fun A B c => c = (redc (r:=r)(R_numlimbs:=sz) p256 A B 1)
)); eexists.
cbv -[Definitions.Z.add_get_carry Definitions.Z.mul_split_at_bitwidth runtime_add runtime_mul Let_In].
- (* TODO: is there a better way to do this? Maybe make runtime_mul_split_at_bitwidth? *)
- cbv [Definitions.Z.mul_split_at_bitwidth].
- change Z.mul with runtime_mul; change Z.shiftr with runtime_shr; change Z.land with runtime_and.
- cbv -[Definitions.Z.add_get_carry runtime_add runtime_mul runtime_and runtime_shr Let_In]. (* unfold Z.ones *)
(*
cbv [
r wt sz p256