| author | blanchet | 
| Thu, 17 Mar 2011 11:18:31 +0100 | |
| changeset 41990 | 7f2793d51efc | 
| parent 41703 | d27950860514 | 
| child 42012 | 2c3fe3cbebae | 
| permissions | -rw-r--r-- | 
| 5828 | 1 | (* Title: Pure/Isar/toplevel.ML | 
| 2 | Author: Markus Wenzel, TU Muenchen | |
| 3 | ||
| 26602 
5534b6a6b810
made purely value-oriented, moved global state to structure Isar (cf. isar.ML);
 wenzelm parents: 
26491diff
changeset | 4 | Isabelle/Isar toplevel transactions. | 
| 5828 | 5 | *) | 
| 6 | ||
| 7 | signature TOPLEVEL = | |
| 8 | sig | |
| 19063 | 9 | exception UNDEF | 
| 5828 | 10 | type state | 
| 26602 
5534b6a6b810
made purely value-oriented, moved global state to structure Isar (cf. isar.ML);
 wenzelm parents: 
26491diff
changeset | 11 | val toplevel: state | 
| 7732 | 12 | val is_toplevel: state -> bool | 
| 18589 | 13 | val is_theory: state -> bool | 
| 14 | val is_proof: state -> bool | |
| 17076 | 15 | val level: state -> int | 
| 30398 | 16 | val presentation_context_of: state -> Proof.context | 
| 30801 | 17 | val previous_context_of: state -> Proof.context option | 
| 21506 | 18 | val context_of: state -> Proof.context | 
| 22089 | 19 | val generic_theory_of: state -> generic_theory | 
| 5828 | 20 | val theory_of: state -> theory | 
| 21 | val proof_of: state -> Proof.state | |
| 18589 | 22 | val proof_position_of: state -> int | 
| 37953 
ddc3b72f9a42
simplified handling of theory begin/end wrt. toplevel and theory loader;
 wenzelm parents: 
37951diff
changeset | 23 | val end_theory: Position.T -> state -> theory | 
| 16815 | 24 | val print_state_context: state -> unit | 
| 25 | val print_state: bool -> state -> unit | |
| 37858 | 26 | val pretty_abstract: state -> Pretty.T | 
| 32738 | 27 | val quiet: bool Unsynchronized.ref | 
| 28 | val debug: bool Unsynchronized.ref | |
| 29 | val interact: bool Unsynchronized.ref | |
| 30 | val timing: bool Unsynchronized.ref | |
| 31 | val profiling: int Unsynchronized.ref | |
| 32 | val skip_proofs: bool Unsynchronized.ref | |
| 20128 
8f0e07d7cf92
keep/transaction: unified execution model (with debugging etc.);
 wenzelm parents: 
