src/HOL/HOL.thy
changeset 15570 8d8c70b41bab
parent 15524 2ef571f80a55
child 15655 157f3988f775
--- a/src/HOL/HOL.thy	Thu Mar 03 09:22:35 2005 +0100
+++ b/src/HOL/HOL.thy	Thu Mar 03 12:43:01 2005 +0100
@@ -771,7 +771,7 @@
   fun wrong_prem (Const ("All", _) $ (Abs (_, _, t))) = wrong_prem t
   |   wrong_prem (Bound _) = true
   |   wrong_prem _ = false
-  val filter_right = filter (fn t => not (wrong_prem (HOLogic.dest_Trueprop (hd (Thm.prems_of t)))))
+  val filter_right = List.filter (fn t => not (wrong_prem (HOLogic.dest_Trueprop (hd (Thm.prems_of t)))))
 in
   fun smp i = funpow i (fn m => filter_right ([spec] RL m)) ([mp])
   fun smp_tac j = EVERY'[dresolve_tac (smp j), atac]