author | Christian Urban <urbanc@in.tum.de> |
Fri, 16 Jul 2010 05:09:45 +0100 | |
changeset 2364 | 2bf351f09317 |
parent 2311 | 4da5c5c29009 |
child 2436 | 3885dc2669f9 |
permissions | -rw-r--r-- |
theory LF imports "../NewParser" begin declare [[STEPS = 9]] atom_decl name atom_decl ident nominal_datatype kind = Type | KPi "ty" n::"name" k::"kind" bind n in k and ty = TConst "ident" | TApp "ty" "trm" | TPi "ty" n::"name" t::"ty" bind n in t and trm = Const "ident" | Var "name" | App "trm" "trm" | Lam "ty" n::"name" t::"trm" bind n in t thm kind_ty_trm.supp end