aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/ZArith/Zgcd_alt.v
diff options
context:
space:
mode:
Diffstat (limited to 'theories/ZArith/Zgcd_alt.v')
-rw-r--r--theories/ZArith/Zgcd_alt.v3
1 files changed, 1 insertions, 2 deletions
diff --git a/theories/ZArith/Zgcd_alt.v b/theories/ZArith/Zgcd_alt.v
index aeddeb70c..fa059313f 100644
--- a/theories/ZArith/Zgcd_alt.v
+++ b/theories/ZArith/Zgcd_alt.v
@@ -105,8 +105,7 @@ Open Scope Z_scope.
Lemma fibonacci_pos : forall n, 0 <= fibonacci n.
Proof.
- cut (forall N n, (n<N)%nat -> 0<=fibonacci n).
- eauto.
+ enough (forall N n, (n<N)%nat -> 0<=fibonacci n) by eauto.
induction N.
inversion 1.
intros.