src/Tools/quickcheck.ML
changeset 35625 9c818cab0dd0
parent 35380 6ac5b81a763d
child 36610 bafd82950e24
equal deleted inserted replaced
35624:c4e29a0bb8c1 35625:9c818cab0dd0
   197     val {goal = st, ...} = Proof.raw_goal state;
   197     val {goal = st, ...} = Proof.raw_goal state;
   198     val (gi, frees) = Logic.goal_params (prop_of st) i;
   198     val (gi, frees) = Logic.goal_params (prop_of st) i;
   199     val gi' = Logic.list_implies (if no_assms then [] else assms,
   199     val gi' = Logic.list_implies (if no_assms then [] else assms,
   200                                   subst_bounds (frees, strip gi))
   200                                   subst_bounds (frees, strip gi))
   201       |> monomorphic_term thy insts default_T
   201       |> monomorphic_term thy insts default_T
   202       |> ObjectLogic.atomize_term thy;
   202       |> Object_Logic.atomize_term thy;
   203   in gen_test_term ctxt quiet report generator_name size iterations gi' end;
   203   in gen_test_term ctxt quiet report generator_name size iterations gi' end;
   204 
   204 
   205 fun pretty_counterex ctxt NONE = Pretty.str "Quickcheck found no counterexample."
   205 fun pretty_counterex ctxt NONE = Pretty.str "Quickcheck found no counterexample."
   206   | pretty_counterex ctxt (SOME cex) =
   206   | pretty_counterex ctxt (SOME cex) =
   207       Pretty.chunks (Pretty.str "Quickcheck found a counterexample:\n" ::
   207       Pretty.chunks (Pretty.str "Quickcheck found a counterexample:\n" ::