Nominal/Test.thy
changeset 1380 dab8d99b37c1
parent 1378 5c6c950812b1
child 1392 baa67b07f436
--- a/Nominal/Test.thy	Tue Mar 09 17:25:35 2010 +0100
+++ b/Nominal/Test.thy	Tue Mar 09 22:08:38 2010 +0100
@@ -66,8 +66,9 @@
   f::"pat' \<Rightarrow> atom set"
 where 
   "f PN = {}"
+| "f (PD x y) = {atom x, atom y}"
 | "f (PS x) = {atom x}"
-| "f (PD x y) = {atom x, atom y}"
+
 
 (* compat should be
 compat (PN) pi (PN) == True