wenzelm [Mon, 12 Mar 2018 11:00:52 +0100] rev 67834
tuned;
wenzelm [Mon, 12 Mar 2018 10:55:02 +0100] rev 67833
tuned signature;
wenzelm [Mon, 12 Mar 2018 10:50:26 +0100] rev 67832
clarified signature -- do not expose socket;
Manuel Eberl <eberlm@in.tum.de> [Mon, 12 Mar 2018 21:03:57 +0100] rev 67831
Removed stray 'sledgehammer' invocation
Manuel Eberl <eberlm@in.tum.de> [Mon, 12 Mar 2018 20:53:29 +0100] rev 67830
Changes to NEWS regarding 2a6ef5ba4822
Manuel Eberl <eberlm@in.tum.de> [Mon, 12 Mar 2018 20:52:53 +0100] rev 67829
Changes to complete distributive lattices due to Viorel Preoteasa
haftmann [Mon, 12 Mar 2018 08:25:35 +0000] rev 67828
eliminiated superfluous class semiring_bits
wenzelm [Sun, 11 Mar 2018 21:08:47 +0100] rev 67827
tuned;
wenzelm [Sun, 11 Mar 2018 20:56:42 +0100] rev 67826
tuned;
wenzelm [Sun, 11 Mar 2018 20:47:17 +0100] rev 67825
update XML cache for slightly modified messages;
wenzelm [Sun, 11 Mar 2018 20:31:25 +0100] rev 67824
more compact markup tree: output messages are already stored in command results (e.g. relevant for XML data representation);
wenzelm [Sun, 11 Mar 2018 15:28:22 +0100] rev 67823
more options;
wenzelm [Sun, 11 Mar 2018 15:21:20 +0100] rev 67822
clarified default server name;
wenzelm [Sun, 11 Mar 2018 15:15:30 +0100] rev 67821
more uniform output: this may be parsed by another program;
wenzelm [Sun, 11 Mar 2018 15:08:14 +0100] rev 67820
clarified argument formats: explicit Unit, allow XML.Elem as well;
tuned messages: prefer single quotes for JSON output;
wenzelm [Sun, 11 Mar 2018 15:06:48 +0100] rev 67819
tuned comments;
wenzelm [Sun, 11 Mar 2018 15:05:43 +0100] rev 67818
convenience to represent XML.Body as single XML.Elem;
wenzelm [Sun, 11 Mar 2018 13:18:41 +0100] rev 67817
clarified AFP partitioning;
haftmann [Sat, 10 Mar 2018 19:36:59 +0000] rev 67816
abstract algebraic bit operations
wenzelm [Sat, 10 Mar 2018 20:24:00 +0100] rev 67815
more balanced AFP partitioning;
wenzelm [Sat, 10 Mar 2018 15:52:47 +0100] rev 67814
workaround for occasional deadlock seen in HOL-Proofs with threads=2;
wenzelm [Sat, 10 Mar 2018 14:43:15 +0100] rev 67813
adapted to 3869b2400e22;
wenzelm [Sat, 10 Mar 2018 14:20:27 +0100] rev 67812
tuned output;
wenzelm [Sat, 10 Mar 2018 14:11:58 +0100] rev 67811
more options: client without implicit server startup;
wenzelm [Sat, 10 Mar 2018 13:54:55 +0100] rev 67810
console interaction with line-editor;
wenzelm [Sat, 10 Mar 2018 13:37:22 +0100] rev 67809
more flexible message formats;
wenzelm [Sat, 10 Mar 2018 13:03:01 +0100] rev 67808
clarified interrupt handling;
wenzelm [Sat, 10 Mar 2018 12:51:04 +0100] rev 67807
clarified signature;
wenzelm [Sat, 10 Mar 2018 12:34:07 +0100] rev 67806
option for console interaction;
wenzelm [Sat, 10 Mar 2018 11:55:54 +0100] rev 67805
more uniform Bytes.read_line/read_block operations;
wenzelm [Sat, 10 Mar 2018 11:40:25 +0100] rev 67804
auto update;
wenzelm [Sat, 10 Mar 2018 11:08:20 +0100] rev 67803
more comments;
wenzelm [Fri, 09 Mar 2018 17:03:10 +0100] rev 67802
more general TTY loop;
wenzelm [Fri, 09 Mar 2018 15:43:54 +0100] rev 67801
added Reply.NOTE for asynchronous notifications;
wenzelm [Fri, 09 Mar 2018 15:36:27 +0100] rev 67800
more operations;
wenzelm [Fri, 09 Mar 2018 15:24:19 +0100] rev 67799
more thorough init: purge inactive entries;
wenzelm [Fri, 09 Mar 2018 15:09:08 +0100] rev 67798
more generous timeout;
wenzelm [Fri, 09 Mar 2018 15:06:35 +0100] rev 67797
Entry.connection: proview password here;
more robust checks;
wenzelm [Fri, 09 Mar 2018 14:35:18 +0100] rev 67796
clarified initial protocol;
wenzelm [Fri, 09 Mar 2018 14:30:13 +0100] rev 67795
ignore empty lines;
wenzelm [Fri, 09 Mar 2018 14:26:08 +0100] rev 67794
tuned;
wenzelm [Fri, 09 Mar 2018 13:36:52 +0100] rev 67793
more robust read_line after shutdown;
wenzelm [Fri, 09 Mar 2018 13:11:47 +0100] rev 67792
more implicit wire protocol;
wenzelm [Fri, 09 Mar 2018 13:07:00 +0100] rev 67791
tuned signature;
wenzelm [Fri, 09 Mar 2018 13:03:55 +0100] rev 67790
clarified server start, notably for invocation within regular Isabelle/Scala process;
wenzelm [Fri, 09 Mar 2018 12:45:53 +0100] rev 67789
tuned signature;
wenzelm [Fri, 09 Mar 2018 12:42:34 +0100] rev 67788
tuned signature;
wenzelm [Fri, 09 Mar 2018 12:38:46 +0100] rev 67787
clarified toString operations;
wenzelm [Fri, 09 Mar 2018 12:29:56 +0100] rev 67786
clarified socket connection;
wenzelm [Fri, 09 Mar 2018 12:07:47 +0100] rev 67785
server commands may access Server;
Server.stop: proper shutdown;
clarified signature;
wenzelm [Thu, 08 Mar 2018 21:09:22 +0100] rev 67784
tuned -- avoid regex matching on potentially large string;
clarified message: command name could be malformed;
wenzelm [Thu, 08 Mar 2018 14:12:25 +0100] rev 67783
more robust build: prevent problems seen with Poly/ML eb94e2820013 on Mac OS X;
wenzelm [Thu, 08 Mar 2018 11:46:37 +0100] rev 67782
clarified notion of unknown files: ignore files outside of a Mercurial repository;
wenzelm [Thu, 08 Mar 2018 11:20:45 +0100] rev 67781
more balanced AFP partitioning;
wenzelm [Wed, 07 Mar 2018 19:02:22 +0100] rev 67780
more abbrevs -- this makes "(=" ambiguous and thus simplifies input of "(=)" (within the context of Main HOL);
wenzelm [Wed, 07 Mar 2018 17:39:18 +0100] rev 67779
tuned -- more uniform;
wenzelm [Wed, 07 Mar 2018 17:27:57 +0100] rev 67778
eliminated somewhat pointless parallelism (from 857da80611ab): usually hundreds of tasks with < 1ms each, also note that the enclosing join_theory happens within theory graph parallelism;
ballarin [Tue, 06 Mar 2018 22:59:00 +0100] rev 67777
Drop rewrite rule arguments of sublocale and interpretation implementations.
wenzelm [Tue, 06 Mar 2018 17:44:19 +0100] rev 67776
more balanced AFP partitioning;
wenzelm [Tue, 06 Mar 2018 17:43:39 +0100] rev 67775
clarified signature;
wenzelm [Tue, 06 Mar 2018 17:41:32 +0100] rev 67774
build_history_base as remote build on lxbroy10: thus self_update has already happened once, and thus avoids conflicts with parallel builds on shared home directory;
wenzelm [Tue, 06 Mar 2018 16:54:13 +0100] rev 67773
more robust: normalize potentially symbolic rev;
wenzelm [Tue, 06 Mar 2018 16:08:12 +0100] rev 67772
proxy setup for lrzcloud1;
wenzelm [Tue, 06 Mar 2018 15:57:34 +0100] rev 67771
tuned signature;
wenzelm [Tue, 06 Mar 2018 15:51:34 +0100] rev 67770
support for permissive connections, for odd situations where host keys are not accepted;
wenzelm [Tue, 06 Mar 2018 14:58:00 +0100] rev 67769
proper target directory;
wenzelm [Tue, 06 Mar 2018 14:41:05 +0100] rev 67768
eliminated dead code from 2a1acc88a180 (presumably left over from ML type-inference experimentation);
wenzelm [Sun, 04 Mar 2018 20:09:09 +0100] rev 67767
document existing Apache2 configuration;
wenzelm [Sun, 04 Mar 2018 15:10:11 +0100] rev 67766
consolidated main cronjob server on virtual machine together with build_log database;
eliminated special tricks for Gentoo;
import plain_identify logs, export all logs for backup;
run build_release, build_history_base in parallel to remote_build_history tasks;
wenzelm [Sun, 04 Mar 2018 13:51:58 +0100] rev 67765
identify closer to main cronjob -- avoid diverging changeset versions;
ballarin [Sun, 04 Mar 2018 12:22:48 +0100] rev 67764
Drop rewrites after defines in interpretations.
wenzelm [Sat, 03 Mar 2018 22:33:25 +0100] rev 67763
proper remote_mac according to Admin/Release/CHECKLIST;
wenzelm [Sat, 03 Mar 2018 21:40:04 +0100] rev 67762
more Java heap, e.g. relevant for hg.graph on Isabelle repository;
wenzelm [Sat, 03 Mar 2018 21:39:24 +0100] rev 67761
more robust check -- do not rely on return code;
wenzelm [Sat, 03 Mar 2018 21:38:27 +0100] rev 67760
more compact ML_Statistics, to make build_status work with less than 2GB heap;
wenzelm [Sat, 03 Mar 2018 17:37:33 +0100] rev 67759
retain latest ml_stats (amending e76c6cb0d461);
wenzelm [Sat, 03 Mar 2018 16:15:21 +0100] rev 67758
accomodate smaller build machine;
wenzelm [Sat, 03 Mar 2018 15:19:25 +0100] rev 67757
clarified signature;
wenzelm [Sat, 03 Mar 2018 15:09:36 +0100] rev 67756
clarified self_update: imitate visible directory state on remote side;
wenzelm [Sat, 03 Mar 2018 14:54:56 +0100] rev 67755
more operations;
wenzelm [Sat, 03 Mar 2018 14:27:33 +0100] rev 67754
self_update implies push_isabelle_home (see also 4c253e84ae62);
wenzelm [Sat, 03 Mar 2018 13:23:09 +0100] rev 67753
uniform setup_repository (pull/clone without update);
tuned signature;
wenzelm [Sat, 03 Mar 2018 13:06:33 +0100] rev 67752
clarified signature: facilitate interactive experimentation;
wenzelm [Sat, 03 Mar 2018 12:54:22 +0100] rev 67751
clarified tasks;
wenzelm [Sat, 03 Mar 2018 12:12:06 +0100] rev 67750
tuned signature;
wenzelm [Fri, 02 Mar 2018 20:46:25 +0100] rev 67749
proper order;
wenzelm [Fri, 02 Mar 2018 20:32:39 +0100] rev 67748
clarified README;
wenzelm [Fri, 02 Mar 2018 19:14:35 +0100] rev 67747
merged
wenzelm [Fri, 02 Mar 2018 18:57:55 +0100] rev 67746
more ssh options;
wenzelm [Fri, 02 Mar 2018 18:45:11 +0100] rev 67745
support for proxy connection, similar to ProxyCommand in ssh config;
wenzelm [Fri, 02 Mar 2018 15:16:10 +0100] rev 67744
prefer https;
wenzelm [Fri, 02 Mar 2018 11:52:27 +0100] rev 67743
avoid hardwired parameters;
less ambitious defaults: low memory requirements;
ballarin [Fri, 02 Mar 2018 15:14:59 +0100] rev 67742
Drop illegitimate optimisation from d5a7f2c54655.
ballarin [Fri, 02 Mar 2018 14:28:39 +0100] rev 67741
Fall back to reading rewrite morphism first if activation fails without it.
ballarin [Fri, 02 Mar 2018 14:19:25 +0100] rev 67740
Proper rewrite morphisms in locale instances.
wenzelm [Thu, 01 Mar 2018 20:44:38 +0100] rev 67739
clarified date for presentation vs. formal pull_date;
wenzelm [Thu, 01 Mar 2018 20:18:24 +0100] rev 67738
reveal raw data in CSV format;
wenzelm [Thu, 01 Mar 2018 20:05:41 +0100] rev 67737
support for CSV files;
wenzelm [Thu, 01 Mar 2018 15:02:45 +0100] rev 67736
tuned comment;
wenzelm [Thu, 01 Mar 2018 12:24:08 +0100] rev 67735
clarified syntax: reject formal comments explicitly, instead of ignoring them silently;
immler [Wed, 28 Feb 2018 17:05:34 +0100] rev 67734
merged
immler [Wed, 28 Feb 2018 15:53:05 +0100] rev 67733
generalized lemmas about orthogonal transformation
wenzelm [Wed, 28 Feb 2018 16:30:25 +0100] rev 67732
more explicit infixl (see initial 1edf0f223c6e);
clarified name;
wenzelm [Wed, 28 Feb 2018 13:37:33 +0100] rev 67731
clarified use of vec type syntax;
haftmann [Mon, 26 Feb 2018 11:52:53 +0000] rev 67730
new lemma
haftmann [Mon, 26 Feb 2018 11:52:52 +0000] rev 67729
dedicated append function for string literals
immler [Mon, 26 Feb 2018 09:58:47 +0100] rev 67728
generalized
immler [Mon, 26 Feb 2018 07:34:05 +0100] rev 67727
moved Lipschitz continuity from AFP/Ordinary_Differential_Equations and AFP/Gromov_Hyperbolicity; moved lemmas from AFP/Gromov_Hyperbolicity/Library_Complements
wenzelm [Sun, 25 Feb 2018 20:05:05 +0100] rev 67726
merged
wenzelm [Sun, 25 Feb 2018 19:43:38 +0100] rev 67725
prefer symbols;
wenzelm [Sun, 25 Feb 2018 19:30:55 +0100] rev 67724
tuned;
wenzelm [Sun, 25 Feb 2018 19:19:11 +0100] rev 67723
more abbrevs;