aboutsummaryrefslogtreecommitdiff
path: root/src/Curves/Edwards
diff options
context:
space:
mode:
authorGravatar Maxime Dénès <mail@maximedenes.fr>2018-10-02 14:57:42 +0200
committerGravatar Jason Gross <jasongross9@gmail.com>2018-10-02 13:57:55 -0400
commitca7dc4f5c6cb59d79e79405572fbb957dd3832ce (patch)
tree81f2f074628905aca7fab294167d32256e3754ee /src/Curves/Edwards
parent94755f0b90af855aa7bf265b37ed101ba95b1103 (diff)
Adapt to Coq's PR#8555
Diffstat (limited to 'src/Curves/Edwards')
-rw-r--r--src/Curves/Edwards/AffineProofs.v12
1 files changed, 6 insertions, 6 deletions
diff --git a/src/Curves/Edwards/AffineProofs.v b/src/Curves/Edwards/AffineProofs.v
index 8fd51e8a0..346567193 100644
--- a/src/Curves/Edwards/AffineProofs.v
+++ b/src/Curves/Edwards/AffineProofs.v
@@ -156,7 +156,7 @@ Module E.
destruct (parity r), p; cbv [negb] in *; congruence. }
Qed.
- Local Ltac t_step :=
+ Local Ltac t'_step :=
match goal with
| _ => progress subst
| _ => progress destruct_head' @E.point
@@ -173,7 +173,7 @@ Module E.
| H:_ |- _ => unique pose proof (exist_option_None _ _ _ H); clear H
| _ => solve [trivial | eapply solve_correct; fsatz]
end.
- Local Ltac t := repeat t_step.
+ Local Ltac t' := repeat t'_step.
Program Definition decompress (b:bool*F) : option point :=
exist_option _
@@ -188,21 +188,21 @@ Module E.
end
end
end _.
- Next Obligation. t. Qed.
+ Next Obligation. t'. Qed.
Lemma decompress_Some b P (H:Logic.eq (decompress b) (Some P))
: Logic.eq (compress P) b.
- Proof using Type. cbv [compress decompress] in *; t. Qed.
+ Proof using Type. cbv [compress decompress] in *; t'. Qed.
Lemma decompress_None b (H:Logic.eq (decompress b) None)
: forall P, not (Logic.eq (compress P) b).
Proof.
cbv [compress decompress exist_option coordinates] in *; intros.
- t.
+ t'.
{ intro.
match goal with
| [ H0 : _ |- False ]
- => apply (H0 f); [t|congruence]; clear H0
+ => apply (H0 f); [t'|congruence]; clear H0
end.
rewrite solve_correct in y; Nsatz.nsatz_power 2%nat. }
{ intro. Prod.inversion_prod; subst.