aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Arith/Max.v
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2006-02-12 18:56:36 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2006-02-12 18:56:36 +0000
commit508603af923a1c0430b19c3cc28720a50ee90667 (patch)
tree60eeeb28610d5827ad6b64454c77b2e6312129a6 /theories/Arith/Max.v
parentcef5ba5017288534c4fb319998981bfac3dfc6ba (diff)
Unification max_case et max_case2
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@8030 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Arith/Max.v')
-rwxr-xr-xtheories/Arith/Max.v10
1 files changed, 2 insertions, 8 deletions
diff --git a/theories/Arith/Max.v b/theories/Arith/Max.v
index 37cc797e5..992bc345a 100755
--- a/theories/Arith/Max.v
+++ b/theories/Arith/Max.v
@@ -69,17 +69,11 @@ induction n; induction m; simpl in |- *; auto with arith.
elim (IHn m); intro H; elim H; auto.
Qed.
-Lemma max_case : forall n m (P:nat -> Set), P n -> P m -> P (max n m).
-Proof.
-induction n; simpl in |- *; auto with arith.
-induction m; intros; simpl in |- *; auto with arith.
-pattern (max n m) in |- *; apply IHn; auto with arith.
-Qed.
-
-Lemma max_case2 : forall n m (P:nat -> Prop), P n -> P m -> P (max n m).
+Lemma max_case : forall n m (P:nat -> Type), P n -> P m -> P (max n m).
Proof.
induction n; simpl in |- *; auto with arith.
induction m; intros; simpl in |- *; auto with arith.
pattern (max n m) in |- *; apply IHn; auto with arith.
Qed.
+Notation max_case2 := max_case (only parsing).