aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Arith/Max.v
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2009-01-01 09:16:30 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2009-01-01 09:16:30 +0000
commit88770a6a1814eb57a161188cda1f4b9ae639c252 (patch)
treea18052a60b0aa331c132d2bc130dabf35234c7da /theories/Arith/Max.v
parent0d03f17a33b43aa87bb201953e4e1a567aac6355 (diff)
- Fixed bug #2021 (uncaught exception with injection/discriminate when
the inductive status of a projectable position comes from a dependency). - Improved doc of the stdlib chapter (see bug #2018), and fixed tex bugs introduced in r11725. - Applied wish #2012 (max_dec transparent). git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@11728 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Arith/Max.v')
-rw-r--r--theories/Arith/Max.v4
1 files changed, 2 insertions, 2 deletions
diff --git a/theories/Arith/Max.v b/theories/Arith/Max.v
index 75e1cdf0c..52beecb74 100644
--- a/theories/Arith/Max.v
+++ b/theories/Arith/Max.v
@@ -74,13 +74,13 @@ Lemma max_dec : forall n m, {max n m = n} + {max n m = m}.
Proof.
induction n; induction m; simpl in |- *; auto with arith.
elim (IHn m); intro H; elim H; auto.
-Qed.
+Defined.
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.
+Defined.
Notation max_case2 := max_case (only parsing).