src/HOL/Set.thy
changeset 33037 b22e44496dc2
parent 32888 ae17e72aac80
child 33038 8f9594c31de4
--- a/src/HOL/Set.thy	Tue Oct 20 13:37:56 2009 +0200
+++ b/src/HOL/Set.thy	Tue Oct 20 16:13:01 2009 +0200
@@ -303,7 +303,7 @@
       fun check (Const ("Ex", _) $ Abs (_, _, P), n) = check (P, n + 1)
         | check (Const ("op &", _) $ (Const ("op =", _) $ Bound m $ e) $ P, n) =
             n > 0 andalso m = n andalso not (loose_bvar1 (P, n)) andalso
-            ((0 upto (n - 1)) subset add_loose_bnos (e, 0, []))
+            gen_subset (op =) (0 upto (n - 1), add_loose_bnos (e, 0, []))
         | check _ = false
 
         fun tr' (_ $ abs) =