author | Cezary Kaliszyk <kaliszyk@in.tum.de> |
Thu, 26 Aug 2010 14:55:15 +0900 | |
changeset 2437 | 319f469b8b67 |
parent 2436 | 3885dc2669f9 |
child 2440 | 0a36825b16c1 |
permissions | -rw-r--r-- |
theory TypeVarsTest imports "../NewParser" begin atom_decl name declare [[STEPS = 21]] class s1 class s2 nominal_datatype ('a, 'b) lam = Var "name" | App "('a::s1, 'b::s2) lam" "('a, 'b) lam" | Lam x::"name" l::"('a, 'b) lam" bind x in l thm lam.distinct thm lam.induct thm lam.exhaust thm lam.fv_defs thm lam.bn_defs thm lam.perm_simps thm lam.eq_iff thm lam.fv_bn_eqvt thm lam.size_eqvt end