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.
more appropriate name for configuration option "meson_max_clauses" (cf. output of 'pront_configs');
2010-08-27, by wenzelm
Sum_Of_Squares: proper configuration options;
2010-08-27, by wenzelm
tuned printed type names, according to ML;
2010-08-27, by wenzelm
eliminated unnecessary ref;
2010-08-27, by wenzelm
clarified iter_deepen_limit vs meson (cf. 7c5896919eb8) -- eliminated global ref;
2010-08-27, by wenzelm
disposed some old debugging tools;
2010-08-27, by wenzelm
proper configuration option "show_proofs";
2010-08-27, by wenzelm
structure Unsynchronized is never opened and set/reset/toggle have been discontinued;
2010-08-27, by wenzelm
expanded some aliases from structure Unsynchronized;
2010-08-27, by wenzelm
merged, resolving some minor conflicts in src/HOL/Tools/Predicate_Compile/code_prolog.ML;
2010-08-27, by wenzelm
merged
2010-08-27, by haftmann
formerly unnamed infix conjunction and disjunction now named HOL.conj and HOL.disj
2010-08-27, by haftmann
tuned fact reference
2010-08-27, by haftmann
merged
2010-08-27, by bulwahn
added support for yet another prolog system (yap); generate has only one option ensure_groundness; added one example of yap invocation in example theory
2010-08-27, by bulwahn
adapted examples; tuned
2010-08-26, by bulwahn
moving options; tuned
2010-08-26, by bulwahn
added generation of predicates for size-limited enumeration of values
2010-08-26, by bulwahn
NEWS
2010-08-26, by haftmann
merged
2010-08-26, by haftmann
formerly unnamed infix impliciation now named HOL.implies
2010-08-26, by haftmann
merged
2010-08-26, by haftmann
proper passing of optional module name
2010-08-26, by haftmann
For sublocale it is sufficient to reconsider ancestors of the target.
2010-08-26, by ballarin
only print qualified implicits
2010-08-26, by haftmann
merged
2010-08-26, by haftmann
stub for (later) correct deresolving of class method names
2010-08-26, by haftmann
tuned serializer interface
2010-08-26, by haftmann
private version of commas, cf. printmode
2010-08-26, by haftmann
merged
2010-08-26, by haftmann
merged
2010-08-26, by haftmann
re-added accidental omission
2010-08-26, by haftmann
tuned includes
2010-08-26, by haftmann
prevent line breaks after Scala symbolic operators
2010-08-26, by haftmann
corrected semantics of presentation_stmt_names; do not print includes on presentation selection
2010-08-26, by haftmann
code_include Scala: qualify module nmae
2010-08-26, by haftmann
merged
2010-08-25, by haftmann
preliminary implementation of hierarchical module name space
2010-08-25, by haftmann
tuned
2010-08-25, by haftmann
proper context for various Thy_Output options, via official configuration options in ML and Isar;
2010-08-27, by wenzelm
Thy_Output: options based on proper context, although Thy_Output.add_wrapper still allows to maintain old-style wrapper combinators (setmp_CRITICAL etc.);
2010-08-27, by wenzelm
eliminated old 'local' command;
2010-08-27, by wenzelm
more uniform descriptions, which end up in the collective output of 'print_attributes' for example;
2010-08-26, by wenzelm
Fast_Lin_Arith.number_of: more conventional merge that prefers the left side -- note that former ordering wrt. serial numbers makes it depend on accidental load order;
2010-08-26, by wenzelm
slightly more abstract data handling in Fast_Lin_Arith;
2010-08-26, by wenzelm
theory data merge: prefer left side uniformly;
2010-08-26, by wenzelm
tuned;
2010-08-26, by wenzelm
simplification/standardization of some theory data;
2010-08-26, by wenzelm
misc tuning and simplification, notably theory data;
2010-08-26, by wenzelm
renamed Local_Theory.theory(_result) to Local_Theory.background_theory(_result) to emphasize that this belongs to the infrastructure and is rarely appropriate in user-space tools;
2010-08-26, by wenzelm
renamed ProofContext.theory(_result) to ProofContext.background_theory(_result) to emphasize that this belongs to the infrastructure and is rarely appropriate in user-space tools;
2010-08-26, by wenzelm
standardized Context.copy_thy to Theory.copy alias, with slightly more direct way of using it;
2010-08-26, by wenzelm
merged
2010-08-26, by wenzelm
merged
2010-08-26, by blanchet
consider "locality" when assigning weights to facts
2010-08-26, by blanchet
add a bonus for chained facts, since they are likely to be relevant;
2010-08-26, by blanchet
merged
2010-08-26, by blanchet
add a penalty for lambda-abstractions;
2010-08-26, by blanchet
renaming
2010-08-26, by blanchet
fiddle with relevance filter
2010-08-26, by blanchet
update docs
2010-08-25, by blanchet
reorganize options regarding to the relevance threshold and decay
2010-08-25, by blanchet
make relevance filter work in term of a "max_relevant" option + use Vampire SOS;
2010-08-25, by blanchet
simplify more code
2010-08-25, by blanchet
cosmetics
2010-08-25, by blanchet
get rid of "defs_relevant" feature;
2010-08-25, by blanchet
make SML/NJ happy
2010-08-25, by blanchet
renamed "relevance_convergence" to "relevance_decay"
2010-08-25, by blanchet
make sure that "undo_ascii_of" is the inverse of "ascii_of", also for non-printable characters -- and avoid those in ``-style facts
2010-08-24, by blanchet
better workaround for E's off-by-one-second issue
2010-08-24, by blanchet
merged
2010-08-26, by bulwahn
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
less
more
|
(0)
-30000
-10000
-3000
-1000
-112
+112
+1000
+3000
+10000
+30000
tip