src/Pure/PIDE/command.ML
author wenzelm
Sun, 24 Feb 2013 14:11:51 +0100
changeset 51266 3007d0bc9cb1
parent 50914 fe4714886d92
child 51284 59a03019f3bf
permissions -rw-r--r--
unified Command.is_proper in ML with Scala (see also 123be08eed88);
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
47336
bed4b2738d8a separate module for prover command execution;
wenzelm
parents:
diff changeset
     1
(*  Title:      Pure/PIDE/command.ML
bed4b2738d8a separate module for prover command execution;
wenzelm
parents:
diff changeset
     2
    Author:     Makarius
bed4b2738d8a separate module for prover command execution;
wenzelm
parents:
diff changeset
     3
bed4b2738d8a separate module for prover command execution;
wenzelm
parents:
diff changeset
     4
Prover command execution.
bed4b2738d8a separate module for prover command execution;
wenzelm
parents:
diff changeset
     5
*)
bed4b2738d8a separate module for prover command execution;
wenzelm
parents:
diff changeset
     6
bed4b2738d8a separate module for prover command execution;
wenzelm
parents:
diff changeset
     7
signature COMMAND =
bed4b2738d8a separate module for prover command execution;
wenzelm
parents:
diff changeset
     8
sig
48771
2ea997196d04 clarified Command.range vs. Command.proper_range according to Scala version, which is potentially relevant for command status markup;
wenzelm
parents: 47395
diff changeset
     9
  val range: Token.T list -> Position.range
2ea997196d04 clarified Command.range vs. Command.proper_range according to Scala version, which is potentially relevant for command status markup;
wenzelm
parents: 47395
diff changeset
    10
  val proper_range: Token.T list -> Position.range
47341
00f6279bb67a Command.memo including physical interrupts (unlike Lazy.lazy);
wenzelm
parents: 47336
diff changeset
    11
  type 'a memo
