(* Title: Pure/Isar/isar_document.ML
Author: Makarius
Interactive Isar documents.
*)
signature ISAR_DOCUMENT =
sig
type state_id = string
type command_id = string
type document_id = string
val define_command: command_id -> Toplevel.transition -> unit
val begin_document: document_id -> Path.T -> unit
val end_document: document_id -> unit
val edit_document: document_id -> document_id -> (command_id * command_id option) list -> unit
end;
structure IsarDocument: ISAR_DOCUMENT =
struct
(* unique identifiers *)
type state_id = string;
type command_id = string;
type document_id = string;
fun new_id () = "isabelle:" ^ serial_string ();
fun err_dup kind id = error ("Duplicate " ^ kind ^ ": " ^ quote id);
fun err_undef kind id = error ("Unknown " ^ kind ^ ": " ^ quote id);
(** documents **)
(* command entries *)
datatype entry = Entry of {next: command_id option, state: state_id option};
fun make_entry next state = Entry {next = next, state = state};
fun the_entry entries (id: command_id) =
(case Symtab.lookup entries id of
NONE => err_undef "document entry" id
| SOME (Entry entry) => entry);
fun put_entry (id: command_id, entry: entry) = Symtab.update (id, entry);
(* document *)
datatype document = Document of
{dir: Path.T, (*master directory*)
name: string, (*theory name*)
start: command_id, (*empty start command*)
entries: entry Symtab.table}; (*unique command entries indexed by command_id*)
fun make_document dir name start entries =
Document {dir = dir, name = name, start = start, entries = entries};
fun map_entries f (Document {dir, name, start, entries}) =
make_document dir name start (f entries);
(* iterate entries *)
fun fold_entries opt_id f (Document {start, entries, ...}) =
let
fun apply NONE x = x
| apply (SOME id) x = apply (#next (the_entry entries id)) (f id x);
in if is_some opt_id then apply opt_id else apply (SOME start) end;
fun find_entries P (Document {start, entries, ...}) =
let
fun find _ NONE = NONE
| find prev (SOME id) =
if P id then SOME (prev, id)
else find (SOME id) (#next (the_entry entries id));
in find NONE (SOME start) end;
(* modify entries *)
fun insert_after (id: command_id) (id2: command_id) = map_entries (fn entries =>
let val {next, state} = the_entry entries id in
entries
|> put_entry (id, make_entry (SOME id2) state)
|> put_entry (id2, make_entry next NONE)
end);
fun delete_after (id: command_id) = map_entries (fn entries =>
let val {next, state} = the_entry entries id in
(case next of
NONE => error ("No next entry to delete: " ^ quote id)
| SOME id2 =>
entries |>
(case #next (the_entry entries id2) of
NONE => put_entry (id, make_entry NONE state)
| SOME id3 =>
put_entry (id, make_entry (SOME id3) state) #>
put_entry (id3, make_entry (#next (the_entry entries id3)) NONE)))
end);
(** global configuration **)
local
val global_states = ref (Symtab.empty: Toplevel.state option future Symtab.table);
val global_commands = ref (Symtab.empty: Toplevel.transition Symtab.table);
val global_documents = ref (Symtab.empty: document Symtab.table);
in
fun change_states f = NAMED_CRITICAL "Isar" (fn () => change global_states f);
fun get_states () = NAMED_CRITICAL "Isar" (fn () => ! global_states);
fun change_commands f = NAMED_CRITICAL "Isar" (fn () => change global_commands f);
fun get_commands () = NAMED_CRITICAL "Isar" (fn () => ! global_commands);
fun change_documents f = NAMED_CRITICAL "Isar" (fn () => change global_documents f);
fun get_documents () = NAMED_CRITICAL "Isar" (fn () => ! global_documents);
fun init () = NAMED_CRITICAL "Isar" (fn () =>
(global_states := Symtab.empty;
global_commands := Symtab.empty;
global_documents := Symtab.empty));
end;
fun define_state (id: state_id) state =
change_states (Symtab.update_new (id, state))
handle Symtab.DUP dup => err_dup "state" dup;
fun the_state (id: state_id) =
(case Symtab.lookup (get_states ()) id of
NONE => err_undef "state" id
| SOME state => state);
fun define_command id tr =
change_commands (Symtab.update_new (id, Toplevel.put_id id tr))
handle Symtab.DUP dup => err_dup "command" dup;
fun the_command (id: command_id) =
(case Symtab.lookup (get_commands ()) id of
NONE => err_undef "command" id
| SOME tr => tr);
fun define_document (id: document_id) document =
change_documents (Symtab.update_new (id, document))
handle Symtab.DUP dup => err_dup "document" dup;
fun the_document (id: document_id) =
(case Symtab.lookup (get_documents ()) id of
NONE => err_undef "document" id
| SOME (Document doc) => doc);
(* begin/end document *)
fun begin_document (id: document_id) path =
let
val (dir, name) = ThyLoad.split_thy_path path;
val _ = define_command id Toplevel.empty;
val _ = define_state id (Future.value (SOME Toplevel.toplevel));
val entries = Symtab.make [(id, make_entry NONE (SOME id))];
val _ = define_document id (make_document dir name id entries);
in () end;
fun end_document (id: document_id) = error "FIXME";
(* document editing *)
fun update_state tr state = Future.fork_deps [state] (fn () =>
(case Future.join state of NONE => NONE | SOME st => Toplevel.run_command tr st));
fun update_entry (id, state_id) entries =
Symtab.map_entry
fun update_states old_document new_document =
let
val Document {entries = old_entries, ...} = old_document;
val Document {entries = new_entries, ...} = new_document;
fun is_changed id =
(case try (the_entry new_entries) id of
SOME {state = SOME _, ...} => false
| _ => true);
fun cancel_state id () =
(case the_entry old_entries id of
{state = SOME state_id, ...} => Future.cancel (the_state state_id)
| _ => ());
fun new_state id (state_id, updates) =
let
val state_id' = new_id ();
val state' = update_state (the_command id) (the_state state_id);
val _ = define_state state_id' state';
in (state_id', (id, state_id') :: updates) end;
fun update_state (id, state_id) entries =
let val _ = Output.status (Markup.markup (Markup.command_state id state_id) "")
in put_entry (id, make_entry (#next (the_entry entries id)) (SOME state_id)) entries end;
in
(case find_entries is_changed old_document of
NONE => new_document
| SOME (prev, id) =>
let
val _ = fold_entries (SOME id) cancel_state old_document ();
val prev_state_id = the (#state (the_entry new_entries (the prev)));
val (_, updates) = fold_entries (SOME id) new_state new_document (prev_state_id, []);
val new_document' = new_document |> map_entries (fold update_state updates);
in new_document' end)
end;
fun edit_document (id: document_id) (id': document_id) edits =
let
val document = Document (the_document id);
val document' =
document
|> fold (fn (id, SOME id2) => insert_after id id2 | (id, NONE) => delete_after id) edits
|> update_states document;
val _ = define_document id' document';
in () end;
(** concrete syntax **)
local structure P = OuterParse structure V = ValueParse in
val _ =
OuterSyntax.internal_command "Isar.define_command"
(P.string -- P.string >> (fn (id, text) =>
Toplevel.imperative (fn () =>
define_command id (OuterSyntax.prepare_command (Position.id id) text))));
val _ =
OuterSyntax.internal_command "Isar.begin_document"
(P.string -- P.string >> (fn (id, path) =>
Toplevel.imperative (fn () => begin_document id (Path.explode path))));
val _ =
OuterSyntax.internal_command "Isar.end_document"
(P.string >> (fn id => Toplevel.imperative (fn () => end_document id)));
val _ =
OuterSyntax.internal_command "Isar.edit_document"
(P.string -- P.string -- V.list (P.string -- (P.string >> SOME) || P.string >> rpair NONE)
>> (fn ((id, new_id), edits) => Toplevel.imperative (fn () => end_document id new_id edits)));
end;
end;