src/Pure/Pure.thy
changeset 70605 048cf2096186
parent 70570 d94456876f2d
child 71166 c9433e8e314e
equal deleted inserted replaced
70604:8088cf2576f3 70605:048cf2096186
  1299     (Scan.option class_bounds -- Scan.option class_bounds >> (fn args =>
  1299     (Scan.option class_bounds -- Scan.option class_bounds >> (fn args =>
  1300       Toplevel.keep (fn st => Class_Deps.class_deps_cmd (Toplevel.context_of st) args)));
  1300       Toplevel.keep (fn st => Class_Deps.class_deps_cmd (Toplevel.context_of st) args)));
  1301 
  1301 
  1302 
  1302 
  1303 val _ =
  1303 val _ =
  1304   Outer_Syntax.command \<^command_keyword>\<open>thm_deps\<close> "visualize theorem dependencies"
  1304   Outer_Syntax.command \<^command_keyword>\<open>thm_deps\<close>
       
  1305     "print theorem dependencies (immediate non-transitive)"
  1305     (Parse.thms1 >> (fn args =>
  1306     (Parse.thms1 >> (fn args =>
  1306       Toplevel.keep (fn st =>
  1307       Toplevel.keep (fn st =>
  1307         let
  1308         let
  1308           val thy = Toplevel.theory_of st;
  1309           val thy = Toplevel.theory_of st;
  1309           val ctxt = Toplevel.context_of st;
  1310           val ctxt = Toplevel.context_of st;
  1310         in Thm_Deps.thm_deps_cmd thy (Attrib.eval_thms ctxt args) end)));
  1311         in Pretty.writeln (Thm_Deps.pretty_thm_deps thy (Attrib.eval_thms ctxt args)) end)));
  1311 
  1312 
  1312 val _ =
  1313 val _ =
  1313   Outer_Syntax.command \<^command_keyword>\<open>thm_oracles\<close>
  1314   Outer_Syntax.command \<^command_keyword>\<open>thm_oracles\<close>
  1314     "print all oracles used in theorems (full graph of transitive dependencies)"
  1315     "print all oracles used in theorems (full graph of transitive dependencies)"
  1315     (Parse.thms1 >> (fn args =>
  1316     (Parse.thms1 >> (fn args =>