aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Vectors/Fin.v
diff options
context:
space:
mode:
authorGravatar pboutill <pboutill@85f007b7-540e-0410-9357-904b9bb8a0f7>2011-02-10 14:11:07 +0000
committerGravatar pboutill <pboutill@85f007b7-540e-0410-9357-904b9bb8a0f7>2011-02-10 14:11:07 +0000
commitc5fa08bbecbc665e1d82d38d2e41f5256efcd545 (patch)
tree28ca895d2615fce2041a7353d06451a9b1e742e8 /theories/Vectors/Fin.v
parent22f3c77a4fbd67eb1a453bab8fcc61e6aea508ce (diff)
Interp a definition with the implicit arguments of its local context
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@13825 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Vectors/Fin.v')
-rw-r--r--theories/Vectors/Fin.v8
1 files changed, 4 insertions, 4 deletions
diff --git a/theories/Vectors/Fin.v b/theories/Vectors/Fin.v
index 97ae56e16..19b4c3b2f 100644
--- a/theories/Vectors/Fin.v
+++ b/theories/Vectors/Fin.v
@@ -57,14 +57,14 @@ Definition rect2 (P: forall {n} (a b: t n), Type)
(H1: forall n (f: t n), P F1 (FS f))
(H2: forall n (f: t n), P (FS f) F1)
(HS: forall n (f g : t n), P f g -> P (FS f) (FS g)):
- forall n (a b: t n), P n a b :=
-fix rect2_fix n (a: t n): forall (b: t n), P n a b :=
+ forall n (a b: t n), P a b :=
+fix rect2_fix n (a: t n): forall (b: t n), P a b :=
match a with
|F1 m => fun (b: t (S m)) => match b as b' in t n'
return match n' as n0
return t n0 -> Type with
|0 => fun _ => @ID
- |S n0 => fun b0 => P _ F1 b0
+ |S n0 => fun b0 => P F1 b0
end b' with
|F1 m' => H0 m'
|FS m' b' => H1 m' b'
@@ -74,7 +74,7 @@ match a with
return t n0 -> Type with
|0 => fun _ => @ID
|S n0 => fun b0 =>
- forall (a0: t n0), P _ (FS a0) b0
+ forall (a0: t n0), P (FS a0) b0
end b' with
|F1 m' => fun aa => H2 m' aa
|FS m' b' => fun aa => HS m' aa b' (rect2_fix m' aa b')