From cdd5ffb086eb647eabe640c81de9d8af7cd0a1dd Mon Sep 17 00:00:00 2001 From: Jason Gross Date: Thu, 17 Jan 2019 15:07:47 -0500 Subject: Split up PushButtonSynthesis.v Closes #497 --- src/SlowPrimeSynthesisExamples.v | 2 +- 1 file changed, 1 insertion(+), 1 deletion(-) (limited to 'src/SlowPrimeSynthesisExamples.v') diff --git a/src/SlowPrimeSynthesisExamples.v b/src/SlowPrimeSynthesisExamples.v index 8da9e8776..74feb7b40 100644 --- a/src/SlowPrimeSynthesisExamples.v +++ b/src/SlowPrimeSynthesisExamples.v @@ -3,7 +3,7 @@ Require Import Coq.Strings.String. Require Import Coq.derive.Derive. Require Import Coq.Lists.List. Require Import Crypto.Arithmetic. -Require Import Crypto.PushButtonSynthesis. +Require Import Crypto.PushButtonSynthesis.UnsaturatedSolinas. Require Import Crypto.CStringification. Require Import Crypto.Util.Notations. -- cgit v1.2.3