Mercurial
Mercurial
>
repos
>
isabelle
/ graph
summary
|
shortlog
|
changelog
| graph |
tags
|
bookmarks
|
branches
|
files
|
gz
|
help
less
more
|
(0)
-30000
-10000
-3000
-1000
-120
+120
+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.
tuned signature;
2013-09-16, by wenzelm
more antiquotations -- avoid unchecked string literals;
2013-09-16, by wenzelm
more explicit exception pattern (NB: unqualified exceptions without arguments are in danger of becoming catch-all patterns by accident);
2013-09-16, by wenzelm
distinguish Proof.context vs. local_theory semantically, with corresponding naming conventions;
2013-09-16, by wenzelm
tuned white space;
2013-09-16, by wenzelm
adhoc check of ML sources, in addition to thy files already covered in Thy_Load;
2013-09-16, by wenzelm
proper Isabelle symbols -- no UTF8 here;
2013-09-16, by wenzelm
proper Cygwin mirror for Isabelle2013-1;
2013-09-16, by wenzelm
explicit test of quick_and_dirty, which is rarely used in practice;
2013-09-16, by wenzelm
updated to cygwin-20130916;
2013-09-16, by wenzelm
more CHECKLIST;
2013-09-16, by wenzelm
updated cygwin snapshot;
2013-09-16, by wenzelm
updated to smlnj 110.76;
2013-09-16, by wenzelm
prefer high-level ML_System.share_common_data, ML_System.save_state -- except for bootstrap images (RAW, Pure);
2013-09-16, by wenzelm
more NEWS;
2013-09-16, by wenzelm
merge
2013-09-16, by panny
prove simp theorems for newly generated definitions
2013-09-16, by panny
example using restoring Transfer/Lifting context
2013-09-16, by kuncar
use lifting_forget for deregistering numeric types as a quotient type
2013-09-16, by kuncar
restoring Transfer/Lifting context
2013-09-16, by kuncar
make ML function for deleting quotients public
2013-09-16, by kuncar
public access to the raw transfer rules - for restoring transferring
2013-09-16, by kuncar
another move to avoid sporadic kill of poly, which is presumably due to resource management on lxbroy2, lxbroy3 etc.;
2013-09-16, by wenzelm
more (co)data docs
2013-09-16, by blanchet
more (co)data docs
2013-09-15, by blanchet
added missing theorems to "simps" collection
2013-09-15, by blanchet
more (co)data docs
2013-09-15, by blanchet
more (co)data docs
2013-09-15, by blanchet
more (co)data docs
2013-09-15, by blanchet
merged
2013-09-14, by wenzelm
tuned proofs;
2013-09-14, by wenzelm
tuned magic number, for improved reactivity on old 2-core machine;
2013-09-14, by wenzelm
tuned proofs;
2013-09-14, by wenzelm
updated keywords
2013-09-14, by krauss
tuned proof
2013-09-14, by haftmann
merged
2013-09-14, by wenzelm
tuned proofs;
2013-09-14, by wenzelm
print find_thms result in reverse order so best result is on top
2013-09-14, by kleing
more useful sorting of find_thms results
2013-09-14, by kleing
proper sharing after change of directory structure (cf. 32ec957e5c3e);
2013-09-13, by wenzelm
restricted heap, which might improve stability of this test;
2013-09-13, by wenzelm
merged
2013-09-13, by wenzelm
tuned proofs;
2013-09-13, by wenzelm
tuned proofs;
2013-09-13, by wenzelm
updated to jdk-7u40;
2013-09-13, by wenzelm
added component jdk-7u40.tar.gz (inactive);
2013-09-13, by wenzelm
merged
2013-09-13, by blanchet
more (co)data docs
2013-09-13, by blanchet
tuning
2013-09-13, by blanchet
more (co)data doc
2013-09-13, by blanchet
generalized and simplified proofs of several theorems about convex sets
2013-09-13, by huffman
more (co)data docs
2013-09-13, by blanchet
removed accidentally submitted line
2013-09-13, by blanchet
more (co)data doc
2013-09-13, by blanchet
more general typing of monadic bind
2013-08-20, by Christian Sternagel
merged
2013-09-13, by krauss
omit automatic Induct.cases_pred declaration, which breaks many existing proofs
2013-09-12, by krauss
NEWS and CONTRIBUTORS
2013-09-10, by krauss
merged
2013-09-10, by krauss
added some examples and tests for fun_cases
2013-09-10, by krauss
dropped unnecessary 'open'
2013-09-09, by krauss
tuned headers
2013-09-09, by krauss
moved cases post-processing under mk_partial_rules_mutual, using existing bookkeeping information;
2013-09-09, by krauss
clarified
2013-09-08, by krauss
clarified, dropping unreachable bool special case
2013-09-08, by krauss
dropped dead code
2013-09-08, by krauss
clarified
2013-09-08, by krauss
generate elim rules for elimination of function equalities;
2013-09-08, by Manuel Eberl
tuned proofs
2013-09-13, by haftmann
merged
2013-09-12, by huffman
make 'linear' into a sublocale of 'bounded_linear';
2013-09-12, by huffman
generalize lemmas
2013-09-12, by huffman
remove unneeded assumption from prime_dvd_power lemmas;
2013-09-12, by huffman
remove duplicate lemmas
2013-09-12, by huffman
new lemmas
2013-09-12, by huffman
prefer theorem name over 'long_thm_list(n)'
2013-09-12, by huffman
prefer attribute 'unfolded thm' to 'simplified'
2013-09-12, by huffman
removed outdated comments
2013-09-12, by huffman
made non-co case more robust as well (cf. b6e2993fd0d3)
2013-09-13, by blanchet
don't wrongly destroy sum types in coiterators
2013-09-13, by blanchet
beware of multi-constructor datatypes (cf. 27c418b7b985)
2013-09-13, by blanchet
beware of single-constructor datatypes, with no discriminators
2013-09-13, by blanchet
more robust tactic to cover another corner case (added as example);
2013-09-12, by traytel
generalized data structure, for extension with SMT solver proofs
2013-09-12, by blanchet
prefixed types and some functions with "atp_" for disambiguation
2013-09-12, by blanchet
merged;
2013-09-12, by wenzelm
absorb final CLASSPATH as well, such that tools might provide that by elementary means, without the "classpath" shell function (e.g. kodkodi/nitpick);
2013-09-12, by wenzelm
more CHECKLIST;
2013-09-12, by wenzelm
more robust System.getProperty with default;
2013-09-12, by wenzelm
generate distribution classpath for cold-start application wrappers;
2013-09-12, by wenzelm
reverse orientation of ISABELLE_CLASSPATH;
2013-09-12, by wenzelm
propagate ISABELLE_CLASSPATH;
2013-09-12, by wenzelm
tuned comments;
2013-09-12, by wenzelm
clarified directory structure;
2013-09-12, by wenzelm
maintain classpath in more elementary manner: turn ISABELLE_CLASSPATH into -classpath option, so that all jars are covered by sun.misc.Launcher.AppClassLoader (e.g. relevant for loading add-on resources);
2013-09-12, by wenzelm
more official initial class path according to sun.misc.Launcher;
2013-09-11, by wenzelm
provide main classpath again, notably for cold-start;
2013-09-11, by wenzelm
cold-start of main application even on Linux;
2013-09-11, by wenzelm
tuned proofs;
2013-09-11, by wenzelm
more explicit indication of 'done' as proof script element;
2013-09-11, by wenzelm
made tactic handle gracefully the case: codatatype ('a, 's) scheduler2 = Combine2 "'s => 'a" "'s => ('a, 's) scheduler2"
2013-09-12, by blanchet
conceal definitions of high-level constructors and (co)iterators
2013-09-12, by traytel
conceal low-level noted facts (+ FIXME to get rid of the notes altogether eventually)
2013-09-12, by traytel
buffer the notes even more
2013-09-12, by traytel
conceal internal bindings
2013-09-12, by traytel
add a notice to myself in doc
2013-09-12, by blanchet
more robust approach to avoid Python byte code -- environment variables get inherited by subprocesses
2013-09-12, by blanchet
unset some spurious executable flags
2013-09-12, by blanchet
handle corner case in tactic
2013-09-12, by traytel
simplified derivation of in_rel
2013-09-12, by traytel
removed unused/inlinable theorems
2013-09-12, by traytel
when pouring in extra features into the goal, only consider facts from the current theory -- the bottom 10 facts of the last import might be completely unrelated
2013-09-12, by blanchet
minor fixes
2013-09-12, by blanchet
commented out code parts leading to runtime errors due to missing gensim module
2013-09-12, by blanchet
invoke Python with "no bytecode" option to avoid litering Isabelle source directory with ".pyc" files (which can be problematic for a number of reasons)
2013-09-12, by blanchet
new version of MaSh
2013-09-12, by blanchet
more (co)data docs
2013-09-12, by blanchet
avoid a keyword
2013-09-12, by blanchet
more (co)datatype docs
2013-09-11, by blanchet
killed dead code
2013-09-11, by blanchet
less
more
|
(0)
-30000
-10000
-3000
-1000
-120
+120
+1000
+3000
+10000
tip