NEWS
Fri, 18 Feb 2022 12:20:30 +0100 wenzelm NEWS;
Thu, 17 Feb 2022 19:42:16 +0000 haftmann Avoid overaggresive splitting.
Thu, 17 Feb 2022 19:42:15 +0000 haftmann Avoid overaggresive simplification.
Wed, 16 Feb 2022 14:35:33 +0100 desharna NEWS
Tue, 01 Feb 2022 08:59:35 +0100 blanchet tuned NEWS
Mon, 31 Jan 2022 16:09:23 +0100 blanchet more NEWS
Mon, 31 Jan 2022 16:09:23 +0100 blanchet updated NEWS
Wed, 26 Jan 2022 14:05:36 +0100 blanchet treat 'using X by meson' as 'by (meson X)' to avoid loss of polymorphism (cf. metis)
Sat, 22 Jan 2022 11:46:25 +0100 desharna renamed run_action to run in Mirabelle.action record
Thu, 20 Jan 2022 13:56:51 +0100 desharna NEWS
Tue, 11 Jan 2022 22:07:04 +0100 desharna split option "sledgehammer_atp_dest_dir" into "sledgehammer_atp_prob_dest_dir" and "sledgehammer_atp_proof_dest_dir"
Tue, 21 Dec 2021 19:31:30 +0100 wenzelm support Gradle as alternative to Maven (again);
Sun, 19 Dec 2021 11:50:54 +0100 desharna NEWS
Mon, 06 Dec 2021 15:34:54 +0100 wenzelm discontinued old-style {* verbatim *} tokens;
Sat, 27 Nov 2021 10:46:57 +0100 desharna redefined less_multiset to be based on multp
Sat, 27 Nov 2021 10:01:40 +0100 desharna added lemma mono_multp
Fri, 26 Nov 2021 11:14:10 +0100 desharna added Multiset.multp as predicate equivalent of Multiset.mult
Fri, 26 Nov 2021 19:44:21 +0100 wenzelm merged
Fri, 26 Nov 2021 13:07:15 +0100 wenzelm NEWS on "isabelle mirabelle";
Fri, 26 Nov 2021 13:05:36 +0100 wenzelm tuned;
Thu, 25 Nov 2021 21:31:50 +0100 wenzelm clarified default for kodkod_scala;
Thu, 25 Nov 2021 19:56:01 +0100 wenzelm maintain option kodkod_scala within theory context, to allow local modification;
Thu, 25 Nov 2021 12:54:21 +0100 wenzelm NEWS for proper release;
Wed, 24 Nov 2021 22:57:33 +0100 wenzelm option document_comment_latex supports e.g. Dagstuhl LIPIcs;
Sun, 21 Nov 2021 17:42:11 +0100 wenzelm clarified system option standard values: avoid oddities like "isabelle build -o document_output" producing directories named "true";
Sat, 20 Nov 2021 18:58:23 +0100 wenzelm Latex.Output.latex_heading depends on option document_heading_prefix, e.g. relevant for Dagstuhl LIPIcs which prefers unaliased \section etc.;
Sat, 20 Nov 2021 12:59:53 +0100 wenzelm tuned;
Sat, 20 Nov 2021 12:53:18 +0100 wenzelm tuned;
Tue, 16 Nov 2021 22:38:34 +0100 wenzelm spelling;
Thu, 25 Nov 2021 14:02:51 +0100 desharna added asymp_{less,greater} to preorder and moved mult1_lessE out
Thu, 25 Nov 2021 12:19:50 +0100 desharna renamed multp_code_iff and multeqp_code_iff
Thu, 25 Nov 2021 12:13:49 +0100 desharna simplified mult_cancel_max and introduced orginal lemma as mult_cancel_max0
Thu, 25 Nov 2021 11:33:38 +0100 desharna renamed Multiset.multp and Multiset.multeqp
Tue, 16 Nov 2021 21:53:09 +0100 wenzelm merged
Tue, 16 Nov 2021 18:45:31 +0100 wenzelm proper version;
Tue, 16 Nov 2021 18:45:02 +0100 wenzelm back to Z3 4.4.0pre for all platforms except arm64-linux: avoid failure e.g. in Padic_Ints (AFP/7a2522dce834);
Mon, 15 Nov 2021 23:52:08 +0100 wenzelm updated NEWS: arm64-linux support is almost complete;
Fri, 12 Nov 2021 18:47:07 +0100 wenzelm back to post-release mode;
Mon, 08 Nov 2021 16:48:42 +0100 wenzelm discontinued redundant document_preprocessor: in the worst case, a plain-old document/build script will do;
Mon, 08 Nov 2021 13:51:24 +0100 wenzelm clarified messages, depending on option "document_echo";
Wed, 03 Nov 2021 21:06:04 +0100 wenzelm improved HTML presentation by Fabian Huch;
Tue, 02 Nov 2021 14:05:02 +0100 wenzelm more robust "isabelle scala_project": Gradle has been replaced by Maven;
Mon, 01 Nov 2021 23:13:14 +0100 wenzelm tuned;
Mon, 01 Nov 2021 15:49:03 +0100 wenzelm updated for release;
Mon, 01 Nov 2021 15:24:53 +0100 wenzelm some reordering for release;
Sat, 30 Oct 2021 13:26:33 +0200 wenzelm tuned;
Sat, 30 Oct 2021 13:12:22 +0200 wenzelm test version of prespective polyml-5.9;
Fri, 29 Oct 2021 11:57:49 +0200 wenzelm added Thm.instantiate_beta;
Thu, 28 Oct 2021 20:38:21 +0200 wenzelm discontinued somewhat pointless antiquotations;
Thu, 28 Oct 2021 20:32:40 +0200 wenzelm NEWS;
Thu, 28 Oct 2021 13:13:48 +0200 wenzelm local fixes for "lemma" antiquotation;
Tue, 26 Oct 2021 15:11:40 +0200 wenzelm more CONTRIBUTORS and NEWS;
Wed, 20 Oct 2021 18:13:17 +0200 wenzelm discontinued obsolete "val extend = I" for data slots;
Fri, 15 Oct 2021 19:25:31 +0200 wenzelm discontinued Term.dest_abs / Logic.dest_all, which are officially superseded by Variable.dest_abs etc., but there are also Term.dest_abs_global to recover existing tools easily;
Sun, 10 Oct 2021 14:45:53 +0000 haftmann avoid overaggressive contraction of conversions
Sat, 09 Oct 2021 16:41:21 +0000 haftmann normalizing NOT (numeral _) (again)
Thu, 07 Oct 2021 23:42:10 +0200 wenzelm recover NEWS from 78d1f73bbeaa;
Thu, 07 Oct 2021 22:46:47 +0200 wenzelm NEWS;
Wed, 06 Oct 2021 14:19:46 +0200 eberlm new notion of infinite sums in HOL-Analysis, ordering on complex numbers
Thu, 07 Oct 2021 10:34:48 +0200 desharna NEWS and CONTRIBUTORS
Wed, 06 Oct 2021 21:18:00 +0200 wenzelm updated to Vampire 4.6, as proposed by Martin Desharnais;
Mon, 04 Oct 2021 20:51:40 +0200 wenzelm removed pointless NEWS: both Docker/ubuntu and Cygwin provide perl by default;
Mon, 04 Oct 2021 20:07:51 +0200 wenzelm discontinued perl;
Mon, 04 Oct 2021 15:01:50 +0200 wenzelm clarified and updated for release;
Mon, 04 Oct 2021 14:02:11 +0200 wenzelm more NEWS and CONTRIBUTORS;
Mon, 04 Oct 2021 13:39:38 +0200 wenzelm support symbol \<Parallel>, based on \bigparallel from stdmaryd (stmary10.pfb: move y=1100, scale 222%, embolden by 40 units, adjust spacing);
Sat, 02 Oct 2021 22:11:34 +0200 wenzelm provide Isabelle/jEdit plugins as services, and thus allow user components do the same;
Sat, 02 Oct 2021 20:27:13 +0200 wenzelm misc tuning for release;
Wed, 29 Sep 2021 11:55:09 +0200 wenzelm clarified examples;
Tue, 28 Sep 2021 17:08:38 +0200 wenzelm more convenient ML arguments: avoid excessive nesting of cartouches;
Sun, 26 Sep 2021 20:13:28 +0200 wenzelm merged
Sun, 26 Sep 2021 18:49:55 +0200 wenzelm improper proof command 'guess' moved to separate theory "Pure-ex.Guess";
Sat, 25 Sep 2021 07:45:27 +0000 haftmann NOT is part of syntax bundle also
Wed, 22 Sep 2021 12:03:59 +0200 wenzelm proper NEWS;
Wed, 22 Sep 2021 11:58:45 +0200 wenzelm tuned NEWS;
Tue, 21 Sep 2021 13:12:14 +0200 wenzelm ML antiquotations for object-logic judgment;
Tue, 21 Sep 2021 00:20:55 +0200 wenzelm NEWS;
Sun, 19 Sep 2021 21:14:14 +0200 wenzelm support ML antiquotations with fn abstraction;
Sat, 11 Sep 2021 21:16:23 +0200 wenzelm ML antiquotations for type constructors and term constants;
Sat, 11 Sep 2021 13:04:32 +0200 wenzelm more antiquotations;
Fri, 10 Sep 2021 23:18:51 +0200 wenzelm tuned;
Fri, 10 Sep 2021 23:03:47 +0200 wenzelm NEWS;
Fri, 10 Sep 2021 15:08:09 +0200 wenzelm NEWS;
Sat, 21 Aug 2021 20:12:15 +0000 haftmann consolidation of rules for bit operations
Wed, 18 Aug 2021 23:04:58 +0200 wenzelm support configuration options "show_results";
Thu, 05 Aug 2021 07:12:49 +0000 haftmann clarified abstract and concrete boolean algebras
Tue, 03 Aug 2021 10:14:48 +0200 desharna fixed typo
Mon, 02 Aug 2021 10:01:06 +0000 haftmann moved theory Bit_Operations into Main corpus
Sun, 01 Aug 2021 10:20:34 +0000 haftmann organize syntax for word operations in bundles
Tue, 27 Jul 2021 15:20:20 +0200 wenzelm various improvements of "isabelle scala_project";
Sun, 18 Jul 2021 22:13:36 +0200 wenzelm tuned;
Sun, 18 Jul 2021 21:47:20 +0200 wenzelm NEWS;
Thu, 15 Jul 2021 22:49:24 +0200 wenzelm NEWS;
Thu, 08 Jul 2021 15:10:52 +0200 desharna added documentation for changes to Sledgehammer option "lam_trans"
Sun, 04 Jul 2021 18:35:57 +0100 paulson Imported lots of material from Stirling_Formula/Gamma_Asymptotics
Mon, 28 Jun 2021 20:10:23 +0200 Andreas Lochbihler move code setup from Cardinality to separate theory
Fri, 25 Jun 2021 21:14:57 +0200 wenzelm support for jEdit font substitution;
Wed, 23 Jun 2021 17:43:31 +0000 haftmann more default simp rules
Wed, 09 Jun 2021 18:04:22 +0000 haftmann global interpretation into nested targets
Wed, 09 Jun 2021 10:58:28 +0200 wenzelm NEWS;
Mon, 07 Jun 2021 14:41:04 +0200 wenzelm tuned;
Mon, 07 Jun 2021 14:40:22 +0200 wenzelm more formal theory and session names;
Mon, 07 Jun 2021 14:34:55 +0200 wenzelm proper NEWS after Isabelle2021;
Mon, 07 Jun 2021 11:42:05 +0200 wenzelm allow system option short form NAME for NAME=true for type string, not just bool;
Sun, 06 Jun 2021 15:49:39 +0000 haftmann moved more legacy to AFP
Fri, 28 May 2021 20:21:23 +0000 haftmann max word moved to Word_Lib in AFP
Mon, 24 May 2021 11:58:06 +0200 wenzelm clarified system_log: make this work independently of the particular "isabelle build" command-line (e.g. "isabelle mirabelle");
Sun, 23 May 2021 22:46:30 +0200 wenzelm syslog option for "isabelle build";
Sun, 23 May 2021 20:12:36 +0200 wenzelm NEWS;
Wed, 19 May 2021 13:19:37 +0200 wenzelm explicit option document_bibliography;
Wed, 19 May 2021 13:00:42 +0200 wenzelm discontinued obsolete "isabelle latex";
Wed, 19 May 2021 11:15:13 +0200 wenzelm clarified bash scripts, with public interfaces for user-defined Document_Build.Engine;
Tue, 18 May 2021 22:02:21 +0200 wenzelm option document_preprocessor;
Tue, 18 May 2021 15:46:03 +0200 wenzelm clarified treatment of Isabelle .sty files;
Tue, 18 May 2021 15:17:55 +0200 wenzelm option document_logo;
Mon, 17 May 2021 23:30:25 +0200 wenzelm option document_build refers to build engine in Isabelle/Scala;
Wed, 12 May 2021 17:05:29 +0000 haftmann explicit type class operations for type-specific implementations
Wed, 12 May 2021 17:05:28 +0000 haftmann obsolete
Tue, 11 May 2021 16:30:24 +0200 wenzelm clarified platforms;
Sun, 09 May 2021 05:48:50 +0000 haftmann more elementary swap
Wed, 05 May 2021 16:09:02 +0000 haftmann tuned theory structure
Wed, 05 May 2021 16:09:02 +0000 haftmann more appropriate location
Sun, 02 May 2021 17:38:49 +0200 wenzelm support nested cases;
Thu, 22 Apr 2021 10:11:11 +0200 wenzelm simplified typesetting of \<guillemotleft>...\<guillemotright>;
Fri, 16 Apr 2021 23:16:00 +0200 wenzelm support for conditional ML text;
Fri, 09 Apr 2021 22:06:59 +0200 wenzelm support for ML special forms: modified evaluation similar to Scheme;
Sat, 27 Mar 2021 18:01:41 +0100 wenzelm clarified output;
Sat, 27 Mar 2021 17:13:15 +0100 wenzelm support repository archives (without full .hg directory);
Thu, 25 Mar 2021 08:52:15 +0000 haftmann dedicated session for combinatorial material
Mon, 22 Mar 2021 17:33:08 +0100 wenzelm more NEWS;
Mon, 22 Mar 2021 10:49:51 +0000 haftmann more lemmas
Mon, 22 Mar 2021 00:07:55 +0100 wenzelm clarified package name (actually both pxfonts and txfonts exist and have this font);
Sun, 21 Mar 2021 23:56:54 +0100 wenzelm tuned;
Sun, 21 Mar 2021 23:03:31 +0100 wenzelm high-quality blackboard-bold fonts from "txmia" (package "txfonts");
Wed, 17 Mar 2021 22:24:57 +0100 wenzelm more Isabelle symbol definitions for Z Notation, based on https://github.com/isabelle-utp/Z_Toolkit 998c9f7880d3 by Simon Foster;
Sun, 14 Mar 2021 21:02:34 +0100 wenzelm removed spurious references to perl / libwww-perl;
Thu, 11 Mar 2021 07:05:38 +0000 haftmann avoid name clash
Thu, 11 Mar 2021 11:22:25 +0100 wenzelm tuned;
Tue, 09 Mar 2021 21:11:05 +0100 wenzelm proper type-setting of cartouches (requires T1);
Sun, 07 Mar 2021 08:24:24 +0100 haftmann follow corresponding precedence on sets
Sat, 06 Mar 2021 18:42:10 +0000 haftmann consolidated names
Fri, 05 Mar 2021 17:29:49 +0100 wenzelm clarified timeouts in Isabelle/ML;
Fri, 05 Mar 2021 10:30:54 +0100 haftmann typo
Mon, 01 Mar 2021 08:16:22 +0100 haftmann NEWS
Sat, 27 Feb 2021 22:17:56 +0100 wenzelm more Isabelle/ML/Scala operations;
Sat, 27 Feb 2021 21:36:58 +0100 wenzelm more Isabelle/ML/Scala operations;
Sat, 27 Feb 2021 21:01:07 +0100 wenzelm more Isabelle/ML/Scala operations;
Tue, 23 Feb 2021 23:00:08 +0100 wenzelm more on Isabelle_System.bash;
Tue, 23 Feb 2021 20:41:48 +0000 haftmann more specific name
Mon, 22 Feb 2021 23:31:59 +0100 wenzelm NEWS;
Mon, 22 Feb 2021 18:28:12 +0000 haftmann NEWS
Mon, 22 Feb 2021 07:49:48 +0000 haftmann get rid of traditional predicate
Fri, 19 Feb 2021 13:42:12 +0100 Manuel Eberl HOL-Analysis/Probability: Hoeffding's inequality, negative binomial distribution, etc.
Sat, 13 Feb 2021 20:39:29 +0100 wenzelm tuned NEWS;
Sun, 07 Feb 2021 20:44:44 +0100 wenzelm updated for release;
Wed, 03 Feb 2021 20:18:34 +0100 wenzelm clarified links to external files, e.g. .pdf within .thy source document;
Tue, 26 Jan 2021 23:34:40 +0100 wenzelm more NEWS;
Fri, 22 Jan 2021 18:44:34 +0100 wenzelm IDE support for Naproche-SAD;
Thu, 21 Jan 2021 16:10:43 +0100 wenzelm support isabelle components -u and -x;
Tue, 19 Jan 2021 14:14:23 +0100 wenzelm clarified documentation concerning macOS Big Sur;
Mon, 18 Jan 2021 20:11:42 +0100 wenzelm obsolete;
Mon, 18 Jan 2021 19:53:20 +0100 wenzelm more NEWS;
Sun, 17 Jan 2021 11:19:15 +0100 wenzelm revert 1105c42722dc on isabelle-release branch;
Sun, 10 Jan 2021 15:48:15 +0100 wenzelm back to post-release mode;
Sun, 10 Jan 2021 15:35:24 +0100 wenzelm tuned;
Sun, 10 Jan 2021 13:17:27 +0100 wenzelm more documentation;
Sat, 09 Jan 2021 19:49:22 +0100 wenzelm clarified default L&F of Isabelle/Scala (not Isabelle/jEdit);
Sat, 09 Jan 2021 00:11:52 +0100 wenzelm clarified default L&F;
Fri, 08 Jan 2021 19:53:44 +0100 Manuel Eberl HOL-Data_Structures: added Selection and time functions for list functions
Thu, 07 Jan 2021 13:23:54 +0100 wenzelm clarified NEWS;
Wed, 06 Jan 2021 12:59:52 +0100 wenzelm more NEWS;
Tue, 05 Jan 2021 03:35:46 +0100 Manuel Eberl HOL-Library.Multiset: new notation for prod_mset, consistent with sum_mset
Mon, 04 Jan 2021 21:25:40 +0100 wenzelm merged
Mon, 04 Jan 2021 21:24:15 +0100 wenzelm more documentation;
Mon, 04 Jan 2021 19:41:38 +0100 Manuel Eberl HOL-Library: Changed notation for sum_mset
Sun, 27 Dec 2020 14:04:16 +0100 wenzelm tuned;
Sun, 27 Dec 2020 13:52:55 +0100 wenzelm proper NEWS according to current situation;
Sun, 27 Dec 2020 13:49:03 +0100 wenzelm updated for release;
Thu, 24 Dec 2020 00:07:51 +0100 wenzelm more NEWS;
Wed, 23 Dec 2020 21:06:31 +0100 wenzelm clarified modules: avoid multiple uses of the same ML file;
Mon, 21 Dec 2020 14:03:12 +0100 wenzelm misc tuning for release;
Mon, 21 Dec 2020 13:58:11 +0100 wenzelm rebuild component with proper ZIPPERPOSITION_HOME for sledgehammer;
Mon, 21 Dec 2020 12:51:28 +0100 wenzelm provide zipperposition-2.0 for experimentation;
Sat, 19 Dec 2020 00:08:14 +0100 wenzelm download auxiliary files via "curl";
Fri, 18 Dec 2020 23:19:07 +0100 wenzelm improved markup for theory header imports;
Wed, 16 Dec 2020 15:39:21 +0100 wenzelm more NEWS;
Wed, 16 Dec 2020 13:47:33 +0100 wenzelm added action isabelle.goto-entity to follow links in a narrow formal sense;
Thu, 10 Dec 2020 22:44:53 +0100 wenzelm clarified session log file: avoid erratic messages;
Thu, 10 Dec 2020 18:38:26 +0100 wenzelm NEWS and documentation for "isabelle log";
Sun, 06 Dec 2020 16:27:37 +0100 wenzelm PIDE support for session ROOTS;
Fri, 04 Dec 2020 18:29:48 +0100 nipkow NEWS
Sat, 28 Nov 2020 21:56:24 +0100 wenzelm added document antiquotation @{tool};
Fri, 27 Nov 2020 23:51:37 +0100 wenzelm merged
Fri, 27 Nov 2020 23:47:06 +0100 wenzelm more flexible syntax for theory load commands via Isabelle/Scala;
Fri, 27 Nov 2020 06:48:35 +0000 haftmann refined syntax for bundle mixins for locale and class specifications
Thu, 26 Nov 2020 17:23:33 +0100 wenzelm clarified options: batch-build has pide_reports disabled by default (requires significant resources);
Sun, 22 Nov 2020 13:11:40 +0100 wenzelm updated to cvc4-1.8;
Sat, 21 Nov 2020 19:48:05 +0100 wenzelm tuned NEWS;
Sat, 21 Nov 2020 18:16:25 +0100 wenzelm more NEWS;
Sat, 21 Nov 2020 17:58:00 +0100 wenzelm NEWS;
Sun, 15 Nov 2020 07:17:06 +0000 haftmann bundles for reflected term syntax
Sat, 14 Nov 2020 12:55:05 +0100 wenzelm official support for document theories from other sessions;
Thu, 12 Nov 2020 09:06:44 +0100 haftmann bundled syntax for state monad combinators
Wed, 11 Nov 2020 21:00:14 +0100 wenzelm build documents in Isabelle/Scala, based on generated tex files as session exports;
Sat, 07 Nov 2020 16:49:51 +0100 wenzelm clarified output of "isabelle process";
Wed, 04 Nov 2020 07:39:17 +0000 haftmann NEWS and CONTRIBUTORS
Fri, 30 Oct 2020 22:56:15 +0100 wenzelm Isabelle/Phabricator supports Ubuntu 20.04 LTS;
Thu, 29 Oct 2020 16:07:41 +0100 desharna Added smt (verit) to Sledgehammer's proof preplay.
Thu, 29 Oct 2020 18:23:28 +0000 haftmann unified Local_Theory.init with Generic_Target.init
Thu, 29 Oct 2020 10:03:03 +0000 haftmann moved most material from session HOL-Word to Word_Lib in the AFP
Tue, 27 Oct 2020 22:34:37 +0100 wenzelm clarified signature: overloaded "+" for Path.append;
Mon, 26 Oct 2020 21:35:39 +0100 wenzelm NEWS;
Thu, 15 Oct 2020 13:24:16 +0200 wenzelm proper Isabelle component settings: prefer standard terminology "ISABELLE_VERIT", avoid conflict of "VERIT_VERSION" with processing of implicit options by veriT;
Tue, 13 Oct 2020 20:28:43 +0200 wenzelm merged
Tue, 13 Oct 2020 16:32:48 +0200 wenzelm tuned;
Tue, 13 Oct 2020 16:45:38 +0200 Mathias Fleury reconstruction of veriT proofs in NEWS
Mon, 12 Oct 2020 18:59:44 +0200 Mathias Fleury add reconstruction for the SMT solver veriT
Mon, 12 Oct 2020 17:42:15 +0200 wenzelm NEWS;
Mon, 12 Oct 2020 07:25:38 +0000 haftmann replaced combinators by more conventional nesting pattern
Mon, 12 Oct 2020 07:25:38 +0000 haftmann consolidated names and operations
Wed, 07 Oct 2020 10:39:14 +0200 haftmann consolidated for the sake of documentation
Tue, 29 Sep 2020 13:19:34 +0200 wenzelm allow Scala function execution on separate thread: better reactivity, but potential overloading of the JVM;
Mon, 28 Sep 2020 13:53:50 +0200 wenzelm clarified "isabelle logo", after discontinuation of DVI output (see 564012e31db1);
Sun, 27 Sep 2020 17:02:59 +0200 wenzelm ISABELLE_PDFLATEX is now lualatex;
Sat, 26 Sep 2020 14:29:46 +0200 wenzelm discontinued obsolete DVI document format and related settings/tools;
Fri, 25 Sep 2020 15:43:53 +0200 wenzelm clarified defaults for nitpick;
Fri, 25 Sep 2020 05:26:09 +0000 haftmann factored out typedef material
Wed, 23 Sep 2020 11:14:38 +0000 haftmann more thorough treatment of division, particularly signed division on int and word
Thu, 17 Sep 2020 13:55:21 +0200 haftmann typo
Thu, 17 Sep 2020 12:06:38 +0200 haftmann NEWS and CONTRIBUTORS
Thu, 10 Sep 2020 21:07:58 +0200 wenzelm more uniform JVM vs. ML status widget;
Tue, 08 Sep 2020 21:14:42 +0200 wenzelm update to official jedit-5.6.0;
Mon, 31 Aug 2020 22:05:05 +0200 wenzelm proper use of SELECT_GOAL to confine distinct_subgoals_tac to original goal range (amending 366d39e95d3c);
Tue, 25 Aug 2020 15:14:46 +0200 wenzelm NEWS;
Mon, 17 Aug 2020 16:26:58 +0200 wenzelm allow user-defined server commands via isabelle_scala_service;
Mon, 17 Aug 2020 13:16:42 +0200 wenzelm more systematic support for special directories;
Thu, 13 Aug 2020 15:52:40 +0200 wenzelm more documentation;
Fri, 07 Aug 2020 23:01:28 +0200 wenzelm NEWS;
Thu, 06 Aug 2020 22:43:40 +0200 wenzelm discontinued old batch-build functionality;
Wed, 05 Aug 2020 19:06:39 +0200 haftmann separation of reversed bit lists from other material
less more (0) -3000 -1000 -240 tip