aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/PArith
diff options
context:
space:
mode:
authorGravatar Pierre Letouzey <pierre.letouzey@inria.fr>2017-03-07 09:16:16 +0100
committerGravatar Jason Gross <jgross@mit.edu>2018-02-20 19:12:35 -0500
commitc1d4048a12441df2977965b186bae9dcd32d4129 (patch)
treecff7fca9f6199a231fb4651de677862d0a88e0dc /theories/PArith
parent960d48790121b876e6be7ca033138f5d28eae0cb (diff)
Decimal: proofs that conversions from/to nat,N,Z are bijections
Diffstat (limited to 'theories/PArith')
-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).