src/Pure/Isar/outer_syntax.ML
author wenzelm
Fri, 29 Mar 2013 22:14:27 +0100
changeset 51580 64ef8260dc60
parent 51271 e8d2ecf6aaac
child 51627 589daaf48dba
permissions -rw-r--r--
Pretty.item markup for improved readability of lists of items;
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
5829
0acb30dd92bc The global Isabelle/Isar outer syntax.
wenzelm
parents:
diff changeset
     1
(*  Title:      Pure/Isar/outer_syntax.ML
0acb30dd92bc The global Isabelle/Isar outer syntax.
wenzelm
parents:
diff changeset
     2
    Author:     Markus Wenzel, TU Muenchen
0acb30dd92bc The global Isabelle/Isar outer syntax.
wenzelm
parents:
diff changeset
     3
27353
71c4dd53d4cb moved global keywords from OuterSyntax to OuterKeyword, tuned interfaces;
wenzelm
parents: 26990
diff changeset
     4
The global Isabelle/Isar outer syntax.
71c4dd53d4cb moved global keywords from OuterSyntax to OuterKeyword, tuned interfaces;
wenzelm
parents: 26990
diff changeset
     5
71c4dd53d4cb moved global keywords from OuterSyntax to OuterKeyword, tuned interfaces;
wenzelm
parents: 26990
diff changeset
     6
Note: the syntax for files is statically determined at the very
71c4dd53d4cb moved global keywords from OuterSyntax to OuterKeyword, tuned interfaces;
wenzelm
parents: 26990
diff changeset
     7
beginning; for interactive processing it may change dynamically.
5829
0acb30dd92bc The global Isabelle/Isar outer syntax.
wenzelm
parents:
diff changeset
     8
*)
0acb30dd92bc The global Isabelle/Isar outer syntax.
wenzelm
parents:
diff changeset
     9
0acb30dd92bc The global Isabelle/Isar outer syntax.
wenzelm
parents:
diff changeset
    10
signature OUTER_SYNTAX =
0acb30dd92bc The global Isabelle/Isar outer syntax.
wenzelm
parents:
diff changeset
    11
sig
43711
608d1b451f67 less stateful outer_syntax;
wenzelm
parents: 43621
diff changeset
    12
  type outer_syntax
43712
3c2c912af2ef moved Outer_Syntax.load_thy to Thy_Load.load_thy;
wenzelm
parents: 43711
diff changeset
    13
  val is_markup: outer_syntax -> Thy_Output.markup -> string -> bool
43711
608d1b451f67 less stateful outer_syntax;
wenzelm
parents: 43621
diff changeset
    14
  val get_syntax: unit -> (Scan.lexicon * Scan.lexicon) * outer_syntax
46970
9667e0dcb5e2 check declared vs. defined commands at end of session;
wenzelm
parents: 46961
diff changeset
    15
  val check_syntax: unit -> unit
48646
91281e9472d8 more official command specifications, including source position;
wenzelm
parents: 48638
diff changeset
    16
  type command_spec = (string * Keyword.T) * Position.T
46961
5c6955f487e5 outer syntax command definitions based on formal command_spec derived from theory header declarations;
wenzelm
parents: 46958
diff changeset
    17
  val command: command_spec -> string ->
29311
4c830711e6f1 added type 'a parser, simplified signature;
wenzelm
parents: 28436
diff changeset
    18
    (Toplevel.transition -> Toplevel.transition) parser -> unit
46961
5c6955f487e5 outer syntax command definitions based on formal command_spec derived from theory header declarations;
wenzelm
parents: 46958
diff changeset
    19
  val markup_command: Thy_Output.markup -> command_spec -> string ->
29311
4c830711e6f1 added type 'a parser, simplified signature;
wenzelm
parents: 28436
diff changeset
    20
    (Toplevel.transition -> Toplevel.transition) parser -> unit
46961
5c6955f487e5 outer syntax command definitions based on formal command_spec derived from theory header declarations;
wenzelm
parents: 46958
diff changeset
    21
  val improper_command: command_spec -> string ->
43711
608d1b451f67 less stateful outer_syntax;
wenzelm
parents: 43621
diff changeset
    22
    (Toplevel.transition -> Toplevel.transition) parser -> unit
46961
5c6955f487e5 outer syntax command definitions based on formal command_spec derived from theory header declarations;
wenzelm
parents: 46958
diff changeset
    23
  val local_theory': command_spec -> string ->
29380
a9ee3475abf4 added local_theory';
wenzelm
parents: 29315
diff changeset
    24
    (bool -> local_theory -> local_theory) parser -> unit
46961
5c6955f487e5 outer syntax command definitions based on formal command_spec derived from theory header declarations;
wenzelm
parents: 46958
diff changeset
    25
  val local_theory: command_spec -> string ->
29311
4c830711e6f1 added type 'a parser, simplified signature;
wenzelm
parents: 28436
diff changeset
    26
    (local_theory -> local_theory) parser -> unit
46961
5c6955f487e5 outer syntax command definitions based on formal command_spec derived from theory header declarations;
wenzelm
parents: 46958
diff changeset
    27
  val local_theory_to_proof': command_spec -> string ->
29311
4c830711e6f1 added type 'a parser, simplified signature;
wenzelm
parents: 28436
diff changeset
    28
    (bool -> local_theory -> Proof.state) parser -> unit
46961
5c6955f487e5 outer syntax command definitions based on formal command_spec derived from theory header declarations;
wenzelm
parents: 46958
diff changeset
    29
  val local_theory_to_proof: command_spec -> string ->
29311
4c830711e6f1 added type 'a parser, simplified signature;
wenzelm
parents: 28436
diff changeset
    30
    (local_theory -> Proof.state) parser -> unit
50213
7b73c0509835 refined outer syntax 'help' command;
wenzelm
parents: 50201
diff changeset
    31
  val help_outer_syntax: string list -> unit
5883
975c984526b0 tuned names;
wenzelm
parents: 5829
diff changeset
    32
  val print_outer_syntax: unit -> unit
36959
f5417836dbea renamed structure OuterLex to Token and type token to Token.T, keeping legacy aliases for some time;
wenzelm
parents: 36955
diff changeset
    33
  val scan: Position.T -> string -> Token.T list
25580
6623674df897 added off-line parse;
wenzelm
parents: 25526
diff changeset
    34
  val parse: Position.T -> string -> Toplevel.transition list
26600
f11515535c83 moved structure Isar to isar.ML;
wenzelm
parents: 26431
diff changeset
    35
  type isar
38253
3d4e521014f7 Isabelle_Process: separate input fifo for commands (still using the old tty protocol);
wenzelm
parents: 38236
diff changeset
    36
  val isar: TextIO.instream -> bool -> isar
