src/Pure/PIDE/command.ML
author wenzelm
Sat, 11 Aug 2012 19:34:36 +0200
changeset 48772 e46cd0d26481
parent 48771 2ea997196d04
child 48918 6e5fd4585512
permissions -rw-r--r--
vacuous execution after first malformed command;
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
48772
e46cd0d26481 vacuous execution after first malformed command;
wenzelm
parents: 48771
diff changeset
    16
  val run_command: Toplevel.transition ->
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
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
    25
fun range [] = (Position.none, Position.none)
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
    26
  | range toks =
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
      let
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
        val start_pos = Token.position_of (hd toks);
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
    29
        val end_pos = Token.end_position_of (List.last toks);
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
    30
      in (start_pos, end_pos) end;
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
    31
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
    32
val proper_range = range o #1 o take_suffix Token.is_space;
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
    33
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
    34
47341
00f6279bb67a Command.memo including physical interrupts (unlike Lazy.lazy);
wenzelm
parents: 47336
diff changeset
    35
(* memo results *)
00f6279bb67a Command.memo including physical interrupts (unlike Lazy.lazy);
wenzelm
parents: 47336
diff changeset
    36
00f6279bb67a Command.memo including physical interrupts (unlike Lazy.lazy);
wenzelm
parents: 47336
diff changeset
    37
datatype 'a expr =
00f6279bb67a Command.memo including physical interrupts (unlike Lazy.lazy);
wenzelm
parents: 47336
diff changeset
    38
  Expr of unit -> 'a |
00f6279bb67a Command.memo including physical interrupts (unlike Lazy.lazy);
wenzelm
parents: 47336
diff changeset
    39
  Result of 'a Exn.result;
00f6279bb67a Command.memo including physical interrupts (unlike Lazy.lazy);
wenzelm
parents: 47336
diff changeset
    40
00f6279bb67a Command.memo including physical interrupts (unlike Lazy.lazy);
wenzelm
parents: 47336
diff changeset
    41
abstype 'a memo = Memo of 'a expr Synchronized.var
00f6279bb67a Command.memo including physical interrupts (unlike Lazy.lazy);
wenzelm
parents: 47336
diff changeset
    42
with
00f6279bb67a Command.memo including physical interrupts (unlike Lazy.lazy);
wenzelm
parents: 47336
diff changeset
    43
00f6279bb67a Command.memo including physical interrupts (unlike Lazy.lazy);
wenzelm
parents: 47336
diff changeset
    44
fun memo e = Memo (Synchronized.var "Command.memo" (Expr e));
00f6279bb67a Command.memo including physical interrupts (unlike Lazy.lazy);
wenzelm
parents: 47336
diff changeset
    45
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
    46
47342
7828c7b3c143 more explicit memo_eval vs. memo_result, to enforce bottom-up execution;
wenzelm
parents: 47341
diff changeset
    47
fun memo_eval (Memo v) =
47341
00f6279bb67a Command.memo including physical interrupts (unlike Lazy.lazy);
wenzelm
parents: 47336
diff changeset
    48
  (case Synchronized.value v of
00f6279bb67a Command.memo including physical interrupts (unlike Lazy.lazy);
wenzelm
parents: 47336
diff changeset
    49
    Result res => res
00f6279bb67a Command.memo including physical interrupts (unlike Lazy.lazy);
wenzelm
parents: 47336
diff changeset
    50
  | _ =>
00f6279bb67a Command.memo including physical interrupts (unlike Lazy.lazy);
wenzelm
parents: 47336
diff changeset
    51
      Synchronized.guarded_access v
00f6279bb67a Command.memo including physical interrupts (unlike Lazy.lazy);
wenzelm
parents: 47336
diff changeset
    52
        (fn Result res => SOME (res, Result res)
00f6279bb67a Command.memo including physical interrupts (unlike Lazy.lazy);
wenzelm
parents: 47336
diff changeset
    53
          | Expr e =>
00f6279bb67a Command.memo including physical interrupts (unlike Lazy.lazy);
wenzelm
parents: 47336
diff changeset
    54
              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
    55
              in SOME (res, Result res) end))
7828c7b3c143 more explicit memo_eval vs. memo_result, to enforce bottom-up execution;
wenzelm
parents: 47341
diff changeset
    56
  |> Exn.release;
7828c7b3c143 more explicit memo_eval vs. memo_result, to enforce bottom-up execution;
wenzelm
parents: 47341
diff changeset
    57
7828c7b3c143 more explicit memo_eval vs. memo_result, to enforce bottom-up execution;
wenzelm
parents: 47341
diff changeset
    58
