Nominal/NewFv.thy
changeset 2071 843e0a2d44d7
parent 2046 73c50e913db6
child 2131 f7ec6f7b152e
--- a/Nominal/NewFv.thy	Thu May 06 14:09:56 2010 +0200
+++ b/Nominal/NewFv.thy	Thu May 06 14:10:26 2010 +0200
@@ -140,7 +140,7 @@
   val non_rec_vars =
     case binds of
       [(SOME bn, i)] =>
-        if i mem bodys
+        if member (op =) bodys i
         then noatoms
         else ((the (AList.lookup (op=) bn_fvbn bn)) $ nth args i)
     | _ => noatoms