diff -r add799cf0817 -r 82e37a4595c7 Nominal/Ex/Foo1.thy --- 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 \ x) y t" - -primrec - permute_bn2_raw -where - "permute_bn2_raw p (As_raw x y t) = As_raw x (p \ y) t" - -primrec - permute_bn3_raw -where - "permute_bn3_raw p (As_raw x y t) = As_raw (p \ x) (p \ y) t" - quotient_definition "permute_bn1 :: perm \ assg \ assg" is