Mercurial
Mercurial
>
repos
>
isabelle
/ graph
summary
|
shortlog
|
changelog
| graph |
tags
|
bookmarks
|
branches
|
files
|
gz
|
help
less
more
|
(0)
-30000
-10000
-3000
-1000
-240
+240
+1000
+3000
+10000
tip
Find changesets by keywords (author, files, the commit message), revision number or hash, or
revset expression
.
The revision graph only works with JavaScript-enabled browsers.
superseded by plain_identify;
2017-11-04, by wenzelm
tolerate odd negative times from old log files (before 1698e9ccef2d);
2017-11-04, by wenzelm
prefer main entry points of HOL;
2017-11-04, by wenzelm
tuned signature;
2017-11-04, by wenzelm
clarified lazy Completion within Outer_Syntax: measurable speedup of Sessions.deps;
2017-11-04, by wenzelm
more robust sorted_entries;
2017-11-04, by wenzelm
more convenient build_log_history;
2017-11-04, by wenzelm
tuned;
2017-11-04, by wenzelm
more portable print_time, notably for occasional negative (!) elapsed time of theory_timing;
2017-11-04, by wenzelm
polyml-test version based on experimental branch NewTestRegisterSave;
2017-11-04, by wenzelm
support for libgmp on x86_64-darwin;
2017-11-03, by wenzelm
avoid slow IntInf.pow in Poly/ML 5.7.1 testing version, e.g. relevant for AFP/Lorenz_C0;
2017-11-03, by wenzelm
delegate boundary cases to existing IntInf.pow;
2017-11-03, by wenzelm
plain identify job for Isabelle + AFP, independent of any Isabelle technology;
2017-11-03, by wenzelm
tuned (non-unique example);
2017-11-03, by wenzelm
clarified situation of global theory names;
2017-11-03, by wenzelm
less global theories -- avoid confusion about special cases;
2017-11-03, by wenzelm
proper deps;
2017-11-02, by wenzelm
allow unrelated ancestor;
2017-11-02, by wenzelm
tuned;
2017-11-02, by wenzelm
support alternative ancestor session;
2017-11-02, by wenzelm
support focus_session, for much faster startup of Isabelle/jEdit;
2017-11-02, by wenzelm
more timing;
2017-11-01, by wenzelm
tuned;
2017-11-01, by wenzelm
init only once (see also c0f776b661fa);
2017-11-01, by wenzelm
proper merge (amending fb46c031c841);
2017-11-01, by wenzelm
build faster without heap images for minor imports;
2017-11-01, by wenzelm
proper order for entries from multiple profiles, notably "AFP";
2017-11-01, by wenzelm
tuned output;
2017-11-01, by wenzelm
tuned;
2017-11-01, by wenzelm
logic_selector refers to raw logic name;
2017-11-01, by wenzelm
clarified terminology;
2017-11-01, by wenzelm
tuned signature;
2017-11-01, by wenzelm
do not store bulky Session.Deps;
2017-11-01, by wenzelm
avoid duplicate invocation of expensive Sessions.deps on full_sessions;
2017-11-01, by wenzelm
added isabelle jedit options -B, -P, clarified -R;
2017-11-01, by wenzelm
no heap sharing for empty session (e.g. HOL-ODE);
2017-11-01, by wenzelm
tuned diagram;
2017-11-01, by wenzelm
clarified ROOT syntax: 'sessions' and 'theories' are optional, but need to be non-empty;
2017-11-01, by wenzelm
removed unused option, which is potentially expensive;
2017-10-31, by wenzelm
allow to augment session context via explicit session infos;
2017-10-31, by wenzelm
synthesize session with all required theories from other session imports;
2017-10-31, by wenzelm
clarified signature;
2017-10-31, by wenzelm
clarified signature;
2017-10-31, by wenzelm
clarified signature;
2017-10-31, by wenzelm
clarified signature;
2017-10-31, by wenzelm
clarified signature: global_theories is always required;
2017-10-31, by wenzelm
tuned;
2017-10-31, by wenzelm
tuned signature;
2017-10-31, by wenzelm
clarified modules;
2017-10-31, by wenzelm
minor performance tuning: avoid mutable variable for plain value, e.g. relevant for GC;
2017-10-31, by wenzelm
more permissive: db could be empty after hard crash;
2017-10-31, by wenzelm
no censorship (in contrast to 2c828c830ad7);
2017-10-31, by wenzelm
A few more topological results. And made some slow proofs faster
2017-10-31, by paulson
removed ancient nat-int transfer
2017-10-31, by haftmann
added lemma
2017-10-30, by haftmann
added 'mlex_iff' lemma and simplified proof
2017-10-30, by blanchet
merged
2017-10-30, by wenzelm
recovered document from 9bfb6978eb80;
2017-10-30, by wenzelm
NEWS;
2017-10-30, by wenzelm
obsolete;
2017-10-30, by wenzelm
tuned;
2017-10-30, by wenzelm
ROOT cleanup: empty 'document_files' means there is no document;
2017-10-30, by wenzelm
eliminated pointless warning (see a35af478aee4): empty 'document_files' means there is no document;
2017-10-30, by wenzelm
more informative timeout message, notably for build_status;
2017-10-30, by wenzelm
clarified: adapted to ML version;
2017-10-30, by wenzelm
proper order of initialization (amending 9953ae603a23);
2017-10-30, by wenzelm
More topological results overlooked last time
2017-10-30, by paulson
merged
2017-10-30, by paulson
New results in topology, mostly from HOL Light's moretop.ml
2017-10-30, by paulson
generalized some lemmas on multisets
2017-10-30, by haftmann
rule out pathologic instances
2017-10-30, by haftmann
tuned some proofs and added some lemmas
2017-10-30, by haftmann
more recent polyml-test version;
2017-10-29, by wenzelm
reduced simp_depth_limit
2017-10-29, by nipkow
generalized
2017-10-28, by immler
reduced heap hierarchy, for potentially improved performance;
2017-10-28, by wenzelm
deactivated old tests;
2017-10-28, by wenzelm
avoid slow proofs due to simp rules from 960509bfd47e;
2017-10-28, by wenzelm
some concrete commands;
2017-10-27, by wenzelm
tuned signature;
2017-10-27, by wenzelm
more formal messages;
2017-10-27, by wenzelm
tuned signature;
2017-10-27, by wenzelm
separate JSON parser, which is slightly more general than (deprecated) scala.util.parsing.json.JSON;
2017-10-27, by wenzelm
more permissive;
2017-10-27, by wenzelm
tuned;
2017-10-27, by wenzelm
separate JSON lexer;
2017-10-26, by wenzelm
clarified command language;
2017-10-26, by wenzelm
use Poly/ML 5.7.1 test version as default;
2017-10-26, by wenzelm
more explicit check;
2017-10-25, by wenzelm
more robust treatment of UTF8 in raw byte sources;
2017-10-25, by wenzelm
clarified check, assuming that load commands are plain ASCII;
2017-10-25, by wenzelm
more documentation;
2017-10-25, by wenzelm
disallow blanks, relevant for session_name / theory_name e.g. in build log files;
2017-10-25, by wenzelm
uniform system name;
2017-10-25, by wenzelm
store session sources stamp;
2017-10-24, by wenzelm
generalized lemmas cancelling real_of_int/real in (in)equalities with power; completed set of related simp rules; lemmas about floorlog/bitlen
2017-10-24, by immler
misc tuning and modernization;
2017-10-24, by wenzelm
tuned output;
2017-10-24, by wenzelm
discontinued Linux 32bit platform support;
2017-10-23, by wenzelm
obsolete;
2017-10-23, by wenzelm
merged
2017-10-23, by wenzelm
updated to jdk-8u152, which is for x86_64 only;
2017-10-23, by wenzelm
added lemma
2017-10-23, by nipkow
minor performance tuning: avoid mutable variable for plain value, e.g. relevant for GC;
2017-10-23, by wenzelm
tuned output;
2017-10-22, by wenzelm
updated test version;
2017-10-22, by wenzelm
merged
2017-10-22, by wenzelm
auto update;
2017-10-22, by wenzelm
more recent polyml-test version;
2017-10-22, by wenzelm
parallel remote_builds2 for the sake of "AFP slow" (with theoretical data race on build_log_dirs);
2017-10-22, by wenzelm
tuned;
2017-10-22, by wenzelm
clarified signature;
2017-10-22, by wenzelm
tuned: build hg_graph only once;
2017-10-22, by wenzelm
tuned
2017-10-22, by nipkow
derived axiom iffI as a lemma (thanks to Alexander Maletzky)
2017-10-22, by nipkow
remove trailing whitespaces in List
2017-10-21, by bulwahn
drop a superfluous assumption that was found by the find_unused_assms command
2017-10-21, by bulwahn
drop a superfluous assumption that was found by the find_unused_assms command and tune proof
2017-10-21, by bulwahn
drop a superfluous assumption that was found by the find_unused_assms command and tune proof
2017-10-21, by bulwahn
algebraic foundation for congruences
2017-10-20, by haftmann
more ambitious test;
2017-10-20, by wenzelm
added lemmas and tuned proofs
2017-10-20, by haftmann
merged
2017-10-19, by paulson
Switching to inverse image and constant_on, plus some new material
2017-10-19, by paulson
proper integer option for Admin/build_history;
2017-10-19, by wenzelm
clarified output;
2017-10-18, by wenzelm
tuned output;
2017-10-18, by wenzelm
more thorough treatment of afp_version and afp_pull_date;
2017-10-18, by wenzelm
tuned options;
2017-10-18, by wenzelm
tuned output;
2017-10-17, by wenzelm
uniform execute, with proper isabelle_identifier (notably for "isabelle components -I");
2017-10-17, by wenzelm
tuned;
2017-10-17, by wenzelm
permissive theory_timings for historic versions;
2017-10-17, by wenzelm
store theory timings in session in build_log database;
2017-10-16, by wenzelm
provide theory timing information, similar to command timing but always considered relevant;
2017-10-16, by wenzelm
tuned;
2017-10-16, by wenzelm
init user settings on fresh test machine;
2017-10-16, by wenzelm
added [simp]
2017-10-16, by nipkow
proper value;
2017-10-15, by wenzelm
more AFP tests;
2017-10-15, by wenzelm
added ml_statistics_step to trim stored properties;
2017-10-15, by wenzelm
proper argument;
2017-10-15, by wenzelm
tuned (graph.all_succs already contains origin);
2017-10-14, by wenzelm
support for AFP versions;
2017-10-14, by wenzelm
clarified afp_pull_date: both repository versions are relevant;
2017-10-14, by wenzelm
clarified stored build_args;
2017-10-14, by wenzelm
partition AFP sessions according to structure, which happens to cut it roughly into equal parts;
2017-10-14, by wenzelm
support for AFP in build_history and remote_build_history;
2017-10-14, by wenzelm
tuned whitespace;
2017-10-13, by wenzelm
support for AFP versions;
2017-10-13, by wenzelm
tuned signature;
2017-10-13, by wenzelm
tuned signature;
2017-10-13, by wenzelm
support for AFP versions;
2017-10-13, by wenzelm
tuned;
2017-10-13, by wenzelm
added lemmas, tuned spaces
2017-10-13, by nipkow
entries_graph requires acyclic graph, but lazy val allows forming the AFP object nonetheless;
2017-10-12, by wenzelm
more informative Imports.Report with actual session imports (minimized);
2017-10-12, by wenzelm
more robust: allow URLs;
2017-10-12, by wenzelm
more robust: allow Windows file names;
2017-10-12, by wenzelm
clarified signature;
2017-10-12, by wenzelm
relaxed assm
2017-10-12, by nipkow
back to build_polyml_component according to 54c6ec4166a4 (amending 808e6ddb5a50);
2017-10-11, by wenzelm
reactivated unfinished tool (cf. a3a847c4fbdb);
2017-10-11, by wenzelm
tuned whitespace;
2017-10-11, by wenzelm
clarified meta_digest;
2017-10-11, by wenzelm
tuned;
2017-10-11, by wenzelm
added isablle build option -f;
2017-10-11, by wenzelm
canonical multiplicative euclidean size
2017-10-09, by haftmann
clarified parity
2017-10-09, by haftmann
clarified uniqueness criterion for euclidean rings
2017-10-09, by haftmann
tuned proofs
2017-10-09, by haftmann
tuned imports
2017-10-09, by haftmann
fixed markup
2017-10-10, by paulson
ignore isolated nodes by default;
2017-10-10, by wenzelm
merged
2017-10-10, by wenzelm
cycle check with informative error;
2017-10-10, by wenzelm
tuned: each session has at most one defining entry;
2017-10-10, by wenzelm
more operations;
2017-10-10, by wenzelm
tuned signature;
2017-10-10, by wenzelm
tuned signature;
2017-10-10, by wenzelm
Divided Topology_Euclidean_Space in two, creating new theory Connected. Also deleted some duplicate / variant theorems
2017-10-10, by paulson
Session HOL-Analysis: Moebius functions and the Riemann mapping theorem.
2017-10-10, by paulson
merged
2017-10-09, by wenzelm
tuned: less oo-non-sense;
2017-10-09, by wenzelm
operations for graph display;
2017-10-09, by wenzelm
tuned signature;
2017-10-09, by wenzelm
dependencies of entries vs. sessions;
2017-10-09, by wenzelm
some administrative support for AFP;
2017-10-09, by wenzelm
tuned;
2017-10-09, by wenzelm
clarified signature: public access to ROOT file syntax;
2017-10-09, by wenzelm
euclidean rings need no normalization
2017-10-08, by haftmann
more fundamental definition of div and mod on int
2017-10-08, by haftmann
one uniform type class for parity structures
2017-10-08, by haftmann
generalized some rules
2017-10-08, by haftmann
avoid variant of mk_sum
2017-10-08, by haftmann
adjusted implementation according to comment
2017-10-08, by haftmann
dropped duplicates
2017-10-08, by haftmann
generalized simproc
2017-10-08, by haftmann
replaced recdef were easy to replace
2017-10-08, by haftmann
elementary definition of division on natural numbers
2017-10-08, by haftmann
tuned structure
2017-10-08, by haftmann
abolished (semi)ring_div in favour of euclidean_(semi)ring_cancel
2017-10-08, by haftmann
Polynomial_Factorial does not depend on Field_as_Ring as such
2017-10-08, by haftmann
avoid name clashes on interpretation of abstract locales
2017-10-08, by haftmann
avoid trivial definition
2017-10-08, by haftmann
canonical introduction and destruction rules for pairwise
2017-10-08, by haftmann
avoid fact name clashes
2017-10-08, by haftmann
spelling and tuned whitespace
2017-10-08, by haftmann
tuned
2017-10-08, by haftmann
fundamental property of division by units
2017-10-08, by haftmann
removed mere toy example from library
2017-10-08, by haftmann
tuned proofs
2017-10-08, by haftmann
dropped dead code
2017-10-08, by haftmann
Fixed the theorem name "closed_imp_fip_compact"
2017-10-09, by paulson
new material about connectedness, etc.
2017-10-09, by paulson
more on Docker;
2017-10-08, by wenzelm
removed obsolete RC tags;
2017-10-08, by wenzelm
build_docker is regular tool (non-admin);
2017-10-08, by wenzelm
merged
2017-10-08, by wenzelm
Added tag Isabelle2017 for changeset 64b47495676d
2017-10-08, by wenzelm
obsolete;
Isabelle2017
2017-10-04, by wenzelm
more NEWS;
2017-10-03, by wenzelm
updated for release;
2017-10-03, by wenzelm
merged
2017-10-08, by wenzelm
proper File.platform_path for SML/NJ on Windows;
2017-10-08, by wenzelm
clarified signature;
2017-10-08, by wenzelm
proper output of raw ML;
2017-10-08, by wenzelm
theory qualifier is always session name (see also 31e8a86971a8);
2017-10-07, by wenzelm
clarified session structure;
2017-10-07, by wenzelm
discontinued somewhat pointless session group: -g ZF may be replaced by -D ~~/src/ZF;
2017-10-07, by wenzelm
merged
2017-10-07, by wenzelm
clarified empty merge;
2017-10-07, by wenzelm
permissive loaded_theories (amending 67dbf5cdc056): user errors are produced e.g. in Known.make;
2017-10-07, by wenzelm
prefer native platform x86-windows, to make this work on x86_64-cygwin;
2017-10-07, by wenzelm
tuned signature;
2017-10-06, by wenzelm
even more robust syntax (amending 122df1fde073);
2017-10-06, by wenzelm
clarified error for bad session-qualified imports;
2017-10-06, by wenzelm
clarified node_syntax (amending ae38b8c0fdd9): default to overall_syntax, e.g. relevant for command spans wrt. bad header;
2017-10-06, by wenzelm
merged
2017-10-05, by wenzelm
less
more
|
(0)
-30000
-10000
-3000
-1000
-240
+240
+1000
+3000
+10000
tip