aboutsummaryrefslogtreecommitdiff
path: root/src/Experiments/SimplyTypedArithmetic.v
diff options
context:
space:
mode:
authorGravatar Jade Philipoom <jadep@google.com>2018-03-07 12:04:48 +0100
committerGravatar jadephilipoom <jade.philipoom@gmail.com>2018-04-03 09:00:55 -0400
commite36523f6d8a34ae8b09aeb77a2533eeb15585443 (patch)
tree7a265497f3d8ce6396cd03c2272a350a06f1085e /src/Experiments/SimplyTypedArithmetic.v
parent502825d2ca27215ae92569df02f82a60c30d9769 (diff)
move some lemmas/hints to ListUtil
Diffstat (limited to 'src/Experiments/SimplyTypedArithmetic.v')
-rw-r--r--src/Experiments/SimplyTypedArithmetic.v13
1 files changed, 0 insertions, 13 deletions
diff --git a/src/Experiments/SimplyTypedArithmetic.v b/src/Experiments/SimplyTypedArithmetic.v
index c872360ba..b0855969a 100644
--- a/src/Experiments/SimplyTypedArithmetic.v
+++ b/src/Experiments/SimplyTypedArithmetic.v
@@ -962,14 +962,6 @@ Module Rows.
Hint Rewrite Positional.eval_nil Positional.eval0 @Positional.eval_snoc
Columns.eval_nil Columns.eval_snoc using (auto; solve [distr_length]) : push_eval.
- (* TODO: move to ListUtil *)
- Lemma sum_app x y : sum (x ++ y) = sum x + sum y.
- Proof. induction x; rewrite ?app_nil_l, <-?app_comm_cons, ?sum_nil, ?sum_cons; omega. Qed.
- (* TODO: move to listUtil or wherever push_map is defined *)
- Hint Rewrite @map_app : push_map.
- Hint Rewrite sum_nil sum_cons sum_app : push_sum.
- Hint Rewrite @combine_nil_r @combine_cons : push_combine.
-
Hint Resolve in_eq in_cons.
Definition eval n (inp : rows) :=
@@ -1093,11 +1085,6 @@ Module Rows.
Proof. apply eval_from_columns'_with_length. Qed.
Hint Rewrite eval_from_columns' using (auto; solve [distr_length]) : push_eval.
- (* TODO: move to ListUtil *)
- Lemma length_tl {A} ls : length (@tl A ls) = (length ls - 1)%nat.
- Proof. destruct ls; cbn [tl length]; lia. Qed.
- Hint Rewrite @length_tl : distr_length.
-
Lemma max_column_size_extract_row inp :
max_column_size (fst (extract_row inp)) = (max_column_size inp - 1)%nat.
Proof.