Mercurial
Mercurial
>
repos
>
isabelle
/ graph
summary
|
shortlog
|
changelog
| graph |
tags
|
bookmarks
|
branches
|
files
|
gz
|
help
less
more
|
(0)
-30000
-10000
-3000
-1000
-112
+112
+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.
include scala-compiler.jar in basic Isabelle/Scala environment, to make Isabelle/jEdit console work with scala-2.10.0-M3;
2012-05-24, by wenzelm
tuned proofs;
2012-05-24, by wenzelm
less warning in scala-2.10.0-M3;
2012-05-24, by wenzelm
avoid scala.tools.nsc.Interpreter -- deprecated in scala-2.9.0;
2012-05-24, by wenzelm
make Nitpick's handling of definitions more robust in the face of formulas that don't have the expected format (needed for soundness, cf. RNG100+1)
2012-05-24, by blanchet
fixed soundness bug in Nitpick related to unfolding -- the unfolding criterion must at least as strict when looking at a definitional axiom as elsewhere, otherwise we end up unfolding a constant's definition in its own definition, yielding a trivial equality
2012-05-24, by blanchet
more robust Swing_Thread.now: allow body to fail;
2012-05-24, by wenzelm
tuned proofs;
2012-05-24, by wenzelm
reparse descendants after update of imports, e.g. required for 'primrec' (line 17 of "src/HOL/Power.thy");
2012-05-24, by wenzelm
merged
2012-05-24, by wenzelm
update Satallax setup based on evaluation
2012-05-24, by blanchet
merged
2012-05-24, by kuncar
drop the feature that more than one quotient type can be defined by quotient_type -> it causes problems
2012-05-24, by kuncar
prove reflexivity also for the quotient composition relation; reflp_preserve renamed to reflexivity_rule
2012-05-24, by kuncar
gracefully handle definition-looking premises
2012-05-24, by blanchet
simplified Poly/ML setup -- 5.3.0 is now the common base-line;
2012-05-24, by wenzelm
discontinued support for Poly/ML 5.2.1;
2012-05-24, by wenzelm
less specific sample usage;
2012-05-24, by wenzelm
some post-release notes;
2012-05-24, by wenzelm
tuned names
2012-05-23, by blanchet
order LEO-II/Satallax definitions so that they build on each other (cf. Satallax's THF policy)
2012-05-23, by blanchet
improved LEO-II definition handling -- still hoping for a fix directly in LEO-II
2012-05-23, by blanchet
augment Satallax unsat cores with all definitions
2012-05-23, by blanchet
better handling of incomplete TSTP proofs
2012-05-23, by blanchet
generate THF definitions
2012-05-23, by blanchet
build hybrid Isabelle component for JDK on x86-linux/x86_64-linux;
2012-05-23, by wenzelm
merged
2012-05-23, by wenzelm
eliminated old 'axioms';
2012-05-23, by wenzelm
discontinued obsolete method fastsimp / tactic fast_simp_tac;
2012-05-23, by wenzelm
eliminated obsolete fastsimp;
2012-05-23, by wenzelm
extend the Z3 proof parser to accept polyadic addition (on integers and reals) due to changes introduced in Z3 4.0
2012-05-23, by boehmes
merged
2012-05-23, by wenzelm
doc updates
2012-05-23, by blanchet
lower the monomorphization thresholds for less scalable provers
2012-05-23, by blanchet
more explicit proof;
2012-05-23, by wenzelm
tuned proof;
2012-05-23, by wenzelm
prefer symbolic "contrib" -- mira should have a symlink to physical contrib_devel;
2012-05-23, by wenzelm
merged, abandoning change of src/HOL/Tools/ATP/atp_problem_generate.ML from 6ea205a4d7fd;
2012-05-23, by wenzelm
compile
2012-05-22, by blanchet
don't apply "ext_cong_neq" to biimplications
2012-05-22, by blanchet
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
less
more
|
(0)
-30000
-10000
-3000
-1000
-112
+112
+1000
+3000
+10000
+30000
tip