merged
authorChristian Urban <urbanc@in.tum.de>
Wed, 03 Feb 2010 14:36:48 +0100
changeset 1054 68bdd5523608
parent 1053 b1ca92ea3a86 (diff)
parent 1052 c1b469325033 (current diff)
child 1055 34220518cccf
merged
Quot/Nominal/Terms.thy
--- a/Quot/Nominal/Terms.thy	Wed Feb 03 14:28:00 2010 +0100
+++ b/Quot/Nominal/Terms.thy	Wed Feb 03 14:36:48 2010 +0100
@@ -822,6 +822,18 @@
 "(alphalts ===> op =) rbv5 rbv5"
 sorry
 
+lemma bv_list_rsp:
+  shows "t \<approx>5 s \<Longrightarrow> True"
+  and "x \<approx>l y \<Longrightarrow> 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