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.
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
less
more
|
(0)
-30000
-10000
-3000
-1000
-120
+120
+1000
+3000
+10000
tip