From 7488682db4cf259e0bb0c886e13301c32a2eeaa2 Mon Sep 17 00:00:00 2001 From: Jason Gross Date: Fri, 2 Jun 2017 00:01:35 -0400 Subject: Don't rely on autogenerated names This fixes all of the private-names warnings emitted by compiling fiat-crypto with https://github.com/coq/coq/pull/268 (minus the ones in coqprime, which I didn't touch). --- src/Curves/Edwards/AffineProofs.v | 7 +++++-- 1 file changed, 5 insertions(+), 2 deletions(-) (limited to 'src/Curves/Edwards/AffineProofs.v') diff --git a/src/Curves/Edwards/AffineProofs.v b/src/Curves/Edwards/AffineProofs.v index e77e39f50..8e69b78fe 100644 --- a/src/Curves/Edwards/AffineProofs.v +++ b/src/Curves/Edwards/AffineProofs.v @@ -44,7 +44,7 @@ Module E. Local Notation mul := (E.mul(nonzero_a:=nonzero_a)(square_a:=square_a)(nonsquare_d:=nonsquare_d)). Program Definition opp (P:point) : point := (Fopp (fst P), (snd P)). - Next Obligation. destruct P as [ [??]?]; cbv; fsatz. Qed. + Next Obligation. match goal with P : point |- _ => destruct P as [ [??]?] end; cbv; fsatz. Qed. Ltac t_step := match goal with @@ -203,7 +203,10 @@ Module E. cbv [compress decompress exist_option coordinates] in *; intros. t. intro. - apply (H0 f); [|congruence]. + match goal with + | [ H0 : _ |- False ] + => apply (H0 f); [|congruence] + end. admit. intro. Prod.inversion_prod; subst. rewrite solve_correct in y. -- cgit v1.2.3