Nominal/Test.thy
changeset 1384 adeb3746ec8f
parent 1380 dab8d99b37c1
child 1392 baa67b07f436
--- a/Nominal/Test.thy	Wed Mar 10 09:09:52 2010 +0100
+++ b/Nominal/Test.thy	Wed Mar 10 09:10:11 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