src/Tools/quickcheck.ML
changeset 57182 79d43c510b84
parent 56467 8d7d6f17c6a7
child 57195 ec0e10f11276
equal deleted inserted replaced
57181:2d13bf9ea77b 57182:79d43c510b84
   360     val _ = message lthy "Quickchecking..."
   360     val _ = message lthy "Quickchecking..."
   361     fun strip (Const (@{const_name Pure.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 = Named_Target.locale_of lthy;
   366       (case (Option.map #target o Named_Target.peek) lthy of
       
   367         NONE => NONE
       
   368       | SOME "" => NONE
       
   369       | SOME locale => SOME locale);
       
   370     val assms =
   366     val assms =
   371       if Config.get lthy no_assms then []
   367       if Config.get lthy no_assms then []
   372       else
   368       else
   373         (case some_locale of
   369         (case some_locale of
   374           NONE => Assumption.all_assms_of lthy
   370           NONE => Assumption.all_assms_of lthy