aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/PArith/BinPosDef.v
diff options
context:
space:
mode:
Diffstat (limited to 'theories/PArith/BinPosDef.v')
-rw-r--r--theories/PArith/BinPosDef.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/theories/PArith/BinPosDef.v b/theories/PArith/BinPosDef.v
index 85c401cf4..a77c26e5a 100644
--- a/theories/PArith/BinPosDef.v
+++ b/theories/PArith/BinPosDef.v
@@ -608,7 +608,7 @@ Fixpoint to_little_uint p :=
| p~0 => Decimal.Little.double (to_little_uint p)
end.
-Definition to_uint p := Decimal.rev (to_little_uint p) Decimal.Nil.
+Definition to_uint p := Decimal.rev (to_little_uint p).
Definition to_int n := Decimal.Pos (to_uint n).