fun memo_result (Memo v) =
7828c7b3c143 more explicit memo_eval vs. memo_result, to enforce bottom-up execution;
wenzelm
parents: 47341
diff changeset
    59
  (case Synchronized.value v of
7828c7b3c143 more explicit memo_eval vs. memo_result, to enforce bottom-up execution;
wenzelm
parents: 47341
diff changeset
    60
    Result res => Exn.release res
7828c7b3c143 more explicit memo_eval vs. memo_result, to enforce bottom-up execution;
wenzelm
parents: 47341
diff changeset
    61
  | _ => raise Fail "Unfinished memo result");
47341
00f6279bb67a Command.memo including physical interrupts (unlike Lazy.lazy);
wenzelm
parents: 47336
diff changeset
    62
00f6279bb67a Command.memo including physical interrupts (unlike Lazy.lazy);
wenzelm
parents: 47336
diff changeset
    63
end;
00f6279bb67a Command.memo including physical interrupts (unlike Lazy.lazy);
wenzelm
parents: 47336
diff changeset
    64
00f6279bb67a Command.memo including physical interrupts (unlike Lazy.lazy);
wenzelm
parents: 47336
diff changeset
    65
00f6279bb67a Command.memo including physical interrupts (unlike Lazy.lazy);
wenzelm
parents: 47336
diff changeset
    66
(* run command *)
47336
bed4b2738d8a separate module for prover command execution;
wenzelm
parents:
diff changeset
    67
bed4b2738d8a separate module for prover command execution;
wenzelm
parents:
diff changeset
    68
local
bed4b2738d8a separate module for prover command execution;
wenzelm
parents:
diff changeset
    69
bed4b2738d8a separate module for prover command execution;
wenzelm
parents:
diff changeset
    70
fun run int tr st =
bed4b2738d8a separate module for prover command execution;
wenzelm
parents:
diff changeset
    71
  (case Toplevel.transition int tr st of
bed4b2738d8a separate module for prover command execution;
wenzelm
parents:
diff changeset
    72
    SOME (st', NONE) => ([], SOME st')
bed4b2738d8a separate module for prover command execution;
wenzelm
parents:
diff changeset
    73
  | SOME (_, SOME (exn, _)) => (ML_Compiler.exn_messages exn, NONE)
bed4b2738d8a separate module for prover command execution;
wenzelm
parents:
diff changeset
    74
  | NONE => ([(serial (), ML_Compiler.exn_message Runtime.TERMINATE)], NONE));
bed4b2738d8a separate module for prover command execution;
wenzelm
parents:
diff changeset
    75
bed4b2738d8a separate module for prover command execution;
wenzelm
parents:
diff changeset
    76
fun timing tr t =
bed4b2738d8a separate module for prover command execution;
wenzelm
parents:
diff changeset
    77
  if Timing.is_relevant t then Toplevel.status tr (Isabelle_Markup.timing t) else ();
bed4b2738d8a separate module for prover command execution;
wenzelm
parents:
diff changeset
    78
bed4b2738d8a separate module for prover command execution;
wenzelm
parents:
diff changeset
    79
fun proof_status tr st =
bed4b2738d8a separate module for prover command execution;
wenzelm
parents:
diff changeset
    80
  (case try Toplevel.proof_of st of
bed4b2738d8a separate module for prover command execution;
wenzelm
parents:
diff changeset
    81
    SOME prf => Toplevel.status tr (Proof.status_markup prf)
bed4b2738d8a separate module for prover command execution;
wenzelm
parents:
diff changeset
    82
  | NONE => ());
bed4b2738d8a separate module for prover command execution;
wenzelm
parents:
diff changeset
    83
bed4b2738d8a separate module for prover command execution;
wenzelm
parents:
diff changeset
    84
val no_print = Lazy.value ();
bed4b2738d8a separate module for prover command execution;
wenzelm
parents:
diff changeset
    85
bed4b2738d8a separate module for prover command execution;
wenzelm
parents:
diff changeset
    86
fun print_state tr st =
bed4b2738d8a separate module for prover command execution;
wenzelm
parents:
diff changeset
    87
  (Lazy.lazy o Toplevel.setmp_thread_position tr)
bed4b2738d8a separate module for prover command execution;
wenzelm
parents:
diff changeset
    88
    (fn () => Toplevel.print_state false st);
bed4b2738d8a separate module for prover command execution;
wenzelm
parents:
diff changeset
    89
bed4b2738d8a separate module for prover command execution;
wenzelm
parents:
diff changeset
    90
in
bed4b2738d8a separate module for prover command execution;
wenzelm
parents:
diff changeset
    91
48772
e46cd0d26481 vacuous execution after first malformed command;
wenzelm
parents: 48771
diff changeset
    92
