Nominal/Nominal2_Base_Exec.thy
changeset 3180 7b5db6c23753
parent 3176 31372760c2fb
child 3182 5335c0ea743a
--- a/Nominal/Nominal2_Base_Exec.thy	Thu May 31 10:05:19 2012 +0100
+++ b/Nominal/Nominal2_Base_Exec.thy	Thu May 31 11:59:56 2012 +0100
@@ -796,6 +796,10 @@
   shows "p \<bullet> (if b then x else y) = (if p \<bullet> b then p \<bullet> x else p \<bullet> y)"
   by (simp add: permute_fun_def permute_bool_def)
 
+lemma Let_eqvt [eqvt]:
+  shows "p \<bullet> Let x y = Let (p \<bullet> x) (p \<bullet> y)"
+  unfolding Let_def permute_fun_app_eq ..
+
 lemma True_eqvt [eqvt]:
   shows "p \<bullet> True = True"
   unfolding permute_bool_def ..