aboutsummaryrefslogtreecommitdiff
path: root/src/Experiments/NewPipeline/AbstractInterpretation.v
diff options
context:
space:
mode:
Diffstat (limited to 'src/Experiments/NewPipeline/AbstractInterpretation.v')
-rw-r--r--src/Experiments/NewPipeline/AbstractInterpretation.v4
1 files changed, 2 insertions, 2 deletions
diff --git a/src/Experiments/NewPipeline/AbstractInterpretation.v b/src/Experiments/NewPipeline/AbstractInterpretation.v
index 72a94e54c..3391c741b 100644
--- a/src/Experiments/NewPipeline/AbstractInterpretation.v
+++ b/src/Experiments/NewPipeline/AbstractInterpretation.v
@@ -52,7 +52,7 @@ Module Compilers.
end%bool.
Fixpoint is_bounded_by {t} : interp t -> binterp t -> bool
:= match t with
- | base.type.Z => fun r z => (lower r <=? z) && (z <=? upper r)
+ | base.type.Z => fun r z => ZRange.is_bounded_by_bool z r
| base.type.nat => Nat.eqb
| base.type.unit => fun _ _ => true
| base.type.bool => bool_eq
@@ -208,7 +208,7 @@ Module Compilers.
| progress cbn in *
| progress destruct_head' option
| solve [ eauto with nocore ]
- | progress cbv [is_tighter_than_bool] in *
+ | progress cbv [ZRange.is_bounded_by_bool is_tighter_than_bool] in *
| progress rewrite ?Bool.andb_true_iff in *
| discriminate
| apply conj