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 9b6081176..b6b7ab7a5 100644
--- a/theories/PArith/BinPosDef.v
+++ b/theories/PArith/BinPosDef.v
@@ -338,7 +338,7 @@ Definition sqrt p := fst (sqrtrem p).
(** ** Greatest Common Divisor *)
-Definition divide p q := exists r, p*r = q.
+Definition divide p q := exists r, q = r*p.
Notation "( p | q )" := (divide p q) (at level 0) : positive_scope.
(** Instead of the Euclid algorithm, we use here the Stein binary