Nominal/Ex/Foo1.thy
changeset 2560 82e37a4595c7
parent 2559 add799cf0817
child 2561 7926f1cb45eb
--- a/Nominal/Ex/Foo1.thy	Wed Nov 10 13:46:21 2010 +0000
+++ b/Nominal/Ex/Foo1.thy	Fri Nov 12 01:20:53 2010 +0000
@@ -42,21 +42,6 @@
 thm foo.supp
 thm foo.fresh
 
-primrec
-  permute_bn1_raw
-where
-  "permute_bn1_raw p (As_raw x y t) = As_raw (p \<bullet> x) y t"
-
-primrec
-  permute_bn2_raw
-where
-  "permute_bn2_raw p (As_raw x y t) = As_raw x (p \<bullet> y) t"
-
-primrec
-  permute_bn3_raw
-where
-  "permute_bn3_raw p (As_raw x y t) = As_raw (p \<bullet> x) (p \<bullet> y) t"
-
 quotient_definition
   "permute_bn1 :: perm \<Rightarrow> assg \<Rightarrow> assg"
 is