Mercurial > urweb
view src/coq/Semantics.v @ 617:5b358e8f9f09
map-only syntax and semantics
author | Adam Chlipala <adamc@hcoop.net> |
---|---|
date | Sat, 21 Feb 2009 11:23:24 -0500 |
parents | d26d1f3acfd6 |
children | be88d2d169f6 |
line wrap: on
line source
(* Copyright (c) 2009, Adam Chlipala * All rights reserved. * * Redistribution and use in source and binary forms, with or without * modification, are permitted provided that the following conditions are met: * * - Redistributions of source code must retain the above copyright notice, * this list of conditions and the following disclaimer. * - Redistributions in binary form must reproduce the above copyright notice, * this list of conditions and the following disclaimer in the documentation * and/or other materials provided with the distribution. * - The names of contributors may not be used to endorse or promote products * derived from this software without specific prior written permission. * * THIS SOFTWARE IS PROVIDED BY THE COPYRIGHT HOLDERS AND CONTRIBUTORS "AS IS" * AND ANY EXPRESS OR IMPLIED WARRANTIES, INCLUDING, BUT NOT LIMITED TO, THE * IMPLIED WARRANTIES OF MERCHANTABILITY AND FITNESS FOR A PARTICULAR PURPOSE * ARE DISCLAIMED. IN NO EVENT SHALL THE COPYRIGHT OWNER OR CONTRIBUTORS BE * LIABLE FOR ANY DIRECT, INDIRECT, INCIDENTAL, SPECIAL, EXEMPLARY, OR * CONSEQUENTIAL DAMAGES (INCLUDING, BUT NOT LIMITED TO, PROCUREMENT OF * SUBSTITUTE GOODS OR SERVICES; LOSS OF USE, DATA, OR PROFITS; OR BUSINESS * INTERRUPTION) HOWEVER CAUSED AND ON ANY THEORY OF LIABILITY, WHETHER IN * CONTRACT, STRICT LIABILITY, OR TORT (INCLUDING NEGLIGENCE OR OTHERWISE) * ARISING IN ANY WAY OUT OF THE USE OF THIS SOFTWARE, EVEN IF ADVISED OF THE * POSSIBILITY OF SUCH DAMAGE. *) Require Import Axioms. Require Import Syntax. Set Implicit Arguments. Definition row (A : Type) : Type := name -> option A. Definition record (r : row Set) := forall n, match r n with | None => unit | Some T => T end. Fixpoint kDen (k : kind) : Type := match k with | KType => Set | KName => name | KArrow k1 k2 => kDen k1 -> kDen k2 | KRecord k1 => row (kDen k1) end. Fixpoint cDen k (c : con kDen k) {struct c} : kDen k := match c in con _ k return kDen k with | CVar _ x => x | Arrow c1 c2 => cDen c1 -> cDen c2 | Poly _ c1 => forall x, cDen (c1 x) | CAbs _ _ c1 => fun x => cDen (c1 x) | CApp _ _ c1 c2 => (cDen c1) (cDen c2) | Name n => n | TRecord c1 => record (cDen c1) | CEmpty _ => fun _ => None | CSingle _ c1 c2 => fun n => if name_eq_dec n (cDen c1) then Some (cDen c2) else None | CConcat _ c1 c2 => fun n => match (cDen c1) n with | None => (cDen c2) n | v => v end | CMap k1 k2 => fun f r n => match r n with | None => None | Some T => Some (f T) end | CGuarded _ _ _ _ c => cDen c end. Theorem subs_correct : forall k1 (c1 : con kDen k1) k2 (c2 : _ -> con kDen k2) c2', subs c1 c2 c2' -> cDen (c2 (cDen c1)) = cDen c2'. induction 1; simpl; intuition; try (apply ext_eq_forallS || apply ext_eq); repeat match goal with | [ H : _ |- _ ] => rewrite H end; intuition. Qed. Definition disjoint T (r1 r2 : row T) := forall n, match r1 n, r2 n with | Some _, Some _ => False | _, _ => True end. Definition dvar k (c1 c2 : con kDen (KRecord k)) := disjoint (cDen c1) (cDen c2). Scheme deq_mut := Minimality for deq Sort Prop with disj_mut := Minimality for disj Sort Prop. Theorem deq_correct : forall k (c1 c2 : con kDen k), deq dvar c1 c2 -> cDen c1 = cDen c2. Ltac t := repeat progress (simpl; intuition; subst). Ltac use_disjoint' notDone E := match goal with | [ H : disjoint _ _ |- _ ] => notDone H; generalize (H E); use_disjoint' ltac:(fun H' => match H' with | H => fail 1 | _ => notDone H' end) E | _ => idtac end. Ltac use_disjoint := use_disjoint' ltac:(fun _ => idtac). apply (deq_mut (dvar := dvar) (fun k (c1 c2 : con kDen k) => cDen c1 = cDen c2) (fun k (c1 c2 : con kDen (KRecord k)) => disjoint (cDen c1) (cDen c2))); t; repeat ((unfold row; apply ext_eq) || (match goal with | [ H : _ |- _ ] => rewrite H | [ H : subs _ _ _ |- _ ] => rewrite <- (subs_correct H) end); t); unfold disjoint; t; repeat (match goal with | [ |- context[match cDen ?C ?E with Some _ => _ | None => _ end] ] => use_disjoint E; destruct (cDen C E) | [ |- context[if name_eq_dec ?N1 ?N2 then _ else _] ] => use_disjoint N1; use_disjoint N2; destruct (name_eq_dec N1 N2) | [ _ : context[match cDen ?C ?E with Some _ => _ | None => _ end] |- _ ] => use_disjoint E; destruct (cDen C E) end; t). Qed.