added a lemma about composition and permutations
authorChristian Urban <urbanc@in.tum.de>
Sat, 12 May 2012 20:54:00 +0100
changeset 3167 c25386402f6a
parent 3166 51c475ceaf09
child 3168 a6f3e1b08494
child 3172 4cf3a4d36799
added a lemma about composition and permutations
Nominal/Nominal2_Base.thy
--- a/Nominal/Nominal2_Base.thy	Tue May 01 12:16:04 2012 +0100
+++ b/Nominal/Nominal2_Base.thy	Sat May 12 20:54:00 2012 +0100
@@ -405,6 +405,9 @@
   shows "p \<bullet> (f x) = (p \<bullet> f) (p \<bullet> x)"
   unfolding permute_fun_def by simp
 
+lemma permute_fun_comp:
+  shows "p \<bullet> f  = (permute p) o f o (permute (-p))"
+by (simp add: comp_def permute_fun_def)
 
 subsection {* Permutations for booleans *}