48918
6e5fd4585512 check side-comments of command spans (normally filtered out in Outer_Syntax.toplevel_source);
wenzelm
parents: 48864
diff changeset
    37
  val span_cmts: Token.T list -> Token.T list
51268
fcc4b89a600d simplified Outer_Syntax.read_span: internalized Toplevel.is_ignored;
wenzelm
parents: 51225
diff changeset
    38
  val read_span: outer_syntax -> Token.T list -> Toplevel.transition
5829
0acb30dd92bc The global Isabelle/Isar outer syntax.
wenzelm
parents:
diff changeset
    39
end;
0acb30dd92bc The global Isabelle/Isar outer syntax.
wenzelm
parents:
diff changeset
    40
36953
2af1ad9aa1a3 renamed structure OuterSyntax to Outer_Syntax, keeping the old name as alias for some time;
wenzelm
parents: 36950
diff changeset
    41
structure Outer_Syntax: OUTER_SYNTAX =
5829
0acb30dd92bc The global Isabelle/Isar outer syntax.
wenzelm
parents:
diff changeset
    42
struct
0acb30dd92bc The global Isabelle/Isar outer syntax.
wenzelm
parents:
diff changeset
    43
0acb30dd92bc The global Isabelle/Isar outer syntax.
wenzelm
parents:
diff changeset
    44
(** outer syntax **)
0acb30dd92bc The global Isabelle/Isar outer syntax.
wenzelm
parents:
diff changeset
    45
29311
4c830711e6f1 added type 'a parser, simplified signature;
wenzelm
parents: 28436
diff changeset
    46
(* command parsers *)
5829
0acb30dd92bc The global Isabelle/Isar outer syntax.
wenzelm
parents:
diff changeset
    47
29311
4c830711e6f1 added type 'a parser, simplified signature;
wenzelm
parents: 28436
diff changeset
    48
datatype command = Command of
24868
2990c327d8c6 simplified interfaces for outer syntax;
wenzelm
parents: 24188
diff changeset
    49
 {comment: string,
37216
3165bc303f66 modernized some structure names, keeping a few legacy aliases;
wenzelm
parents: 36959
diff changeset
    50
  markup: Thy_Output.markup option,
24868
2990c327d8c6 simplified interfaces for outer syntax;
wenzelm
parents: 24188
diff changeset
    51
  int_only: bool,
48647
a5144c4c26a2 report commands as formal entities, with def/ref positions;
wenzelm
parents: 48646
diff changeset
    52
  parse: (Toplevel.transition -> Toplevel.transition) parser,
a5144c4c26a2 report commands as formal entities, with def/ref positions;
wenzelm
parents: 48646
diff changeset
    53
  pos: Position.T,
a5144c4c26a2 report commands as formal entities, with def/ref positions;
wenzelm
parents: 48646
diff changeset
    54
  id: serial};
5829
0acb30dd92bc The global Isabelle/Isar outer syntax.
wenzelm
parents:
diff changeset
    55
48647
a5144c4c26a2 report commands as formal entities, with def/ref positions;
wenzelm
parents: 48646
diff changeset
    56
fun new_command comment markup int_only parse pos =
a5144c4c26a2 report commands as formal entities, with def/ref positions;
wenzelm
parents: 48646
diff changeset
    57
  Command {comment = comment, markup = markup, int_only = int_only, parse = parse,
a5144c4c26a2 report commands as formal entities, with def/ref positions;
wenzelm
parents: 48646
diff changeset
    58
    pos = pos, id = serial ()};
a5144c4c26a2 report commands as formal entities, with def/ref positions;
wenzelm
parents: 48646
diff changeset
    59
a5144c4c26a2 report commands as formal entities, with def/ref positions;
wenzelm
parents: 48646
diff changeset
    60
fun command_markup def (name, Command {pos, id, ...}) =
a5144c4c26a2 report commands as formal entities, with def/ref positions;
wenzelm
parents: 48646
diff changeset
    61
  Markup.properties (Position.entity_properties_of def id pos)
50201
c26369c9eda6 Isabelle-specific implementation of quasi-abstract markup elements -- back to module arrangement before d83797ef0d2d;
wenzelm
parents: 49564
diff changeset
    62
    (Markup.entity Markup.commandN name);
5829
0acb30dd92bc The global Isabelle/Isar outer syntax.
wenzelm
parents:
diff changeset
    63
50213
7b73c0509835 refined outer syntax 'help' command;
wenzelm
parents: 50201
diff changeset
    64
fun pretty_command (cmd as (name, Command {comment, ...})) =
7b73c0509835 refined outer syntax 'help' command;
wenzelm
parents: 50201
diff changeset
    65
  Pretty.block
7b73c0509835 refined outer syntax 'help' command;
wenzelm
parents: 50201
diff changeset
    66
    (Pretty.marks_str
50450
358b6020f8b6 generalized notion of active area, where sendback is just one application;
wenzelm
parents: 50215
diff changeset
    67
      ([Active.make_markup Markup.sendbackN {implicit = true, properties = [Markup.padding_line]},
50215
97959912840a more general sendback properties;
wenzelm
parents: 50213
diff changeset
    68
        command_markup false cmd], name) :: Pretty.str ":" :: Pretty.brk 2 :: Pretty.text comment);
50213
7b73c0509835 refined outer syntax 'help' command;
wenzelm
parents: 50201
diff changeset
    69
5829
0acb30dd92bc The global Isabelle/Isar outer syntax.
wenzelm
parents:
diff changeset
    70
0acb30dd92bc The global Isabelle/Isar outer syntax.
wenzelm
parents:
diff changeset
    71
(* parse command *)
0acb30dd92bc The global Isabelle/Isar outer syntax.
wenzelm
parents:
diff changeset
    72
6860
8dc6a1e6fa13 added sync;
wenzelm
parents: 6733
diff changeset
    73
local
6199
9b1be867e21a removed load;
wenzelm
parents: 6107
diff changeset
    74
14925
0f86a8a694f8 added read (provides transition names and sources);
wenzelm
parents: 14687
diff changeset
    75
fun terminate false = Scan.succeed ()
44357
5f5649ac8235 tuned Parse.group: delayed failure message;
wenzelm
parents: 44187
diff changeset
    76
  | terminate true =
5f5649ac8235 tuned Parse.group: delayed failure message;
wenzelm
parents: 44187
diff changeset
    77
      Parse.group (fn () => "end of input")
5f5649ac8235 tuned Parse.group: delayed failure message;
wenzelm
parents: 44187
diff changeset
    78
        (Scan.option Parse.sync -- Parse.semicolon >> K ());
14925
0f86a8a694f8 added read (provides transition names and sources);
wenzelm
parents: 14687
diff changeset
    79
26620
722cf4fdd4dd eliminated unused trace, read;
wenzelm
parents: 26611
diff changeset
    80
