From d1f2e143ff56e53d6feee4158bc9f69b8d3e9ee1 Mon Sep 17 00:00:00 2001 From: letouzey Date: Thu, 17 Dec 2009 16:46:56 +0000 Subject: Reverse order of arguments in min_case_strong for better uniformity (and compatibility...) git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@12595 85f007b7-540e-0410-9357-904b9bb8a0f7 --- theories/Structures/GenericMinMax.v | 2 +- 1 file changed, 1 insertion(+), 1 deletion(-) (limited to 'theories/Structures/GenericMinMax.v') diff --git a/theories/Structures/GenericMinMax.v b/theories/Structures/GenericMinMax.v index ed9c035a1..49daacabd 100644 --- a/theories/Structures/GenericMinMax.v +++ b/theories/Structures/GenericMinMax.v @@ -303,7 +303,7 @@ Proof. intros. exact (MPRev.max_spec_le m n). Qed. Lemma min_case_strong : forall n m (P:O.t -> Type), (forall x y, x == y -> P x -> P y) -> - (m<=n -> P m) -> (n<=m -> P n) -> P (min n m). + (n<=m -> P n) -> (m<=n -> P m) -> P (min n m). Proof. intros. apply (MPRev.max_case_strong m n P); auto. Qed. Lemma min_case : forall n m (P:O.t -> Type), -- cgit v1.2.3