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.
added canonical screenshot;
2013-09-21, by wenzelm
removed obsolete README;
2013-09-21, by wenzelm
tuned;
2013-09-21, by wenzelm
added/updated material from src/Tools/jEdit/README.html;
2013-09-21, by wenzelm
basic setup for Isabelle/jEdit documentation;
2013-09-21, by wenzelm
updated keywords;
2013-09-21, by wenzelm
updated CONTRIBUTORS
2013-09-20, by blanchet
updated NEWS
2013-09-20, by blanchet
document option
2013-09-20, by blanchet
merged "isar_try0" and "isar_minimize" options
2013-09-20, by blanchet
hardcoded obscure option
2013-09-20, by blanchet
hard-coded an obscure option
2013-09-20, by blanchet
use configuration mechanism for low-level tracing
2013-09-20, by blanchet
moved focus to Isabell/jEdit and away from Proof General
2013-09-20, by blanchet
took out Waldmeister from list of default provers -- it's usually just visual noise, and its integration in Sledgehammer leaves much to be desired
2013-09-20, by blanchet
tuning (use a blacklist instead of a whitelist)
2013-09-20, by blanchet
reduce the number of emitted MaSh commands (among others to facilitate debugging)
2013-09-20, by blanchet
MaSh tweaks to facilitate debugging
2013-09-20, by blanchet
tuned proofs
2013-09-20, by haftmann
make SML/NJ happy
2013-09-20, by kuncar
renamed "primcorec" to "primcorecursive", to open the door to a 'theory -> theory' command called "primcorec" (cf. "fun" vs. "function")
2013-09-20, by blanchet
more primcorec docs
2013-09-20, by blanchet
added primcorec examples with lambdas
2013-09-20, by blanchet
more primcorec docs
2013-09-20, by blanchet
adapted primcorec documentation to reflect the three views
2013-09-20, by blanchet
updated docs
2013-09-20, by blanchet
took out spurious attributes (no need for several code equations / simps for thesame constants)
2013-09-20, by blanchet
have "datatype_new_compat" register induction and recursion theorems in nested case
2013-09-20, by blanchet
prefer Code.abort over code_abort
2013-09-20, by Andreas Lochbihler
setting the stage for safe constructor simp rules
2013-09-20, by blanchet
added TODO
2013-09-19, by blanchet
made tactic more reliable
2013-09-19, by blanchet
killed exceptional code that is anyway no longer needed, now that the 'simp' attribute has been taken away -- this solves issues in 'primcorec'
2013-09-19, by blanchet
cleaner handling of collapse theorems
2013-09-19, by blanchet
repaired latex (cf. 84522727f9d3);
2013-09-19, by wenzelm
updated NEWS
2013-09-19, by blanchet
dropped dead code
2013-09-19, by haftmann
don't declare ctr view primcorec theorems as simp (they loop)
2013-09-19, by traytel
simplified code; eliminated some dummyTs
2013-09-19, by panny
avoid infinite loop for unapplied terms + tuning
2013-09-19, by blanchet
generalize code to handle zero-argument case gracefully (e.g. for nullay functions defined over codatatypes that corecurse through "fun"
2013-09-19, by blanchet
give lambda abstractions a chance, as an alternative to function composition, for corecursion via "fun"
2013-09-19, by blanchet
added auxiliary function
2013-09-19, by blanchet
avoid parameter
2013-09-19, by blanchet
added helper function for code equations in primcorec
2013-09-19, by blanchet
updated NEWS and CONTRIBUTORS
2013-09-19, by blanchet
split functionality into two functions to avoid redoing work over and over
2013-09-19, by blanchet
added massaging function for primcorec code equations
2013-09-19, by blanchet
simplified code
2013-09-19, by blanchet
no need for beta-eta contraction
2013-09-19, by blanchet
generalize helper function
2013-09-19, by blanchet
generate more theorems (e.g. for types with only one constructor)
2013-09-19, by panny
added two functions to List (one contributed by Manuel Eberl)
2013-09-18, by traytel
generate constructor view theorems
2013-09-18, by panny
merged;
2013-09-18, by wenzelm
merged;
2013-09-18, by wenzelm
tuned proofs;
2013-09-18, by wenzelm
tuned proofs;
2013-09-18, by wenzelm
added option "jedit_auto_load";
2013-09-18, by wenzelm
limit for text height;
2013-09-18, by wenzelm
improved layout, with special treatment for ScrollPane;
2013-09-18, by wenzelm
tuned signature;
2013-09-18, by wenzelm
improved FlowLayout for wrapping of components over multiple lines;
2013-09-18, by wenzelm
updated to polyml-5.5.1;
2013-09-18, by wenzelm
improved printing of exception trace in Poly/ML 5.5.1;
2013-09-18, by wenzelm
more antiquotations;
2013-09-18, by wenzelm
moved module into plain Isabelle/ML user space;
2013-09-18, by wenzelm
more primcorec tactics
2013-09-18, by blanchet
enrich data structure
2013-09-18, by blanchet
include more "discI" rules
2013-09-18, by blanchet
updated docs
2013-09-18, by blanchet
tuning (alphabetical order)
2013-09-18, by blanchet
removed spurious "simp"
2013-09-18, by blanchet
note "discI"
2013-09-18, by blanchet
tuned tactics
2013-09-18, by blanchet
no need thanks to "Code.abort"
2013-09-18, by blanchet
minor change related to code equations in primcorec
2013-09-18, by blanchet
don't unfold as eager as in 11a77e4aa98b
2013-09-18, by traytel
tuned proofs
2013-09-18, by traytel
use singular to avoid confusion
2013-09-18, by blanchet
new tactics for constructor view
2013-09-18, by blanchet
tuning
2013-09-18, by blanchet
fixed embarrassing typo in example
2013-09-18, by blanchet
avoid duplicate simp rule warnings
2013-09-18, by blanchet
added and tuned lemmas
2013-09-18, by nipkow
tuned proofs;
2013-09-18, by wenzelm
updated to official polyml-5.5.1;
2013-09-17, by wenzelm
updated to polyml-5.5.1;
2013-09-17, by wenzelm
actually use x86_64 machine;
2013-09-17, by wenzelm
correct merging of restore data
2013-09-17, by kuncar
order_bot, order_top
2013-09-17, by lammich
include Int_Pow into Quotient_Examples; add end of the theory
2013-09-17, by kuncar
NEWS: Simps_Case_Conv
2013-09-17, by noschinl
added lemmas and made concerse executable
2013-09-17, by nipkow
merge
2013-09-17, by blanchet
return right theorems
2013-09-17, by blanchet
more (co)data docs
2013-09-17, by blanchet
tuned proofs about 'convex'
2013-09-13, by huffman
more (co)data docs
2013-09-17, by blanchet
tuned proofs;
2013-09-17, by wenzelm
treat all dummy type variables separately (in contrast to fca432074fb2);
2013-09-16, by wenzelm
removed dead code (see also 69d4543811d0);
2013-09-16, by wenzelm
merged
2013-09-16, by wenzelm
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
get rid of another complication in relevance filter
2013-09-11, by blanchet
tuning
2013-09-11, by blanchet
renamed config option
2013-09-11, by blanchet
more correct NEWS
2013-09-11, by haftmann
kick out totally hopeless facts after 5 iterations to speed things up
2013-09-11, by blanchet
reintroduced 8d8f72aa5c0b, which does make a small difference in practice, but implemented more efficiently
2013-09-11, by blanchet
more (co)data docs
2013-09-11, by blanchet
more (co)data docs
2013-09-11, by blanchet
more (co)data docs
2013-09-11, by blanchet
merged
2013-09-11, by wenzelm
prefer explicit type constraint (again, see also Type.appl_error);
2013-09-11, by wenzelm
tuned signature;
2013-09-11, by wenzelm
tuned whitespace;
2013-09-11, by wenzelm
tuned message;
2013-09-11, by wenzelm
do not expose internal flags to attribute name space;
2013-09-11, by wenzelm
more (co)data docs
2013-09-11, by blanchet
more (co)datatype documentation
2013-09-11, by blanchet
less
more
|
(0)
-30000
-10000
-3000
-1000
-240
+240
+1000
+3000
+10000
tip