Nominal/Ex/LetPat.thy
author Christian Urban <urbanc@in.tum.de>
Sat, 06 Nov 2010 06:18:41 +0000
changeset 2556 8ed62410236e
parent 2454 9ffee4eb1ae1
child 2648 5d9724ad543d
permissions -rw-r--r--
added a test about subtyping; disabled two tests, because of problem with function package

theory LetPat
imports "../Nominal2"
begin

declare [[STEPS = 100]]

atom_decl name

nominal_datatype trm =
  Var "name"
| App "trm" "trm"
| Lam x::"name" t::"trm"       bind (set) x in t
| Let p::"pat" "trm" t::"trm"  bind (set) "f p" in t
and pat =
  PN
| PS "name"
| PD "name" "name"
binder
  f::"pat \<Rightarrow> atom set"
where
  "f PN = {}"
| "f (PD x y) = {atom x, atom y}"
| "f (PS x) = {atom x}"

thm trm_pat.distinct
thm trm_pat.induct
thm trm_pat.exhaust
thm trm_pat.fv_defs
thm trm_pat.bn_defs
thm trm_pat.perm_simps
thm trm_pat.eq_iff
thm trm_pat.fv_bn_eqvt
thm trm_pat.size_eqvt


end