fun body cmd (name, _) =
7026
69724548fad1 separate command tokens;
wenzelm
parents: 6868
diff changeset
    81
  (case cmd name of
29311
4c830711e6f1 added type 'a parser, simplified signature;
wenzelm
parents: 28436
diff changeset
    82
    SOME (Command {int_only, parse, ...}) =>
36950
75b8f26f2f07 refer directly to structure Keyword and Parse;
wenzelm
parents: 33223
diff changeset
    83
      Parse.!!! (Scan.prompt (name ^ "# ") (Parse.tags |-- parse >> pair int_only))
48191
c1def7433a72 internalize error into command transaction -- relevant for commands that are declared via 'keywords', but not defined yet;
wenzelm
parents: 47416
diff changeset
    84
  | NONE =>
c1def7433a72 internalize error into command transaction -- relevant for commands that are declared via 'keywords', but not defined yet;
wenzelm
parents: 47416
diff changeset
    85
      Scan.succeed (false, Toplevel.imperative (fn () =>
c1def7433a72 internalize error into command transaction -- relevant for commands that are declared via 'keywords', but not defined yet;
wenzelm
parents: 47416
diff changeset
    86
        error ("Bad parser for outer syntax command " ^ quote name))));
6860
8dc6a1e6fa13 added sync;
wenzelm
parents: 6733
diff changeset
    87
8dc6a1e6fa13 added sync;
wenzelm
parents: 6733
diff changeset
    88
in
5829
0acb30dd92bc The global Isabelle/Isar outer syntax.
wenzelm
parents:
diff changeset
    89
26620
722cf4fdd4dd eliminated unused trace, read;
wenzelm
parents: 26611
diff changeset
    90
fun parse_command do_terminate cmd =
36950
75b8f26f2f07 refer directly to structure Keyword and Parse;
wenzelm
parents: 33223
diff changeset
    91
  Parse.semicolon >> K NONE ||
75b8f26f2f07 refer directly to structure Keyword and Parse;
wenzelm
parents: 33223
diff changeset
    92
  Parse.sync >> K NONE ||
75b8f26f2f07 refer directly to structure Keyword and Parse;
wenzelm
parents: 33223
diff changeset
    93
  (Parse.position Parse.command :-- body cmd) --| terminate do_terminate
6860
8dc6a1e6fa13 added sync;
wenzelm
parents: 6733
diff changeset
    94
    >> (fn ((name, pos), (int_only, f)) =>
15531
08c8dad8e399 Deleted Library.option type.
skalberg
parents: 15224
diff changeset
    95
      SOME (Toplevel.empty |> Toplevel.name name |> Toplevel.position pos |>
6860
8dc6a1e6fa13 added sync;
wenzelm
parents: 6733
diff changeset
    96
        Toplevel.interactive int_only |> f));
5829
0acb30dd92bc The global Isabelle/Isar outer syntax.
wenzelm
parents:
diff changeset
    97
6199
9b1be867e21a removed load;
wenzelm
parents: 6107
diff changeset
    98
end;
9b1be867e21a removed load;
wenzelm
parents: 6107
diff changeset
    99
5829
0acb30dd92bc The global Isabelle/Isar outer syntax.
wenzelm
parents:
diff changeset
   100
43711
608d1b451f67 less stateful outer_syntax;
wenzelm
parents: 43621
diff changeset
   101
(* type outer_syntax *)
608d1b451f67 less stateful outer_syntax;
wenzelm
parents: 43621
diff changeset
   102
608d1b451f67 less stateful outer_syntax;
wenzelm
parents: 43621
diff changeset
   103
datatype outer_syntax = Outer_Syntax of
608d1b451f67 less stateful outer_syntax;
wenzelm
parents: 43621
diff changeset
   104
 {commands: command Symtab.table,
608d1b451f67 less stateful outer_syntax;
wenzelm
parents: 43621
diff changeset
   105
  markups: (string * Thy_Output.markup) list};
608d1b451f67 less stateful outer_syntax;
wenzelm
parents: 43621
diff changeset
   106
608d1b451f67 less stateful outer_syntax;
wenzelm
parents: 43621
diff changeset
   107
fun make_outer_syntax commands markups =
608d1b451f67 less stateful outer_syntax;
wenzelm
parents: 43621
diff changeset
   108
  Outer_Syntax {commands = commands, markups = markups};
608d1b451f67 less stateful outer_syntax;
wenzelm
parents: 43621
diff changeset
   109
608d1b451f67 less stateful outer_syntax;
wenzelm
parents: 43621
diff changeset
   110
val empty_outer_syntax = make_outer_syntax Symtab.empty [];
608d1b451f67 less stateful outer_syntax;
wenzelm
parents: 43621
diff changeset
   111
608d1b451f67 less stateful outer_syntax;
wenzelm
parents: 43621
diff changeset
   112
608d1b451f67 less stateful outer_syntax;
wenzelm
parents: 43621
diff changeset
   113
fun map_commands f (Outer_Syntax {commands, ...}) =
608d1b451f67 less stateful outer_syntax;
wenzelm
parents: 43621
diff changeset
   114
  let
608d1b451f67 less stateful outer_syntax;
wenzelm
parents: 43621
diff changeset
   115
    val commands' = f commands;
608d1b451f67 less stateful outer_syntax;
wenzelm
parents: 43621
diff changeset
   116
    val markups' =
608d1b451f67 less stateful outer_syntax;
wenzelm
parents: 43621
diff changeset
   117
      Symtab.fold (fn (name, Command {markup = SOME m, ...}) => cons (name, m) | _ => I)
608d1b451f67 less stateful outer_syntax;
wenzelm
parents: 43621
diff changeset
   118
        commands' [];
608d1b451f67 less stateful outer_syntax;
wenzelm
parents: 43621
diff changeset
   119
  in make_outer_syntax commands' markups' end;
608d1b451f67 less stateful outer_syntax;
wenzelm
parents: 43621
diff changeset
   120
608d1b451f67 less stateful outer_syntax;
wenzelm
parents: 43621
diff changeset
   121
fun dest_commands (Outer_Syntax {commands, ...}) =
50213
7b73c0509835 refined outer syntax 'help' command;
wenzelm
parents: 50201
diff changeset
   122
  commands |> Symtab.dest |> sort_wrt #1;
43711
608d1b451f67 less stateful outer_syntax;
wenzelm
parents: 43621
diff changeset
   123
608d1b451f67 less stateful outer_syntax;
wenzelm
parents: 43621
diff changeset
   124
fun lookup_commands (Outer_Syntax {commands, ...}) = Symtab.lookup commands;
608d1b451f67 less stateful outer_syntax;
wenzelm
parents: 43621
diff changeset
   125
608d1b451f67 less stateful outer_syntax;
wenzelm
parents: 43621
diff changeset
   126
