# HG changeset patch # User Christian Urban # Date 1265204182 -3600 # Node ID b1ca92ea3a86e5cdf55339841b3ccbae3ecd4776 # Parent 277301dc5c4c7336ebff7332b4da9d9ef6d24d91 proved that bv for lists respects alpha for terms diff -r 277301dc5c4c -r b1ca92ea3a86 Quot/Nominal/Terms.thy --- a/Quot/Nominal/Terms.thy Wed Feb 03 14:22:25 2010 +0100 +++ b/Quot/Nominal/Terms.thy Wed Feb 03 14:36:22 2010 +0100 @@ -822,6 +822,18 @@ "(alphalts ===> op =) rbv5 rbv5" sorry +lemma bv_list_rsp: + shows "t \5 s \ True" + and "x \l y \ rbv5 x = rbv5 y" +apply(induct rule: alpha5_alphalts.inducts) +apply(simp_all) +done + +lemma + shows "(alphalts ===> op =) rbv5 rbv5" + by (simp add: bv_list_rsp) + + instantiation trm5 and lts :: pt begin