aboutsummaryrefslogtreecommitdiff
path: root/src/Compilers/TestCase.v
diff options
context:
space:
mode:
Diffstat (limited to 'src/Compilers/TestCase.v')
-rw-r--r--src/Compilers/TestCase.v6
1 files changed, 3 insertions, 3 deletions
diff --git a/src/Compilers/TestCase.v b/src/Compilers/TestCase.v
index 36774e4e3..e1fb0087a 100644
--- a/src/Compilers/TestCase.v
+++ b/src/Compilers/TestCase.v
@@ -212,17 +212,17 @@ Module bounds.
Definition add_bounded_pf (x y : bounded_pf) : bounded_pf.
Proof.
exists (map_bounded_f2 plus false (proj1_sig x) (proj1_sig y)).
- simpl; abstract (destruct x, y; simpl; omega).
+ simpl; let x := x in let y := y in abstract (destruct x, y; simpl; omega).
Defined.
Definition mul_bounded_pf (x y : bounded_pf) : bounded_pf.
Proof.
exists (map_bounded_f2 mult false (proj1_sig x) (proj1_sig y)).
- simpl; abstract (destruct x, y; simpl; nia).
+ simpl; let x := x in let y := y in abstract (destruct x, y; simpl; nia).
Defined.
Definition sub_bounded_pf (x y : bounded_pf) : bounded_pf.
Proof.
exists (map_bounded_f2 minus true (proj1_sig x) (proj1_sig y)).
- simpl; abstract (destruct x, y; simpl; omega).
+ simpl; let x := x in let y := y in abstract (destruct x, y; simpl; omega).
Defined.
Definition interp_base_type_bounds (v : base_type) : Type :=
match v with