fun is_markup (Outer_Syntax {markups, ...}) kind name =
608d1b451f67 less stateful outer_syntax;
wenzelm
parents: 43621
diff changeset
   127
  AList.lookup (op =) markups name = SOME kind;
608d1b451f67 less stateful outer_syntax;
wenzelm
parents: 43621
diff changeset
   128
608d1b451f67 less stateful outer_syntax;
wenzelm
parents: 43621
diff changeset
   129
5829
0acb30dd92bc The global Isabelle/Isar outer syntax.
wenzelm
parents:
diff changeset
   130
9132
52286129faa5 moved header stuff to thy_header.ML;
wenzelm
parents: 9056
diff changeset
   131
(** global outer syntax **)
5829
0acb30dd92bc The global Isabelle/Isar outer syntax.
wenzelm
parents:
diff changeset
   132
48646
91281e9472d8 more official command specifications, including source position;
wenzelm
parents: 48638
diff changeset
   133
type command_spec = (string * Keyword.T) * Position.T;
46961
5c6955f487e5 outer syntax command definitions based on formal command_spec derived from theory header declarations;
wenzelm
parents: 46958
diff changeset
   134
7026
69724548fad1 separate command tokens;
wenzelm
parents: 6868
diff changeset
   135
local
69724548fad1 separate command tokens;
wenzelm
parents: 6868
diff changeset
   136
43711
608d1b451f67 less stateful outer_syntax;
wenzelm
parents: 43621
diff changeset
   137
(*synchronized wrt. Keywords*)
608d1b451f67 less stateful outer_syntax;
wenzelm
parents: 43621
diff changeset
   138
val global_outer_syntax = Unsynchronized.ref empty_outer_syntax;
5952
7d4ec8992b23 added commands;
wenzelm
parents: 5923
diff changeset
   139
48647
a5144c4c26a2 report commands as formal entities, with def/ref positions;
wenzelm
parents: 48646
diff changeset
   140
fun add_command (name, kind) cmd = CRITICAL (fn () =>
46950
d0181abdbdac declare command keywords via theory header, including strict checking outside Pure;
wenzelm
parents: 46876
diff changeset
   141
  let
d0181abdbdac declare command keywords via theory header, including strict checking outside Pure;
wenzelm
parents: 46876
diff changeset
   142
    val thy = ML_Context.the_global_context ();
48647
a5144c4c26a2 report commands as formal entities, with def/ref positions;
wenzelm
parents: 48646
diff changeset
   143
    val Command {pos, ...} = cmd;
46950
d0181abdbdac declare command keywords via theory header, including strict checking outside Pure;
wenzelm
parents: 46876
diff changeset
   144
    val _ =
d0181abdbdac declare command keywords via theory header, including strict checking outside Pure;
wenzelm
parents: 46876
diff changeset
   145
      (case try (Thy_Header.the_keyword thy) name of
46961
5c6955f487e5 outer syntax command definitions based on formal command_spec derived from theory header declarations;
wenzelm
parents: 46958
diff changeset
   146
        SOME spec =>
48864
3ee314ae1e0a added keyword kind "thy_load" (with optional list of file extensions);
wenzelm
parents: 48771
diff changeset
   147
          if Option.map #1 spec = SOME (Keyword.kind_files_of kind) then ()
48646
91281e9472d8 more official command specifications, including source position;
wenzelm
parents: 48638
diff changeset
   148
          else error ("Inconsistent outer syntax keyword declaration " ^
48992
0518bf89c777 renamed Position.str_of to Position.here;
wenzelm
parents: 48918
diff changeset
   149
            quote name ^ Position.here pos)
46950
d0181abdbdac declare command keywords via theory header, including strict checking outside Pure;
wenzelm
parents: 46876
diff changeset
   150
      | NONE =>
46961
5c6955f487e5 outer syntax command definitions based on formal command_spec derived from theory header declarations;
wenzelm
parents: 46958
diff changeset
   151
          if Context.theory_name thy = Context.PureN
5c6955f487e5 outer syntax command definitions based on formal command_spec derived from theory header declarations;
wenzelm
parents: 46958
diff changeset
   152
          then Keyword.define (name, SOME kind)
48992
0518bf89c777 renamed Position.str_of to Position.here;
wenzelm
parents: 48918
diff changeset
   153
          else error ("Undeclared outer syntax command " ^ quote name ^ Position.here pos));
48647
a5144c4c26a2 report commands as formal entities, with def/ref positions;
wenzelm
parents: 48646
diff changeset
   154
    val _ = Position.report pos (command_markup true (name, cmd));
46950
d0181abdbdac declare command keywords via theory header, including strict checking outside Pure;
wenzelm
parents: 46876
diff changeset
   155
  in
d0181abdbdac declare command keywords via theory header, including strict checking outside Pure;
wenzelm
parents: 46876
diff changeset
   156
    Unsynchronized.change global_outer_syntax (map_commands (fn commands =>
d0181abdbdac declare command keywords via theory header, including strict checking outside Pure;
wenzelm
parents: 46876
diff changeset
   157
     (if not (Symtab.defined commands name) then ()
d0181abdbdac declare command keywords via theory header, including strict checking outside Pure;
wenzelm
parents: 46876
diff changeset
   158
      else warning ("Redefining outer syntax command " ^ quote name);
d0181abdbdac declare command keywords via theory header, including strict checking outside Pure;
wenzelm
parents: 46876
diff changeset
   159
      Symtab.update (name, cmd) commands)))
d0181abdbdac declare command keywords via theory header, including strict checking outside Pure;
wenzelm
parents: 46876
diff changeset
   160
  end);
6722
5e82c7196789 added keyword classification;
wenzelm
parents: 6685
diff changeset
   161
7026
69724548fad1 separate command tokens;
wenzelm
parents: 6868
diff changeset
   162
in
69724548fad1 separate command tokens;
wenzelm
parents: 6868
diff changeset
   163
43711
608d1b451f67 less stateful outer_syntax;
wenzelm
parents: 43621
diff changeset
   164
fun get_syntax () = CRITICAL (fn () => (Keyword.get_lexicons (), ! global_outer_syntax));
7789
57d20133224e verbatim markup tokens;
wenzelm
parents: 7774
diff changeset
   165
46970
9667e0dcb5e2 check declared vs. defined commands at end of session;
wenzelm
parents: 46961
diff changeset
   166
fun check_syntax () =
9667e0dcb5e2 check declared vs. defined commands at end of session;
wenzelm
parents: 46961
diff changeset
   167
  let
9667e0dcb5e2 check declared vs. defined commands at end of session;
wenzelm
parents: 46961
diff changeset
   168
    val ((_, major), syntax) = CRITICAL (fn () => (Keyword.dest (), ! global_outer_syntax));
9667e0dcb5e2 check declared vs. defined commands at end of session;
wenzelm
parents: 46961
diff changeset
   169
  in