19996diff
changeset | 33 | val program: (unit -> 'a) -> 'a | 
| 33604 
d4220df6fde2
Toplevel.thread provides Isar-style exception output;
 wenzelm parents: 
33553diff
changeset | 34 | val thread: bool -> (unit -> unit) -> Thread.thread | 
| 16682 | 35 | type transition | 
| 5828 | 36 | val empty: transition | 
| 27441 | 37 | val init_of: transition -> string option | 
| 38888 
8248cda328de
moved Toplevel.run_command to Pure/PIDE/document.ML;
 wenzelm parents: 
38876diff
changeset | 38 | val print_of: transition -> bool | 
| 27427 | 39 | val name_of: transition -> string | 
| 28105 | 40 | val pos_of: transition -> Position.T | 
| 27500 | 41 | val str_of: transition -> string | 
| 5828 | 42 | val name: string -> transition -> transition | 
| 43 | val position: Position.T -> transition -> transition | |
| 44 | val interactive: bool -> transition -> transition | |
| 38888 
8248cda328de
moved Toplevel.run_command to Pure/PIDE/document.ML;
 wenzelm parents: 
38876diff
changeset | 45 | val set_print: bool -> transition -> transition | 
| 5828 | 46 | val print: transition -> transition | 
| 9010 | 47 | val no_timing: transition -> transition | 
| 41536 
47fef6afe756
Toplevel.init_theory: maintain optional master directory, to allow bypassing global Thy_Load.master_path;
 wenzelm parents: 
40960diff
changeset | 48 | val init_theory: Path.T option -> string -> (Path.T option -> theory) -> transition -> transition | 
| 
47fef6afe756
Toplevel.init_theory: maintain optional master directory, to allow bypassing global Thy_Load.master_path;
 wenzelm parents: 
40960diff
changeset | 49 | val modify_master: Path.T option -> transition -> transition | 
| 
47fef6afe756
Toplevel.init_theory: maintain optional master directory, to allow bypassing global Thy_Load.master_path;
 wenzelm parents: 
40960diff
changeset | 50 | val modify_init: (Path.T option -> theory) -> transition -> transition | 
| 6689 | 51 | val exit: transition -> transition | 
| 5828 | 52 | val keep: (state -> unit) -> transition -> transition | 
| 7612 | 53 | val keep': (bool -> state -> unit) -> transition -> transition | 
| 5828 | 54 | val imperative: (unit -> unit) -> transition -> transition | 
| 27840 | 55 | val ignored: Position.T -> transition | 
| 56 | val malformed: Position.T -> string -> transition | |
| 5828 | 57 | val theory: (theory -> theory) -> transition -> transition | 
| 26491 | 58 | val generic_theory: (generic_theory -> generic_theory) -> transition -> transition | 
| 7612 | 59 | val theory': (bool -> theory -> theory) -> transition -> transition | 
| 20985 | 60 | val begin_local_theory: bool -> (theory -> local_theory) -> transition -> transition | 
| 21007 | 61 | val end_local_theory: transition -> transition | 
| 29380 | 62 | val local_theory': xstring option -> (bool -> local_theory -> local_theory) -> | 
| 63 | transition -> transition | |
| 20963 
a7fd8f05a2be
added type global_theory -- theory or local_theory;
 wenzelm parents: 
20928diff
changeset | 64 | val local_theory: xstring option -> (local_theory -> local_theory) -> transition -> transition | 
| 30366 
e3d788b9dffb
simplified presentation: built into transaction, pass state directly;
 wenzelm parents: 
29516diff
changeset | 65 | val present_local_theory: xstring option -> (state -> unit) -> transition -> transition | 
| 24453 | 66 | val local_theory_to_proof': xstring option -> (bool -> local_theory -> Proof.state) -> | 
| 67 | transition -> transition | |
| 21007 | 68 | val local_theory_to_proof: xstring option -> (local_theory -> Proof.state) -> | 
| 69 | transition -> transition | |
| 17363 | 70 | val theory_to_proof: (theory -> Proof.state) -> transition -> transition | 
| 21007 | 71 | val end_proof: (bool -> Proof.state -> Proof.context) -> transition -> transition | 
| 72 | val forget_proof: transition -> transition | |
| 30366 
e3d788b9dffb
simplified presentation: built into transaction, pass state directly;
 wenzelm parents: 
29516diff
changeset | 73 | val present_proof: (state -> unit) -> transition -> transition | 
| 21177 | 74 | val proofs': (bool -> Proof.state -> Proof.state Seq.seq) -> transition -> transition | 
| 17904 
21c6894b5998
simplified interfaces proof/proof' etc.: perform ProofHistory.apply(s)/current internally;
 wenzelm parents: 
17513diff
changeset | 75 | val proof': (bool -> Proof.state -> Proof.state) -> transition -> transition | 
| 21177 | 76 | val proofs: (Proof.state -> Proof.state Seq.seq) -> transition -> transition | 
| 77 | val proof: (Proof.state -> Proof.state) -> transition -> transition | |
| 33390 | 78 | val actual_proof: (Proof_Node.T -> Proof_Node.T) -> transition -> transition | 
| 27564 
fc6d34e49e17
replaced obsolete ProofHistory by ProofNode (backtracking only);
 wenzelm parents: 
27500diff
changeset | 79 | val skip_proof: (int -> int) -> transition -> transition | 
| 17904 
21c6894b5998
simplified interfaces proof/proof' etc.: perform ProofHistory.apply(s)/current internally;
 wenzelm parents: 
17513diff
changeset | 80 | val skip_proof_to_theory: (int -> bool) -> transition -> transition | 
| 27427 | 81 | val get_id: transition -> string option | 
| 82 | val put_id: string -> transition -> transition | |
| 9512 | 83 | val unknown_theory: transition -> transition | 
| 84 | val unknown_proof: transition -> transition | |
| 85 | val unknown_context: transition -> transition | |
| 28425 | 86 |   val setmp_thread_position: transition -> ('a -> 'b) -> 'a -> 'b
 | 
| 27606 | 87 | val status: transition -> Markup.T -> unit | 
| 38876 
ec7045139e70
Toplevel.run_command: more careful treatment of interrupts stemming from nested multi-exceptions etc.;
 wenzelm parents: 
38875diff
changeset | 88 | val error_msg: transition -> string -> unit | 
| 28103 
b79e61861f0f
simplified Toplevel.add_hook: cover successful transactions only;
 wenzelm parents: 
28095diff
changeset | 89 | val add_hook: (transition -> state -> state -> unit) -> unit | 
| 26602 
5534b6a6b810
made purely value-oriented, moved global state to structure Isar (cf. isar.ML);
 wenzelm parents: 
26491diff
changeset | 90 | val transition: bool -> transition -> state -> (state * (exn * string) option) option | 
| 28425 | 91 | val command: transition -> state -> state | 
| 37953 
ddc3b72f9a42
simplified handling of theory begin/end wrt. toplevel and theory loader;
 wenzelm parents: 
37951diff
changeset | 92 | val excursion: (transition * transition list) list -> (transition * state) list lazy * theory | 
| 5828 | 93 | end; | 
| 94 | ||
| 6965 | 95 | structure Toplevel: TOPLEVEL = | 
| 5828 | 96 | struct | 
| 97 | ||
| 98 | (** toplevel state **) | |
| 99 | ||
| 31476 
c5d2899b6de9
moved Isar toplevel runtime support to runtime.ML, which is loaded early (before ml_compiler.ML);
 wenzelm parents: 
31431diff
changeset | 100 | exception UNDEF = Runtime.UNDEF; | 
| 19063 | 101 | |
| 102 | ||
| 21294 | 103 | (* local theory wrappers *) | 
| 5828 | 104 | |
| 38350 
480b2de9927c
renamed Theory_Target to the more appropriate Named_Target
 haftmann parents: 
38236diff
changeset | 105 | val loc_init = Named_Target.context_cmd; | 
| 33671 | 106 | val loc_exit = Local_Theory.exit_global; | 
| 21294 | 107 | |
| 25292 | 108 | fun loc_begin loc (Context.Theory thy) = loc_init (the_default "-" loc) thy | 
| 21294 | 109 | | loc_begin NONE (Context.Proof lthy) = lthy | 
| 38391 
ba1cc1815ce1
named target is optional; explicit Name_Target.reinit
 haftmann parents: 
38389diff
changeset | 110 | | loc_begin (SOME loc) (Context.Proof lthy) = (loc_init loc o loc_exit) lthy; | 
| 21294 | 111 | |
| 112 | fun loc_finish _ (Context.Theory _) = Context.Theory o loc_exit | |
| 33671 | 113 | | loc_finish NONE (Context.Proof _) = Context.Proof o Local_Theory.restore | 
| 38391 
ba1cc1815ce1
named target is optional; explicit Name_Target.reinit
 haftmann parents: 
38389diff
changeset | 114 | | loc_finish (SOME _) (Context.Proof lthy) = Context.Proof o Named_Target.reinit lthy; | 
| 21294 | 115 | |
| 116 | ||
| 21958 
9dfd1ca4c0a0
refined notion of empty toplevel, admits undo of 'end';
 wenzelm parents: 
21861diff
changeset | 117 | (* datatype node *) | 
| 21294 | 118 | |
| 5828 | 119 | datatype node = | 
| 27576 
7afff36043e6
eliminated internal command history -- superceeded by global Isar state (cf. isar.ML);
 wenzelm parents: 
27564diff
changeset | 120 | Theory of generic_theory * Proof.context option | 
| 
7afff36043e6
eliminated internal command history -- superceeded by global Isar state (cf. isar.ML);
 wenzelm parents: 
27564diff
changeset | 121 | (*theory with presentation context*) | | 
| 33390 | 122 | Proof of Proof_Node.T * ((Proof.context -> generic_theory) * generic_theory) | 
| 27576 
7afff36043e6
eliminated internal command history -- superceeded by global Isar state (cf. isar.ML);
 wenzelm parents: 
27564diff
changeset | 123 | (*proof node, finish, original theory*) | | 
| 27564 
fc6d34e49e17
replaced obsolete ProofHistory by ProofNode (backtracking only);
 wenzelm parents: 
27500diff
changeset | 124 | SkipProof of int * (generic_theory * generic_theory); | 
| 
fc6d34e49e17
replaced obsolete ProofHistory by ProofNode (backtracking only);
 wenzelm parents: 
27500diff
changeset | 125 | (*proof depth, resulting theory, original theory*) | 
| 5828 | 126 | |
| 20963 
a7fd8f05a2be
added type global_theory -- theory or local_theory;
 wenzelm parents: 
20928diff
changeset | 127 | val theory_node = fn Theory (gthy, _) => SOME gthy | _ => NONE; | 
| 18589 | 128 | val proof_node = fn Proof (prf, _) => SOME prf | _ => NONE; | 
| 129 | ||
| 20963 
a7fd8f05a2be
added type global_theory -- theory or local_theory;
 wenzelm parents: 
20928diff
changeset | 130 | fun cases_node f _ (Theory (gthy, _)) = f gthy | 
| 33390 | 131 | | cases_node _ g (Proof (prf, _)) = g (Proof_Node.current prf) | 
| 21007 | 132 | | cases_node f _ (SkipProof (_, (gthy, _))) = f gthy; | 
| 19063 | 133 | |
| 29066 | 134 | val context_node = cases_node Context.proof_of Proof.context_of; | 
| 135 | ||
| 21958 
9dfd1ca4c0a0
refined notion of empty toplevel, admits undo of 'end';
 wenzelm parents: 
21861diff
changeset | 136 | |
| 
9dfd1ca4c0a0
refined notion of empty toplevel, admits undo of 'end';
 wenzelm parents: 
21861diff
changeset | 137 | (* datatype state *) | 
| 
9dfd1ca4c0a0
refined notion of empty toplevel, admits undo of 'end';
 wenzelm parents: 
21861diff
changeset | 138 | |
| 37953 
ddc3b72f9a42
simplified handling of theory begin/end wrt. toplevel and theory loader;
 wenzelm parents: 
37951diff
changeset | 139 | datatype state = State of node option * node option; (*current, previous*) | 
| 5828 | 140 | |
| 27576 
7afff36043e6
eliminated internal command history -- superceeded by global Isar state (cf. isar.ML);
 wenzelm parents: 
27564diff
changeset | 141 | val toplevel = State (NONE, NONE); | 
| 5828 | 142 | |
| 27576 
7afff36043e6
eliminated internal command history -- superceeded by global Isar state (cf. isar.ML);
 wenzelm parents: 
27564diff
changeset | 143 | fun is_toplevel (State (NONE, _)) = true | 
| 7732 | 144 | | is_toplevel _ = false; | 
| 145 | ||
| 27576 
7afff36043e6
eliminated internal command history -- superceeded by global Isar state (cf. isar.ML);
 wenzelm parents: 
27564diff
changeset | 146 | fun level (State (NONE, _)) = 0 | 
| 37953 
ddc3b72f9a42
simplified handling of theory begin/end wrt. toplevel and theory loader;
 wenzelm parents: 
37951diff
changeset | 147 | | level (State (SOME (Theory _), _)) = 0 | 
| 
ddc3b72f9a42
simplified handling of theory begin/end wrt. toplevel and theory loader;
 wenzelm parents: 
37951diff
changeset | 148 | | level (State (SOME (Proof (prf, _)), _)) = Proof.level (Proof_Node.current prf) | 
| 
ddc3b72f9a42
simplified handling of theory begin/end wrt. toplevel and theory loader;
 wenzelm parents: 
37951diff
changeset | 149 | | level (State (SOME (SkipProof (d, _)), _)) = d + 1; (*different notion of proof depth!*) | 
| 17076 | 150 | |
| 27576 
7afff36043e6
eliminated internal command history -- superceeded by global Isar state (cf. isar.ML);
 wenzelm parents: 
27564diff
changeset | 151 | fun str_of_state (State (NONE, _)) = "at top level" | 
| 37953 
ddc3b72f9a42
simplified handling of theory begin/end wrt. toplevel and theory loader;
 wenzelm parents: 
37951diff
changeset | 152 | | str_of_state (State (SOME (Theory (Context.Theory _, _)), _)) = "in theory mode" | 
| 
ddc3b72f9a42
simplified handling of theory begin/end wrt. toplevel and theory loader;
 wenzelm parents: 
37951diff
changeset | 153 | | str_of_state (State (SOME (Theory (Context.Proof _, _)), _)) = "in local theory mode" | 
| 
ddc3b72f9a42
simplified handling of theory begin/end wrt. toplevel and theory loader;
 wenzelm parents: 
37951diff
changeset | 154 | | str_of_state (State (SOME (Proof _), _)) = "in proof mode" | 
| 
ddc3b72f9a42
simplified handling of theory begin/end wrt. toplevel and theory loader;
 wenzelm parents: 
37951diff
changeset | 155 | | str_of_state (State (SOME (SkipProof _), _)) = "in skipped proof mode"; | 
| 5946 
a4600d21b59b
print_state hook, obeys Goals.current_goals_markers by default;
 wenzelm parents: 
5939diff
changeset | 156 | |
| 
a4600d21b59b
print_state hook, obeys Goals.current_goals_markers by default;
 wenzelm parents: 
5939diff
changeset | 157 | |
| 27576 
7afff36043e6
eliminated internal command history -- superceeded by global Isar state (cf. isar.ML);
 wenzelm parents: 
27564diff
changeset | 158 | (* current node *) | 
| 5828 | 159 | |
| 27576 
7afff36043e6
eliminated internal command history -- superceeded by global Isar state (cf. isar.ML);
 wenzelm parents: 
27564diff
changeset | 160 | fun node_of (State (NONE, _)) = raise UNDEF | 
| 37953 
ddc3b72f9a42
simplified handling of theory begin/end wrt. toplevel and theory loader;
 wenzelm parents: 
37951diff
changeset | 161 | | node_of (State (SOME node, _)) = node; | 
| 5828 | 162 | |
| 18589 | 163 | fun is_theory state = not (is_toplevel state) andalso is_some (theory_node (node_of state)); | 
| 164 | fun is_proof state = not (is_toplevel state) andalso is_some (proof_node (node_of state)); | |
| 165 | ||
| 19063 | 166 | fun node_case f g state = cases_node f g (node_of state); | 
| 5828 | 167 | |
| 30398 | 168 | fun presentation_context_of state = | 
| 169 | (case try node_of state of | |
| 170 | SOME (Theory (_, SOME ctxt)) => ctxt | |
| 171 | | SOME node => context_node node | |
| 172 | | NONE => raise UNDEF); | |
| 30366 
e3d788b9dffb
simplified presentation: built into transaction, pass state directly;
 wenzelm parents: 
29516diff
changeset | 173 | |
| 30801 | 174 | fun previous_context_of (State (_, NONE)) = NONE | 
| 37953 
ddc3b72f9a42
simplified handling of theory begin/end wrt. toplevel and theory loader;
 wenzelm parents: 
37951diff
changeset | 175 | | previous_context_of (State (_, SOME prev)) = SOME (context_node prev); | 
| 30801 | 176 | |
| 21506 | 177 | val context_of = node_case Context.proof_of Proof.context_of; | 
| 22089 | 178 | val generic_theory_of = node_case I (Context.Proof o Proof.context_of); | 
| 20963 
a7fd8f05a2be
added type global_theory -- theory or local_theory;
 wenzelm parents: 
20928diff
changeset | 179 | val theory_of = node_case Context.theory_of Proof.theory_of; | 
| 18589 | 180 | val proof_of = node_case (fn _ => raise UNDEF) I; | 
| 17208 | 181 | |
| 18589 | 182 | fun proof_position_of state = | 
| 183 | (case node_of state of | |
| 33390 | 184 | Proof (prf, _) => Proof_Node.position prf | 
| 18589 | 185 | | _ => raise UNDEF); | 
| 6664 | 186 | |
| 37953 
ddc3b72f9a42
simplified handling of theory begin/end wrt. toplevel and theory loader;
 wenzelm parents: 
37951diff
changeset | 187 | fun end_theory _ (State (NONE, SOME (Theory (Context.Theory thy, _)))) = Theory.end_theory thy | 
| 
ddc3b72f9a42
simplified handling of theory begin/end wrt. toplevel and theory loader;
 wenzelm parents: 
37951diff
changeset | 188 |   | end_theory pos _ = error ("Unfinished theory at end of input" ^ Position.str_of pos);
 | 
| 
ddc3b72f9a42
simplified handling of theory begin/end wrt. toplevel and theory loader;
 wenzelm parents: 
37951diff
changeset | 189 | |
| 5828 | 190 | |
| 16815 | 191 | (* print state *) | 
| 192 | ||
| 38388 | 193 | val pretty_context = Local_Theory.pretty o Context.cases (Named_Target.theory_init) I; | 
| 16815 | 194 | |
| 23640 
baec2e674461
toplevel prompt/print_state: proper markup, removed hooks;
 wenzelm parents: 
23619diff
changeset | 195 | fun print_state_context state = | 
| 24795 
6f5cb7885fd7
print_state_context: local theory context, not proof context;
 wenzelm parents: 
24780diff
changeset | 196 | (case try node_of state of | 
| 21506 | 197 | NONE => [] | 
| 24795 
6f5cb7885fd7
print_state_context: local theory context, not proof context;
 wenzelm parents: 
24780diff
changeset | 198 | | SOME (Theory (gthy, _)) => pretty_context gthy | 
| 
6f5cb7885fd7
print_state_context: local theory context, not proof context;
 wenzelm parents: 
24780diff
changeset | 199 | | SOME (Proof (_, (_, gthy))) => pretty_context gthy | 
| 
6f5cb7885fd7
print_state_context: local theory context, not proof context;
 wenzelm parents: 
24780diff
changeset | 200 | | SOME (SkipProof (_, (gthy, _))) => pretty_context gthy) | 
| 23640 
baec2e674461
toplevel prompt/print_state: proper markup, removed hooks;
 wenzelm parents: 
23619diff
changeset | 201 | |> Pretty.chunks |> Pretty.writeln; | 
| 16815 | 202 | |
| 23640 
baec2e674461
toplevel prompt/print_state: proper markup, removed hooks;
 wenzelm parents: 
23619diff
changeset | 203 | fun print_state prf_only state = | 
| 23701 | 204 | (case try node_of state of | 
| 205 | NONE => [] | |
| 206 | | SOME (Theory (gthy, _)) => if prf_only then [] else pretty_context gthy | |
| 207 | | SOME (Proof (prf, _)) => | |
| 33390 | 208 | Proof.pretty_state (Proof_Node.position prf) (Proof_Node.current prf) | 
| 27564 
fc6d34e49e17
replaced obsolete ProofHistory by ProofNode (backtracking only);
 wenzelm parents: 
27500diff
changeset | 209 |   | SOME (SkipProof (d, _)) => [Pretty.str ("skipped proof: depth " ^ string_of_int d)])
 | 
| 23701 | 210 | |> Pretty.markup_chunks Markup.state |> Pretty.writeln; | 
| 16815 | 211 | |
| 37858 | 212 | fun pretty_abstract state = Pretty.str ("<Isar " ^ str_of_state state ^ ">");
 | 
| 213 | ||
| 16815 | 214 | |
| 15668 | 215 | |
| 5828 | 216 | (** toplevel transitions **) | 
| 217 | ||
| 32738 | 218 | val quiet = Unsynchronized.ref false; | 
| 39513 
fce2202892c4
discontinued Output.debug, which belongs to early PGIP experiments (b6788dbd2ef9) and causes just too many problems (like spamming the message channel if it is used by more than one module);
 wenzelm parents: 
39285diff
changeset | 219 | val debug = Runtime.debug; | 
| 32738 | 220 | val interact = Unsynchronized.ref false; | 
| 16682 | 221 | val timing = Output.timing; | 
| 32738 | 222 | val profiling = Unsynchronized.ref 0; | 
| 223 | val skip_proofs = Unsynchronized.ref false; | |
| 16682 | 224 | |
| 33604 
d4220df6fde2
Toplevel.thread provides Isar-style exception output;
 wenzelm parents: 
33553diff
changeset | 225 | fun program body = | 
| 
d4220df6fde2
Toplevel.thread provides Isar-style exception output;
 wenzelm parents: 
33553diff
changeset | 226 | (body | 
| 31476 
c5d2899b6de9
moved Isar toplevel runtime support to runtime.ML, which is loaded early (before ml_compiler.ML);
 wenzelm parents: 
31431diff
changeset | 227 | |> Runtime.controlled_execution | 
| 33604 
d4220df6fde2
Toplevel.thread provides Isar-style exception output;
 wenzelm parents: 
33553diff
changeset | 228 | |> Runtime.toplevel_error (Output.error_msg o ML_Compiler.exn_message)) (); | 
| 
d4220df6fde2
Toplevel.thread provides Isar-style exception output;
 wenzelm parents: 
33553diff
changeset | 229 | |
| 
d4220df6fde2
Toplevel.thread provides Isar-style exception output;
 wenzelm parents: 
33553diff
changeset | 230 | fun thread interrupts body = | 
| 
d4220df6fde2
Toplevel.thread provides Isar-style exception output;
 wenzelm parents: 
33553diff
changeset | 231 | Thread.fork | 
| 39232 
69c6d3e87660
more abstract treatment of interrupts in structure Exn -- hardly ever need to mention Interrupt literally;
 wenzelm parents: 
38888diff
changeset | 232 | (((fn () => body () handle exn => if Exn.is_interrupt exn then () else reraise exn) | 
| 33604 
d4220df6fde2
Toplevel.thread provides Isar-style exception output;
 wenzelm parents: 
33553diff
changeset | 233 | |> Runtime.debugging | 
| 
d4220df6fde2
Toplevel.thread provides Isar-style exception output;
 wenzelm parents: 
33553diff
changeset | 234 | |> Runtime.toplevel_error | 
| 40132 
7ee65dbffa31
renamed Output.priority to Output.urgent_message to emphasize its special role more clearly;
 wenzelm parents: 
39513diff
changeset | 235 | (fn exn => | 
| 
7ee65dbffa31
renamed Output.priority to Output.urgent_message to emphasize its special role more clearly;
 wenzelm parents: 
39513diff
changeset | 236 |             Output.urgent_message ("## INTERNAL ERROR ##\n" ^ ML_Compiler.exn_message exn))),
 | 
| 37216 
3165bc303f66
modernized some structure names, keeping a few legacy aliases;
 wenzelm parents: 
37208diff
changeset | 237 | Simple_Thread.attributes interrupts); | 
| 20128 
8f0e07d7cf92
keep/transaction: unified execution model (with debugging etc.);
 wenzelm parents: 
19996diff
changeset | 238 | |
| 5828 | 239 | |
| 27601 
6683cdb94af8
simplified commit_exit: operate on previous node of final state, include warning here;
 wenzelm parents: 
27583diff
changeset | 240 | (* node transactions -- maintaining stable checkpoints *) | 
| 7022 | 241 | |
| 31476 
c5d2899b6de9
moved Isar toplevel runtime support to runtime.ML, which is loaded early (before ml_compiler.ML);
 wenzelm parents: 
31431diff
changeset | 242 | exception FAILURE of state * exn; | 
| 
c5d2899b6de9
moved Isar toplevel runtime support to runtime.ML, which is loaded early (before ml_compiler.ML);
 wenzelm parents: 
31431diff
changeset | 243 | |
| 6689 | 244 | local | 
| 245 | ||
| 30366 
e3d788b9dffb
simplified presentation: built into transaction, pass state directly;
 wenzelm parents: 
29516diff
changeset | 246 | fun reset_presentation (Theory (gthy, _)) = Theory (gthy, NONE) | 
| 
e3d788b9dffb
simplified presentation: built into transaction, pass state directly;
 wenzelm parents: 
29516diff
changeset | 247 | | reset_presentation node = node; | 
| 
e3d788b9dffb
simplified presentation: built into transaction, pass state directly;
 wenzelm parents: 
29516diff
changeset | 248 | |
| 26624 
770265032999
transaction/init: ensure stable theory (non-draft);
 wenzelm parents: 
26621diff
changeset | 249 | fun is_draft_theory (Theory (gthy, _)) = Context.is_draft (Context.theory_of gthy) | 
| 
770265032999
transaction/init: ensure stable theory (non-draft);
 wenzelm parents: 
26621diff
changeset | 250 | | is_draft_theory _ = false; | 
| 
770265032999
transaction/init: ensure stable theory (non-draft);
 wenzelm parents: 
26621diff
changeset | 251 | |
| 31476 
c5d2899b6de9
moved Isar toplevel runtime support to runtime.ML, which is loaded early (before ml_compiler.ML);
 wenzelm parents: 
31431diff
changeset | 252 | fun is_stale state = Context.is_stale (theory_of state) handle Runtime.UNDEF => false; | 
| 27601 
6683cdb94af8
simplified commit_exit: operate on previous node of final state, include warning here;
 wenzelm parents: 
27583diff
changeset | 253 | |
| 26624 
770265032999
transaction/init: ensure stable theory (non-draft);
 wenzelm parents: 
26621diff
changeset | 254 | fun stale_error NONE = SOME (ERROR "Stale theory encountered after successful execution!") | 
| 
770265032999
transaction/init: ensure stable theory (non-draft);
 wenzelm parents: 
26621diff
changeset | 255 | | stale_error some = some; | 
| 16815 | 256 | |
| 27576 
7afff36043e6
eliminated internal command history -- superceeded by global Isar state (cf. isar.ML);
 wenzelm parents: 
27564diff
changeset | 257 | fun map_theory f (Theory (gthy, ctxt)) = | 
| 33671 | 258 | Theory (Context.mapping f (Local_Theory.raw_theory f) gthy, ctxt) | 
| 27576 
7afff36043e6
eliminated internal command history -- superceeded by global Isar state (cf. isar.ML);
 wenzelm parents: 
27564diff
changeset | 259 | | map_theory _ node = node; | 
| 6689 | 260 | |
| 261 | in | |
| 262 | ||
| 37953 
ddc3b72f9a42
simplified handling of theory begin/end wrt. toplevel and theory loader;
 wenzelm parents: 
37951diff
changeset | 263 | fun apply_transaction f g node = | 
| 20128 
8f0e07d7cf92
keep/transaction: unified execution model (with debugging etc.);
 wenzelm parents: 
19996diff
changeset | 264 | let | 
| 27576 
7afff36043e6
eliminated internal command history -- superceeded by global Isar state (cf. isar.ML);
 wenzelm parents: 
27564diff
changeset | 265 | val _ = is_draft_theory node andalso error "Illegal draft theory in toplevel state"; | 
| 
7afff36043e6
eliminated internal command history -- superceeded by global Isar state (cf. isar.ML);
 wenzelm parents: 
27564diff
changeset | 266 | val cont_node = reset_presentation node; | 
| 
7afff36043e6
eliminated internal command history -- superceeded by global Isar state (cf. isar.ML);
 wenzelm parents: 
27564diff
changeset | 267 | val back_node = map_theory (Theory.checkpoint o Theory.copy) cont_node; | 
| 37953 
ddc3b72f9a42
simplified handling of theory begin/end wrt. toplevel and theory loader;
 wenzelm parents: 
37951diff
changeset | 268 | fun state_error e nd = (State (SOME nd, SOME node), e); | 
| 6689 | 269 | |
| 20128 
8f0e07d7cf92
keep/transaction: unified execution model (with debugging etc.);
 wenzelm parents: 
19996diff
changeset | 270 | val (result, err) = | 
| 
8f0e07d7cf92
keep/transaction: unified execution model (with debugging etc.);
 wenzelm parents: 
19996diff
changeset | 271 | cont_node | 
| 31476 
c5d2899b6de9
moved Isar toplevel runtime support to runtime.ML, which is loaded early (before ml_compiler.ML);
 wenzelm parents: 
31431diff
changeset | 272 | |> Runtime.controlled_execution f | 
| 26624 
770265032999
transaction/init: ensure stable theory (non-draft);
 wenzelm parents: 
26621diff
changeset | 273 | |> map_theory Theory.checkpoint | 
| 
770265032999
transaction/init: ensure stable theory (non-draft);
 wenzelm parents: 
26621diff
changeset | 274 | |> state_error NONE | 
| 
770265032999
transaction/init: ensure stable theory (non-draft);
 wenzelm parents: 
26621diff
changeset | 275 | handle exn => state_error (SOME exn) cont_node; | 
| 
770265032999
transaction/init: ensure stable theory (non-draft);
 wenzelm parents: 
26621diff
changeset | 276 | |
| 
770265032999
transaction/init: ensure stable theory (non-draft);
 wenzelm parents: 
26621diff
changeset | 277 | val (result', err') = | 
| 
770265032999
transaction/init: ensure stable theory (non-draft);
 wenzelm parents: 
26621diff
changeset | 278 | if is_stale result then state_error (stale_error err) back_node | 
| 
770265032999
transaction/init: ensure stable theory (non-draft);
 wenzelm parents: 
26621diff
changeset | 279 | else (result, err); | 
| 20128 
8f0e07d7cf92
keep/transaction: unified execution model (with debugging etc.);
 wenzelm parents: 
19996diff
changeset | 280 | in | 
| 26624 
770265032999
transaction/init: ensure stable theory (non-draft);
 wenzelm parents: 
26621diff
changeset | 281 | (case err' of | 
| 30366 
e3d788b9dffb
simplified presentation: built into transaction, pass state directly;
 wenzelm parents: 
29516diff
changeset | 282 | NONE => tap g result' | 
| 26624 
770265032999
transaction/init: ensure stable theory (non-draft);
 wenzelm parents: 
26621diff
changeset | 283 | | SOME exn => raise FAILURE (result', exn)) | 
| 20128 
8f0e07d7cf92
keep/transaction: unified execution model (with debugging etc.);
 wenzelm parents: 
19996diff
changeset | 284 | end; | 
| 6689 | 285 | |
| 286 | end; | |
| 287 | ||
| 288 | ||
| 289 | (* primitive transitions *) | |
| 290 | ||
| 5828 | 291 | datatype trans = | 
| 41536 
47fef6afe756
Toplevel.init_theory: maintain optional master directory, to allow bypassing global Thy_Load.master_path;
 wenzelm parents: 
40960diff
changeset | 292 | Init of Path.T option * string * (Path.T option -> theory) | (*master dir, theory name, init*) | 
| 37953 
ddc3b72f9a42
simplified handling of theory begin/end wrt. toplevel and theory loader;
 wenzelm parents: 
37951diff
changeset | 293 | Exit | (*formal exit of theory*) | 
| 
ddc3b72f9a42
simplified handling of theory begin/end wrt. toplevel and theory loader;
 wenzelm parents: 
37951diff
changeset | 294 | Keep of bool -> state -> unit | (*peek at state*) | 
| 30366 
e3d788b9dffb
simplified presentation: built into transaction, pass state directly;
 wenzelm parents: 
29516diff
changeset | 295 | Transaction of (bool -> node -> node) * (state -> unit); (*node transaction and presentation*) | 
| 21958 
9dfd1ca4c0a0
refined notion of empty toplevel, admits undo of 'end';
 wenzelm parents: 
21861diff
changeset | 296 | |
| 6689 | 297 | local | 
| 5828 | 298 | |
| 41536 
47fef6afe756
Toplevel.init_theory: maintain optional master directory, to allow bypassing global Thy_Load.master_path;
 wenzelm parents: 
40960diff
changeset | 299 | fun apply_tr _ (Init (master, _, f)) (State (NONE, _)) = | 
| 33727 
e2d5d7f51aa3
init_theory: Runtime.controlled_execution for proper exception trace etc.;
 wenzelm parents: 
33725diff
changeset | 300 | State (SOME (Theory (Context.Theory | 
| 41536 
47fef6afe756
Toplevel.init_theory: maintain optional master directory, to allow bypassing global Thy_Load.master_path;
 wenzelm parents: 
40960diff
changeset | 301 | (Theory.checkpoint (Runtime.controlled_execution f master)), NONE)), NONE) | 
| 37953 
ddc3b72f9a42
simplified handling of theory begin/end wrt. toplevel and theory loader;
 wenzelm parents: 
37951diff
changeset | 302 | | apply_tr _ Exit (State (prev as SOME (Theory (Context.Theory _, _)), _)) = | 
| 27603 | 303 | State (NONE, prev) | 
| 32792 | 304 | | apply_tr int (Keep f) state = | 
| 31476 
c5d2899b6de9
moved Isar toplevel runtime support to runtime.ML, which is loaded early (before ml_compiler.ML);
 wenzelm parents: 
31431diff
changeset | 305 | Runtime.controlled_execution (fn x => tap (f int) x) state | 
| 32792 | 306 | | apply_tr int (Transaction (f, g)) (State (SOME state, _)) = | 
| 307 | apply_transaction (fn x => f int x) g state | |
| 308 | | apply_tr _ _ _ = raise UNDEF; | |
| 5828 | 309 | |
| 32792 | 310 | fun apply_union _ [] state = raise FAILURE (state, UNDEF) | 
| 311 | | apply_union int (tr :: trs) state = | |
| 312 | apply_union int trs state | |
| 313 | handle Runtime.UNDEF => apply_tr int tr state | |
| 314 | | FAILURE (alt_state, UNDEF) => apply_tr int tr alt_state | |
| 6689 | 315 | | exn as FAILURE _ => raise exn | 
| 316 | | exn => raise FAILURE (state, exn); | |
| 317 | ||
| 318 | in | |
| 319 | ||
| 32792 | 320 | fun apply_trans int trs state = (apply_union int trs state, NONE) | 
| 15531 | 321 | handle FAILURE (alt_state, exn) => (alt_state, SOME exn) | exn => (state, SOME exn); | 
| 6689 | 322 | |
| 323 | end; | |
| 5828 | 324 | |
| 325 | ||
| 326 | (* datatype transition *) | |
| 327 | ||
| 328 | datatype transition = Transition of | |
| 26621 
78b3ad7af5d5
eliminated unused name_of, source, source_of, print', print3, three_buffersN;
 wenzelm parents: 
26602diff
changeset | 329 |  {name: string,              (*command name*)
 | 
| 
78b3ad7af5d5
eliminated unused name_of, source, source_of, print', print3, three_buffersN;
 wenzelm parents: 
26602diff
changeset | 330 | pos: Position.T, (*source position*) | 
| 
78b3ad7af5d5
eliminated unused name_of, source, source_of, print', print3, three_buffersN;
 wenzelm parents: 
26602diff
changeset | 331 | int_only: bool, (*interactive-only*) | 
| 
78b3ad7af5d5
eliminated unused name_of, source, source_of, print', print3, three_buffersN;
 wenzelm parents: 
26602diff
changeset | 332 | print: bool, (*print result state*) | 
| 
78b3ad7af5d5
eliminated unused name_of, source, source_of, print', print3, three_buffersN;
 wenzelm parents: 
26602diff
changeset | 333 | no_timing: bool, (*suppress timing*) | 
| 
78b3ad7af5d5
eliminated unused name_of, source, source_of, print', print3, three_buffersN;
 wenzelm parents: 
26602diff
changeset | 334 | trans: trans list}; (*primitive transitions (union)*) | 
| 5828 | 335 | |
| 26621 
78b3ad7af5d5
eliminated unused name_of, source, source_of, print', print3, three_buffersN;
 wenzelm parents: 
26602diff
changeset | 336 | fun make_transition (name, pos, int_only, print, no_timing, trans) = | 
| 
78b3ad7af5d5
eliminated unused name_of, source, source_of, print', print3, three_buffersN;
 wenzelm parents: 
26602diff
changeset | 337 |   Transition {name = name, pos = pos, int_only = int_only, print = print, no_timing = no_timing,
 | 
| 
78b3ad7af5d5
eliminated unused name_of, source, source_of, print', print3, three_buffersN;
 wenzelm parents: 
26602diff
changeset | 338 | trans = trans}; | 
| 5828 | 339 | |
| 26621 
78b3ad7af5d5
eliminated unused name_of, source, source_of, print', print3, three_buffersN;
 wenzelm parents: 
26602diff
changeset | 340 | fun map_transition f (Transition {name, pos, int_only, print, no_timing, trans}) =
 | 
| 
78b3ad7af5d5
eliminated unused name_of, source, source_of, print', print3, three_buffersN;
 wenzelm parents: 
26602diff
changeset | 341 | make_transition (f (name, pos, int_only, print, no_timing, trans)); | 
| 5828 | 342 | |
| 27441 | 343 | val empty = make_transition ("", Position.none, false, false, false, []);
 | 
| 5828 | 344 | |
| 345 | ||
| 346 | (* diagnostics *) | |
| 347 | ||
| 41536 
47fef6afe756
Toplevel.init_theory: maintain optional master directory, to allow bypassing global Thy_Load.master_path;
 wenzelm parents: 
40960diff
changeset | 348 | fun get_init (Transition {trans = [Init args], ...}) = SOME args
 | 
| 
47fef6afe756
Toplevel.init_theory: maintain optional master directory, to allow bypassing global Thy_Load.master_path;
 wenzelm parents: 
40960diff
changeset | 349 | | get_init _ = NONE; | 
| 27441 | 350 | |
| 41536 
47fef6afe756
Toplevel.init_theory: maintain optional master directory, to allow bypassing global Thy_Load.master_path;
 wenzelm parents: 
40960diff
changeset | 351 | val init_of = Option.map #2 o get_init; | 
| 38888 
8248cda328de
moved Toplevel.run_command to Pure/PIDE/document.ML;
 wenzelm parents: 
38876diff
changeset | 352 | fun print_of (Transition {print, ...}) = print;
 | 
| 27427 | 353 | fun name_of (Transition {name, ...}) = name;
 | 
| 28105 | 354 | fun pos_of (Transition {pos, ...}) = pos;
 | 
| 355 | fun str_of tr = quote (name_of tr) ^ Position.str_of (pos_of tr); | |
| 5828 | 356 | |
| 27427 | 357 | fun command_msg msg tr = msg ^ "command " ^ str_of tr; | 
| 38875 
c7a66b584147
tuned messages: discontinued spurious full-stops (messages are occasionally composed unexpectedly);
 wenzelm parents: 
38721diff
changeset | 358 | fun at_command tr = command_msg "At " tr; | 
| 5828 | 359 | |
| 360 | fun type_error tr state = | |
| 18685 | 361 | ERROR (command_msg "Illegal application of " tr ^ " " ^ str_of_state state); | 
| 5828 | 362 | |
| 363 | ||
| 364 | (* modify transitions *) | |
| 365 | ||
| 28451 
0586b855c2b5
datatype transition: internal trans field is maintained in reverse order;
 wenzelm parents: 
28446diff
changeset | 366 | fun name name = map_transition (fn (_, pos, int_only, print, no_timing, trans) => | 
| 
0586b855c2b5
datatype transition: internal trans field is maintained in reverse order;
 wenzelm parents: 
28446diff
changeset | 367 | (name, pos, int_only, print, no_timing, trans)); | 
| 9010 | 368 | |
| 26621 
78b3ad7af5d5
eliminated unused name_of, source, source_of, print', print3, three_buffersN;
 wenzelm parents: 
26602diff
changeset | 369 | fun position pos = map_transition (fn (name, _, int_only, print, no_timing, trans) => | 
| 
78b3ad7af5d5
eliminated unused name_of, source, source_of, print', print3, three_buffersN;
 wenzelm parents: 
26602diff
changeset | 370 | (name, pos, int_only, print, no_timing, trans)); | 
| 5828 | 371 | |
| 26621 
78b3ad7af5d5
eliminated unused name_of, source, source_of, print', print3, three_buffersN;
 wenzelm parents: 
26602diff
changeset | 372 | fun interactive int_only = map_transition (fn (name, pos, _, print, no_timing, trans) => | 
| 
78b3ad7af5d5
eliminated unused name_of, source, source_of, print', print3, three_buffersN;
 wenzelm parents: 
26602diff
changeset | 373 | (name, pos, int_only, print, no_timing, trans)); | 
| 14923 | 374 | |
| 26621 
78b3ad7af5d5
eliminated unused name_of, source, source_of, print', print3, three_buffersN;
 wenzelm parents: 
26602diff
changeset | 375 | val no_timing = map_transition (fn (name, pos, int_only, print, _, trans) => | 
| 
78b3ad7af5d5
eliminated unused name_of, source, source_of, print', print3, three_buffersN;
 wenzelm parents: 
26602diff
changeset | 376 | (name, pos, int_only, print, true, trans)); | 
| 17363 | 377 | |
| 26621 
78b3ad7af5d5
eliminated unused name_of, source, source_of, print', print3, three_buffersN;
 wenzelm parents: 
26602diff
changeset | 378 | fun add_trans tr = map_transition (fn (name, pos, int_only, print, no_timing, trans) => | 
| 28451 
0586b855c2b5
datatype transition: internal trans field is maintained in reverse order;
 wenzelm parents: 
28446diff
changeset | 379 | (name, pos, int_only, print, no_timing, tr :: trans)); | 
| 16607 | 380 | |
| 28433 
b3dab95f098f
begin_proof: avoid race condition wrt. skip_proofs flag;
 wenzelm parents: 
28425diff
changeset | 381 | val reset_trans = map_transition (fn (name, pos, int_only, print, no_timing, _) => | 
| 
b3dab95f098f
begin_proof: avoid race condition wrt. skip_proofs flag;
 wenzelm parents: 
28425diff
changeset | 382 | (name, pos, int_only, print, no_timing, [])); | 
| 
b3dab95f098f
begin_proof: avoid race condition wrt. skip_proofs flag;
 wenzelm parents: 
28425diff
changeset | 383 | |
| 28453 
06702e7acd1d
excursion/unit_result: no print for forked end, finish into global theory, pick resul from presentation context;
 wenzelm parents: 
28451diff
changeset | 384 | fun set_print print = map_transition (fn (name, pos, int_only, _, no_timing, trans) => | 
| 
06702e7acd1d
excursion/unit_result: no print for forked end, finish into global theory, pick resul from presentation context;
 wenzelm parents: 
28451diff
changeset | 385 | (name, pos, int_only, print, no_timing, trans)); | 
| 
06702e7acd1d
excursion/unit_result: no print for forked end, finish into global theory, pick resul from presentation context;
 wenzelm parents: 
28451diff
changeset | 386 | |
| 
06702e7acd1d
excursion/unit_result: no print for forked end, finish into global theory, pick resul from presentation context;
 wenzelm parents: 
28451diff
changeset | 387 | val print = set_print true; | 
| 5828 | 388 | |
| 389 | ||
| 21007 | 390 | (* basic transitions *) | 
| 5828 | 391 | |
| 41536 
47fef6afe756
Toplevel.init_theory: maintain optional master directory, to allow bypassing global Thy_Load.master_path;
 wenzelm parents: 
40960diff
changeset | 392 | fun init_theory master name f = add_trans (Init (master, name, f)); | 
| 
47fef6afe756
Toplevel.init_theory: maintain optional master directory, to allow bypassing global Thy_Load.master_path;
 wenzelm parents: 
40960diff
changeset | 393 | |
| 
47fef6afe756
Toplevel.init_theory: maintain optional master directory, to allow bypassing global Thy_Load.master_path;
 wenzelm parents: 
40960diff
changeset | 394 | fun modify_master master tr = | 
| 
47fef6afe756
Toplevel.init_theory: maintain optional master directory, to allow bypassing global Thy_Load.master_path;
 wenzelm parents: 
40960diff
changeset | 395 | (case get_init tr of | 
| 
47fef6afe756
Toplevel.init_theory: maintain optional master directory, to allow bypassing global Thy_Load.master_path;
 wenzelm parents: 
40960diff
changeset | 396 | SOME (_, name, f) => init_theory master name f (reset_trans tr) | 
| 
47fef6afe756
Toplevel.init_theory: maintain optional master directory, to allow bypassing global Thy_Load.master_path;
 wenzelm parents: 
40960diff
changeset | 397 | | NONE => tr); | 
| 37977 
3ceccd415145
simplified/clarified theory loader: more explicit task management, kill old versions at start, commit results only in the very end, non-optional master dependency, do not store text in deps;
 wenzelm parents: 
37953diff
changeset | 398 | |
| 
3ceccd415145
simplified/clarified theory loader: more explicit task management, kill old versions at start, commit results only in the very end, non-optional master dependency, do not store text in deps;
 wenzelm parents: 
37953diff
changeset | 399 | fun modify_init f tr = | 
| 41536 
47fef6afe756
Toplevel.init_theory: maintain optional master directory, to allow bypassing global Thy_Load.master_path;
 wenzelm parents: 
40960diff
changeset | 400 | (case get_init tr of | 
| 
47fef6afe756
Toplevel.init_theory: maintain optional master directory, to allow bypassing global Thy_Load.master_path;
 wenzelm parents: 
40960diff
changeset | 401 | SOME (master, name, _) => init_theory master name f (reset_trans tr) | 
| 37977 
3ceccd415145
simplified/clarified theory loader: more explicit task management, kill old versions at start, commit results only in the very end, non-optional master dependency, do not store text in deps;
 wenzelm parents: 
37953diff
changeset | 402 | | NONE => tr); | 
| 
3ceccd415145
simplified/clarified theory loader: more explicit task management, kill old versions at start, commit results only in the very end, non-optional master dependency, do not store text in deps;
 wenzelm parents: 
37953diff
changeset | 403 | |
| 6689 | 404 | val exit = add_trans Exit; | 
| 7612 | 405 | val keep' = add_trans o Keep; | 
| 30366 
e3d788b9dffb
simplified presentation: built into transaction, pass state directly;
 wenzelm parents: 
29516diff
changeset | 406 | |
| 
e3d788b9dffb
simplified presentation: built into transaction, pass state directly;
 wenzelm parents: 
29516diff
changeset | 407 | fun present_transaction f g = add_trans (Transaction (f, g)); | 
| 
e3d788b9dffb
simplified presentation: built into transaction, pass state directly;
 wenzelm parents: 
29516diff
changeset | 408 | fun transaction f = present_transaction f (K ()); | 
| 5828 | 409 | |
| 7612 | 410 | fun keep f = add_trans (Keep (fn _ => f)); | 
| 5828 | 411 | fun imperative f = keep (fn _ => f ()); | 
| 412 | ||
| 27840 | 413 | fun ignored pos = empty |> name "<ignored>" |> position pos |> imperative I; | 
| 414 | fun malformed pos msg = | |
| 415 | empty |> name "<malformed>" |> position pos |> imperative (fn () => error msg); | |
| 416 | ||
| 21007 | 417 | val unknown_theory = imperative (fn () => warning "Unknown theory context"); | 
| 418 | val unknown_proof = imperative (fn () => warning "Unknown proof context"); | |
| 419 | val unknown_context = imperative (fn () => warning "Unknown context"); | |
| 15668 | 420 | |
| 21007 | 421 | |
| 422 | (* theory transitions *) | |
| 15668 | 423 | |
| 27601 
6683cdb94af8
simplified commit_exit: operate on previous node of final state, include warning here;
 wenzelm parents: 
27583diff
changeset | 424 | fun generic_theory f = transaction (fn _ => | 
| 26491 | 425 | (fn Theory (gthy, _) => Theory (f gthy, NONE) | 
| 426 | | _ => raise UNDEF)); | |
| 427 | ||
| 27601 
6683cdb94af8
simplified commit_exit: operate on previous node of final state, include warning here;
 wenzelm parents: 
27583diff
changeset | 428 | fun theory' f = transaction (fn int => | 
| 33725 
a8481da77270
implicit name space grouping for theory/local_theory transactions;
 wenzelm parents: 
33671diff
changeset | 429 | (fn Theory (Context.Theory thy, _) => | 
| 
a8481da77270
implicit name space grouping for theory/local_theory transactions;
 wenzelm parents: 
33671diff
changeset | 430 | let val thy' = thy | 
| 
a8481da77270
implicit name space grouping for theory/local_theory transactions;
 wenzelm parents: 
33671diff
changeset | 431 | |> Sign.new_group | 
| 
a8481da77270
implicit name space grouping for theory/local_theory transactions;
 wenzelm parents: 
33671diff
changeset | 432 | |> Theory.checkpoint | 
| 
a8481da77270
implicit name space grouping for theory/local_theory transactions;
 wenzelm parents: 
33671diff
changeset | 433 | |> f int | 
| 
a8481da77270
implicit name space grouping for theory/local_theory transactions;
 wenzelm parents: 
33671diff
changeset | 434 | |> Sign.reset_group; | 
| 
a8481da77270
implicit name space grouping for theory/local_theory transactions;
 wenzelm parents: 
33671diff
changeset | 435 | in Theory (Context.Theory thy', NONE) end | 
| 20963 
a7fd8f05a2be
added type global_theory -- theory or local_theory;
 wenzelm parents: 
20928diff
changeset | 436 | | _ => raise UNDEF)); | 
| 
a7fd8f05a2be
added type global_theory -- theory or local_theory;
 wenzelm parents: 
20928diff
changeset | 437 | |
| 
a7fd8f05a2be
added type global_theory -- theory or local_theory;
 wenzelm parents: 
20928diff
changeset | 438 | fun theory f = theory' (K f); | 
| 
a7fd8f05a2be
added type global_theory -- theory or local_theory;
 wenzelm parents: 
20928diff
changeset | 439 | |
| 27601 
6683cdb94af8
simplified commit_exit: operate on previous node of final state, include warning here;
 wenzelm parents: 
27583diff
changeset | 440 | fun begin_local_theory begin f = transaction (fn _ => | 
| 20963 
a7fd8f05a2be
added type global_theory -- theory or local_theory;
 wenzelm parents: 
20928diff
changeset | 441 | (fn Theory (Context.Theory thy, _) => | 
| 
a7fd8f05a2be
added type global_theory -- theory or local_theory;
 wenzelm parents: 
20928diff
changeset | 442 | let | 
| 20985 | 443 | val lthy = f thy; | 
| 21294 | 444 | val gthy = if begin then Context.Proof lthy else Context.Theory (loc_exit lthy); | 
| 445 | in Theory (gthy, SOME lthy) end | |
| 20963 
a7fd8f05a2be
added type global_theory -- theory or local_theory;
 wenzelm parents: 
20928diff
changeset | 446 | | _ => raise UNDEF)); | 
| 17076 | 447 | |
| 27601 
6683cdb94af8
simplified commit_exit: operate on previous node of final state, include warning here;
 wenzelm parents: 
27583diff
changeset | 448 | val end_local_theory = transaction (fn _ => | 
| 21294 | 449 | (fn Theory (Context.Proof lthy, _) => Theory (Context.Theory (loc_exit lthy), SOME lthy) | 
| 21007 | 450 | | _ => raise UNDEF)); | 
| 451 | ||
| 452 | local | |
| 453 | ||
| 30366 
e3d788b9dffb
simplified presentation: built into transaction, pass state directly;
 wenzelm parents: 
29516diff
changeset | 454 | fun local_theory_presentation loc f = present_transaction (fn int => | 
| 21294 | 455 | (fn Theory (gthy, _) => | 
| 456 | let | |
| 457 | val finish = loc_finish loc gthy; | |
| 33725 
a8481da77270
implicit name space grouping for theory/local_theory transactions;
 wenzelm parents: 
33671diff
changeset | 458 | val lthy' = loc_begin loc gthy | 
| 
a8481da77270
implicit name space grouping for theory/local_theory transactions;
 wenzelm parents: 
33671diff
changeset | 459 | |> Local_Theory.new_group | 
| 
a8481da77270
implicit name space grouping for theory/local_theory transactions;
 wenzelm parents: 
33671diff
changeset | 460 | |> f int | 
| 
a8481da77270
implicit name space grouping for theory/local_theory transactions;
 wenzelm parents: 
33671diff
changeset | 461 | |> Local_Theory.reset_group; | 
| 21294 | 462 | in Theory (finish lthy', SOME lthy') end | 
| 30366 
e3d788b9dffb
simplified presentation: built into transaction, pass state directly;
 wenzelm parents: 
29516diff
changeset | 463 | | _ => raise UNDEF)); | 
| 15668 | 464 | |
| 21007 | 465 | in | 
| 466 | ||
| 30366 
e3d788b9dffb
simplified presentation: built into transaction, pass state directly;
 wenzelm parents: 
29516diff
changeset | 467 | fun local_theory' loc f = local_theory_presentation loc f (K ()); | 
| 29380 | 468 | fun local_theory loc f = local_theory' loc (K f); | 
| 30366 
e3d788b9dffb
simplified presentation: built into transaction, pass state directly;
 wenzelm parents: 
29516diff
changeset | 469 | fun present_local_theory loc = local_theory_presentation loc (K I); | 
| 18955 | 470 | |
| 21007 | 471 | end; | 
| 472 | ||
| 473 | ||
| 474 | (* proof transitions *) | |
| 475 | ||
| 27601 
6683cdb94af8
simplified commit_exit: operate on previous node of final state, include warning here;
 wenzelm parents: 
27583diff
changeset | 476 | fun end_proof f = transaction (fn int => | 
| 24795 
6f5cb7885fd7
print_state_context: local theory context, not proof context;
 wenzelm parents: 
24780diff
changeset | 477 | (fn Proof (prf, (finish, _)) => | 
| 33390 | 478 | let val state = Proof_Node.current prf in | 
| 21007 | 479 | if can (Proof.assert_bottom true) state then | 
| 480 | let | |
| 481 | val ctxt' = f int state; | |
| 482 | val gthy' = finish ctxt'; | |
| 483 | in Theory (gthy', SOME ctxt') end | |
| 484 | else raise UNDEF | |
| 485 | end | |
| 27564 
fc6d34e49e17
replaced obsolete ProofHistory by ProofNode (backtracking only);
 wenzelm parents: 
27500diff
changeset | 486 | | SkipProof (0, (gthy, _)) => Theory (gthy, NONE) | 
| 21007 | 487 | | _ => raise UNDEF)); | 
| 488 | ||
| 21294 | 489 | local | 
| 490 | ||
| 27601 
6683cdb94af8
simplified commit_exit: operate on previous node of final state, include warning here;
 wenzelm parents: 
27583diff
changeset | 491 | fun begin_proof init finish = transaction (fn int => | 
| 21294 | 492 | (fn Theory (gthy, _) => | 
| 493 | let | |
| 24453 | 494 | val prf = init int gthy; | 
| 28433 
b3dab95f098f
begin_proof: avoid race condition wrt. skip_proofs flag;
 wenzelm parents: 
28425diff
changeset | 495 | val skip = ! skip_proofs; | 
| 40960 | 496 | val (is_goal, no_skip) = | 
| 497 | (true, Proof.schematic_goal prf) handle ERROR _ => (false, true); | |
| 21294 | 498 | in | 
| 40960 | 499 | if is_goal andalso skip andalso no_skip then | 
| 21294 | 500 | warning "Cannot skip proof of schematic goal statement" | 
| 501 | else (); | |
| 40960 | 502 | if skip andalso not no_skip then | 
| 27564 
fc6d34e49e17
replaced obsolete ProofHistory by ProofNode (backtracking only);
 wenzelm parents: 
27500diff
changeset | 503 | SkipProof (0, (finish gthy (Proof.global_skip_proof int prf), gthy)) | 
| 33390 | 504 | else Proof (Proof_Node.init prf, (finish gthy, gthy)) | 
| 21294 | 505 | end | 
| 506 | | _ => raise UNDEF)); | |
| 507 | ||
| 508 | in | |
| 509 | ||
| 24780 
47bb1e380d83
local_theory transactions: more careful treatment of context position;
 wenzelm parents: 
24634diff
changeset | 510 | fun local_theory_to_proof' loc f = begin_proof | 
| 33725 
a8481da77270
implicit name space grouping for theory/local_theory transactions;
 wenzelm parents: 
33671diff
changeset | 511 | (fn int => fn gthy => f int (Local_Theory.new_group (loc_begin loc gthy))) | 
| 
a8481da77270
implicit name space grouping for theory/local_theory transactions;
 wenzelm parents: 
33671diff
changeset | 512 | (fn gthy => loc_finish loc gthy o Local_Theory.reset_group); | 
| 24780 
47bb1e380d83
local_theory transactions: more careful treatment of context position;
 wenzelm parents: 
24634diff
changeset | 513 | |
| 24453 | 514 | fun local_theory_to_proof loc f = local_theory_to_proof' loc (K f); | 
| 21294 | 515 | |
| 516 | fun theory_to_proof f = begin_proof | |
| 33725 
a8481da77270
implicit name space grouping for theory/local_theory transactions;
 wenzelm parents: 
33671diff
changeset | 517 | (K (fn Context.Theory thy => f (Theory.checkpoint (Sign.new_group thy)) | _ => raise UNDEF)) | 
| 
a8481da77270
implicit name space grouping for theory/local_theory transactions;
 wenzelm parents: 
33671diff
changeset | 518 | (K (Context.Theory o Sign.reset_group o ProofContext.theory_of)); | 
| 21294 | 519 | |
| 520 | end; | |
| 521 | ||
| 27601 
6683cdb94af8
simplified commit_exit: operate on previous node of final state, include warning here;
 wenzelm parents: 
27583diff
changeset | 522 | val forget_proof = transaction (fn _ => | 
| 21007 | 523 | (fn Proof (_, (_, orig_gthy)) => Theory (orig_gthy, NONE) | 
| 524 | | SkipProof (_, (_, orig_gthy)) => Theory (orig_gthy, NONE) | |
| 525 | | _ => raise UNDEF)); | |
| 526 | ||
| 30366 
e3d788b9dffb
simplified presentation: built into transaction, pass state directly;
 wenzelm parents: 
29516diff
changeset | 527 | val present_proof = present_transaction (fn _ => | 
| 33390 | 528 | (fn Proof (prf, x) => Proof (Proof_Node.apply I prf, x) | 
| 27564 
fc6d34e49e17
replaced obsolete ProofHistory by ProofNode (backtracking only);
 wenzelm parents: 
27500diff
changeset | 529 | | skip as SkipProof _ => skip | 
| 30366 
e3d788b9dffb
simplified presentation: built into transaction, pass state directly;
 wenzelm parents: 
29516diff
changeset | 530 | | _ => raise UNDEF)); | 
| 21177 | 531 | |
| 27601 
6683cdb94af8
simplified commit_exit: operate on previous node of final state, include warning here;
 wenzelm parents: 
27583diff
changeset | 532 | fun proofs' f = transaction (fn int => | 
| 33390 | 533 | (fn Proof (prf, x) => Proof (Proof_Node.applys (f int) prf, x) | 
| 27564 
fc6d34e49e17
replaced obsolete ProofHistory by ProofNode (backtracking only);
 wenzelm parents: 
27500diff
changeset | 534 | | skip as SkipProof _ => skip | 
| 16815 | 535 | | _ => raise UNDEF)); | 
| 15668 | 536 | |
| 17904 
21c6894b5998
simplified interfaces proof/proof' etc.: perform ProofHistory.apply(s)/current internally;
 wenzelm parents: 
17513diff
changeset | 537 | fun proof' f = proofs' (Seq.single oo f); | 
| 
21c6894b5998
simplified interfaces proof/proof' etc.: perform ProofHistory.apply(s)/current internally;
 wenzelm parents: 
17513diff
changeset | 538 | val proofs = proofs' o K; | 
| 6689 | 539 | val proof = proof' o K; | 
| 16815 | 540 | |
| 27601 
6683cdb94af8
simplified commit_exit: operate on previous node of final state, include warning here;
 wenzelm parents: 
27583diff
changeset | 541 | fun actual_proof f = transaction (fn _ => | 
| 21007 | 542 | (fn Proof (prf, x) => Proof (f prf, x) | 
| 20963 
a7fd8f05a2be
added type global_theory -- theory or local_theory;
 wenzelm parents: 
20928diff
changeset | 543 | | _ => raise UNDEF)); | 
| 16815 | 544 | |
| 27601 
6683cdb94af8
simplified commit_exit: operate on previous node of final state, include warning here;
 wenzelm parents: 
27583diff
changeset | 545 | fun skip_proof f = transaction (fn _ => | 
| 21007 | 546 | (fn SkipProof (h, x) => SkipProof (f h, x) | 
| 18563 | 547 | | _ => raise UNDEF)); | 
| 548 | ||
| 27601 
6683cdb94af8
simplified commit_exit: operate on previous node of final state, include warning here;
 wenzelm parents: 
27583diff
changeset | 549 | fun skip_proof_to_theory pred = transaction (fn _ => | 
| 27564 
fc6d34e49e17
replaced obsolete ProofHistory by ProofNode (backtracking only);
 wenzelm parents: 
27500diff
changeset | 550 | (fn SkipProof (d, (gthy, _)) => if pred d then Theory (gthy, NONE) else raise UNDEF | 
| 33725 
a8481da77270
implicit name space grouping for theory/local_theory transactions;
 wenzelm parents: 
33671diff
changeset | 551 | | _ => raise UNDEF)); | 
| 5828 | 552 | |
| 553 | ||
| 554 | ||
| 555 | (** toplevel transactions **) | |
| 556 | ||
| 27427 | 557 | (* identification *) | 
| 558 | ||
| 559 | fun get_id (Transition {pos, ...}) = Position.get_id pos;
 | |
| 560 | fun put_id id (tr as Transition {pos, ...}) = position (Position.put_id id pos) tr;
 | |
| 561 | ||
| 562 | ||
| 25960 | 563 | (* thread position *) | 
| 25799 | 564 | |
| 25960 | 565 | fun setmp_thread_position (Transition {pos, ...}) f x =
 | 
| 25819 
e6feb08b7f4b
replaced thread_properties by simplified version in position.ML;
 wenzelm parents: 
25809diff
changeset | 566 | Position.setmp_thread_data pos f x; | 
| 25799 | 567 | |
| 27606 | 568 | fun status tr m = | 
| 569 | setmp_thread_position tr (fn () => Output.status (Markup.markup m "")) (); | |
| 570 | ||
| 38876 
ec7045139e70
Toplevel.run_command: more careful treatment of interrupts stemming from nested multi-exceptions etc.;
 wenzelm parents: 
38875diff
changeset | 571 | fun error_msg tr msg = | 
| 
ec7045139e70
Toplevel.run_command: more careful treatment of interrupts stemming from nested multi-exceptions etc.;
 wenzelm parents: 
38875diff
changeset | 572 | setmp_thread_position tr (fn () => Output.error_msg msg) (); | 
| 26602 
5534b6a6b810
made purely value-oriented, moved global state to structure Isar (cf. isar.ML);
 wenzelm parents: 
26491diff
changeset | 573 | |
| 25799 | 574 | |
| 28095 
7eaf0813bdc3
added add_hook interface for post-transition hooks;
 wenzelm parents: 
27859diff
changeset | 575 | (* post-transition hooks *) | 
| 
7eaf0813bdc3
added add_hook interface for post-transition hooks;
 wenzelm parents: 
27859diff
changeset | 576 | |
| 37905 | 577 | local | 
| 578 | val hooks = Unsynchronized.ref ([]: (transition -> state -> state -> unit) list); | |
| 579 | in | |
| 28095 
7eaf0813bdc3
added add_hook interface for post-transition hooks;
 wenzelm parents: 
27859diff
changeset | 580 | |
| 32738 | 581 | fun add_hook f = CRITICAL (fn () => Unsynchronized.change hooks (cons f)); | 
| 33223 | 582 | fun get_hooks () = ! hooks; | 
| 28095 
7eaf0813bdc3
added add_hook interface for post-transition hooks;
 wenzelm parents: 
27859diff
changeset | 583 | |
| 
7eaf0813bdc3
added add_hook interface for post-transition hooks;
 wenzelm parents: 
27859diff
changeset | 584 | end; | 
| 
7eaf0813bdc3
added add_hook interface for post-transition hooks;
 wenzelm parents: 
27859diff
changeset | 585 | |
| 
7eaf0813bdc3
added add_hook interface for post-transition hooks;
 wenzelm parents: 
27859diff
changeset | 586 | |
| 5828 | 587 | (* apply transitions *) | 
| 588 | ||
| 6664 | 589 | local | 
| 590 | ||
| 32792 | 591 | fun app int (tr as Transition {trans, print, no_timing, ...}) =
 | 
| 25819 
e6feb08b7f4b
replaced thread_properties by simplified version in position.ML;
 wenzelm parents: 
25809diff
changeset | 592 | setmp_thread_position tr (fn state => | 
| 25799 | 593 | let | 
| 594 | fun do_timing f x = (warning (command_msg "" tr); timeap f x); | |
| 595 | fun do_profiling f x = profile (! profiling) f x; | |
| 596 | ||
| 26256 
3e7939e978c6
added exception CONTEXT, indicating context of another exception;
 wenzelm parents: 
26081diff
changeset | 597 | val (result, status) = | 
| 37905 | 598 | state |> | 
| 599 | (apply_trans int trans | |
| 600 | |> (! profiling > 0 andalso not no_timing) ? do_profiling | |
| 601 | |> (! profiling > 0 orelse ! timing andalso not no_timing) ? do_timing); | |
| 26256 
3e7939e978c6
added exception CONTEXT, indicating context of another exception;
 wenzelm parents: 
26081diff
changeset | 602 | |
| 26621 
78b3ad7af5d5
eliminated unused name_of, source, source_of, print', print3, three_buffersN;
 wenzelm parents: 
26602diff
changeset | 603 | val _ = if int andalso not (! quiet) andalso print then print_state false result else (); | 
| 26256 
3e7939e978c6
added exception CONTEXT, indicating context of another exception;
 wenzelm parents: 
26081diff
changeset | 604 | in (result, Option.map (fn UNDEF => type_error tr state | exn => exn) status) end); | 
| 6664 | 605 | |
| 606 | in | |
| 5828 | 607 | |
| 26602 
5534b6a6b810
made purely value-oriented, moved global state to structure Isar (cf. isar.ML);
 wenzelm parents: 
26491diff
changeset | 608 | fun transition int tr st = | 
| 28095 
7eaf0813bdc3
added add_hook interface for post-transition hooks;
 wenzelm parents: 
27859diff
changeset | 609 | let | 
| 
7eaf0813bdc3
added add_hook interface for post-transition hooks;
 wenzelm parents: 
27859diff
changeset | 610 | val hooks = get_hooks (); | 
| 28103 
b79e61861f0f
simplified Toplevel.add_hook: cover successful transactions only;
 wenzelm parents: 
28095diff
changeset | 611 | fun apply_hooks st' = hooks |> List.app (fn f => (try (fn () => f tr st st') (); ())); | 
| 28095 
7eaf0813bdc3
added add_hook interface for post-transition hooks;
 wenzelm parents: 
