From cca0eb7decb313fc22865881c6923d7e48258c69 Mon Sep 17 00:00:00 2001 From: Jason Gross Date: Tue, 1 Nov 2016 16:41:59 -0400 Subject: Move hlist to new file --- src/Util/HList.v | 33 +++++++++++++++++++++++++++++++++ 1 file changed, 33 insertions(+) create mode 100644 src/Util/HList.v (limited to 'src/Util/HList.v') diff --git a/src/Util/HList.v b/src/Util/HList.v new file mode 100644 index 000000000..addb0e40d --- /dev/null +++ b/src/Util/HList.v @@ -0,0 +1,33 @@ +Require Import Coq.Classes.Morphisms. +Require Import Coq.Relations.Relation_Definitions. +Require Import Coq.Lists.List. +Require Import Crypto.Util.Decidable. +Require Import Crypto.Util.ListUtil. +Require Import Crypto.Util.Tuple. +Require Export Crypto.Util.FixCoqMistakes. + +Fixpoint hlist' T n (f : T -> Type) : tuple' T n -> Type := + match n return tuple' _ n -> Type with + | 0 => fun T => f T + | S n' => fun Ts => (hlist' T n' f (fst Ts) * f (snd Ts))%type + end. +Global Arguments hlist' {T n} f _. + +Definition hlist {T n} (f : T -> Type) : forall (Ts : tuple T n), Type := + match n return tuple _ n -> Type with + | 0 => fun _ => unit + | S n' => @hlist' T n' f + end. + +(* tuple map *) +Fixpoint mapt' {n A F B} (f : forall x : A, F x -> B) : forall ts : tuple' A n, hlist' F ts -> tuple' B n + := match n return forall ts : tuple' A n, hlist' F ts -> tuple' B n with + | 0 => fun ts v => f _ v + | S n' => fun ts v => (@mapt' n' A F B f _ (fst v), f _ (snd v)) + end. +Definition mapt {n A F B} (f : forall x : A, F x -> B) + : forall ts : tuple A n, hlist F ts -> tuple B n + := match n return forall ts : tuple A n, hlist F ts -> tuple B n with + | 0 => fun ts v => tt + | S n' => @mapt' n' A F B f + end. -- cgit v1.2.3