wenzelm [Tue, 30 Jan 2024 12:48:27 +0100] rev 79545
more robust message;
paulson <lp15@cam.ac.uk> [Tue, 30 Jan 2024 16:39:21 +0000] rev 79544
A few more new theorems taken from AFP entries
nipkow [Mon, 29 Jan 2024 21:18:11 +0100] rev 79543
merged
nipkow [Mon, 29 Jan 2024 21:17:57 +0100] rev 79542
define_time_function: avoid unused let's
haftmann [Mon, 29 Jan 2024 19:35:07 +0000] rev 79541
common type class for trivial properties on div/mod
wenzelm [Mon, 29 Jan 2024 11:54:44 +0100] rev 79540
more robust (amending 1600fb749c54), to support the following corner case:
schematic_goal "PROP ((?f :: ?'a \<Rightarrow> _) (x :: ?'a))"
apply (tactic \<open>PRIMITIVE (Thm.instantiate (TVars.make1 ((("'a", 0), []), @{ctyp prop}), Vars.empty))\<close>)
oops
wenzelm [Sun, 28 Jan 2024 19:22:33 +0100] rev 79539
proper test options;
wenzelm [Sat, 27 Jan 2024 23:05:00 +0100] rev 79538
proper history_base for linux_arm;
wenzelm [Sat, 27 Jan 2024 22:35:14 +0100] rev 79537
updated to PostgreSQL 12 on Ubuntu 20.04;
more accurate command-line;
wenzelm [Sat, 27 Jan 2024 22:15:40 +0100] rev 79536
routine build + test for linux_arm;
wenzelm [Sat, 27 Jan 2024 21:12:16 +0100] rev 79535
disable test on "augsburg1": machine will be dismantled;
Fabian Huch <huch@in.tum.de> [Fri, 26 Jan 2024 16:06:48 +0100] rev 79534
add approximation factors in build schedule to estimate build times more conservatively;
paulson [Fri, 26 Jan 2024 11:19:30 +0000] rev 79533
merged
paulson <lp15@cam.ac.uk> [Fri, 26 Jan 2024 11:19:22 +0000] rev 79532
Type class patch suggested by Achim Brucker, plus tidied lemma
haftmann [Thu, 25 Jan 2024 11:19:03 +0000] rev 79531
rearranged and reformulated abstract classes for bit structures and operations
paulson <lp15@cam.ac.uk> [Thu, 25 Jan 2024 17:08:07 +0000] rev 79530
Three new lemmas
wenzelm [Wed, 24 Jan 2024 23:53:51 +0100] rev 79529
tuned proof: avoid z3 to make it work on arm64-linux;
wenzelm [Wed, 24 Jan 2024 22:43:41 +0100] rev 79528
update to jdk-21.0.2;
enforce rebuild of Isabelle/Scala + Isabelle/ML;
Fabian Huch <huch@in.tum.de> [Wed, 24 Jan 2024 18:41:21 +0100] rev 79527
make build process state protected to avoid copying in subclasses (e.g. for database connections);
Fabian Huch <huch@in.tum.de> [Wed, 24 Jan 2024 17:30:49 +0100] rev 79526
add build_sync tag to sync certain options (e.g., build_engine) across build processes;
wenzelm [Tue, 23 Jan 2024 23:15:51 +0100] rev 79525
clarified Mercurial version: presumably the last version that supports both python2 and python3;
wenzelm [Tue, 23 Jan 2024 21:00:54 +0100] rev 79524
more robust: avoid crash on non-Linux systems;
wenzelm [Tue, 23 Jan 2024 20:50:24 +0100] rev 79523
clarified webserver names;
wenzelm [Tue, 23 Jan 2024 20:10:40 +0100] rev 79522
proper Apache.php_name;
wenzelm [Tue, 23 Jan 2024 19:56:52 +0100] rev 79521
proper packages for mercurial_setup on Ubuntu 22.04: building from source provides hgweb modules, and also provides a defined version (6.1.1 is also provided by Ubuntu 22.04);
wenzelm [Tue, 23 Jan 2024 19:39:49 +0100] rev 79520
tuned source structure;
wenzelm [Tue, 23 Jan 2024 16:30:29 +0100] rev 79519
more robust systemd configuration;
wenzelm [Tue, 23 Jan 2024 15:02:52 +0100] rev 79518
more robust nginx configuration, notably for "certbot --nginx -d DOMAIN";
wenzelm [Tue, 23 Jan 2024 12:28:35 +0100] rev 79517
tuned whitespace in generated file;
wenzelm [Tue, 23 Jan 2024 12:28:02 +0100] rev 79516
tuned;