aboutsummaryrefslogtreecommitdiff
path: root/src/ModularArithmetic/ModularBaseSystem.v
diff options
context:
space:
mode:
Diffstat (limited to 'src/ModularArithmetic/ModularBaseSystem.v')
-rw-r--r--src/ModularArithmetic/ModularBaseSystem.v4
1 files changed, 2 insertions, 2 deletions
diff --git a/src/ModularArithmetic/ModularBaseSystem.v b/src/ModularArithmetic/ModularBaseSystem.v
index a48ec2536..c25f89785 100644
--- a/src/ModularArithmetic/ModularBaseSystem.v
+++ b/src/ModularArithmetic/ModularBaseSystem.v
@@ -94,11 +94,11 @@ Section Canonicalization.
Fixpoint modulus_digits' i :=
match i with
| O => max_bound i - c + 1 :: nil
- | S i' => max_bound i :: modulus_digits' i'
+ | S i' => modulus_digits' i' ++ max_bound i :: nil
end.
(* compute at compile time *)
- Definition modulus_digits := modulus_digits' (length base).
+ Definition modulus_digits := modulus_digits' (length base - 1).
Fixpoint map2 {A B C} (f : A -> B -> C) (la : list A) (lb : list B) : list C :=
match la with