aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/ZArith/Zminmax.v
diff options
context:
space:
mode:
Diffstat (limited to 'theories/ZArith/Zminmax.v')
-rw-r--r--theories/ZArith/Zminmax.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/theories/ZArith/Zminmax.v b/theories/ZArith/Zminmax.v
index 5fa90487b..e4d290ab2 100644
--- a/theories/ZArith/Zminmax.v
+++ b/theories/ZArith/Zminmax.v
@@ -74,7 +74,7 @@ Lemma Zmax_monotone: forall f,
Proof. intros; apply max_monotone; auto. congruence. Qed.
Lemma Zmin_case_strong : forall n m (P:Z -> Type),
- (m<=n -> P m) -> (n<=m -> P n) -> P (Zmin n m).
+ (n<=m -> P n) -> (m<=n -> P m) -> P (Zmin n m).
Proof. intros; apply min_case_strong; auto. congruence. Defined.
Lemma Zmin_case : forall n m (P:Z -> Type),