diff -r e54cf66928e6 -r 5e0455e29339 src/HOL/Quickcheck_Narrowing.thy --- a/src/HOL/Quickcheck_Narrowing.thy Thu Aug 23 12:44:52 2012 +0200 +++ b/src/HOL/Quickcheck_Narrowing.thy Thu Aug 23 12:55:23 2012 +0200 @@ -5,9 +5,6 @@ theory Quickcheck_Narrowing imports Quickcheck_Exhaustive keywords "find_unused_assms" :: diag -uses (* FIXME session files *) - ("Tools/Quickcheck/PNF_Narrowing_Engine.hs") - ("Tools/Quickcheck/Narrowing_Engine.hs") begin subsection {* Counterexample generator *}