diff -r 30e9720cc0b9 -r 2520cd337056 src/HOL/Tools/Quickcheck/PNF_Narrowing_Engine.hs --- a/src/HOL/Tools/Quickcheck/PNF_Narrowing_Engine.hs Fri Feb 03 18:00:55 2012 +0100 +++ b/src/HOL/Tools/Quickcheck/PNF_Narrowing_Engine.hs Sat Feb 04 07:40:02 2012 +0100 @@ -3,11 +3,12 @@ -} module Narrowing_Engine where -import Monad +import Control.Monad import Control.Exception +import System.IO import System.Exit -import Maybe -import List (partition, findIndex) +import Data.Maybe +import Data.List (partition, findIndex) import qualified Generated_Code @@ -35,7 +36,7 @@ termListOf' i [] = [] termListOf' i (e : es) = let - (ts, rs) = List.partition (\e -> head (posOf e) == i) (e : es) + (ts, rs) = Data.List.partition (\e -> head (posOf e) == i) (e : es) t = termOf (pos ++ [i]) (map tailPosEdge ts) in (t : termListOf' (i + 1) rs)