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.
renaming variables to conform to prolog names
2010-08-25, by bulwahn
changing hotel trace definition; adding simple handling of numerals on natural numbers
2010-08-25, by bulwahn
added quickcheck generator for prolog generation; first example of counterexample search with prolog for hotel key card system
2010-08-25, by bulwahn
moving preprocessing to values in prolog generation
2010-08-25, by bulwahn
invocation of values for prolog execution does not require invocation of code_pred anymore
2010-08-25, by bulwahn
adding hotel keycard example for prolog generation
2010-08-25, by bulwahn
improving output of set comprehensions; adding style_check flags
2010-08-25, by bulwahn
improving ensure_groundness in prolog generation; added further example
2010-08-25, by bulwahn
adding very basic transformation to ensure groundness before negations
2010-08-25, by bulwahn
Markup_Tree.select: uniform treatment of root_range wrt. singularities, yielding empty result stream;
2010-08-26, by wenzelm
tuned signature;
2010-08-26, by wenzelm
Pretty: tuned markup objects;
2010-08-25, by wenzelm
tuned;
2010-08-25, by wenzelm
organized markup properties via apply/unapply patterns;
2010-08-25, by wenzelm
added some proof state markup, notably number of subgoals (e.g. for indentation);
2010-08-25, by wenzelm
ML_Context.eval: produce antiquotation environment preferably in invisible context, to avoid displaced report messages from ML_Compiler;
2010-08-25, by wenzelm
merged
2010-08-25, by wenzelm
tuned code
2010-08-25, by Christian Urban
quotient package: deal correctly with frees in lifted theorems
2010-08-25, by Christian Urban
approximation_oracle: actually match true/false in ML, not arbitrary values;
2010-08-25, by wenzelm
renamed Simplifier.simproc(_i) to Simplifier.simproc_global(_i) to emphasize that this is not the real thing;
2010-08-25, by wenzelm
more precise Command.State accumulation;
2010-08-25, by wenzelm
eliminated some old camel case stuff;
2010-08-25, by wenzelm
some attempts to recover Isabelle/ML style from the depths of time;
2010-08-25, by wenzelm
keep persistent production tables as immutable vectors -- potential performance improvement on modern hardware;
2010-08-25, by wenzelm
select tangible text ranges here -- more robust against ongoing changes of the markup query model
2010-08-25, by wenzelm
structure Thm: less pervasive names;
2010-08-25, by wenzelm
discontinued obsolete 'global' and 'local' commands;
2010-08-25, by wenzelm
merged
2010-08-25, by wenzelm
merged
2010-08-25, by hoelzl
moved generic lemmas in Probability to HOL
2010-08-24, by hoelzl
merged
2010-08-25, by wenzelm
traling newline on standard output
2010-08-25, by haftmann
Quotient Package / lemma for regularization of bex1_rel for equivalence relations
2010-08-25, by Cezary Kaliszyk
merged
2010-08-24, by blanchet
make Mirabelle happy
2010-08-24, by blanchet
compute names lazily;
2010-08-24, by blanchet
clean handling of whether a fact is chained or not;
2010-08-24, by blanchet
don't backtick facts that contain schematic variables, since this doesn't work (for some reason)
2010-08-24, by blanchet
quote facts whose names collide with a keyword or command name (cf. "subclass" in "Jinja/J/TypeSafe.thy")
2010-08-24, by blanchet
revert this idea of automatically invoking "metisFT" when "metis" fails;
2010-08-24, by blanchet
use matching of types than just equality - this is needed in nominal to cope with type variables
2010-08-24, by Christian Urban
merge
2010-08-24, by blanchet
cosmetics
2010-08-24, by blanchet
use a soft time limit for E
2010-08-24, by blanchet
make remote ATP versions more robust, by starting with "preferred" version numbers and falling back on any version
2010-08-24, by blanchet
cosmetics
2010-08-23, by blanchet
optimize fact filter some more
2010-08-23, by blanchet
cache previous iteration's weights, and keep track of what's dirty and what's clean;
2010-08-23, by blanchet
modified relevance filter
2010-08-23, by blanchet
adjust fudge factors in the light of experiments
2010-08-23, by blanchet
invert semantics of "relevance_convergence", to make it more intuitive
2010-08-23, by blanchet
if no facts were selected on first iteration, try again with a lower threshold
2010-08-23, by blanchet
weed out junk in relevance filter
2010-08-23, by blanchet
no need for "eq" facts -- good old "=" is good enough for us
2010-08-23, by blanchet
revert unintended change
2010-08-23, by blanchet
destroy elim rules before checking for finite exhaustive facts
2010-08-23, by blanchet
prevent double inclusion of the fact "True_or_False" in TPTP problems
2010-08-23, by blanchet
merged
2010-08-24, by haftmann
tuned
2010-08-24, by haftmann
merged
2010-08-23, by haftmann
dropped pre_post_conv
2010-08-23, by haftmann
use conv alias
2010-08-23, by haftmann
preliminary versions of static_eval_conv(_simple)
2010-08-23, by haftmann
use Code_Thingol.static_eval_conv_simple
2010-08-23, by haftmann
added static_eval_conv
2010-08-23, by haftmann
refined and unified naming convention for dynamic code evaluation techniques
2010-08-23, by haftmann
tap_thy conversional
2010-08-23, by haftmann
dropped now obsolete purge_data -- happens implicitly on change of theory identity
2010-08-23, by haftmann
merged
2010-08-24, by bulwahn
introducing simplification equations for inductive sets; added data structure for storing equations; rewriting retrieval of simplification equation for inductive predicates and sets
2010-08-23, by bulwahn
added support for xsymbol syntax for mode annotations in code_pred command
2010-08-23, by bulwahn
tuned raw Sidekick output;
2010-08-25, by wenzelm
Text.Range.is_singleton;
2010-08-24, by wenzelm
Markup_Tree.+: new info tends to sink to bottom, where it is prefered by select;
2010-08-24, by wenzelm
tuned;
2010-08-24, by wenzelm
Markup_Tree.select: more straight-forward recursion producing one main stream, avoid fragmentation of parent info due to ignored subtree;
2010-08-24, by wenzelm
tuned root markup;
2010-08-24, by wenzelm
misc tuning of important special cases;
2010-08-23, by wenzelm
Rewrite the Probability theory.
2010-08-23, by hoelzl
merged
2010-08-23, by wenzelm
merged
2010-08-23, by blanchet
use different name for debugging purposes
2010-08-23, by blanchet
perform eta-expansion of quantifier bodies in Sledgehammer translation when needed + transform elim rules later;
2010-08-23, by blanchet
"no_atp" fact that leads to unsound Sledgehammer proofs
2010-08-23, by blanchet
"no_atp" fact that leads to unsound proofs in Sledgehammer
2010-08-23, by blanchet
"no_atp" fact that leads to unsound proofs
2010-08-23, by blanchet
"no_atp" a few facts that often lead to unsound proofs
2010-08-23, by blanchet
play with fudge factor + parse one more Vampire error
2010-08-23, by blanchet
fiddle a bit with the SPASS fudge number
2010-08-23, by blanchet
be more generous towards SPASS's -SOS mode
2010-08-22, by blanchet
don't penalize abstractions in relevance filter + support nameless `foo`-style facts
2010-08-22, by blanchet
merged
2010-08-23, by haftmann
dropped type classes mult_mono and mult_mono1; tuned names of technical rule duplicates
2010-08-23, by haftmann
Document_Model.token_marker: lock jEdit buffer here, which is presumably a critical spot (the model is not necessarily accessed from the Swing thread);
2010-08-23, by wenzelm
sporadic locking of jEdit buffer;
2010-08-23, by wenzelm
main session actor as independent thread, to avoid starvation via regular worker pool;
2010-08-23, by wenzelm
optional daemon flag;
2010-08-23, by wenzelm
tuned;
2010-08-23, by wenzelm
module for simplified thread operations (Scala version);
2010-08-23, by wenzelm
added ML toplevel pretty-printing for tables, using dummy for anything other than Poly/ML 5.3.0 (or later);
2010-08-23, by wenzelm
recognize more "smlnj" variants;
2010-08-23, by wenzelm
merged
2010-08-23, by wenzelm
treat "using X by metis" (more or less) the same as "by (metis X)"
2010-08-22, by blanchet
prefer TPTP "conjecture" tag to "hypothesis" on ATPs where this is possible;
2010-08-22, by blanchet
merged
2010-08-22, by blanchet
more work on finite axiom detection
2010-08-22, by blanchet
revert junk submitted by mistake
2010-08-22, by blanchet
make sure minimizer facts go through "transform_elim_theorems"
2010-08-20, by blanchet
use a smaller simpset in order to not solve refl-instances
2010-08-22, by Christian Urban
allow for pre-simplification of lifted theorems
2010-08-22, by Christian Urban
changed to a more convenient argument order
2010-08-22, by Christian Urban
merged
2010-08-20, by haftmann
split and enriched theory SetsAndFunctions
2010-08-20, by haftmann
more concise characterization of of_nat operation and class semiring_char_0
2010-08-20, by haftmann
inj_comp and inj_fun
2010-08-20, by haftmann
tuned: less formal noise in Named_Target, more coherence in Class
2010-08-20, by haftmann
remove trivial facts
2010-08-20, by blanchet
unbreak "only" option of Sledgehammer
2010-08-20, by blanchet
merged
2010-08-20, by blanchet
less
more
|
(0)
-30000
-10000
-3000
-1000
-120
+120
+1000
+3000
+10000
+30000
tip