27859diff
changeset | 612 | |
| 
7eaf0813bdc3
added add_hook interface for post-transition hooks;
 wenzelm parents: 
27859diff
changeset | 613 | val ctxt = try context_of st; | 
| 
7eaf0813bdc3
added add_hook interface for post-transition hooks;
 wenzelm parents: 
27859diff
changeset | 614 | val res = | 
| 
7eaf0813bdc3
added add_hook interface for post-transition hooks;
 wenzelm parents: 
27859diff
changeset | 615 | (case app int tr st of | 
| 38888 
8248cda328de
moved Toplevel.run_command to Pure/PIDE/document.ML;
 wenzelm parents: 
38876diff
changeset | 616 | (_, SOME Runtime.TERMINATE) => NONE | 
| 
8248cda328de
moved Toplevel.run_command to Pure/PIDE/document.ML;
 wenzelm parents: 
38876diff
changeset | 617 | | (st', SOME (Runtime.EXCURSION_FAIL exn_info)) => SOME (st', SOME exn_info) | 
| 31476 
c5d2899b6de9
moved Isar toplevel runtime support to runtime.ML, which is loaded early (before ml_compiler.ML);
 wenzelm parents: 
31431diff
changeset | 618 | | (st', SOME exn) => SOME (st', SOME (Runtime.exn_context ctxt exn, at_command tr)) | 
| 28103 
b79e61861f0f
simplified Toplevel.add_hook: cover successful transactions only;
 wenzelm parents: 
28095diff
changeset | 619 | | (st', NONE) => SOME (st', NONE)); | 
| 
b79e61861f0f
simplified Toplevel.add_hook: cover successful transactions only;
 wenzelm parents: 
