obsolete -- cf. isabelle.Keywords in Scala;
authorwenzelm
Mon, 24 Jun 2013 23:39:17 +0200
changeset 52440 67f57dc115b9
parent 52439 4cf3f6153eb8
child 52441 ffc3f1659a25
obsolete -- cf. isabelle.Keywords in Scala;
src/Pure/Isar/keyword.ML
src/Pure/System/session.ML
--- a/src/Pure/Isar/keyword.ML	Mon Jun 24 23:33:14 2013 +0200
+++ b/src/Pure/Isar/keyword.ML	Mon Jun 24 23:39:17 2013 +0200
@@ -52,7 +52,6 @@
   val command_files: string -> string list
   val command_tags: string -> string list
   val dest: unit -> string list * string list
-  val status: unit -> unit
   val define: string * T option -> unit
   val is_diag: string -> bool
   val is_control: string -> bool
@@ -199,18 +198,6 @@
 fun dest () = pairself (sort_strings o Scan.dest_lexicon) (get_lexicons ());
 
 
-(* status *)
-
-fun status () =
-  let
-    val Keywords {lexicons = (minor, _), commands} = get_keywords ();
-    val _ = sort_strings (Scan.dest_lexicon minor) |> List.app (fn name =>
-      writeln ("\fOuter syntax keyword " ^ quote name));
-    val _ = sort_wrt #1 (Symtab.dest commands) |> List.app (fn (name, kind) =>
-      writeln ("\fOuter syntax keyword " ^ quote name ^ " :: " ^ kind_of kind));
-  in () end;
-
-
 (* define *)
 
 fun define (name, opt_kind) = change_keywords (fn ((minor, major), commands) =>
--- a/src/Pure/System/session.ML	Mon Jun 24 23:33:14 2013 +0200
+++ b/src/Pure/System/session.ML	Mon Jun 24 23:39:17 2013 +0200
@@ -54,7 +54,6 @@
  (Goal.shutdown_futures ();
   Thy_Info.finish ();
   Present.finish ();
-  Keyword.status ();
   Outer_Syntax.check_syntax ();
   Future.shutdown ();
   Event_Timer.shutdown ();