author | Christian Urban <urbanc@in.tum.de> |
Mon, 10 May 2010 17:55:54 +0100 | |
changeset 2099 | 9454feb74b45 |
parent 2083 | 9568f9f31822 |
child 2104 | 2205b572bc9b |
permissions | -rw-r--r-- |
theory LF imports "../NewParser" begin atom_decl name atom_decl ident nominal_datatype kind = Type | KPi "ty" n::"name" k::"kind" bind_set n in k and ty = TConst "ident" | TApp "ty" "trm" | TPi "ty" n::"name" t::"ty" bind_set n in t and trm = Const "ident" | Var "name" | App "trm" "trm" | Lam "ty" n::"name" t::"trm" bind_set n in t thm kind_ty_trm.supp declare permute_kind_raw_permute_ty_raw_permute_trm_raw.simps[eqvt] declare alpha_gen_eqvt[eqvt] equivariance alpha_trm_raw end