aboutsummaryrefslogtreecommitdiff
path: root/src/Util/ListUtil.v
diff options
context:
space:
mode:
authorGravatar Jason Gross <jagro@google.com>2016-07-06 11:42:35 -0700
committerGravatar Jason Gross <jagro@google.com>2016-07-06 11:42:35 -0700
commit930c791bd99a13e211098627109e240ecd0b815d (patch)
tree57703e179fdaf80eec0fb1b3bad0dd53d8419ff2 /src/Util/ListUtil.v
parent9bf4094f3a9cba14c9106a2fb49c121540c1372e (diff)
Fix for broken 8.5 build in ListUtil
Diffstat (limited to 'src/Util/ListUtil.v')
-rw-r--r--src/Util/ListUtil.v11
1 files changed, 6 insertions, 5 deletions
diff --git a/src/Util/ListUtil.v b/src/Util/ListUtil.v
index ed20cd15c..060372341 100644
--- a/src/Util/ListUtil.v
+++ b/src/Util/ListUtil.v
@@ -2,6 +2,7 @@ Require Import Coq.Lists.List.
Require Import Coq.omega.Omega.
Require Import Coq.Arith.Peano_dec.
Require Import Crypto.Tactics.VerdiTactics.
+Require Import Coq.Numbers.Natural.Peano.NPeano.
Definition sum_firstn l n := fold_right Z.add 0%Z (firstn n l).
@@ -686,15 +687,15 @@ Lemma sum_firstn_succ : forall l i x,
Proof.
unfold sum_firstn; induction l;
[intros; rewrite (@nth_error_nil_error Z) in *; congruence | ].
- intros ? x nth_err_x; destruct (NPeano.Nat.eq_dec i 0).
+ intros ? x nth_err_x; destruct (Nat.eq_dec i 0).
+ subst; simpl in *; unfold value in *.
congruence.
- + rewrite <- (NPeano.Nat.succ_pred i) at 2 by auto.
- rewrite <- (NPeano.Nat.succ_pred i) in nth_err_x by auto.
+ + rewrite <- (Nat.succ_pred i) at 2 by auto.
+ rewrite <- (Nat.succ_pred i) in nth_err_x by auto.
simpl. simpl in nth_err_x.
specialize (IHl (pred i) x).
- rewrite NPeano.Nat.succ_pred in IHl by auto.
- destruct (NPeano.Nat.eq_dec (pred i) 0).
+ rewrite Nat.succ_pred in IHl by auto.
+ destruct (Nat.eq_dec (pred i) 0).
- replace i with 1%nat in * by omega.
simpl. replace (pred 1) with 0%nat in * by auto.
apply nth_error_exists_first in nth_err_x.