src/Pure/Pure.thy
Wed, 07 Sep 2022 11:25:49 +0200 wenzelm clarified message channel for 'print_state' (NB: the command was originally for TTY or Proof General);
Fri, 22 Jul 2022 15:28:56 +0200 wenzelm removed obsolete commands;
Fri, 22 Jul 2022 15:15:26 +0200 wenzelm command 'scala_build_generated_files' with proper management of source dependencies;
Tue, 12 Jul 2022 15:42:57 +0200 wenzelm support for classpath artifacts within session structure:
Fri, 08 Jul 2022 22:29:26 +0200 wenzelm support for Isabelle/Scala/Java modules in Isabelle/ML;
Mon, 06 Dec 2021 15:34:54 +0100 wenzelm discontinued old-style {* verbatim *} tokens;
Thu, 28 Oct 2021 12:09:58 +0200 wenzelm clarified keywords: major take precedence for commands, but not used for antiquotations;
Sun, 26 Sep 2021 18:49:55 +0200 wenzelm improper proof command 'guess' moved to separate theory "Pure-ex.Guess";
Tue, 21 Sep 2021 12:08:41 +0200 wenzelm clarified modules;
Mon, 20 Sep 2021 23:15:02 +0200 wenzelm localized command 'syntax' and 'no_syntax';
Mon, 20 Sep 2021 20:22:32 +0200 wenzelm clarified signature;
Mon, 23 Aug 2021 14:24:57 +0200 wenzelm clarified signature;
Mon, 23 Aug 2021 12:54:28 +0200 wenzelm clarified signature;
Wed, 26 May 2021 18:07:49 +0200 wenzelm more robust syntax;
Sat, 27 Feb 2021 13:39:06 +0100 wenzelm more checks;
Mon, 07 Dec 2020 16:09:06 +0100 wenzelm more accurate markup (refining 1c59b555ac4a);
Sun, 06 Dec 2020 20:49:44 +0100 wenzelm more accurate syntax, following Sessions.parse_roots in Scala;
Sun, 06 Dec 2020 16:27:37 +0100 wenzelm PIDE support for session ROOTS;
Sat, 05 Dec 2020 12:14:40 +0100 wenzelm support for PIDE markup for auxiliary files ("blobs");
Fri, 27 Nov 2020 23:51:37 +0100 wenzelm merged
Fri, 27 Nov 2020 21:59:23 +0100 wenzelm clarified theory keywords: loaded_files are determined statically in Scala, but ML needs to do it semantically;
Fri, 27 Nov 2020 06:48:35 +0000 haftmann refined syntax for bundle mixins for locale and class specifications
Sun, 01 Nov 2020 16:54:49 +0100 haftmann bundle mixins for locale and class specifications
Mon, 12 Oct 2020 07:25:38 +0000 haftmann dedicated module for toplevel target handling
Sat, 10 Oct 2020 18:43:09 +0000 haftmann consolidated terminology
Mon, 02 Mar 2020 14:58:37 +0000 haftmann infrastructure for extraction of equations x = t from premises beneath meta-all
Tue, 26 Nov 2019 08:09:44 +0100 ballarin Remove diagnostic command 'print_dependencies'.
Fri, 23 Aug 2019 14:32:51 +0200 wenzelm clarified 'thm_deps' command;
Sat, 17 Aug 2019 19:04:03 +0200 wenzelm clarified signature;
Sat, 17 Aug 2019 12:44:22 +0200 wenzelm added command 'thm_oracles';
Sun, 28 Apr 2019 13:09:15 +0200 wenzelm tuned signature;
Wed, 17 Apr 2019 16:57:06 +0000 haftmann backed out experimental b67bab2b132c, which slipped in accidentally
Tue, 16 Apr 2019 19:50:30 +0000 haftmann hierarchically inclusive named theorem collections
Sat, 13 Apr 2019 13:30:02 +0200 wenzelm more abbrevs;
Thu, 04 Apr 2019 22:17:37 +0200 wenzelm tuned;
Thu, 04 Apr 2019 20:45:55 +0200 wenzelm type Path.binding may be empty: check later via proper_binding;
Thu, 04 Apr 2019 16:47:09 +0200 wenzelm clarified export_files: Isabelle_System.copy_file_base preserves given directory sub-structure;
Thu, 04 Apr 2019 14:30:58 +0200 wenzelm added command 'compile_generated_files';
Wed, 03 Apr 2019 21:50:00 +0200 wenzelm clarified signature: more explicit operations for corresponding Isar commands;
Thu, 28 Mar 2019 21:24:55 +0100 wenzelm "export_code ... file_prefix ..." is the preferred way to produce output within the logical file-system within the theory context, as well as session exports;
Thu, 14 Mar 2019 16:55:06 +0100 wenzelm more specific keyword kinds;
Sun, 10 Mar 2019 21:12:29 +0100 wenzelm document markers are formal comments, and may thus occur anywhere in the command-span;
Sun, 10 Mar 2019 00:21:34 +0100 wenzelm added semantic document markers;
Tue, 15 Jan 2019 20:03:53 +0100 wenzelm added command 'export_generated_files';
Thu, 20 Dec 2018 12:40:24 +0000 haftmann disregard historic keyword
Sat, 01 Dec 2018 16:11:59 +0100 wenzelm clarified modules;
Fri, 30 Nov 2018 23:43:10 +0100 wenzelm more general command 'generate_file' for registered file types, notably Haskell;
Tue, 27 Nov 2018 21:07:39 +0100 wenzelm more accurate positions for "name" (quoted string) and "embedded" (cartouche): refer to content without delimiters, which is e.g. relevant for systematic selection/renaming of scope groups;
Thu, 08 Nov 2018 13:42:36 +0100 wenzelm more standard Resources.provide_parse_files: avoid duplicate markup reports;
Mon, 24 Sep 2018 19:53:45 +0200 wenzelm tuned signature: prefer value-oriented pretty-printing;
Mon, 24 Sep 2018 19:34:14 +0200 wenzelm tuned signature: prefer value-oriented pretty-printing;
Sun, 02 Sep 2018 14:14:43 +0200 wenzelm no reset_proof for notepad: begin/end structure takes precedence over goal/proof structure;
Tue, 28 Aug 2018 11:22:04 +0200 wenzelm tuned signature;
Tue, 28 Aug 2018 11:13:33 +0200 wenzelm clarified ML_environment: ML_write_global requires "Isabelle";
Mon, 27 Aug 2018 17:30:13 +0200 wenzelm clarified environment: allow "read>write" specification;
Mon, 27 Aug 2018 14:42:24 +0200 wenzelm support named ML environments, notably "Isabelle", "SML";
Sun, 26 Aug 2018 17:28:38 +0200 wenzelm clarified signature;
Tue, 26 Jun 2018 14:01:46 +0200 wenzelm clarified default tag;
Thu, 21 Jun 2018 14:49:21 +0200 wenzelm clarified signature;
Fri, 25 May 2018 22:47:57 +0200 wenzelm added command 'ML_export';
Tue, 06 Mar 2018 22:59:00 +0100 ballarin Drop rewrite rule arguments of sublocale and interpretation implementations.
Sun, 04 Mar 2018 12:22:48 +0100 ballarin Drop rewrites after defines in interpretations.
Fri, 02 Mar 2018 14:19:25 +0100 ballarin Proper rewrite morphisms in locale instances.
Sun, 25 Feb 2018 19:30:55 +0100 wenzelm tuned;
Tue, 16 Jan 2018 19:28:05 +0100 ballarin Experimental support for rewrite morphisms in locale instances.
Tue, 16 Jan 2018 11:27:52 +0100 wenzelm discontinued old form of marginal comments;
Tue, 09 Jan 2018 15:40:12 +0100 wenzelm clarified modules;
Thu, 28 Dec 2017 12:07:52 +0100 wenzelm prefer existing Resources.check_path;
Thu, 28 Dec 2017 11:49:54 +0100 wenzelm added command 'bibtex_file' (for PIDE interaction only);
Fri, 22 Dec 2017 18:32:59 +0100 wenzelm discontinued 'display_drafts' command;
Wed, 06 Dec 2017 18:59:33 +0100 wenzelm prefer control symbol antiquotations;
Sun, 03 Dec 2017 13:22:09 +0100 wenzelm discontinued old 'def' command;
Wed, 29 Nov 2017 10:27:56 +0100 wenzelm clarified dependencies: "isabelle build -S" should be invariant wrt. change of ML system or platform;
Wed, 08 Nov 2017 17:34:32 +0100 wenzelm formal dependency on "poly" executable;
Sun, 05 Nov 2017 17:45:17 +0100 wenzelm more uniform header syntax, in contrast to the former etc/abbrevs file-format (see 73939a9b70a3);
Mon, 02 Oct 2017 19:28:18 +0200 wenzelm added command 'external_file';
Sun, 02 Jul 2017 20:13:38 +0200 haftmann proper concept of code declaration wrt. atomicity and Isar declarations
Mon, 03 Jul 2017 13:51:55 +0200 wenzelm added command 'alias' and 'type_alias';
Mon, 26 Jun 2017 11:07:48 +0200 wenzelm clarified indentation;
Wed, 28 Dec 2016 10:39:50 +0100 wenzelm more uniform treatment of "bad" like other messages (with serial number);
Sun, 18 Dec 2016 12:34:31 +0100 wenzelm tuned;
Wed, 14 Sep 2016 14:37:38 +0200 wenzelm discontinued global etc/abbrevs;
Tue, 06 Sep 2016 13:26:14 +0200 wenzelm strictly sequential abbrevs;
Tue, 02 Aug 2016 17:35:18 +0200 wenzelm support 'abbrevs' within theory header;
Sat, 16 Jul 2016 00:38:33 +0200 wenzelm information about proof outline with cases (sendback);
Fri, 15 Jul 2016 23:46:28 +0200 wenzelm singleton result for 'proof' command (without backtracking), e.g. relevant for well-defined output;
Mon, 11 Jul 2016 20:58:00 +0200 wenzelm clarified indentation;
Mon, 11 Jul 2016 16:36:29 +0200 wenzelm explicit kind "before_command";
Mon, 11 Jul 2016 10:43:54 +0200 wenzelm more indentation for quasi_command keywords;
Thu, 23 Jun 2016 11:01:14 +0200 wenzelm tuned signature;
Tue, 21 Jun 2016 17:35:45 +0200 wenzelm tuned;
Sat, 11 Jun 2016 16:41:11 +0200 wenzelm clarified syntax;
Fri, 10 Jun 2016 22:47:25 +0200 wenzelm added command 'unbundle';
Fri, 10 Jun 2016 12:45:34 +0200 wenzelm prefer hybrid 'bundle' command;
Thu, 09 Jun 2016 17:13:52 +0200 wenzelm clarified;
Thu, 09 Jun 2016 15:41:49 +0200 wenzelm support for bundle definition via target;
Sun, 29 May 2016 15:40:25 +0200 wenzelm clarified check_open_spec / read_open_spec;
Sat, 28 May 2016 21:38:58 +0200 wenzelm clarified 'axiomatization';
Sat, 14 May 2016 19:49:10 +0200 wenzelm toplevel theorem statements support 'if'/'for' eigen-context;
Thu, 28 Apr 2016 09:43:11 +0200 wenzelm support 'assumes' in specifications, e.g. 'definition', 'inductive';
Tue, 26 Apr 2016 22:39:17 +0200 wenzelm 'obtain' supports structured statements (similar to 'define');
Mon, 25 Apr 2016 19:41:39 +0200 wenzelm old 'def' is legacy;
Sun, 24 Apr 2016 21:31:14 +0200 wenzelm added Isar command 'define';
Wed, 13 Apr 2016 18:01:05 +0200 wenzelm eliminated "xname" and variants;
Sun, 10 Apr 2016 21:46:12 +0200 wenzelm more standard session build process, including browser_info;
Fri, 08 Apr 2016 20:15:20 +0200 wenzelm eliminated unused simproc identifier;
Thu, 07 Apr 2016 16:53:43 +0200 wenzelm more conventional theory syntax for ML bootstrap, with 'ML_file' instead of 'use';
Thu, 07 Apr 2016 12:13:11 +0200 wenzelm Pure attribute setup is back to Pure/Isar/attrib.ML, where it can be editing continuously (see also 7eb0c04e4c40);
Tue, 05 Apr 2016 18:20:25 +0200 wenzelm support bootstrap from fresh SML environment, with syntax of Isabelle/ML or SML;
Tue, 05 Apr 2016 15:53:48 +0200 wenzelm tuned;
Mon, 04 Apr 2016 23:58:48 +0200 wenzelm more uniform ML file commands;
Mon, 04 Apr 2016 23:08:43 +0200 wenzelm tuned whitespace;
Mon, 04 Apr 2016 22:13:08 +0200 wenzelm tuned -- more explicit sections;
Mon, 04 Apr 2016 17:25:53 +0200 wenzelm clarified bootstrap -- avoid 'ML_file' in Pure.thy for uniformity;
Mon, 04 Apr 2016 17:02:34 +0200 wenzelm clarified bootstrap -- more uniform use of ML files;
Tue, 01 Mar 2016 19:42:59 +0100 wenzelm ML debugger support in Pure (again, see 3565c9f407ec);
Sun, 14 Feb 2016 16:30:27 +0100 wenzelm command '\<proof>' is an alias for 'sorry', with different typesetting;
Wed, 13 Jan 2016 16:55:56 +0100 wenzelm removed old 'defs' command;
Sat, 19 Dec 2015 11:05:04 +0100 haftmann abandoned attempt to unify sublocale and interpretation into global theories
Wed, 16 Dec 2015 16:31:36 +0100 wenzelm rule_attribute and declaration_attribute implicitly support abstract closure, but mixed_attribute implementations need to be aware of Thm.is_free_dummy;
less more (0) -120 tip