src/HOL/Set.thy
changeset 33038 8f9594c31de4
parent 33037 b22e44496dc2
child 33039 5018f6a76b3f
--- a/src/HOL/Set.thy	Tue Oct 20 16:13:01 2009 +0200
+++ b/src/HOL/Set.thy	Wed Oct 21 08:14:38 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
-            gen_subset (op =) (0 upto (n - 1), add_loose_bnos (e, 0, []))
+            subset (op =) (0 upto (n - 1), add_loose_bnos (e, 0, []))
         | check _ = false
 
         fun tr' (_ $ abs) =