Mercurial > cpdt > repo
view src/DepList.v @ 162:df02642f93b8
Evaluation contexts ahoy
author | Adam Chlipala <adamc@hcoop.net> |
---|---|
date | Tue, 04 Nov 2008 12:39:28 -0500 |
parents | e70fbfc56c46 |
children | ba306bf9ec80 |
line wrap: on
line source
(* Copyright (c) 2008, Adam Chlipala * * This work is licensed under a * Creative Commons Attribution-Noncommercial-No Derivative Works 3.0 * Unported License. * The license text is available at: * http://creativecommons.org/licenses/by-nc-nd/3.0/ *) (* Dependent list types presented in Chapter 8 *) Require Import Arith List. Set Implicit Arguments. Section ilist. Variable A : Type. Fixpoint ilist (n : nat) : Type := match n with | O => unit | S n' => A * ilist n' end%type. Definition inil : ilist O := tt. Definition icons n x (ls : ilist n) : ilist (S n) := (x, ls). Definition hd n (ls : ilist (S n)) : A := fst ls. Definition tl n (ls : ilist (S n)) : ilist n := snd ls. Implicit Arguments icons [n]. Fixpoint index (n : nat) : Type := match n with | O => Empty_set | S n' => option (index n') end. Fixpoint get (n : nat) : ilist n -> index n -> A := match n return ilist n -> index n -> A with | O => fun _ idx => match idx with end | S n' => fun ls idx => match idx with | None => fst ls | Some idx' => get n' (snd ls) idx' end end. Section everywhere. Variable x : A. Fixpoint everywhere (n : nat) : ilist n := match n return ilist n with | O => inil | S n' => icons x (everywhere n') end. End everywhere. Section singleton. Variables x default : A. Fixpoint singleton (n m : nat) {struct n} : ilist n := match n return ilist n with | O => inil | S n' => match m with | O => icons x (everywhere default n') | S m' => icons default (singleton n' m') end end. End singleton. Section map2. Variable f : A -> A -> A. Fixpoint map2 (n : nat) : ilist n -> ilist n -> ilist n := match n return ilist n -> ilist n -> ilist n with | O => fun _ _ => inil | S n' => fun ls1 ls2 => icons (f (hd ls1) (hd ls2)) (map2 _ (tl ls1) (tl ls2)) end. End map2. End ilist. Implicit Arguments icons [A n]. Implicit Arguments get [A n]. Implicit Arguments map2 [A n]. Section hlist. Variable A : Type. Variable B : A -> Type. Fixpoint hlist (ls : list A) : Type := match ls with | nil => unit | x :: ls' => B x * hlist ls' end%type. Definition hnil : hlist nil := tt. Definition hcons (x : A) (ls : list A) (v : B x) (hls : hlist ls) : hlist (x :: ls) := (v, hls). Variable elm : A. Fixpoint member (ls : list A) : Type := match ls with | nil => Empty_set | x :: ls' => (x = elm) + member ls' end%type. Definition hfirst (x : A) (ls : list A) (pf : x = elm) : member (x :: ls) := inl _ pf. Definition hnext (x : A) (ls : list A) (m : member ls) : member (x :: ls) := inr _ m. Fixpoint hget (ls : list A) : hlist ls -> member ls -> B elm := match ls return hlist ls -> member ls -> B elm with | nil => fun _ idx => match idx with end | _ :: ls' => fun mls idx => match idx with | inl pf => match pf with | refl_equal => fst mls end | inr idx' => hget ls' (snd mls) idx' end end. Fixpoint happ (ls1 ls2 : list A) {struct ls1} : hlist ls1 -> hlist ls2 -> hlist (ls1 ++ ls2) := match ls1 return hlist ls1 -> hlist ls2 -> hlist (ls1 ++ ls2) with | nil => fun _ hls2 => hls2 | _ :: _ => fun hls1 hls2 => (fst hls1, happ _ _ (snd hls1) hls2) end. End hlist. Implicit Arguments hnil [A B]. Implicit Arguments hcons [A B x ls]. Implicit Arguments hget [A B elm ls]. Implicit Arguments happ [A B ls1 ls2]. Implicit Arguments hfirst [A elm x ls]. Implicit Arguments hnext [A elm x ls]. Infix ":::" := hcons (right associativity, at level 60). Infix "+++" := happ (right associativity, at level 60).