aboutsummaryrefslogtreecommitdiff
path: root/src/Arithmetic/PrimeFieldTheorems.v
diff options
context:
space:
mode:
authorGravatar Andres Erbsen <andreser@mit.edu>2017-06-14 00:36:23 -0400
committerGravatar Andres Erbsen <andreser@mit.edu>2017-06-14 13:05:52 -0400
commit53d6e0a991ce110864b2293eb25feca4042186eb (patch)
tree5a63e122cd2444aa12531f5f7a3bef159c7cca69 /src/Arithmetic/PrimeFieldTheorems.v
parent362eaa5da1f291b86aa04e8d745738a647ee34ce (diff)
ScalarMult: Z -> G -> G (closes #193)
Diffstat (limited to 'src/Arithmetic/PrimeFieldTheorems.v')
-rw-r--r--src/Arithmetic/PrimeFieldTheorems.v6
1 files changed, 3 insertions, 3 deletions
diff --git a/src/Arithmetic/PrimeFieldTheorems.v b/src/Arithmetic/PrimeFieldTheorems.v
index 3d6260bba..2184d20c6 100644
--- a/src/Arithmetic/PrimeFieldTheorems.v
+++ b/src/Arithmetic/PrimeFieldTheorems.v
@@ -251,9 +251,8 @@ Module F.
{phi'_opp : forall a : H, Logic.eq (phi' (opp a)) (F.opp (phi' a))}
{phi'_add : forall a b : H, Logic.eq (phi' (add a b)) (F.add (phi' a) (phi' b))}
{phi'_sub : forall a b : H, Logic.eq (phi' (sub a b)) (F.sub (phi' a) (phi' b))}
- {phi'_mul : forall a b : H, Logic.eq (phi' (mul a b)) (F.mul (phi' a) (phi' b))}
- {P:Type} {pow : H -> P -> H} {NtoP:N->P}
- {pow_is_scalarmult:ScalarMult.is_scalarmult(G:=H)(eq:=eq)(add:=mul)(zero:=one)(mul:=fun (n:nat) (k:H) => pow k (NtoP (N.of_nat n)))}.
+ {phi'_mul : forall a b : H, Logic.eq (phi' (mul a b)) (F.mul (phi' a) (phi' b))}.
+ (* TODO: revive this once we figure out how to spec the pow impl
Definition inv (x:H) := pow x (NtoP (Z.to_N (q - 2)%Z)).
Definition div x y := mul (inv y) x.
@@ -289,6 +288,7 @@ Module F.
/\ @Ring.is_homomorphism H eq one add mul (F q) Logic.eq F.one F.add F.mul phi'.
Proof using Type*. eapply @Field.field_and_homomorphism_from_redundant_representation;
assumption || exact _ || exact inv_proof || exact div_proof. Qed.
+ *)
End IsomorphicRings.
End Iso.
End F.