aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/PArith
diff options
context:
space:
mode:
Diffstat (limited to 'theories/PArith')
-rw-r--r--theories/PArith/BinPos.v2
1 files changed, 2 insertions, 0 deletions
diff --git a/theories/PArith/BinPos.v b/theories/PArith/BinPos.v
index 4747cfe14..be5858718 100644
--- a/theories/PArith/BinPos.v
+++ b/theories/PArith/BinPos.v
@@ -1486,6 +1486,8 @@ Qed.
Include UsualMinMaxLogicalProperties <+ UsualMinMaxDecProperties.
+Ltac order := Private_Tac.order.
+
(** Minimum, maximum and constant one *)
Lemma max_1_l n : max 1 n = n.