History log of /seL4-l4v-master/isabelle/src/HOL/ex/Cartouche_Examples.thy
Revision Date Author Comments
# 56af848c 06-Jan-2019 wenzelm <none@none>

isabelle update -u control_cartouches;


# ed7a971e 05-Jan-2019 wenzelm <none@none>

isabelle update -u control_cartouches;


# 1e9e4316 31-Oct-2018 wenzelm <none@none>

clarified ML_Context.expression: it is a closed expression, not a let-declaration -- thus source positions are more accurate (amending d8849cfad60f, 162a4c2e97bc);


# 240e33b8 25-Oct-2018 wenzelm <none@none>

clarified ML position: proper markup for def/ref scopes (see also 162a4c2e97bc);


# 15f64c17 27-Aug-2018 wenzelm <none@none>

clarified signature;


# 3a4a7136 24-Apr-2018 haftmann <none@none>

proper datatype for 8-bit characters


# 610fd638 08-Jan-2018 wenzelm <none@none>

updated to 146757999c8d;


# 8faaa443 23-May-2016 wenzelm <none@none>

embedded content may be delimited via cartouches;


# f5e47925 26-Apr-2016 wenzelm <none@none>

misc tuning and modernization;


# 4eb81afa 07-Apr-2016 wenzelm <none@none>

explicit handling of recursive ML name space, e.g. relevant for ML_Bootstrap;
handle bootstrap signatures as well;


# a7d79152 04-Apr-2016 wenzelm <none@none>

clarified conditional compilation;


# 8175ce0f 12-Mar-2016 haftmann <none@none>

model characters directly as range 0..255
* * *
operate on syntax terms rather than asts


# 36e39dcf 26-Dec-2015 wenzelm <none@none>

isabelle update_cartouches -c -t;


# 6a6a64be 16-Oct-2015 wenzelm <none@none>

clarified Antiquote.antiq_reports;
Thy_Output.output_text: support for markdown (inactive);
eliminared Thy_Output.check_text -- uniform use of Thy_Output.output_text;


# 7f7de75b 18-Jul-2015 wenzelm <none@none>

prefer tactics with explicit context;


# 4aa541f4 06-Apr-2015 wenzelm <none@none>

@{command_spec} is superseded by @{command_keyword};


# f739ffa6 25-Mar-2015 wenzelm <none@none>

tuned signature;


# 986c7f6c 23-Dec-2014 wenzelm <none@none>

explicit message channels for "state", "information";
separate state_message_color;


# 8bec48b7 11-Dec-2014 wenzelm <none@none>

tuned;


# 509a45fc 10-Dec-2014 wenzelm <none@none>

more examples;


# 54c11317 08-Dec-2014 wenzelm <none@none>

expand ML cartouches to Input.source;
tuned signature;


# 142cfa6d 04-Dec-2014 wenzelm <none@none>

tuned header;


# 97306d3c 30-Nov-2014 wenzelm <none@none>

update_cartouches;


# fb314c8c 30-Nov-2014 wenzelm <none@none>

tuned signature;


# 9bbace2c 29-Nov-2014 wenzelm <none@none>

more abstract type Input.source;


# d552e1f7 22-Apr-2015 wenzelm <none@none>

tuned signature;


# 8acf1ce1 13-Nov-2014 wenzelm <none@none>

uniform treatment of all document markup commands: 'text' and 'txt' merely differ in LaTeX style;
discontinued obsolete 'txt_raw' (superseded by 'text_raw');
eliminated obsolete Outer_Syntax.markup (superseded by keyword kinds);
'text' and 'txt' no longer appear in Sidekick tree due to change of keyword kind;
changed tagging of diagnostic commands within proof;


# 65238ad7 12-Nov-2014 wenzelm <none@none>

more careful ML source positions, for improved PIDE markup;


# f19e7944 11-Nov-2014 wenzelm <none@none>

more position information, e.g. relevant for errors in generated ML source;


# c12ca051 07-Nov-2014 wenzelm <none@none>

plain value Keywords.keywords, which might be used outside theory for bootstrap purposes;
plain value Outer_Syntax within theory: parsing requires current theory context;
clarified name of Keyword.is_literal according to its semantics;
eliminated pointless type Keyword.T;
simplified @{command_spec};
clarified bootstrap keywords and syntax: take it as basis instead of side-branch;


# 7ee8e540 03-Nov-2014 wenzelm <none@none>

eliminated unused int_only flag (see also c12484a27367);
just proper commands;


# 794edf80 02-Nov-2014 wenzelm <none@none>

modernized header uniformly as section;


# 6635fc4f 09-Apr-2014 wenzelm <none@none>

proper Args.name vs. Args.text as documented (in contrast to adhoc union in 75aaee32893d, which had to cope with more limited Args.T);


# e5385d18 09-Apr-2014 wenzelm <none@none>

allow text cartouches in regular outer syntax categories "text" and "altstring";


# 2ff916cd 27-Mar-2014 wenzelm <none@none>

redirect ML_Compiler reports more directly: only the (big) parse tree report is deferred via Execution.print (NB: this does not work for asynchronous "diag" commands);
more explicit ML_Compiler.flags;


# 86334bff 25-Mar-2014 wenzelm <none@none>

separate tokenization and language context for SML: no symbols, no antiquotes;


# bcd9b054 25-Mar-2014 wenzelm <none@none>

added command 'SML_file' for Standard ML without Isabelle/ML add-ons;


# 42ab7e1e 12-Mar-2014 wenzelm <none@none>

tuned signature -- clarified module name;

--HG--
rename : src/Pure/ML/ml_antiquote.ML => src/Pure/ML/ml_antiquotation.ML


# 0e1799d7 01-Mar-2014 wenzelm <none@none>

clarified language markup: added "delimited" property;
type Symbol_Pos.source preserves information about delimited outer tokens (e.g string, cartouche);
observe Completion.Language_Context only for delimited languages, which is important to complete keywords after undelimited inner tokens, e.g. "lemma A pro";


# fd3490fe 25-Jan-2014 wenzelm <none@none>

simplified inner syntax;


# 08a19319 22-Jan-2014 wenzelm <none@none>

avoid breakdown of document preparation, which does not understand cartouche tokens yet;


# 8355749f 22-Jan-2014 wenzelm <none@none>

more cartouche examples, including uniform nesting of sub-languages;


# 3286e50f 19-Jan-2014 wenzelm <none@none>

implicit "cartouche" method (experimental, undocumented);


# b59e95b0 19-Jan-2014 wenzelm <none@none>

more examples;


# d6c7b394 18-Jan-2014 wenzelm <none@none>

proper \<newline>;


# 42b5b84f 18-Jan-2014 wenzelm <none@none>

support for nested text cartouches;
clarified Symbol.is_symbolic: exclude \<open> and \<close>;