00f6279bb67a Command.memo including physical interrupts (unlike Lazy.lazy);
wenzelm
parents: 47336
diff changeset
    12
  val memo: (unit -> 'a) -> 'a memo
00f6279bb67a Command.memo including physical interrupts (unlike Lazy.lazy);
wenzelm
parents: 47336
diff changeset
    13
  val memo_value: 'a -> 'a memo
47342
7828c7b3c143 more explicit memo_eval vs. memo_result, to enforce bottom-up execution;
wenzelm
parents: 47341
diff changeset
    14
  val memo_eval: 'a memo -> 'a
7828c7b3c143 more explicit memo_eval vs. memo_result, to enforce bottom-up execution;
wenzelm
parents: 47341
diff changeset
    15
  val memo_result: 'a memo -> 'a
48918
6e5fd4585512 check side-comments of command spans (normally filtered out in Outer_Syntax.toplevel_source);
wenzelm
parents: 48772
diff changeset
    16
  val run_command: Toplevel.transition * Token.T list ->
48772
e46cd0d26481 vacuous execution after first malformed command;
wenzelm
parents: 48771
diff changeset
    17
    Toplevel.state * bool -> (Toplevel.state * bool) * unit lazy
47336
bed4b2738d8a separate module for prover command execution;
wenzelm
parents:
diff changeset
    18
end;
bed4b2738d8a separate module for prover command execution;
wenzelm
parents:
diff changeset
    19
bed4b2738d8a separate module for prover command execution;
wenzelm
parents:
diff changeset
    20
structure Command: COMMAND =
bed4b2738d8a separate module for prover command execution;
wenzelm
parents:
diff changeset
    21
struct
bed4b2738d8a separate module for prover command execution;
wenzelm
parents:
diff changeset
    22
48771
2ea997196d04 clarified Command.range vs. Command.proper_range according to Scala version, which is potentially relevant for command status markup;
wenzelm
parents: 47395
diff changeset
    23
(* span range *)
2ea997196d04 clarified Command.range vs. Command.proper_range according to Scala version, which is potentially relevant for command status markup;
wenzelm
parents: 47395
diff changeset
    24
49866
619acbd72664 more proof method text position information;
wenzelm
parents: 49036
diff changeset
    25
val range = Token.position_range_of;
51266
3007d0bc9cb1 unified Command.is_proper in ML with Scala (see also 123be08eed88);
wenzelm
parents: 50914
diff changeset
    26
val proper_range = Token.position_range_of o #1 o take_suffix Token.is_improper;
48771
2ea997196d04 clarified Command.range vs. Command.proper_range according to Scala version, which is potentially relevant for command status markup;
wenzelm
parents: 47395
diff changeset
    27
2ea997196d04 clarified Command.range vs. Command.proper_range according to Scala version, which is potentially relevant for command status markup;
wenzelm
parents: 47395
diff changeset
    28
47341
00f6279bb67a Command.memo including physical interrupts (unlike Lazy.lazy);
wenzelm
parents: 47336
diff changeset
    29
(* memo results *)
00f6279bb67a Command.memo including physical interrupts (unlike Lazy.lazy);
wenzelm
parents: 47336
diff changeset
    30
00f6279bb67a Command.memo including physical interrupts (unlike Lazy.lazy);
wenzelm
parents: 47336
diff changeset
    31
datatype 'a expr =
00f6279bb67a Command.memo including physical interrupts (unlike Lazy.lazy);
wenzelm
parents: 47336
diff changeset
    32
  Expr of unit -> 'a |
00f6279bb67a Command.memo including physical interrupts (unlike Lazy.lazy);
wenzelm
parents: 47336
diff changeset
    33
  Result of 'a Exn.result;
00f6279bb67a Command.memo including physical interrupts (unlike Lazy.lazy);
wenzelm
parents: 47336
diff changeset
    34
00f6279bb67a Command.memo including physical interrupts (unlike Lazy.lazy);
wenzelm
parents: 47336
diff changeset
    35
abstype 'a memo = Memo of 'a expr Synchronized.var
00f6279bb67a Command.memo including physical interrupts (unlike Lazy.lazy);
wenzelm
parents: 47336
diff changeset
    36
with
00f6279bb67a Command.memo including physical interrupts (unlike Lazy.lazy);
wenzelm
parents: 47336
diff changeset
    37
00f6279bb67a Command.memo including physical interrupts (unlike Lazy.lazy);
wenzelm
parents: 47336
diff changeset
    38
fun memo e = Memo (Synchronized.var "Command.memo" (Expr e));
00f6279bb67a Command.memo including physical interrupts (unlike Lazy.lazy);
wenzelm
parents: 47336
diff changeset
    39
fun memo_value a = Memo (Synchronized.var "Command.memo" (Result (Exn.Res a)));
00f6279bb67a Command.memo including physical interrupts (unlike Lazy.lazy);
wenzelm
parents: 47336
diff changeset
    40
47342
7828c7b3c143 more explicit memo_eval vs. memo_result, to enforce bottom-up execution;
wenzelm
parents: 47341
diff changeset
    41
fun memo_eval (Memo v) =
47341
00f6279bb67a Command.memo including physical interrupts (unlike Lazy.lazy);
wenzelm
parents: 47336
diff changeset
    42
  (case Synchronized.value v of
00f6279bb67a Command.memo including physical interrupts (unlike Lazy.lazy);
wenzelm
parents: 47336
diff changeset
    43
    Result res => res
00f6279bb67a Command.memo including physical interrupts (unlike Lazy.lazy);
wenzelm
parents: 47336
diff changeset
    44
  | _ =>
00f6279bb67a Command.memo including physical interrupts (unlike Lazy.lazy);
wenzelm
parents: 47336
diff changeset
    45
      Synchronized.guarded_access v
00f6279bb67a Command.memo including physical interrupts (unlike Lazy.lazy);
wenzelm
parents: 47336
diff changeset
    46
        (fn Result res => SOME (res, Result res)
00f6279bb67a Command.memo including physical interrupts (unlike Lazy.lazy);
wenzelm
parents: 47336
diff changeset
    47
          | Expr e =>
00f6279bb67a Command.memo including physical interrupts (unlike Lazy.lazy);
wenzelm
parents: 47336
diff changeset
    48
              let val res = Exn.capture e ();  (*memoing of physical interrupts!*)
47342
7828c7b3c143 more explicit memo_eval vs. memo_result, to enforce bottom-up execution;
wenzelm
parents: 47341
diff changeset
    49
              in SOME (res, Result res) end))
7828c7b3c143 more explicit memo_eval vs. memo_result, to enforce bottom-up execution;
wenzelm
parents: 47341
diff changeset
    50
  |> Exn.release;
7828c7b3c143 more explicit memo_eval vs. memo_result, to enforce bottom-up execution;
wenzelm
parents: 47341
diff changeset
    51
7828c7b3c143 more explicit memo_eval vs. memo_result, to enforce bottom-up execution;
wenzelm
parents: 47341
diff changeset
    52
fun memo_result (Memo v) =
7828c7b3c143 more explicit memo_eval vs. memo_result, to enforce bottom-up execution;
wenzelm
parents: 47341
diff changeset
    53
  (case Synchronized.value v of
7828c7b3c143 more explicit memo_eval vs. memo_result, to enforce bottom-up execution;
wenzelm
parents: 47341
diff changeset
    54
    Result res => Exn.release res
7828c7b3c143 more explicit memo_eval vs. memo_result, to enforce bottom-up execution;
wenzelm
parents: 47341
diff changeset
    55
  | _ => raise Fail "Unfinished memo result");
47341
00f6279bb67a Command.memo including physical interrupts (unlike Lazy.lazy);
wenzelm
parents: 47336
diff changeset
    56
00f6279bb67a Command.memo including physical interrupts (unlike Lazy.lazy);
wenzelm
parents: 47336
diff changeset
    57
end;
00f6279bb67a Command.memo including physical interrupts (unlike Lazy.lazy);
wenzelm
parents: 47336
diff changeset
    58
00f6279bb67a Command.memo including physical interrupts (unlike Lazy.lazy);
wenzelm
parents: 47336
diff changeset
    59
00f6279bb67a Command.memo including physical interrupts (unlike Lazy.lazy);
wenzelm
parents: 47336
diff changeset
    60
(* run command *)
47336
bed4b2738d8a separate module for prover command execution;
wenzelm
parents:
diff changeset
    61
bed4b2738d8a separate module for prover command execution;
wenzelm
parents:
diff changeset
    62
local
bed4b2738d8a separate module for prover command execution;
wenzelm
parents:
diff changeset
    63
bed4b2738d8a separate module for prover command execution;
wenzelm
parents:
diff changeset
    64
fun run int tr st =
bed4b2738d8a separate module for prover command execution;
wenzelm
parents:
diff changeset
    65
  (case Toplevel.transition int tr st of
bed4b2738d8a separate module for prover command execution;
wenzelm
parents:
diff changeset
    66
    SOME (st', NONE) => ([], SOME st')
50914
fe4714886d92 identify future results more carefully, to avoid odd duplication of error messages, notably from forked goals;
wenzelm
parents: 50911
diff changeset
    67
  | SOME (_, SOME (exn, _)) => (ML_Compiler.exn_messages_ids exn, NONE)
fe4714886d92 identify future results more carefully, to avoid odd duplication of error messages, notably from forked goals;
wenzelm
parents: 50911
diff changeset
    68
  | NONE => (ML_Compiler.exn_messages_ids Runtime.TERMINATE, NONE));
47336
bed4b2738d8a separate module for prover command execution;
wenzelm
parents:
diff changeset
    69
48918
6e5fd4585512 check side-comments of command spans (normally filtered out in Outer_Syntax.toplevel_source);
wenzelm
parents: 48772
diff changeset
    70
fun check_cmts tr cmts st =
6e5fd4585512 check side-comments of command spans (normally filtered out in Outer_Syntax.toplevel_source);
wenzelm
parents: 48772
diff changeset
    71
  Toplevel.setmp_thread_position tr
6e5fd4585512 check side-comments of command spans (normally filtered out in Outer_Syntax.toplevel_source);
wenzelm
parents: 48772
diff changeset
    72
    (fn () => cmts
6e5fd4585512 check side-comments of command spans (normally filtered out in Outer_Syntax.toplevel_source);
wenzelm
parents: 48772
diff changeset
    73
      |> maps (fn cmt =>
6e5fd4585512 check side-comments of command spans (normally filtered out in Outer_Syntax.toplevel_source);
wenzelm
parents: 48772
diff changeset
    74
        (Thy_Output.check_text (Token.source_position_of cmt) st; [])
50914
fe4714886d92 identify future results more carefully, to avoid odd duplication of error messages, notably from forked goals;
wenzelm
parents: 50911
diff changeset
    75
          handle exn => ML_Compiler.exn_messages_ids exn)) ();
48918
6e5fd4585512 check side-comments of command spans (normally filtered out in Outer_Syntax.toplevel_source);
wenzelm
parents: 48772
diff changeset
    76
47336
bed4b2738d8a separate module for prover command execution;
wenzelm
parents:
diff changeset
    77
fun timing tr t =
50201
c26369c9eda6 Isabelle-specific implementation of quasi-abstract markup elements -- back to module arrangement before d83797ef0d2d;
wenzelm
parents: 49866
diff changeset
    78
  if Timing.is_relevant t then Toplevel.status tr (Markup.timing t) else ();
47336
bed4b2738d8a separate module for prover command execution;
wenzelm
parents:
diff changeset
    79
bed4b2738d8a separate module for prover command execution;
wenzelm
parents:
diff changeset
    80
fun proof_status tr st =
bed4b2738d8a separate module for prover command execution;
wenzelm
parents:
diff changeset
    81
  (case try Toplevel.proof_of st of
bed4b2738d8a separate module for prover command execution;
wenzelm
parents:
diff changeset
    82
    SOME prf => Toplevel.status tr (Proof.status_markup prf)
bed4b2738d8a separate module for prover command execution;
wenzelm
parents:
diff changeset
    83
  | NONE => ());
bed4b2738d8a separate module for prover command execution;
wenzelm
parents:
diff changeset
    84
bed4b2738d8a separate module for prover command execution;
wenzelm
parents:
diff changeset
    85
val no_print = Lazy.value ();
bed4b2738d8a separate module for prover command execution;
wenzelm
parents:
diff changeset
    86
bed4b2738d8a separate module for prover command execution;
wenzelm
parents:
diff changeset
    87
fun print_state tr st =
bed4b2738d8a separate module for prover command execution;
wenzelm
parents:
diff changeset
    88
  (Lazy.lazy o Toplevel.setmp_thread_position tr)
bed4b2738d8a separate module for prover command execution;
wenzelm
parents:
diff changeset
    89
    (fn () => Toplevel.print_state false st);
bed4b2738d8a separate module for prover command execution;
wenzelm
parents:
diff changeset
    90
bed4b2738d8a separate module for prover command execution;
wenzelm
parents:
diff changeset
    91
in
bed4b2738d8a separate module for prover command execution;
wenzelm
parents:
diff changeset
    92
48918
6e5fd4585512 check side-comments of command spans (normally filtered out in Outer_Syntax.toplevel_source);
wenzelm
parents: 48772
diff changeset
    93
fun run_command (tr, cmts) (st, malformed) =
48772
e46cd0d26481 vacuous execution after first malformed command;
wenzelm
parents: 48771
diff changeset
    94
  if malformed then ((Toplevel.toplevel, malformed), no_print)
e46cd0d26481 vacuous execution after first malformed command;
wenzelm
parents: 48771
diff changeset
    95
  else
e46cd0d26481 vacuous execution after first malformed command;
wenzelm
parents: 48771
diff changeset
    96
    let
e46cd0d26481 vacuous execution after first malformed command;
wenzelm
parents: 48771
diff changeset
    97
      val malformed' = Toplevel.is_malformed tr;
e46cd0d26481 vacuous execution after first malformed command;
wenzelm
parents: 48771
diff changeset
    98
      val is_init = Toplevel.is_init tr;
e46cd0d26481 vacuous execution after first malformed command;
wenzelm
parents: 48771
diff changeset
    99
      val is_proof = Keyword.is_proof (Toplevel.name_of tr);
47336
bed4b2738d8a separate module for prover command execution;
wenzelm
parents:
diff changeset
   100
48772
e46cd0d26481 vacuous execution after first malformed command;
wenzelm
parents: 48771
diff changeset
   101
      val _ = Multithreading.interrupted ();
50201
c26369c9eda6 Isabelle-specific implementation of quasi-abstract markup elements -- back to module arrangement before d83797ef0d2d;
wenzelm
parents: 49866
diff changeset
   102
      val _ = Toplevel.status tr Markup.running;
48772
e46cd0d26481 vacuous execution after first malformed command;
wenzelm
parents: 48771
diff changeset
   103
      val start = Timing.start ();
48918
6e5fd4585512 check side-comments of command spans (normally filtered out in Outer_Syntax.toplevel_source);
wenzelm
parents: 48772
diff changeset
   104
      val (errs1, result) = run (is_init orelse is_proof) (Toplevel.set_print false tr) st;
6e5fd4585512 check side-comments of command spans (normally filtered out in Outer_Syntax.toplevel_source);
wenzelm
parents: 48772
diff changeset
   105
      val errs2 = (case result of NONE => [] | SOME st' => check_cmts tr cmts st');
6e5fd4585512 check side-comments of command spans (normally filtered out in Outer_Syntax.toplevel_source);
wenzelm
parents: 48772
diff changeset
   106
      val errs = errs1 @ errs2;
48772
e46cd0d26481 vacuous execution after first malformed command;
wenzelm
parents: 48771
diff changeset
   107
      val _ = timing tr (Timing.result start);
50201
c26369c9eda6 Isabelle-specific implementation of quasi-abstract markup elements -- back to module arrangement before d83797ef0d2d;
wenzelm
parents: 49866
diff changeset
   108
      val _ = Toplevel.status tr Markup.finished;
50914
fe4714886d92 identify future results more carefully, to avoid odd duplication of error messages, notably from forked goals;
wenzelm
parents: 50911
diff changeset
   109
      val _ = List.app (Future.error_msg (Toplevel.pos_of tr)) errs;
48772
e46cd0d26481 vacuous execution after first malformed command;
wenzelm
parents: 48771
diff changeset
   110
    in
e46cd0d26481 vacuous execution after first malformed command;
wenzelm
parents: 48771
diff changeset
   111
      (case result of
e46cd0d26481 vacuous execution after first malformed command;
wenzelm
parents: 48771
diff changeset
   112
        NONE =>
e46cd0d26481 vacuous execution after first malformed command;
wenzelm
parents: 48771
diff changeset
   113
          let
e46cd0d26481 vacuous execution after first malformed command;
wenzelm
parents: 48771
diff changeset
   114
            val _ = if null errs then Exn.interrupt () else ();
50201
c26369c9eda6 Isabelle-specific implementation of quasi-abstract markup elements -- back to module arrangement before d83797ef0d2d;
wenzelm
parents: 49866
diff changeset
   115
            val _ = Toplevel.status tr Markup.failed;
48772
e46cd0d26481 vacuous execution after first malformed command;
wenzelm
parents: 48771
diff changeset
   116
          in ((st, malformed'), no_print) end
e46cd0d26481 vacuous execution after first malformed command;
wenzelm
parents: 48771
diff changeset
   117
      | SOME st' =>
e46cd0d26481 vacuous execution after first malformed command;
wenzelm
parents: 48771
diff changeset
   118
          let
e46cd0d26481 vacuous execution after first malformed command;
wenzelm
parents: 48771
diff changeset
   119
            val _ = proof_status tr st';
e46cd0d26481 vacuous execution after first malformed command;
wenzelm
parents: 48771
diff changeset
   120
            val do_print =
e46cd0d26481 vacuous execution after first malformed command;
wenzelm
parents: 48771
diff changeset
   121
              not is_init andalso
e46cd0d26481 vacuous execution after first malformed command;
wenzelm
parents: 48771
diff changeset
   122
                (Toplevel.print_of tr orelse (is_proof andalso Toplevel.is_proof st'));
e46cd0d26481 vacuous execution after first malformed command;
wenzelm
parents: 48771
diff changeset
   123
          in ((st', malformed'), if do_print then print_state tr st' else no_print) end)
e46cd0d26481 vacuous execution after first malformed command;
wenzelm
parents: 48771
diff changeset
   124
    end;
47336
bed4b2738d8a separate module for prover command execution;
wenzelm
parents:
diff changeset
   125
bed4b2738d8a separate module for prover command execution;
wenzelm
parents:
diff changeset
   126
end;
bed4b2738d8a separate module for prover command execution;
wenzelm
parents:
diff changeset
   127
bed4b2738d8a separate module for prover command execution;
wenzelm
parents:
diff changeset
   128
end;
bed4b2738d8a separate module for prover command execution;
wenzelm
parents:
diff changeset
   129