aboutsummaryrefslogtreecommitdiffstats
path: root/src/bva/BVList.v
diff options
context:
space:
mode:
Diffstat (limited to 'src/bva/BVList.v')
-rw-r--r--src/bva/BVList.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/src/bva/BVList.v b/src/bva/BVList.v
index 261f660..dc8660c 100644
--- a/src/bva/BVList.v
+++ b/src/bva/BVList.v
@@ -668,7 +668,7 @@ Fixpoint mult_bool_step_k_h (a b: list bool) (c: bool) (k: Z) : list bool :=
Local Open Scope int63_scope.
Fixpoint top_k_bools (a: list bool) (k: int) : list bool :=
- if (k == 0) then nil
+ if (k =? 0) then nil
else match a with
| nil => nil
| ai :: a' => ai :: top_k_bools a' (k - 1)