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
+30000
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 one slice with configurable simplification turned off
2012-05-22, by blanchet
make higher-order goals more first-order via extensionality
2012-05-22, by blanchet
added "ext_cong_neq" lemma (not used yet); tuning
2012-05-22, by blanchet
use quot_del instead of ML code in Rat.thy
2012-05-21, by kuncar
quot_del attribute, it allows us to deregister quotient types
2012-05-21, by kuncar
invite users to upgrade their SPASS (so we can get rid of old code)
2012-05-21, by blanchet
start phasing out old SPASS
2012-05-21, by blanchet
minor tweak in Vampire setup
2012-05-21, by blanchet
include "ext" in all Satallax proofs
2012-05-21, by blanchet
add an experimental "aggressive" mode to Sledgehammer, to experiment with more complete translations of higher-order features without breaking "metis"
2012-05-21, by blanchet
tuning
2012-05-21, by blanchet
added helper -- cf. SET616^5
2012-05-21, by blanchet
note Quotient theorem for typedefs in setup_lifting
2012-05-18, by kuncar
added a timeout to "try0" in Mirabelle
2012-05-18, by blanchet
don't generate code in Word because it breaks the current code setup
2012-05-18, by kuncar
robustly parse Z3 4.0's output (with outcome appearing on first rather than last line)
2012-05-17, by blanchet
added "Collect_cong" to cover extensionality of "Collect" (special cases of "ext" pass through the relevant filter)
2012-05-17, by blanchet
remove the generation of a code certificate from the Quotient package (mainly from quotient_def), because it's in lift_definition now
2012-05-16, by kuncar
generate abs_eq, use it as a code equation for total quotients; no_abs_code renamed to no_code; added no_code for quotient_type command
2012-05-16, by kuncar
infrastructure that makes possible to prove that a relation is reflexive
2012-05-16, by kuncar
temporarily disable "ext" rule helpers until Metis supports them (and until they are properly evaluated)
2012-05-16, by blanchet
lower skolem penalty to ensure that some useful facts with existentials, e.g. congruence of "setsum", eventually get picked up
2012-05-16, by blanchet
treat sets specially in relevance filter, as they used to, to avoid cluttering the problem with facts about Set.member and Collect
2012-05-16, by blanchet
get ready for automatic generation of extensionality helpers
2012-05-16, by blanchet
minor slice tweaking (swapped two slices to move polymorphic encoding up a bit)
2012-05-16, by blanchet
more helpful error message
2012-05-16, by blanchet
transfer rules for many more list constants
2012-05-15, by huffman
made SML/NJ happy
2012-05-15, by blanchet
repair the Waldmeister endgame only for Waldmeister proofs
2012-05-15, by blanchet
fixed Waldmeister commutativity hack
2012-05-15, by blanchet
imported patch atp_tuning
2012-05-15, by blanchet
add transfer rules for nat_rec and funpow
2012-05-15, by huffman
add transfer rule for constant List.lists
2012-05-14, by huffman
add transfer rule for set_rel
2012-05-14, by huffman
ensure the "show" equation is not reoriented by Waldmeister
2012-05-14, by blanchet
ensure consistent naming of Waldmeister proof steps, so that they are not cleaned away by "clean_up_atp_proof_dependencies"
2012-05-14, by blanchet
repaired snag in debug function
2012-05-14, by blanchet
graceful handling of Waldmeister endgame
2012-05-14, by blanchet
improve parsing of Waldmeister dependencies (and kill obsolete hack)
2012-05-14, by blanchet
tuning
2012-05-14, by blanchet
added debugging function
2012-05-14, by blanchet
LEO-II's "--sos" option confusingly disables rather than enables SOS, and SOS seems to be ignored anyway; also, pass a number of facts that's more appropriate for each prover
2012-05-13, by blanchet
eta-reduce definition-like equations for THF provers; Satallax in particular seems to love that
2012-05-13, by blanchet
get rid of "conj_sym_kind" -- most interesting provers now have built-in sorts, and for the others (e.g. E) "Hypothesis" isn't too bad a default
2012-05-13, by blanchet
extend ATP data structure to avoid having to perform ((non-)capture avoiding) beta reduction -- fixes a bug in the THF translation of "is_measure.simps"
2012-05-13, by blanchet
reintroduced example now that it's no longer broken
2012-05-11, by blanchet
fixed "real" after they were redefined as a 'quotient_type'
2012-05-11, by blanchet
temporarily comment out broken nitpick example;
2012-05-10, by huffman
simplify instance proofs for rat
2012-05-10, by huffman
convert Rat.thy to use lift_definition/transfer
2012-05-10, by huffman
cleaner handling of bi-implication for THF output of first-order type encodings
2012-05-10, by blanchet
distinguish between instantiated and uninstantiated inductions -- the latter are OK for first-order provers
2012-05-10, by blanchet
temporarily comment out broken nitpick example
2012-05-10, by huffman
convert real number theory to use lifting/transfer
2012-05-10, by huffman
tuned ordering of lemmas
2012-05-07, by huffman
pass fewer facts to LEO-II and Satallax
2012-05-10, by blanchet
tweak LEO-II setup
2012-05-10, by blanchet
use raw monomorphic encoding with Waldmeister, to avoid overloading it with too many function symbols (as would be the case using mangled monomorphic encodings)
2012-05-10, by blanchet
build Pure_64 with new settings
2012-05-09, by bulwahn
tuned
2012-05-09, by bulwahn
playing around with mira settings
2012-05-09, by bulwahn
defining and proving Executable_Relation with lift_definition and transfer
2012-05-08, by bulwahn
specialised fact in the Record theory should not be appear in proofs discovered by sledgehammer
2012-05-08, by bulwahn
prevent spurious timeouts
2012-05-07, by blanchet
added "try0" tool to Mirabelle
2012-05-07, by blanchet
use latest E (1.5)
2012-05-07, by blanchet
lifting package produces abs_eq_iff rules for total quotients
2012-05-04, by huffman
using the new transfer method to obtain abstract properties of RBT trees
2012-05-04, by bulwahn
back to post-release mode -- after fork point;
2012-05-02, by wenzelm
removed obsolete RC tags;
2012-05-23, by wenzelm
Added tag Isabelle2012 for changeset 21c42b095c84
2012-05-22, by wenzelm
try to avoid races again (cf. 8c37cb84065f and fd3a36e48b09);
Isabelle2012
2012-05-20, by wenzelm
Added tag Isabelle2012-RC3 for changeset ed5f56b8f90a
2012-05-17, by wenzelm
some message;
2012-05-17, by wenzelm
tuned error -- reduce potential for confusion in a higher-level context, e.g. partial checking of theory sub-graph;
2012-05-17, by wenzelm
Fixed disambiguation of names (cf. 5759ecd5c905)
2012-05-11, by berghofe
merged
2012-05-10, by wenzelm
file.encoding=UTF-8 for java.ext.dirs, to agree with java runtime invocation;
2012-05-10, by wenzelm
prefer absolute paths, to allow launching from a different context (e.g. via file associations);
2012-05-10, by wenzelm
tweaked Inductive.prove_eqs to allow degenerate definition like "inductive TRUE where TRUE";
2012-05-10, by wenzelm
allow spaces in target directory;
2012-05-09, by wenzelm
Added tag Isabelle2012-RC2 for changeset 1636ff4c6243
2012-05-07, by wenzelm
init Cygwin after unpacking;
2012-05-07, by wenzelm
tuned proofs;
2012-05-06, by wenzelm
more accurate ROOT.ML;
2012-05-06, by wenzelm
prefer http://isabelle.in.tum.de/library alias, which is available at TUM only;
2012-05-06, by wenzelm
some highlights of Isabelle2012;
2012-05-05, by wenzelm
refrain from SIGHUP handling (cf. 5f629ee2502b), which does not work on Cygwin and appears to be redundant anyway (no extra output produced within pipe);
2012-05-04, by wenzelm
some attempts to make critical errors fit on screen;
2012-05-04, by wenzelm
more NEWS;
2012-05-03, by wenzelm
backout 9579464d00f9 to avoid odd crash of polyml-5.2.1 (according to Jasmin, this change is not essential for now);
2012-05-03, by wenzelm
Added tag Isabelle2012-RC1 for changeset ec5d54029664
2012-05-02, by wenzelm
clarified;
2012-05-02, by wenzelm
makedist for release;
2012-05-02, by wenzelm
merged
2012-05-02, by wenzelm
more contributors;
2012-05-02, by wenzelm
tuned latex sources;
2012-05-02, by wenzelm
more CHECKLIST;
2012-05-02, by wenzelm
save 90MB by removing foreign binaries -- multi-platform installations are unlikely on Windows;
2012-05-02, by wenzelm
some re-ordering;
2012-05-02, by wenzelm
some re-ordering;
2012-05-02, by wenzelm
tuned spelling;
2012-05-02, by wenzelm
resolved maxidx bug
2012-05-02, by kuncar
documentation of the Lifting package on the ML level & tuned
2012-05-02, by kuncar
edit NEWS items for transfer/lifting
2012-05-02, by huffman
avoid interference of markup for literal tokens, which may contain slightly odd \<^bsub> \<^esub> counted as pseudo-markup (especially relevant for HTML output, e.g. of thm power3_eq_cube);
2012-05-02, by wenzelm
accomodate scala-2.10.0-M3 with its extra jar;
2012-05-02, by wenzelm
more robust wrt. spaces in directory names;
2012-05-02, by wenzelm
updated headers;
2012-05-02, by wenzelm
back to "Tools" in conformance with toplevel Isabelle layout (cf. 3fabf352243e, 15f4309bb9eb);
2012-05-02, by wenzelm
export more symbols
2012-04-30, by blanchet
merged
2012-04-30, by bulwahn
adding configuration to pass options to the ghc call in quickcheck[narrowing]
2012-04-30, by bulwahn
provide [[record_codegen]] option for skipping codegen setup for records
2012-04-30, by Gerwin Klein
making sorted_list_of_set executable
2012-04-30, by bulwahn
removing obsolete setup for sets now that sets are executable
2012-04-30, by bulwahn
update references in HOLCF README
2012-04-30, by huffman
basic setup for self-extracting 7zip installer;
2012-04-29, by wenzelm
merged
2012-04-29, by krauss
added test case for dependency graph (cf. 2d48bf79b725)
2012-04-29, by krauss
less
more
|
(0)
-30000
-10000
-3000
-1000
-120
+120
+1000
+3000
+10000
+30000
tip