fun run_command tr (st, malformed) =
e46cd0d26481 vacuous execution after first malformed command;
wenzelm
parents: 48771
diff changeset
    93
  if malformed then ((Toplevel.toplevel, malformed), no_print)
e46cd0d26481 vacuous execution after first malformed command;
wenzelm
parents: 48771
diff changeset
    94
  else
e46cd0d26481 vacuous execution after first malformed command;
wenzelm
parents: 48771
diff changeset
    95
    let
e46cd0d26481 vacuous execution after first malformed command;
wenzelm
parents: 48771
diff changeset
    96
      val malformed' = Toplevel.is_malformed tr;
e46cd0d26481 vacuous execution after first malformed command;
wenzelm
parents: 48771
diff changeset
    97
      val is_init = Toplevel.is_init tr;
e46cd0d26481 vacuous execution after first malformed command;
wenzelm
parents: 48771
diff changeset
    98
      val is_proof = Keyword.is_proof (Toplevel.name_of tr);
47336
bed4b2738d8a separate module for prover command execution;
wenzelm
parents:
diff changeset
    99
48772
e46cd0d26481 vacuous execution after first malformed command;
wenzelm
parents: 48771
diff changeset
   100
      val _ = Multithreading.interrupted ();
e46cd0d26481 vacuous execution after first malformed command;
wenzelm
parents: 48771
diff changeset
   101
      val _ = Toplevel.status tr Isabelle_Markup.forked;
e46cd0d26481 vacuous execution after first malformed command;
wenzelm
parents: 48771
diff changeset
   102
      val start = Timing.start ();
e46cd0d26481 vacuous execution after first malformed command;
wenzelm
parents: 48771
diff changeset
   103
      val (errs, result) = run (is_init orelse is_proof) (Toplevel.set_print false tr) st;
e46cd0d26481 vacuous execution after first malformed command;
wenzelm
parents: 48771
diff changeset
   104
      val _ = timing tr (Timing.result start);
e46cd0d26481 vacuous execution after first malformed command;
wenzelm
parents: 48771
diff changeset
   105
      val _ = Toplevel.status tr Isabelle_Markup.joined;
e46cd0d26481 vacuous execution after first malformed command;
wenzelm
parents: 48771
diff changeset
   106
      val _ = List.app (Toplevel.error_msg tr) errs;
e46cd0d26481 vacuous execution after first malformed command;
wenzelm
parents: 48771
diff changeset
   107
    in
e46cd0d26481 vacuous execution after first malformed command;
wenzelm
parents: 48771
diff changeset
   108
      (case result of
e46cd0d26481 vacuous execution after first malformed command;
wenzelm
parents: 48771
diff changeset
   109
        NONE =>
e46cd0d26481 vacuous execution after first malformed command;
wenzelm
parents: 48771
diff changeset
   110
          let
e46cd0d26481 vacuous execution after first malformed command;
wenzelm
parents: 48771
diff changeset
   111
            val _ = if null errs then Exn.interrupt () else ();
e46cd0d26481 vacuous execution after first malformed command;
wenzelm
parents: 48771
diff changeset
   112
            val _ = Toplevel.status tr Isabelle_Markup.failed;
e46cd0d26481 vacuous execution after first malformed command;
wenzelm
parents: 48771
diff changeset
   113
          in ((st, malformed'), no_print) end
e46cd0d26481 vacuous execution after first malformed command;
wenzelm
parents: 48771
diff changeset
   114
      | SOME st' =>
e46cd0d26481 vacuous execution after first malformed command;
wenzelm
parents: 48771
diff changeset
   115
          let
e46cd0d26481 vacuous execution after first malformed command;
wenzelm
parents: 48771
diff changeset
   116
            val _ = Toplevel.status tr Isabelle_Markup.finished;
e46cd0d26481 vacuous execution after first malformed command;
wenzelm
parents: 48771
diff changeset
   117
            val _ = proof_status tr st';
e46cd0d26481 vacuous execution after first malformed command;
wenzelm
parents: 48771
diff changeset
   118
            val do_print =
e46cd0d26481 vacuous execution after first malformed command;
wenzelm
parents: 48771
diff changeset
   119
              not is_init andalso
e46cd0d26481 vacuous execution after first malformed command;
wenzelm
parents: 48771
diff changeset
   120
                (Toplevel.print_of tr orelse (is_proof andalso Toplevel.is_proof st'));
e46cd0d26481 vacuous execution after first malformed command;
wenzelm
parents: 48771
diff changeset
   121
          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
   122
    end;
47336
bed4b2738d8a separate module for prover command execution;
wenzelm
parents:
diff changeset
   123
bed4b2738d8a separate module for prover command execution;
wenzelm
parents:
diff changeset
   124
end;
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