From 1f21c2be76a6f84fa90669876e425ee006978899 Mon Sep 17 00:00:00 2001 From: Andres Erbsen Date: Fri, 12 Feb 2016 17:11:15 -0500 Subject: fix imports --- src/CompleteEdwardsCurve/ExtendedCoordinatesIssue.v | 2 +- 1 file changed, 1 insertion(+), 1 deletion(-) (limited to 'src/CompleteEdwardsCurve/ExtendedCoordinatesIssue.v') diff --git a/src/CompleteEdwardsCurve/ExtendedCoordinatesIssue.v b/src/CompleteEdwardsCurve/ExtendedCoordinatesIssue.v index b9baf1498..37bc8cca5 100644 --- a/src/CompleteEdwardsCurve/ExtendedCoordinatesIssue.v +++ b/src/CompleteEdwardsCurve/ExtendedCoordinatesIssue.v @@ -1,5 +1,5 @@ Require Import Crypto.ModularArithmetic.PrimeFieldTheorems. -Require Import Crypto.CompleteEdwardsCurve.Pre. +Require Import Crypto.Spec.CompleteEdwardsCurve. Section ExtendedCoordinates. Local Open Scope F_scope. -- cgit v1.2.3