aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/NArith/BinPos.v
diff options
context:
space:
mode:
authorGravatar emakarov <emakarov@85f007b7-540e-0410-9357-904b9bb8a0f7>2007-03-14 13:23:43 +0000
committerGravatar emakarov <emakarov@85f007b7-540e-0410-9357-904b9bb8a0f7>2007-03-14 13:23:43 +0000
commita305642ea1bd5389b08f7a1d29d55a1587919bbd (patch)
treec210165e1a282ce51cfed43d938bcabc61d9c795 /theories/NArith/BinPos.v
parentbed901fd770c13c1f9825f51b4ed80c9bce280bc (diff)
Removed an unnecessary argument (p : positive) in Prect_base.
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@9701 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/NArith/BinPos.v')
-rw-r--r--theories/NArith/BinPos.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/theories/NArith/BinPos.v b/theories/NArith/BinPos.v
index 8123d8d85..dc6156d6a 100644
--- a/theories/NArith/BinPos.v
+++ b/theories/NArith/BinPos.v
@@ -578,7 +578,7 @@ trivial.
Qed.
Theorem Prect_base : forall (P:positive->Type) (a:P xH)
- (f:forall p, P p -> P (Psucc p)) (p:positive), Prect P a f xH = a.
+ (f:forall p, P p -> P (Psucc p)), Prect P a f xH = a.
Proof.
trivial.
Qed.