9667e0dcb5e2 check declared vs. defined commands at end of session;
wenzelm
parents: 46961
diff changeset
   170
    (case subtract (op =) (map #1 (dest_commands syntax)) major of
9667e0dcb5e2 check declared vs. defined commands at end of session;
wenzelm
parents: 46961
diff changeset
   171
      [] => ()
9667e0dcb5e2 check declared vs. defined commands at end of session;
wenzelm
parents: 46961
diff changeset
   172
    | missing => error ("Missing outer syntax command(s) " ^ commas_quote missing))
9667e0dcb5e2 check declared vs. defined commands at end of session;
wenzelm
parents: 46961
diff changeset
   173
  end;
9667e0dcb5e2 check declared vs. defined commands at end of session;
wenzelm
parents: 46961
diff changeset
   174
43711
608d1b451f67 less stateful outer_syntax;
wenzelm
parents: 43621
diff changeset
   175
fun lookup_commands_dynamic () = lookup_commands (! global_outer_syntax);
5829
0acb30dd92bc The global Isabelle/Isar outer syntax.
wenzelm
parents:
diff changeset
   176
48647
a5144c4c26a2 report commands as formal entities, with def/ref positions;
wenzelm
parents: 48646
diff changeset
   177
fun command (spec, pos) comment parse =
a5144c4c26a2 report commands as formal entities, with def/ref positions;
wenzelm
parents: 48646
diff changeset
   178
  add_command spec (new_command comment NONE false parse pos);
24868
2990c327d8c6 simplified interfaces for outer syntax;
wenzelm
parents: 24188
diff changeset
   179
48647
a5144c4c26a2 report commands as formal entities, with def/ref positions;
wenzelm
parents: 48646
diff changeset
   180
fun markup_command markup (spec, pos) comment parse =
a5144c4c26a2 report commands as formal entities, with def/ref positions;
wenzelm
parents: 48646
diff changeset
   181
  add_command spec (new_command comment (SOME markup) false parse pos);
7026
69724548fad1 separate command tokens;
wenzelm
parents: 6868
diff changeset
   182
48647
a5144c4c26a2 report commands as formal entities, with def/ref positions;
wenzelm
parents: 48646
diff changeset
   183
fun improper_command (spec, pos) comment parse =
a5144c4c26a2 report commands as formal entities, with def/ref positions;
wenzelm
parents: 48646
diff changeset
   184
  add_command spec (new_command comment NONE true parse pos);
29311
4c830711e6f1 added type 'a parser, simplified signature;
wenzelm
parents: 28436
diff changeset
   185
43711
608d1b451f67 less stateful outer_syntax;
wenzelm
parents: 43621
diff changeset
   186
end;
608d1b451f67 less stateful outer_syntax;
wenzelm
parents: 43621
diff changeset
   187
5829
0acb30dd92bc The global Isabelle/Isar outer syntax.
wenzelm
parents:
diff changeset
   188
26990
a91f7741967a added local_theory command wrappers;
wenzelm
parents: 26881
diff changeset
   189
(* local_theory commands *)
a91f7741967a added local_theory command wrappers;
wenzelm
parents: 26881
diff changeset
   190
46961
5c6955f487e5 outer syntax command definitions based on formal command_spec derived from theory header declarations;
wenzelm
parents: 46958
diff changeset
   191
fun local_theory_command do_print trans command_spec comment parse =
5c6955f487e5 outer syntax command definitions based on formal command_spec derived from theory header declarations;
wenzelm
parents: 46958
diff changeset
   192
  command command_spec comment (Parse.opt_target -- parse
26990
a91f7741967a added local_theory command wrappers;
wenzelm
parents: 26881
diff changeset
   193
    >> (fn (loc, f) => (if do_print then Toplevel.print else I) o trans loc f));
a91f7741967a added local_theory command wrappers;
wenzelm
parents: 26881
diff changeset
   194
29380
a9ee3475abf4 added local_theory';
wenzelm
parents: 29315
diff changeset
   195
val local_theory' = local_theory_command false Toplevel.local_theory';
29311
4c830711e6f1 added type 'a parser, simplified signature;
wenzelm
parents: 28436
diff changeset
   196
val local_theory = local_theory_command false Toplevel.local_theory;
26990
a91f7741967a added local_theory command wrappers;
wenzelm
parents: 26881
diff changeset
   197
val local_theory_to_proof' = local_theory_command true Toplevel.local_theory_to_proof';
29311
4c830711e6f1 added type 'a parser, simplified signature;
wenzelm
parents: 28436
diff changeset
   198
val local_theory_to_proof = local_theory_command true Toplevel.local_theory_to_proof;
26990
a91f7741967a added local_theory command wrappers;
wenzelm
parents: 26881
diff changeset
   199
a91f7741967a added local_theory command wrappers;
wenzelm
parents: 26881
diff changeset
   200
24872
7fd1aa6671a4 report on keyword/command declarations;
wenzelm
parents: 24868
diff changeset
   201
(* inspect syntax *)
7026
69724548fad1 separate command tokens;
wenzelm
parents: 6868
diff changeset
   202
50213
7b73c0509835 refined outer syntax 'help' command;
wenzelm
parents: 50201
diff changeset
   203
fun help_outer_syntax pats =
7b73c0509835 refined outer syntax 'help' command;
wenzelm
parents: 50201
diff changeset
   204
  dest_commands (#2 (get_syntax ()))
7b73c0509835 refined outer syntax 'help' command;
wenzelm
parents: 50201
diff changeset
   205
  |> filter (fn (name, _) => forall (fn pat => match_string pat name) pats)
7b73c0509835 refined outer syntax 'help' command;
wenzelm
parents: 50201
diff changeset
   206
  |> map pretty_command
7b73c0509835 refined outer syntax 'help' command;
wenzelm
parents: 50201
diff changeset
   207
  |> Pretty.chunks |> Pretty.writeln;
7b73c0509835 refined outer syntax 'help' command;
wenzelm
parents: 50201
diff changeset
   208
9223
eb752c2fac22 removed help;
wenzelm
parents: 9213
diff changeset
   209
fun print_outer_syntax () =
7026
69724548fad1 separate command tokens;
wenzelm
parents: 6868
diff changeset
   210
  let
46957
0c15caf47040 clarified Keyword.is_keyword: union of minor and major;
wenzelm
parents: 46950
diff changeset
   211
    val ((keywords, _), outer_syntax) =
0c15caf47040 clarified Keyword.is_keyword: union of minor and major;
wenzelm
parents: 46950
diff changeset
   212
      CRITICAL (fn () => (Keyword.dest (), #2 (get_syntax ())));
50213
7b73c0509835 refined outer syntax 'help' command;
wenzelm
parents: 50201
diff changeset
   213
    val (int_cmds, cmds) =
7b73c0509835 refined outer syntax 'help' command;
wenzelm
parents: 50201
diff changeset
   214
      List.partition (fn (_, Command {int_only, ...}) => int_only) (dest_commands outer_syntax);
7026
69724548fad1 separate command tokens;
wenzelm
parents: 6868
diff changeset
   215
  in
43711
608d1b451f67 less stateful outer_syntax;
wenzelm
parents: 43621
diff changeset
   216
    [Pretty.strs ("syntax keywords:" :: map quote keywords),
50213
7b73c0509835 refined outer syntax 'help' command;
wenzelm
parents: 50201
diff changeset
   217
      Pretty.big_list "commands:" (map pretty_command cmds),
7b73c0509835 refined outer syntax 'help' command;
wenzelm
parents: 50201
diff changeset
   218
      Pretty.big_list "interactive-only commands:" (map pretty_command int_cmds)]
9223
eb752c2fac22 removed help;
wenzelm
parents: 9213
diff changeset
   219
    |> Pretty.chunks |> Pretty.writeln
7026
69724548fad1 separate command tokens;
wenzelm
parents: 6868
diff changeset
   220
  end;
5829
0acb30dd92bc The global Isabelle/Isar outer syntax.
wenzelm
parents:
diff changeset
   221
0acb30dd92bc The global Isabelle/Isar outer syntax.
wenzelm
parents:
diff changeset
   222
0acb30dd92bc The global Isabelle/Isar outer syntax.
wenzelm
parents:
diff changeset
   223
9132
52286129faa5 moved header stuff to thy_header.ML;
wenzelm
parents: 9056
diff changeset
   224
(** toplevel parsing **)
5829
0acb30dd92bc The global Isabelle/Isar outer syntax.
wenzelm
parents:
diff changeset
   225
9132
52286129faa5 moved header stuff to thy_header.ML;
wenzelm
parents: 9056
diff changeset
   226
(* basic sources *)
6860
8dc6a1e6fa13 added sync;
wenzelm
parents: 6733
diff changeset
   227
26620
722cf4fdd4dd eliminated unused trace, read;
wenzelm
parents: 26611
diff changeset
   228
fun toplevel_source term do_recover cmd src =
9132
52286129faa5 moved header stuff to thy_header.ML;
wenzelm
parents: 9056
diff changeset
   229
  let
52286129faa5 moved header stuff to thy_header.ML;
wenzelm
parents: 9056
diff changeset
   230
    val no_terminator =
36959
f5417836dbea renamed structure OuterLex to Token and type token to Token.T, keeping legacy aliases for some time;
wenzelm
parents: 36955
diff changeset
   231
      Scan.unless Parse.semicolon (Scan.one (Token.not_sync andf Token.not_eof));
23682
cf4773532006 nested source: explicit interactive flag for recover avoids duplicate errors;
wenzelm
parents: 23679
diff changeset
   232
    fun recover int =
cf4773532006 nested source: explicit interactive flag for recover avoids duplicate errors;
wenzelm
parents: 23679
diff changeset
   233
      (int, fn _ => Scan.prompt "recover# " (Scan.repeat no_terminator) >> K [NONE]);
9132
52286129faa5 moved header stuff to thy_header.ML;
wenzelm
parents: 9056
diff changeset
   234
  in
52286129faa5 moved header stuff to thy_header.ML;
wenzelm
parents: 9056
diff changeset
   235
    src
36959
f5417836dbea renamed structure OuterLex to Token and type token to Token.T, keeping legacy aliases for some time;
wenzelm
parents: 36955
diff changeset
   236
    |> Token.source_proper
f5417836dbea renamed structure OuterLex to Token and type token to Token.T, keeping legacy aliases for some time;
wenzelm
parents: 36955
diff changeset
   237
    |> Source.source Token.stopper
36950
75b8f26f2f07 refer directly to structure Keyword and Parse;
wenzelm
parents: 33223
diff changeset
   238
      (Scan.bulk (Parse.$$$ "--" -- Parse.!!! Parse.doc_source >> K NONE || Parse.not_eof >> SOME))
23682
cf4773532006 nested source: explicit interactive flag for recover avoids duplicate errors;
wenzelm
parents: 23679
diff changeset
   239
        (Option.map recover do_recover)
19482
9f11af8f7ef9 tuned basic list operators (flat, maps, map_filter);
wenzelm
parents: 19060
diff changeset
   240
    |> Source.map_filter I
36959
f5417836dbea renamed structure OuterLex to Token and type token to Token.T, keeping legacy aliases for some time;
wenzelm
parents: 36955
diff changeset
   241
    |> Source.source Token.stopper
36950
75b8f26f2f07 refer directly to structure Keyword and Parse;
wenzelm
parents: 33223
diff changeset
   242
        (Scan.bulk (fn xs => Parse.!!! (parse_command term (cmd ())) xs))
23682
cf4773532006 nested source: explicit interactive flag for recover avoids duplicate errors;
wenzelm
parents: 23679
diff changeset
   243
        (Option.map recover do_recover)
19482
9f11af8f7ef9 tuned basic list operators (flat, maps, map_filter);
wenzelm
parents: 19060
diff changeset
   244
    |> Source.map_filter I
9132
52286129faa5 moved header stuff to thy_header.ML;
wenzelm
parents: 9056
diff changeset
   245
  end;
5829
0acb30dd92bc The global Isabelle/Isar outer syntax.
wenzelm
parents:
diff changeset
   246
7746
b52c1a632e6a simplified;
wenzelm
parents: 7735
diff changeset
   247
25580
6623674df897 added off-line parse;
wenzelm
parents: 25526
diff changeset
   248
(* off-line scanning/parsing *)
14925
0f86a8a694f8 added read (provides transition names and sources);
wenzelm
parents: 14687
diff changeset
   249
27839
0be8644c45eb Symbol.source/OuterLex.source: more explicit do_recover argument;
wenzelm
parents: 27831
diff changeset
   250
fun scan pos str =
16195
wenzelm
parents: 15989
diff changeset
   251
  Source.of_string str
40523
1050315f6ee2 simplified/robustified treatment of malformed symbols, which are now fully internalized (total Symbol.explode etc.);
wenzelm
parents: 38422
diff changeset
   252
  |> Symbol.source
36959
f5417836dbea renamed structure OuterLex to Token and type token to Token.T, keeping legacy aliases for some time;
wenzelm
parents: 36955
diff changeset
   253
  |> Token.source {do_recover = SOME false} Keyword.get_lexicons pos
16195
wenzelm
parents: 15989
diff changeset
   254
  |> Source.exhaust;
wenzelm
parents: 15989
diff changeset
   255
25580
6623674df897 added off-line parse;
wenzelm
parents: 25526
diff changeset
   256
fun parse pos str =
6623674df897 added off-line parse;
wenzelm
parents: 25526
diff changeset
   257
  Source.of_string str
40523
1050315f6ee2 simplified/robustified treatment of malformed symbols, which are now fully internalized (total Symbol.explode etc.);
wenzelm
parents: 38422
diff changeset
   258
  |> Symbol.source
36959
f5417836dbea renamed structure OuterLex to Token and type token to Token.T, keeping legacy aliases for some time;
wenzelm
parents: 36955
diff changeset
   259
  |> Token.source {do_recover = SOME false} Keyword.get_lexicons pos
43711
608d1b451f67 less stateful outer_syntax;
wenzelm
parents: 43621
diff changeset
   260
  |> toplevel_source false NONE lookup_commands_dynamic
25580
6623674df897 added off-line parse;
wenzelm
parents: 25526
diff changeset
   261
  |> Source.exhaust;
6623674df897 added off-line parse;
wenzelm
parents: 25526
diff changeset
   262
14091
ad6ba9c55190 A patch by david aspinall
nipkow
parents: 12943
diff changeset
   263
24868
2990c327d8c6 simplified interfaces for outer syntax;
wenzelm
parents: 24188
diff changeset
   264
(* interactive source of toplevel transformers *)
2990c327d8c6 simplified interfaces for outer syntax;
wenzelm
parents: 24188
diff changeset
   265
26600
f11515535c83 moved structure Isar to isar.ML;
wenzelm
parents: 26431
diff changeset
   266
type isar =
f11515535c83 moved structure Isar to isar.ML;
wenzelm
parents: 26431
diff changeset
   267
  (Toplevel.transition, (Toplevel.transition option,
36959
f5417836dbea renamed structure OuterLex to Token and type token to Token.T, keeping legacy aliases for some time;
wenzelm
parents: 36955
diff changeset
   268
    (Token.T, (Token.T option, (Token.T, (Token.T,
30573
49899f26fbd1 de-camelized Symbol_Pos;
wenzelm
parents: 30513
diff changeset
   269
      (Symbol_Pos.T, Position.T * (Symbol.symbol, (string, unit) Source.source)
27770
10d84e124a2f updated type of nested sources;
wenzelm
parents: 27720
diff changeset
   270
  Source.source) Source.source) Source.source) Source.source)
10d84e124a2f updated type of nested sources;
wenzelm
parents: 27720
diff changeset
   271
  Source.source) Source.source) Source.source) Source.source;
26600
f11515535c83 moved structure Isar to isar.ML;
wenzelm
parents: 26431
diff changeset
   272
38253
3d4e521014f7 Isabelle_Process: separate input fifo for commands (still using the old tty protocol);
wenzelm
parents: 38236
diff changeset
   273
fun isar in_stream term : isar =
3d4e521014f7 Isabelle_Process: separate input fifo for commands (still using the old tty protocol);
wenzelm
parents: 38236
diff changeset
   274
  Source.tty in_stream
40523
1050315f6ee2 simplified/robustified treatment of malformed symbols, which are now fully internalized (total Symbol.explode etc.);
wenzelm
parents: 38422
diff changeset
   275
  |> Symbol.source
36959
f5417836dbea renamed structure OuterLex to Token and type token to Token.T, keeping legacy aliases for some time;
wenzelm
parents: 36955
diff changeset
   276
  |> Token.source {do_recover = SOME true} Keyword.get_lexicons Position.none
43711
608d1b451f67 less stateful outer_syntax;
wenzelm
parents: 43621
diff changeset
   277
  |> toplevel_source term (SOME true) lookup_commands_dynamic;
24868
2990c327d8c6 simplified interfaces for outer syntax;
wenzelm
parents: 24188
diff changeset
   278
2990c327d8c6 simplified interfaces for outer syntax;
wenzelm
parents: 24188
diff changeset
   279
48918
6e5fd4585512 check side-comments of command spans (normally filtered out in Outer_Syntax.toplevel_source);
wenzelm
parents: 48864
diff changeset
   280
(* side-comments *)
6e5fd4585512 check side-comments of command spans (normally filtered out in Outer_Syntax.toplevel_source);
wenzelm
parents: 48864
diff changeset
   281
6e5fd4585512 check side-comments of command spans (normally filtered out in Outer_Syntax.toplevel_source);
wenzelm
parents: 48864
diff changeset
   282
local
6e5fd4585512 check side-comments of command spans (normally filtered out in Outer_Syntax.toplevel_source);
wenzelm
parents: 48864
diff changeset
   283
6e5fd4585512 check side-comments of command spans (normally filtered out in Outer_Syntax.toplevel_source);
wenzelm
parents: 48864
diff changeset
   284
fun cmts (t1 :: t2 :: toks) =
6e5fd4585512 check side-comments of command spans (normally filtered out in Outer_Syntax.toplevel_source);
wenzelm
parents: 48864
diff changeset
   285
      if Token.keyword_with (fn s => s = "--") t1 then t2 :: cmts toks
6e5fd4585512 check side-comments of command spans (normally filtered out in Outer_Syntax.toplevel_source);
wenzelm
parents: 48864
diff changeset
   286
      else cmts (t2 :: toks)
49564
wenzelm
parents: 48992
diff changeset
   287
  | cmts _ = [];
48918
6e5fd4585512 check side-comments of command spans (normally filtered out in Outer_Syntax.toplevel_source);
wenzelm
parents: 48864
diff changeset
   288
6e5fd4585512 check side-comments of command spans (normally filtered out in Outer_Syntax.toplevel_source);
wenzelm
parents: 48864
diff changeset
   289
in
6e5fd4585512 check side-comments of command spans (normally filtered out in Outer_Syntax.toplevel_source);
wenzelm
parents: 48864
diff changeset
   290
6e5fd4585512 check side-comments of command spans (normally filtered out in Outer_Syntax.toplevel_source);
wenzelm
parents: 48864
diff changeset
   291
val span_cmts = filter Token.is_proper #> cmts;
6e5fd4585512 check side-comments of command spans (normally filtered out in Outer_Syntax.toplevel_source);
wenzelm
parents: 48864
diff changeset
   292
6e5fd4585512 check side-comments of command spans (normally filtered out in Outer_Syntax.toplevel_source);
wenzelm
parents: 48864
diff changeset
   293
end;
6e5fd4585512 check side-comments of command spans (normally filtered out in Outer_Syntax.toplevel_source);
wenzelm
parents: 48864
diff changeset
   294
6e5fd4585512 check side-comments of command spans (normally filtered out in Outer_Syntax.toplevel_source);
wenzelm
parents: 48864
diff changeset
   295
51271
e8d2ecf6aaac tuned comment;
wenzelm
parents: 51268
diff changeset
   296
(* read command span -- fail-safe *)
27839
0be8644c45eb Symbol.source/OuterLex.source: more explicit do_recover argument;
wenzelm
parents: 27831
diff changeset
   297
44658
5bec9c15ef29 more direct Token.range_pos and Outer_Syntax.read_command, bypassing Thy_Syntax.span;
wenzelm
parents: 44478
diff changeset
   298
fun read_span outer_syntax toks =
27839
0be8644c45eb Symbol.source/OuterLex.source: more explicit do_recover argument;
wenzelm
parents: 27831
diff changeset
   299
  let
43711
608d1b451f67 less stateful outer_syntax;
wenzelm
parents: 43621
diff changeset
   300
    val commands = lookup_commands outer_syntax;
48749
c197b3c3e7fa some attempts to keep malformed syntax errors focussed, without too much red spilled onto the document view;
wenzelm
parents: 48647
diff changeset
   301
48771
2ea997196d04 clarified Command.range vs. Command.proper_range according to Scala version, which is potentially relevant for command status markup;
wenzelm
parents: 48768
diff changeset
   302
    val proper_range = Position.set_range (Command.proper_range toks);
48749
c197b3c3e7fa some attempts to keep malformed syntax errors focussed, without too much red spilled onto the document view;
wenzelm
parents: 48647
diff changeset
   303
    val pos =
c197b3c3e7fa some attempts to keep malformed syntax errors focussed, without too much red spilled onto the document view;
wenzelm
parents: 48647
diff changeset
   304
      (case find_first Token.is_command toks of
c197b3c3e7fa some attempts to keep malformed syntax errors focussed, without too much red spilled onto the document view;
wenzelm
parents: 48647
diff changeset
   305
        SOME tok => Token.position_of tok
48771
2ea997196d04 clarified Command.range vs. Command.proper_range according to Scala version, which is potentially relevant for command status markup;
wenzelm
parents: 48768
diff changeset
   306
      | NONE => proper_range);
48647
a5144c4c26a2 report commands as formal entities, with def/ref positions;
wenzelm
parents: 48646
diff changeset
   307
a5144c4c26a2 report commands as formal entities, with def/ref positions;
wenzelm
parents: 48646
diff changeset
   308
    fun command_reports tok =
48749
c197b3c3e7fa some attempts to keep malformed syntax errors focussed, without too much red spilled onto the document view;
wenzelm
parents: 48647
diff changeset
   309
      if Token.is_command tok then
48647
a5144c4c26a2 report commands as formal entities, with def/ref positions;
wenzelm
parents: 48646
diff changeset
   310
        let val name = Token.content_of tok in
a5144c4c26a2 report commands as formal entities, with def/ref positions;
wenzelm
parents: 48646
diff changeset
   311
          (case commands name of
a5144c4c26a2 report commands as formal entities, with def/ref positions;
wenzelm
parents: 48646
diff changeset
   312
            NONE => []
48768
abc45de5bb22 clarified "bad" markup: proper body text, invent missing serial on Scala side (counting backwards);
wenzelm
parents: 48749
diff changeset
   313
          | SOME cmd => [((Token.position_of tok, command_markup false (name, cmd)), "")])
48647
a5144c4c26a2 report commands as formal entities, with def/ref positions;
wenzelm
parents: 48646
diff changeset
   314
        end
a5144c4c26a2 report commands as formal entities, with def/ref positions;
wenzelm
parents: 48646
diff changeset
   315
      else [];
48749
c197b3c3e7fa some attempts to keep malformed syntax errors focussed, without too much red spilled onto the document view;
wenzelm
parents: 48647
diff changeset
   316
c197b3c3e7fa some attempts to keep malformed syntax errors focussed, without too much red spilled onto the document view;
wenzelm
parents: 48647
diff changeset
   317
    val (is_malformed, token_reports) = Thy_Syntax.reports_of_tokens toks;
48768
abc45de5bb22 clarified "bad" markup: proper body text, invent missing serial on Scala side (counting backwards);
wenzelm
parents: 48749
diff changeset
   318
    val _ = Position.reports_text (token_reports @ maps command_reports toks);
27839
0be8644c45eb Symbol.source/OuterLex.source: more explicit do_recover argument;
wenzelm
parents: 27831
diff changeset
   319
  in
51268
fcc4b89a600d simplified Outer_Syntax.read_span: internalized Toplevel.is_ignored;
wenzelm
parents: 51225
diff changeset
   320
    if is_malformed then Toplevel.malformed pos "Malformed command syntax"
48749
c197b3c3e7fa some attempts to keep malformed syntax errors focussed, without too much red spilled onto the document view;
wenzelm
parents: 48647
diff changeset
   321
    else
c197b3c3e7fa some attempts to keep malformed syntax errors focussed, without too much red spilled onto the document view;
wenzelm
parents: 48647
diff changeset
   322
      (case Source.exhaust (toplevel_source false NONE (K commands) (Source.of_list toks)) of
c197b3c3e7fa some attempts to keep malformed syntax errors focussed, without too much red spilled onto the document view;
wenzelm
parents: 48647
diff changeset
   323
        [tr] =>
c197b3c3e7fa some attempts to keep malformed syntax errors focussed, without too much red spilled onto the document view;
wenzelm
parents: 48647
diff changeset
   324
          if Keyword.is_control (Toplevel.name_of tr) then
51268
fcc4b89a600d simplified Outer_Syntax.read_span: internalized Toplevel.is_ignored;
wenzelm
parents: 51225
diff changeset
   325
            Toplevel.malformed pos "Illegal control command"
fcc4b89a600d simplified Outer_Syntax.read_span: internalized Toplevel.is_ignored;
wenzelm
parents: 51225
diff changeset
   326
          else tr
fcc4b89a600d simplified Outer_Syntax.read_span: internalized Toplevel.is_ignored;
wenzelm
parents: 51225
diff changeset
   327
      | [] => Toplevel.ignored (Position.set_range (Command.range toks))
fcc4b89a600d simplified Outer_Syntax.read_span: internalized Toplevel.is_ignored;
wenzelm
parents: 51225
diff changeset
   328
      | _ => Toplevel.malformed proper_range "Exactly one command expected")
fcc4b89a600d simplified Outer_Syntax.read_span: internalized Toplevel.is_ignored;
wenzelm
parents: 51225
diff changeset
   329
      handle ERROR msg => Toplevel.malformed proper_range msg
28436
4faf705a177d load_thy: more precise treatment of improper cmd or proof (notably 'oops');
wenzelm
parents: 28432
diff changeset
   330
  end;
28432
944cb67f809a load_thy: Toplevel.excursion based on units of command/proof pairs;
wenzelm
parents: 28424
diff changeset
   331
5829
0acb30dd92bc The global Isabelle/Isar outer syntax.
wenzelm
parents:
diff changeset
   332
end;
36953
2af1ad9aa1a3 renamed structure OuterSyntax to Outer_Syntax, keeping the old name as alias for some time;
wenzelm
parents: 36950
diff changeset
   333