--- a/Nominal/Abs.thy Tue Mar 02 17:48:41 2010 +0100
+++ b/Nominal/Abs.thy Tue Mar 02 17:48:56 2010 +0100
@@ -500,5 +500,14 @@
oops
*)
+
+fun
+ distinct_perms
+where
+ "distinct_perms [] = True"
+| "distinct_perms (p # ps) = (supp p \<inter> supp ps = {} \<and> distinct_perms ps)"
+
+
+
end