aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Vectors/Fin.v
diff options
context:
space:
mode:
Diffstat (limited to 'theories/Vectors/Fin.v')
-rw-r--r--theories/Vectors/Fin.v12
1 files changed, 3 insertions, 9 deletions
diff --git a/theories/Vectors/Fin.v b/theories/Vectors/Fin.v
index 980a5f706..d6ffef6c4 100644
--- a/theories/Vectors/Fin.v
+++ b/theories/Vectors/Fin.v
@@ -31,10 +31,7 @@ Definition case0 P (p: t 0): P p :=
Definition caseS (P: forall {n}, t (S n) -> Type)
(P1: forall n, @P n F1) (PS : forall {n} (p: t n), P (FS p))
{n} (p: t (S n)): P p :=
- match p as p0 in t n0
- return match n0 as nn return t nn -> Type with
- |0 => fun _ => @ID |S n' => fun p' => P p'
- end p0 with
+ match p with
|F1 k => P1 k
|FS k pp => PS pp
end.
@@ -43,10 +40,7 @@ Definition rectS (P: forall {n}, t (S n) -> Type)
(P1: forall n, @P n F1) (PS : forall {n} (p: t (S n)), P p -> P (FS p)):
forall {n} (p: t (S n)), P p :=
fix rectS_fix {n} (p: t (S n)): P p:=
- match p as p0 in t n0
- return match n0 as nn return t nn -> Type with
- |0 => fun _ => @ID |S n' => fun p' => P p'
- end p0 with
+ match p with
|F1 k => P1 k
|FS 0 pp => case0 (fun f => P (FS f)) pp
|FS (S k) pp => PS pp (rectS_fix pp)
@@ -187,4 +181,4 @@ induction o ; simpl.
rewrite R_sanity. rewrite IHo.
rewrite Plus.plus_assoc. destruct (to_nat o); simpl; rewrite Mult.mult_succ_r.
now rewrite (Plus.plus_comm n).
-Qed. \ No newline at end of file
+Qed.