28095diff
changeset | 620 | val _ = (case res of SOME (st', NONE) => apply_hooks st' | _ => ()); | 
| 28095 
7eaf0813bdc3
added add_hook interface for post-transition hooks;
 wenzelm parents: 
27859diff
changeset | 621 | in res end; | 
| 6664 | 622 | |
| 623 | end; | |
| 5828 | 624 | |
| 625 | ||
| 28425 | 626 | (* nested commands *) | 
| 5828 | 627 | |
| 28425 | 628 | fun command tr st = | 
| 27576 
7afff36043e6
eliminated internal command history -- superceeded by global Isar state (cf. isar.ML);
 wenzelm parents: 
27564diff
changeset | 629 | (case transition (! interact) tr st of | 
| 28425 | 630 | SOME (st', NONE) => st' | 
| 39285 | 631 | | SOME (_, SOME (exn, info)) => | 
| 632 | if Exn.is_interrupt exn then reraise exn else raise Runtime.EXCURSION_FAIL (exn, info) | |
| 38888 
8248cda328de
moved Toplevel.run_command to Pure/PIDE/document.ML;
 wenzelm parents: 
38876diff
changeset | 633 | | NONE => raise Runtime.EXCURSION_FAIL (Runtime.TERMINATE, at_command tr)); | 
| 27576 
7afff36043e6
eliminated internal command history -- superceeded by global Isar state (cf. isar.ML);
 wenzelm parents: 
27564diff
changeset | 634 | |
| 29483 | 635 | fun command_result tr st = | 
| 636 | let val st' = command tr st | |
| 637 | in (st', st') end; | |
| 638 | ||
| 28433 
b3dab95f098f
begin_proof: avoid race condition wrt. skip_proofs flag;
 wenzelm parents: 
28425diff
changeset | 639 | |
| 
b3dab95f098f
begin_proof: avoid race condition wrt. skip_proofs flag;
 wenzelm parents: 
28425diff
changeset | 640 | (* excursion of units, consisting of commands with proof *) | 
| 
b3dab95f098f
begin_proof: avoid race condition wrt. skip_proofs flag;
 wenzelm parents: 
28425diff
changeset | 641 | |
| 33519 | 642 | structure States = Proof_Data | 
| 28974 
d6b190efa01a
excursion: pass explicit proof states as result of future proof, replaced low-level Thm.join_futures by PureThy.force_proofs;
 wenzelm parents: 
28645diff
changeset | 643 | ( | 
| 
d6b190efa01a
excursion: pass explicit proof states as result of future proof, replaced low-level Thm.join_futures by PureThy.force_proofs;
 wenzelm parents: 
28645diff
changeset | 644 | type T = state list future option; | 
| 
d6b190efa01a
excursion: pass explicit proof states as result of future proof, replaced low-level Thm.join_futures by PureThy.force_proofs;
 wenzelm parents: 
28645diff
changeset | 645 | fun init _ = NONE; | 
| 
d6b190efa01a
excursion: pass explicit proof states as result of future proof, replaced low-level Thm.join_futures by PureThy.force_proofs;
 wenzelm parents: 
28645diff
changeset | 646 | ); | 
| 
d6b190efa01a
excursion: pass explicit proof states as result of future proof, replaced low-level Thm.join_futures by PureThy.force_proofs;
 wenzelm parents: 
28645diff
changeset | 647 | |
| 
d6b190efa01a
excursion: pass explicit proof states as result of future proof, replaced low-level Thm.join_futures by PureThy.force_proofs;
 wenzelm parents: 
28645diff
changeset | 648 | fun proof_result immediate (tr, proof_trs) st = | 
| 28433 
b3dab95f098f
begin_proof: avoid race condition wrt. skip_proofs flag;
 wenzelm parents: 
28425diff
changeset | 649 | let val st' = command tr st in | 
| 36315 
e859879079c8
added keyword category "schematic goal", which prevents any attempt to fork the proof;
 wenzelm parents: 
35205diff
changeset | 650 | if immediate orelse | 
| 
e859879079c8
added keyword category "schematic goal", which prevents any attempt to fork the proof;
 wenzelm parents: 
35205diff
changeset | 651 | null proof_trs orelse | 
| 36950 | 652 | Keyword.is_schematic_goal (name_of tr) orelse | 
| 653 | exists (Keyword.is_qed_global o name_of) proof_trs orelse | |
| 36315 
e859879079c8
added keyword category "schematic goal", which prevents any attempt to fork the proof;
 wenzelm parents: 
35205diff
changeset | 654 | not (can proof_of st') orelse | 
| 
e859879079c8
added keyword category "schematic goal", which prevents any attempt to fork the proof;
 wenzelm parents: 
35205diff
changeset | 655 | Proof.is_relevant (proof_of st') | 
| 28433 
b3dab95f098f
begin_proof: avoid race condition wrt. skip_proofs flag;
 wenzelm parents: 
28425diff
changeset | 656 | then | 
| 28453 
06702e7acd1d
excursion/unit_result: no print for forked end, finish into global theory, pick resul from presentation context;
 wenzelm parents: 
28451diff
changeset | 657 | let val (states, st'') = fold_map command_result proof_trs st' | 
| 28974 
d6b190efa01a
excursion: pass explicit proof states as result of future proof, replaced low-level Thm.join_futures by PureThy.force_proofs;
 wenzelm parents: 
28645diff
changeset | 658 | in (Lazy.value ((tr, st') :: (proof_trs ~~ states)), st'') end | 
| 28453 
06702e7acd1d
excursion/unit_result: no print for forked end, finish into global theory, pick resul from presentation context;
 wenzelm parents: 
28451diff
changeset | 659 | else | 
| 28433 
b3dab95f098f
begin_proof: avoid race condition wrt. skip_proofs flag;
 wenzelm parents: 
28425diff
changeset | 660 | let | 
| 
b3dab95f098f
begin_proof: avoid race condition wrt. skip_proofs flag;
 wenzelm parents: 
28425diff
changeset | 661 | val (body_trs, end_tr) = split_last proof_trs; | 
| 28453 
06702e7acd1d
excursion/unit_result: no print for forked end, finish into global theory, pick resul from presentation context;
 wenzelm parents: 
28451diff
changeset | 662 | val finish = Context.Theory o ProofContext.theory_of; | 
| 28974 
d6b190efa01a
excursion: pass explicit proof states as result of future proof, replaced low-level Thm.join_futures by PureThy.force_proofs;
 wenzelm parents: 
28645diff
changeset | 663 | |
| 29386 | 664 | val future_proof = Proof.global_future_proof | 
| 28974 
d6b190efa01a
excursion: pass explicit proof states as result of future proof, replaced low-level Thm.join_futures by PureThy.force_proofs;
 wenzelm parents: 
28645diff
changeset | 665 | (fn prf => | 
| 41703 
d27950860514
parallelization of nested Isar proofs is subject to Goal.parallel_proofs_threshold;
 wenzelm parents: 
41674diff
changeset | 666 | Goal.fork_name "Toplevel.future_proof" | 
| 41673 | 667 | (fn () => | 
| 668 | let val (states, result_state) = | |
| 669 | (case st' of State (SOME (Proof (_, (_, orig_gthy))), prev) | |
| 670 | => State (SOME (Proof (Proof_Node.init prf, (finish, orig_gthy))), prev)) | |
| 671 | |> fold_map command_result body_trs | |
| 672 | ||> command (end_tr |> set_print false); | |
| 673 | in (states, presentation_context_of result_state) end)) | |
| 28974 
d6b190efa01a
excursion: pass explicit proof states as result of future proof, replaced low-level Thm.join_futures by PureThy.force_proofs;
 wenzelm parents: 
28645diff
changeset | 674 | #> (fn (states, ctxt) => States.put (SOME states) ctxt); | 
| 
d6b190efa01a
excursion: pass explicit proof states as result of future proof, replaced low-level Thm.join_futures by PureThy.force_proofs;
 wenzelm parents: 
28645diff
changeset | 675 | |
| 
d6b190efa01a
excursion: pass explicit proof states as result of future proof, replaced low-level Thm.join_futures by PureThy.force_proofs;
 wenzelm parents: 
28645diff
changeset | 676 | val st'' = st' |> command (end_tr |> reset_trans |> end_proof (K future_proof)); | 
| 
d6b190efa01a
excursion: pass explicit proof states as result of future proof, replaced low-level Thm.join_futures by PureThy.force_proofs;
 wenzelm parents: 
28645diff
changeset | 677 | |
| 
d6b190efa01a
excursion: pass explicit proof states as result of future proof, replaced low-level Thm.join_futures by PureThy.force_proofs;
 wenzelm parents: 
28645diff
changeset | 678 | val states = | 
| 30398 | 679 | (case States.get (presentation_context_of st'') of | 
| 37852 
a902f158b4fc
eliminated old-style sys_error/SYS_ERROR in favour of exception Fail -- after careful checking that there is no overlap with existing handling of that;
 wenzelm parents: 
37711diff
changeset | 680 |             NONE => raise Fail ("No future states for " ^ name_of tr ^ Position.str_of (pos_of tr))
 | 
| 28974 
d6b190efa01a
excursion: pass explicit proof states as result of future proof, replaced low-level Thm.join_futures by PureThy.force_proofs;
 wenzelm parents: 
28645diff
changeset | 681 | | SOME states => states); | 
| 
d6b190efa01a
excursion: pass explicit proof states as result of future proof, replaced low-level Thm.join_futures by PureThy.force_proofs;
 wenzelm parents: 
28645diff
changeset | 682 | val result = Lazy.lazy | 
| 
d6b190efa01a
excursion: pass explicit proof states as result of future proof, replaced low-level Thm.join_futures by PureThy.force_proofs;
 wenzelm parents: 
28645diff
changeset | 683 | (fn () => (tr, st') :: (body_trs ~~ Future.join states) @ [(end_tr, st'')]); | 
| 
d6b190efa01a
excursion: pass explicit proof states as result of future proof, replaced low-level Thm.join_futures by PureThy.force_proofs;
 wenzelm parents: 
28645diff
changeset | 684 | |
| 
d6b190efa01a
excursion: pass explicit proof states as result of future proof, replaced low-level Thm.join_futures by PureThy.force_proofs;
 wenzelm parents: 
28645diff
changeset | 685 | in (result, st'') end | 
| 28433 
b3dab95f098f
begin_proof: avoid race condition wrt. skip_proofs flag;
 wenzelm parents: 
28425diff
changeset | 686 | end; | 
| 
b3dab95f098f
begin_proof: avoid race condition wrt. skip_proofs flag;
 wenzelm parents: 
28425diff
changeset | 687 | |
| 29068 | 688 | fun excursion input = | 
| 28425 | 689 | let | 
| 28433 
b3dab95f098f
begin_proof: avoid race condition wrt. skip_proofs flag;
 wenzelm parents: 
28425diff
changeset | 690 | val end_pos = if null input then error "No input" else pos_of (fst (List.last input)); | 
| 29448 
34b9652b2f45
added Goal.future_enabled abstraction -- now also checks that this is already
 wenzelm parents: 
29435diff
changeset | 691 | val immediate = not (Goal.future_enabled ()); | 
| 29427 
7ba952481e29
excursion: commit_exit internally -- checkpoints are fully persistent now;
 wenzelm parents: 
29386diff
changeset | 692 | val (results, end_state) = fold_map (proof_result immediate) input toplevel; | 
| 37953 
ddc3b72f9a42
simplified handling of theory begin/end wrt. toplevel and theory loader;
 wenzelm parents: 
37951diff
changeset | 693 | val thy = end_theory end_pos end_state; | 
| 
ddc3b72f9a42
simplified handling of theory begin/end wrt. toplevel and theory loader;
 wenzelm parents: 
37951diff
changeset | 694 | in (Lazy.lazy (fn () => maps Lazy.force results), thy) end; | 
| 7062 | 695 | |
| 6664 | 696 | end; |