aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Numbers/NatInt/NZDomain.v
diff options
context:
space:
mode:
Diffstat (limited to 'theories/Numbers/NatInt/NZDomain.v')
-rw-r--r--theories/Numbers/NatInt/NZDomain.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/theories/Numbers/NatInt/NZDomain.v b/theories/Numbers/NatInt/NZDomain.v
index 2ab7413e3..9c01ba8cd 100644
--- a/theories/Numbers/NatInt/NZDomain.v
+++ b/theories/Numbers/NatInt/NZDomain.v
@@ -59,7 +59,7 @@ Module NZDomainProp (Import NZ:NZDomainSig').
(** We prove that any points in NZ have a common descendant by [succ] *)
-Definition common_descendant n m := exists k, exists l, (S^k) n == (S^l) m.
+Definition common_descendant n m := exists k l, (S^k) n == (S^l) m.
Instance common_descendant_wd : Proper (eq==>eq==>iff) common_descendant.
Proof.