aboutsummaryrefslogtreecommitdiff
path: root/src/BaseSystemProofs.v
diff options
context:
space:
mode:
authorGravatar Jason Gross <jagro@google.com>2016-07-18 13:32:06 -0700
committerGravatar Jason Gross <jagro@google.com>2016-07-18 13:32:06 -0700
commit19dbf8eb3fd57262c6c66677f71e7a6617e0df9d (patch)
tree4391f972c5d36aff777775968ed2aea8e1c47f7b /src/BaseSystemProofs.v
parent45474c87340288731ba0783325278406bec0c147 (diff)
Add more distr_length proofs in BaseSystemProofs
Diffstat (limited to 'src/BaseSystemProofs.v')
-rw-r--r--src/BaseSystemProofs.v50
1 files changed, 40 insertions, 10 deletions
diff --git a/src/BaseSystemProofs.v b/src/BaseSystemProofs.v
index eb7f31ba6..8bd390635 100644
--- a/src/BaseSystemProofs.v
+++ b/src/BaseSystemProofs.v
@@ -1,7 +1,7 @@
-Require Import List.
-Require Import Util.ListUtil Util.CaseUtil Util.ZUtil.
-Require Import ZArith.ZArith ZArith.Zdiv.
-Require Import Omega NPeano Arith.
+Require Import Coq.Lists.List.
+Require Import Crypto.Util.ListUtil Crypto.Util.CaseUtil Crypto.Util.ZUtil.
+Require Import Coq.ZArith.ZArith Coq.ZArith.Zdiv.
+Require Import Coq.omega.Omega Coq.Numbers.Natural.Peano.NPeano Coq.Arith.Arith.
Require Import Crypto.BaseSystem.
Require Import Crypto.Util.Notations.
Local Open Scope Z.
@@ -532,9 +532,13 @@ Section BaseSystemProofs.
induction us; destruct vs; boring.
Qed.
- Lemma mul'_length_exact: forall us vs,
- (length us <= length vs)%nat -> us <> nil ->
- (length (mul' us vs) = pred (length us + length vs))%nat.
+ Hint Rewrite add_length_exact : distr_length.
+
+ Lemma mul'_length_exact_full: forall us vs,
+ (length (mul' us vs) = match length us with
+ | 0 => 0%nat
+ | _ => pred (length us + length vs)
+ end)%nat.
Proof.
induction us; intros; try solve [boring].
unfold mul'; fold mul'.
@@ -544,9 +548,33 @@ Section BaseSystemProofs.
+ rewrite Max.max_0_r. simpl; omega.
+ rewrite Max.max_l; [ omega | ].
rewrite IHus by ( congruence || simpl in *; omega).
- omega.
+ simpl; omega.
+ Qed.
+
+ Hint Rewrite mul'_length_exact_full : distr_length.
+
+ (* TODO(@jadephilipoom, from jgross): one of these conditions isn't
+ needed. Should it be dropped, or was there a reason to keep it? *)
+ Lemma mul'_length_exact: forall us vs,
+ (length us <= length vs)%nat -> us <> nil ->
+ (length (mul' us vs) = pred (length us + length vs))%nat.
+ Proof.
+ intros; rewrite mul'_length_exact_full; destruct us; simpl; congruence.
+ Qed.
+
+ Lemma mul_length_exact_full: forall us vs,
+ (length (mul us vs) = match length us with
+ | 0 => 0
+ | _ => pred (length us + length vs)
+ end)%nat.
+ Proof.
+ intros; unfold mul; autorewrite with distr_length; reflexivity.
Qed.
+ Hint Rewrite mul_length_exact_full : distr_length.
+
+ (* TODO(@jadephilipoom, from jgross): one of these conditions isn't
+ needed. Should it be dropped, or was there a reason to keep it? *)
Lemma mul_length_exact: forall us vs,
(length us <= length vs)%nat -> us <> nil ->
(length (mul us vs) = pred (length us + length vs))%nat.
@@ -559,7 +587,7 @@ Section BaseSystemProofs.
reflexivity.
Qed.
Definition encode'_zero z max : encode' base z max 0%nat = nil := eq_refl.
- Definition encode'_succ z max i : encode' base z max (S i) =
+ Definition encode'_succ z max i : encode' base z max (S i) =
encode' base z max i ++ ((z mod (nth_default max base (S i))) / (nth_default max base i)) :: nil := eq_refl.
Opaque encode'.
Hint Resolve encode'_zero encode'_succ.
@@ -606,4 +634,6 @@ Section BaseSystemProofs.
apply Z.mod_small; omega.
Qed.
-End BaseSystemProofs. \ No newline at end of file
+End BaseSystemProofs.
+
+Hint Rewrite @add_length_exact @mul'_length_exact_full @mul_length_exact_full @encode'_length @sub_length : distr_length.