aboutsummaryrefslogtreecommitdiff
path: root/src/Util/ListUtil.v
diff options
context:
space:
mode:
authorGravatar Jason Gross <jasongross9@gmail.com>2016-07-22 15:33:31 -0700
committerGravatar GitHub <noreply@github.com>2016-07-22 15:33:31 -0700
commit2abb4b5ea3440d478540aad852cfe81e65596189 (patch)
tree3851f94e613e595bc99da6c932ec99e033694fa3 /src/Util/ListUtil.v
parent29bb3dd531be45ba7960b34ef759b44436e48905 (diff)
parent4519b114c66b184611068b2cc9bdad644f4a5a47 (diff)
Merge pull request #37 from JasonGross/fix-intuition
Redesign intuition, speeding up overall compilation by 20%
Diffstat (limited to 'src/Util/ListUtil.v')
-rw-r--r--src/Util/ListUtil.v7
1 files changed, 4 insertions, 3 deletions
diff --git a/src/Util/ListUtil.v b/src/Util/ListUtil.v
index 1032e1dc2..74c2b8537 100644
--- a/src/Util/ListUtil.v
+++ b/src/Util/ListUtil.v
@@ -5,6 +5,7 @@ Require Import Coq.Classes.Morphisms.
Require Import Crypto.Tactics.VerdiTactics.
Require Import Coq.Numbers.Natural.Peano.NPeano.
Require Import Crypto.Util.NatUtil.
+Require Export Crypto.Util.FixCoqMistakes.
Create HintDb distr_length discriminated.
Create HintDb simpl_set_nth discriminated.
@@ -72,14 +73,14 @@ Definition splice_nth {T} n (x:T) xs := firstn n xs ++ x :: skipn (S n) xs.
Hint Unfold splice_nth.
Ltac boring :=
- simpl; intuition;
+ simpl; intuition auto with zarith datatypes;
repeat match goal with
| [ H : _ |- _ ] => rewrite H; clear H
| [ |- appcontext[match ?pf with end] ] => solve [ case pf ]
| _ => progress autounfold in *
| _ => progress autorewrite with core
| _ => progress simpl in *
- | _ => progress intuition
+ | _ => progress intuition auto with zarith datatypes
end; eauto.
Ltac boring_list :=
@@ -1133,7 +1134,7 @@ Proof.
induction n as [|n IHn]; destruct l as [|? l]; autorewrite with simpl_sum_firstn; simpl; try omega.
{ specialize (IHn l).
destruct n; simpl; autorewrite with simpl_sum_firstn simpl_nth_default in *;
- intuition. }
+ intuition auto with zarith. }
Qed.
Hint Resolve sum_firstn_nonnegative : znonzero.