misc tuning: more concise operations on prems (without change of exceptions);
discontinue odd clone Drule.cprems_of (see also 991a3feaf270);
(* Title: Tools/profiling.ML
Author: Makarius
Session profiling based on loaded ML image.
*)
theory Profiling
imports Pure
begin
ML_file "profiling.ML"
ML_command \<open>Profiling.main ()\<close>
end