aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Arith/Max.v
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2009-10-03 12:05:59 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2009-10-03 12:05:59 +0000
commit60622d207ebbeffb8e0c3d7861858e8ca9819e6e (patch)
tree8c75e9450007945cd162b821f06a72d60253b093 /theories/Arith/Max.v
parent32222d67e21922966a49dccff81f99dd7ef5ec05 (diff)
A few additions in Min.v.
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@12368 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Arith/Max.v')
-rw-r--r--theories/Arith/Max.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/theories/Arith/Max.v b/theories/Arith/Max.v
index dcc973a96..c7e81505c 100644
--- a/theories/Arith/Max.v
+++ b/theories/Arith/Max.v
@@ -12,7 +12,7 @@ Require Import Le Plus.
Open Local Scope nat_scope.
-Implicit Types m n : nat.
+Implicit Types m n p : nat.
(** * Maximum of two natural numbers *)