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
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.
merged
2021-11-04, by wenzelm
clarified Theory_Cache: prefer immutable data with Synchronized variable;
2021-11-04, by wenzelm
tuned signature;
2021-11-04, by wenzelm
unused;
2021-11-04, by wenzelm
proper support of verit's return code for timeout
2021-11-04, by Mathias Fleury
tuned whitespace;
2021-11-04, by wenzelm
updated to verit-2021.06.1-rmx, to address "Abnormal termination with exit code 14";
2021-11-04, by wenzelm
clarified signature;
2021-11-04, by wenzelm
prefer official Export.explode_name;
2021-11-04, by wenzelm
tuned;
2021-11-04, by wenzelm
avoid conflict with future keyword;
2021-11-04, by wenzelm
tuned messages;
2021-11-04, by wenzelm
clarified signature: more direct XML.symbol_length;
2021-11-04, by wenzelm
more direct Symbol.length: Symbol.decode is redundant, symbol counts are invariant under it;
2021-11-04, by wenzelm
tuned -- eliminate clones stemming from d28a51dd9da6;
2021-11-04, by wenzelm
more to ANNOUNCE;
2021-11-03, by wenzelm
clarified link style: similar to Isabelle/jEdit;
2021-11-03, by wenzelm
tuned;
2021-11-03, by wenzelm
improved HTML presentation by Fabian Huch;
2021-11-03, by wenzelm
proper HTTPS;
2021-11-03, by wenzelm
proper markup type (amending be49c660ebbf);
2021-11-03, by wenzelm
merged;
2021-11-03, by wenzelm
more PIDE markup;
2021-11-03, by wenzelm
tuned signature;
2021-11-03, by wenzelm
more PIDE markup;
2021-11-03, by wenzelm
recover library_index_content.template from c337c798f64c: required for website/build/main;
2021-11-03, by wenzelm
merged
2021-11-03, by paulson
simplified some ugly proofs
2021-11-02, by paulson
more generous timeout: support build on Raspberry Pi;
2021-11-03, by wenzelm
add documentation for pred_mono
2021-11-03, by traytel
merged
2021-11-03, by desharna
added "mono" attribute to BNF generated pred_mono theorems
2021-11-02, by desharna
merged
2021-11-02, by desharna
do not declare $let-bound variables in TPTP output
2021-10-29, by desharna
IDE build actually works (but somewhat pointless);
2021-11-03, by wenzelm
suppress sources from jEdit/test, which prevent regular build of the generated scala_project;
2021-11-03, by wenzelm
removed junk;
2021-11-03, by wenzelm
improve pagebreaks by *not* using supertabular too much;
2021-11-02, by wenzelm
updated to scala-2.13.7 --- problems with jline disappear after purging $HOME/.inputrc;
2021-11-02, by wenzelm
more robust "isabelle scala_project": Gradle has been replaced by Maven;
2021-11-02, by wenzelm
tuned;
2021-11-01, by wenzelm
support linux_arm as well, e.g. native Docker on Apple Silicon;
2021-11-01, by wenzelm
update paths at TUM;
2021-11-01, by wenzelm
Added tag Isabelle2021-1-RC1 for changeset 81cc8f2ea9e7
2021-11-01, by wenzelm
updated for release;
2021-11-01, by wenzelm
some reordering for release;
2021-11-01, by wenzelm
updated to jdk-17.0.1+12;
2021-11-01, by wenzelm
tuned message;
2021-11-01, by wenzelm
clarified antiquotations;
2021-10-31, by wenzelm
tuned;
2021-10-31, by wenzelm
minor performance tuning;
2021-10-31, by wenzelm
more robust;
2021-10-30, by wenzelm
provide native executables for arm64-darwin, for more robust startup without Rosetta 2;
2021-10-30, by wenzelm
tuned proofs -- avoid z3, which is unavailable on arm64-linux;
2021-10-30, by wenzelm
prefer "sat_solver = MiniSat", to make examples work uniformly on all platforms;
2021-10-30, by wenzelm
discontinued pointless check of kodkodi_version, it is implicit in the bundled component;
2021-10-30, by wenzelm
tuned proofs -- avoid z3, which is unavailable on arm64-linux;
2021-10-30, by wenzelm
tuned;
2021-10-30, by wenzelm
test version of prespective polyml-5.9;
2021-10-30, by wenzelm
clarified antiquotations;
2021-10-30, by wenzelm
updated for pre-5.9 testing;
2021-10-30, by wenzelm
clarified antiquotations;
2021-10-30, by wenzelm
clarified antiquotations;
2021-10-30, by wenzelm
clarified antiquotations;
2021-10-29, by wenzelm
more robust subgoal addressing;
2021-10-29, by wenzelm
proper subgoal addressing;
2021-10-29, by wenzelm
clarified antiquotations;
2021-10-29, by wenzelm
recursive find_eq, not find_dist;
2021-10-29, by wenzelm
misc tuning and clarification;
2021-10-29, by wenzelm
clarified antiquotations;
2021-10-29, by wenzelm
order_tac: prevent potential bug, improve perf and tracing
2021-10-29, by Lukas Stevens
misc tuning and clarification;
2021-10-29, by wenzelm
clarified antiquotations;
2021-10-29, by wenzelm
clarified antiquotations: no need for Thm.beta_conversion, due to Thm.instantiate_beta;
2021-10-29, by wenzelm
clarified antiquotations: no need for Thm.beta_conversion, due to Thm.instantiate_beta;
2021-10-29, by wenzelm
avoid persistence of static context: instantiation arguments should provide proper dynamic context (see also e2e2bc1f9570);
2021-10-29, by wenzelm
added Thm.instantiate_beta;
2021-10-29, by wenzelm
moved generic implementation into HOL-Main
2021-10-28, by haftmann
tuned;
2021-10-29, by wenzelm
tuned;
2021-10-28, by wenzelm
clarified antiquotations;
2021-10-28, by wenzelm
clarified antiquotations;
2021-10-28, by wenzelm
discontinued somewhat pointless antiquotations;
2021-10-28, by wenzelm
NEWS;
2021-10-28, by wenzelm
clarified antiquotations, assuming that Drule.instantiate_normalize was merely a historical relic;
2021-10-28, by wenzelm
clarified antiquotations;
2021-10-28, by wenzelm
clarified antiquotations;
2021-10-28, by wenzelm
clarified antiquotations;
2021-10-28, by wenzelm
clarified antiquotations;
2021-10-28, by wenzelm
support for "lemma";
2021-10-28, by wenzelm
tuned;
2021-10-28, by wenzelm
local fixes for "lemma" antiquotation;
2021-10-28, by wenzelm
clarified signature;
2021-10-28, by wenzelm
tuned;
2021-10-28, by wenzelm
clarified keywords: major take precedence for commands, but not used for antiquotations;
2021-10-28, by wenzelm
tuned modules;
2021-10-28, by wenzelm
more antiquotations;
2021-10-27, by wenzelm
moved a theorem to a sensible place
2021-10-27, by paulson
merged
2021-10-26, by wenzelm
tuned, continuing e955964d89cb;
2021-10-26, by wenzelm
avoid waste of resources due to dynamic simpset (amending 45c09620f726);
2021-10-26, by wenzelm
fix latex
2021-10-26, by Norbert Schirmer
clarified modules;
2021-10-26, by wenzelm
more generic bit/word lemmas for distribution
2021-10-26, by haftmann
merged
2021-10-26, by paulson
Added / moved some simple set-theoretic lemmas
2021-10-26, by paulson
more CONTRIBUTORS and NEWS;
2021-10-26, by wenzelm
cleanup; add Apple reference
2021-10-19, by Norbert Schirmer
refine interface
2021-07-15, by Norbert Schirmer
generalized component lookup for syntax and distinctness proofs. added some tracing.
2020-11-12, by Norbert Schirmer
merged
2021-10-25, by wenzelm
tuned;
2021-10-25, by wenzelm
more antiquotations;
2021-10-25, by wenzelm
more antiquotations;
2021-10-25, by wenzelm
more robust: genuinely free variables need to be instantiated;
2021-10-25, by wenzelm
tuned comments;
2021-10-25, by wenzelm
clarified errors;
2021-10-25, by wenzelm
tuned;
2021-10-25, by wenzelm
clarified instantiation: local beta reduction after substitution, as for Envir.expand_term_defs;
2021-10-25, by wenzelm
tuned;
2021-10-25, by wenzelm
clarified signature -- avoid clones;
2021-10-25, by wenzelm
Refinement of partitions
2021-10-25, by paulson
avoid persistence of static context: instantiation arguments should provide proper dynamic context;
2021-10-24, by wenzelm
more antiquotations;
2021-10-24, by wenzelm
more markup;
2021-10-24, by wenzelm
clarified name, syntax, messages;
2021-10-24, by wenzelm
more antiquotations;
2021-10-24, by wenzelm
more control symbols;
2021-10-24, by wenzelm
tuned signature;
2021-10-24, by wenzelm
ML antiquotations to instantiate types/terms/props;
2021-10-24, by wenzelm
tuned;
2021-10-21, by wenzelm
clarified modules;
2021-10-21, by wenzelm
clarified modules;
2021-10-20, by wenzelm
clarified modules;
2021-10-20, by wenzelm
discontinued obsolete "val extend = I" for data slots;
2021-10-20, by wenzelm
clarified modules;
2021-10-20, by wenzelm
clarified modules;
2021-10-20, by wenzelm
clarified signature;
2021-10-20, by wenzelm
tuned;
2021-10-20, by wenzelm
clarified keywords and reports;
2021-10-20, by wenzelm
clarified signature;
2021-10-20, by wenzelm
merged
2021-10-20, by desharna
proper veriT --max-time option
2021-10-19, by desharna
refactored tptp_builtins in Sledgehammer
2021-10-19, by desharna
merged
2021-10-19, by wenzelm
tuned ML --- clarified use of context;
2021-10-19, by wenzelm
tuned --- fewer clones;
2021-10-19, by wenzelm
updated to jEdit plugin Highlight 2.5;
2021-10-19, by wenzelm
proper tactic combinator;
2021-10-19, by wenzelm
proper file headers;
2021-10-19, by wenzelm
clarified context;
2021-10-19, by wenzelm
more accurate treatment of context;
2021-10-19, by wenzelm
updated email address
2021-10-19, by Manuel Eberl
removed some 'private' modifiers from HOL-Computational_Algebra
2021-10-15, by Manuel Eberl
merged
2021-10-18, by wenzelm
merged
2021-10-18, by wenzelm
more robust Variable.revert_bounds (see also b12f2cef3ee5);
2021-10-18, by wenzelm
more accurate treatment of context;
2021-10-17, by wenzelm
tuned -- proper names/scopes for contexts;
2021-10-17, by wenzelm
clarified context;
2021-10-16, by wenzelm
clarified context;
2021-10-16, by wenzelm
tuned;
2021-10-16, by wenzelm
unused;
2021-10-16, by wenzelm
more accurate treatment of context;
2021-10-16, by wenzelm
isabelle regenerate_cooper;
2021-10-15, by wenzelm
revert bbfed17243af, breaks HOL-Proofs extraction;
2021-10-15, by wenzelm
tuned;
2021-10-15, by wenzelm
tuned;
2021-10-15, by wenzelm
proper p' instead of p (amending 52c7c42e7e27);
2021-10-15, by wenzelm
proper context for Goal.prove_internal;
2021-10-15, by 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;
2021-10-15, by wenzelm
more accurate treatment of context, notably for nested Goal.proof / SUBPROOF;
2021-10-15, by wenzelm
tuned;
2021-10-15, by wenzelm
tuned;
2021-10-15, by wenzelm
tuned;
2021-10-15, by wenzelm
spelling;
2021-10-15, by wenzelm
clarified context;
2021-10-15, by wenzelm
clarified signature;
2021-10-14, by wenzelm
tuned Vampire configuration to use TFX in Sledgehammer
2021-10-14, by desharna
added Mirabelle action presburger
2021-10-18, by desharna
added timing to Mirabelle action arith
2021-10-18, by desharna
added error message on invalid Mirabelle action
2021-10-18, by desharna
A few new lemmas plus some refinements
2021-10-15, by paulson
merged
2021-10-14, by desharna
produced Mirabelle output directly in ML until Scala output gets fixed
2021-09-20, by desharna
clarified signature;
2021-10-13, by wenzelm
clarified signature;
2021-10-13, by wenzelm
clarified signature;
2021-10-13, by wenzelm
removed unused material (left-over from fd0c85d7da38);
2021-10-13, by wenzelm
support HOL-Isar_Examples.Hoare as well (amending 403ce50e6a2a);
2021-10-13, by wenzelm
removed junk;
2021-10-13, by wenzelm
merged
2021-10-12, by nipkow
separated commands from annotations to be able to abstract about the latter only
2021-10-12, by nipkow
prefer standard Term.dest_abs, with minor deviation of generated names;
2021-10-12, by wenzelm
tuned comments;
2021-10-12, by wenzelm
more examples
2021-10-11, by nipkow
workaround for old macOS versions, after change of Let's Encrypt root certificate --- see also https://letsencrypt.org/docs/dst-root-ca-x3-expiration-september-2021 --- Java/Scala Isabelle_System.download() works, but curl doens't;
2021-10-11, by wenzelm
more complete simp rules
2021-10-11, by haftmann
more complete simp rules
2021-10-10, by haftmann
avoid overaggressive contraction of conversions
2021-10-10, by haftmann
normalizing NOT (numeral _) (again)
2021-10-09, by haftmann
tuned text;
2021-10-08, by wenzelm
recover NEWS from 78d1f73bbeaa;
2021-10-07, by wenzelm
save 90 MB by excluding rlwrap and thus perl;
2021-10-07, by wenzelm
save 45 MB by excluding rlwrap and thus perl;
2021-10-07, by wenzelm
NEWS;
2021-10-07, by wenzelm
clarified test of directories;
2021-10-07, by wenzelm
misc tuning for release;
2021-10-07, by wenzelm
merged
2021-10-07, by wenzelm
updated to kodkodi-1.5.7. with more robust/portable management of files and processes;
2021-10-07, by wenzelm
provide minisat-2.2.1 on all currently supported platforms, notably as external solver for Nitpick;
2021-10-07, by wenzelm
tuned message;
2021-10-07, by wenzelm
proper build on macOS;
2021-10-07, by wenzelm
build minisat, using recent fork from original sources;
2021-10-07, by wenzelm
proper platform_path for executables run from Java;
2021-10-07, by wenzelm
tuned message;
2021-10-07, by wenzelm
tuned;
2021-10-06, by wenzelm
tuned whitespace;
2021-10-06, by wenzelm
merged
2021-10-07, by desharna
added timeout to veriT
2021-10-07, by desharna
new notion of infinite sums in HOL-Analysis, ordering on complex numbers
2021-10-06, by eberlm
NEWS and CONTRIBUTORS
2021-10-07, by desharna
merged
2021-10-07, by desharna
added offset to Mirabelle's tptp output names
2021-09-20, by desharna
tuned zipperposition config in sledgehammer
2021-10-04, by desharna
considered slices overhead in sledgehammer
2021-10-04, by desharna
tuned atp_prover sliding
2021-09-29, by desharna
tuned Zipperposition slides in sledgehammer
2021-09-29, by desharna
include arm64-linux;
2021-10-06, by wenzelm
updated to Vampire 4.6, as proposed by Martin Desharnais;
2021-10-06, by wenzelm
build from official downloads;
2021-10-06, by wenzelm
build just one vampire version;
2021-10-06, by wenzelm
clarified signature;
2021-10-06, by wenzelm
maintain previous theory identifier to support semantic caching, notably in Isabelle/Naproche;
2021-10-05, by wenzelm
more exports, notably for Isabelle/Naproche;
2021-10-05, by wenzelm
include arm64-linux;
2021-10-05, by wenzelm
prefer existing OCaml installation;
2021-10-05, by wenzelm
include arm64-linux;
2021-10-04, by wenzelm
no patchelf on macOS (undetected due to cached executables?);
2021-10-04, by wenzelm
provide opam-2.1.0 for experimentation;
2021-10-04, by wenzelm
less
more
|
(0)
-30000
-10000
-3000
-1000
-240
+240
+1000
+3000
tip