aboutsummaryrefslogtreecommitdiff
path: root/src
diff options
context:
space:
mode:
authorGravatar Jason Gross <jgross@mit.edu>2016-11-10 13:23:30 -0500
committerGravatar Jason Gross <jgross@mit.edu>2016-11-10 13:23:40 -0500
commitf6f124ca138d49e88c8b7b9ee5d3777e374760c1 (patch)
tree749fa9d35595a8e2371ffbd34bec049ae3866446 /src
parentd82fad78d2c09f75a5fadaded2dd3bd056288739 (diff)
More proof fixes
Diffstat (limited to 'src')
-rw-r--r--src/Reflection/Z/Interpretations.v13
1 files changed, 6 insertions, 7 deletions
diff --git a/src/Reflection/Z/Interpretations.v b/src/Reflection/Z/Interpretations.v
index c418a2926..8a31b3947 100644
--- a/src/Reflection/Z/Interpretations.v
+++ b/src/Reflection/Z/Interpretations.v
@@ -237,8 +237,10 @@ Module Word64.
apply Z.log2_lt_pow2; assumption.
Qed.
- Lemma word64ToZ_land : bounds_2statement land Z.land. Proof. w64ToZ_t. Qed.
- Lemma word64ToZ_lor : bounds_2statement lor Z.lor. Proof. w64ToZ_t. Qed.
+ Lemma word64ToZ_land : bounds_2statement land Z.land.
+ Proof. w64ToZ_t. Qed.
+ Lemma word64ToZ_lor : bounds_2statement lor Z.lor.
+ Proof. w64ToZ_t. Qed.
Lemma word64ToZ_neg : bounds_2statement neg ModularBaseSystemListZOperations.neg.
Proof. w64ToZ_t; w64ToZ_extra_t. Qed.
Lemma word64ToZ_cmovne : bounds_4statement cmovne ModularBaseSystemListZOperations.cmovne.
@@ -677,9 +679,6 @@ Module BoundedWord64.
=> apply (Z.max_case_strong x y)
end ].
- Ltac ktrans k := do k (etransitivity; [|eassumption]); assumption.
- Ltac trans' := first [ assumption | ktrans ltac:(1) | ktrans ltac:(2) ].
-
(** TODO(jadep): Use the bounds lemma here to prove that if each
component of [ret_val] is [Some (l, v, u)], then we can fill in
[pf] and return the tuple of [{| lower := l ; value := v ; upper
@@ -813,13 +812,13 @@ Module BoundedWord64.
Proof.
refine (t_map2 Word64.land ZBounds.land _);
abstract (t_prestart; eapply land_valid_update; eauto).
- Qed.
+ Defined.
Definition lor : t -> t -> t.
Proof.
refine (t_map2 Word64.lor ZBounds.lor _);
abstract (t_prestart; eapply lor_valid_update; eauto).
- Qed.
+ Defined.
Definition shl : t -> t -> t.
Proof.