# HG changeset patch # User blanchet # Date 1256727348 -3600 # Node ID b12ab081e5d1cc7e16e290b1ded52ef944b1fdc5 # Parent 63925777ccf9cb168488ffd0300df9dedb6501d8 use "get_goal" rather than "flat_goal" in Auto Quickcheck, since we don't need the extra facts for counterexample generation diff -r 63925777ccf9 -r b12ab081e5d1 src/Tools/quickcheck.ML --- a/src/Tools/quickcheck.ML Tue Oct 27 21:53:13 2009 +0100 +++ b/src/Tools/quickcheck.ML Wed Oct 28 11:55:48 2009 +0100 @@ -143,7 +143,7 @@ val thy = Proof.theory_of state; fun strip (Const ("all", _) $ Abs (_, _, t)) = strip t | strip t = t; - val (_, st) = Proof.flat_goal state; + val (_, (_, st)) = Proof.get_goal state; val (gi, frees) = Logic.goal_params (prop_of st) i; val gi' = Logic.list_implies (assms, subst_bounds (frees, strip gi)) |> monomorphic_term thy insts default_T