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
less more (0) -3000 -1000 -120 tip