Library MenhirLib.Tuples
A curryfied function with multiple parameters
A curryfied function with multiple parameters
A tuple is a heterogeneous list. For convenience, we use pairs.
Fixpoint tuple (types : list Type) : Type :=
match types with
| nil => unit
| t::q => prod t (tuple q)
end.
Fixpoint uncurry {args:list Type} {res:Type}:
arrows_left args res -> tuple args -> res :=
match args return forall res, arrows_left args res -> tuple args -> res with
| [] => fun _ f _ => f
| t::q => fun res f p => let (d, t) := p in
(@uncurry q _ f t) d
end res.
Lemma JMeq_eqrect:
forall (U:Type) (a b:U) (P:U -> Type) (x:P a) (e:a=b),
eq_rect a P x b e ~= x.
Proof.
destruct e.
reflexivity.
Qed.
match types with
| nil => unit
| t::q => prod t (tuple q)
end.
Fixpoint uncurry {args:list Type} {res:Type}:
arrows_left args res -> tuple args -> res :=
match args return forall res, arrows_left args res -> tuple args -> res with
| [] => fun _ f _ => f
| t::q => fun res f p => let (d, t) := p in
(@uncurry q _ f t) d
end res.
Lemma JMeq_eqrect:
forall (U:Type) (a b:U) (P:U -> Type) (x:P a) (e:a=b),
eq_rect a P x b e ~= x.
Proof.
destruct e.
reflexivity.
Qed.