diff -r 2f47291b6ff9 -r 9ffee4eb1ae1 Nominal/Ex/SingleLet.thy --- a/Nominal/Ex/SingleLet.thy Sun Aug 29 12:17:25 2010 +0800 +++ b/Nominal/Ex/SingleLet.thy Sun Aug 29 13:36:03 2010 +0800 @@ -1,5 +1,5 @@ theory SingleLet -imports "../NewParser" +imports "../Nominal2" begin atom_decl name @@ -38,17 +38,19 @@ - +(* lemma test: "(\p. (bs, x) \lst (op=) f p (cs, y)) \ (\p. (bs, x) \lst (op=) supp p (cs, y))" -sorry +oops lemma Abs_eq_iff: shows "Abs bs x = Abs cs y \ (\p. (bs, x) \gen (op =) supp p (cs, y))" and "Abs_res bs x = Abs_res cs y \ (\p. (bs, x) \res (op =) supp p (cs, y))" and "Abs_lst bsl x = Abs_lst csl y \ (\p. (bsl, x) \lst (op =) supp p (csl, y))" by (lifting alphas_abs) +*) +(* lemma supp_fv: "supp t = fv_trm t \ supp b = fv_bn b" apply(rule single_let.induct) @@ -73,7 +75,7 @@ apply(subst test) apply(rule refl) sorry - +*) (* consts perm_bn_trm :: "perm \ trm \ trm" consts perm_bn_assg :: "perm \ assg \ assg"