src/Tools/quickcheck.ML
changeset 56245 84fc7dfa3cd4
parent 55630 47286c847749
child 56467 8d7d6f17c6a7
equal deleted inserted replaced
56244:3298b7a2795a 56245:84fc7dfa3cd4
   356 fun test_goal (time_limit, is_interactive) (insts, eval_terms) i state =
   356 fun test_goal (time_limit, is_interactive) (insts, eval_terms) i state =
   357   let
   357   let
   358     val lthy = Proof.context_of state;
   358     val lthy = Proof.context_of state;
   359     val thy = Proof.theory_of state;
   359     val thy = Proof.theory_of state;
   360     val _ = message lthy "Quickchecking..."
   360     val _ = message lthy "Quickchecking..."
   361     fun strip (Const ("all", _) $ Abs (_, _, t)) = strip t
   361     fun strip (Const (@{const_name Pure.all}, _) $ Abs (_, _, t)) = strip t
   362       | strip t = t;
   362       | strip t = t;
   363     val {goal = st, ...} = Proof.raw_goal state;
   363     val {goal = st, ...} = Proof.raw_goal state;
   364     val (gi, frees) = Logic.goal_params (prop_of st) i;
   364     val (gi, frees) = Logic.goal_params (prop_of st) i;
   365     val some_locale =
   365     val some_locale =
   366       (case (Option.map #target o Named_Target.peek) lthy of
   366       (case (Option.map #target o Named_Target.peek) lthy of