Nominal/Ex/Classical.thy
author Christian Urban <urbanc@in.tum.de>
Sun, 29 Aug 2010 13:36:03 +0800
changeset 2454 9ffee4eb1ae1
parent 2436 3885dc2669f9
child 2617 e44551d067e6
permissions -rw-r--r--
renamed NewParser to Nominal2

theory Classical
imports "../Nominal2"
begin

(* example from my Urban's PhD *)

atom_decl name
atom_decl coname

nominal_datatype trm =
   Ax "name" "coname"
|  Cut n::"coname" t1::"trm" c::"coname" t2::"trm"             bind n in t1, bind c in t2
|  AndR c1::"coname" t1::"trm" c2::"coname" t2::"trm" "coname" bind c1 in t1, bind c2 in t2
|  AndL1 n::"name" t::"trm" "name"                             bind n in t
|  AndL2 n::"name" t::"trm" "name"                             bind n in t
|  ImpL c::"coname" t1::"trm" n::"name" t2::"trm" "name"       bind c in t1, bind n in t2
|  ImpR c::"coname" n::"name" t::"trm" "coname"                bind n c in t

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




end