Nominal/Ex/LF.thy
author Christian Urban <urbanc@in.tum.de>
Thu, 31 Mar 2011 15:25:35 +0200
changeset 2751 3b8232f56941
parent 2617 e44551d067e6
child 2779 3c769bf10e63
permissions -rw-r--r--
final version of slides

theory LF
imports "../Nominal2"
begin

atom_decl name
atom_decl ident

nominal_datatype lf:
    kind =
      Type
    | KPi "ty" n::"name" k::"kind" bind n in k
and ty =
      TConst "ident"
    | TApp "ty" "trm"
    | TPi "ty" n::"name" ty::"ty"   bind n in ty
and trm =
      Const "ident"
    | Var "name"
    | App "trm" "trm"
    | Lam "ty" n::"name" t::"trm"  bind n in t

thm lf.distinct
thm lf.induct
thm lf.inducts
thm lf.exhaust
thm lf.strong_exhaust
thm lf.fv_defs
thm lf.bn_defs
thm lf.perm_simps
thm lf.eq_iff
thm lf.fv_bn_eqvt
thm lf.size_eqvt
thm lf.supports
thm lf.fsupp
thm lf.supp
thm lf.fresh
thm lf.fresh[simplified]



end