Mercurial
Mercurial
>
repos
>
isabelle
/ graph
summary
|
shortlog
|
changelog
| graph |
tags
|
bookmarks
|
branches
|
files
|
gz
|
help
less
more
|
(0)
-30000
-10000
-3000
-1000
-256
+256
+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 generation of lambdas in THF
2011-07-05, by nik
add support for lambdas in TPTP THF generator + killed an unsound type encoding (because the monotonicity calculus assumes first-order)
2011-07-05, by nik
simplified Symbol.iterator: produce strings, which are mostly preallocated;
2011-07-05, by wenzelm
tuned comment (cf. e9f26e66692d);
2011-07-05, by wenzelm
Thy_Info.dependencies: ignore already loaded theories, according to initial prover session status;
2011-07-05, by wenzelm
theory name needs to conform to Path syntax;
2011-07-05, by wenzelm
hard-wired print mode "xsymbols" increases chance that "iff" in HOL will print symbolic arrow;
2011-07-05, by wenzelm
prefer space_explode/split_lines as in Isabelle/ML;
2011-07-05, by wenzelm
Path.split convenience;
2011-07-05, by wenzelm
get theory from last executation state;
2011-07-05, by wenzelm
explicit exit_transaction with Theory.end_theory (which could include sanity checks as in HOL-SPARK for example);
2011-07-05, by wenzelm
clarified cancel_execution/await_cancellation;
2011-07-05, by wenzelm
tuned signature;
2011-07-05, by wenzelm
tuned;
2011-07-05, by wenzelm
re-check to explicitly propagate a given type constraint to lhs -- necessary to trigger type improvement in an instantiation target
2011-07-05, by krauss
Document.no_id/new_id as in ML (new_id *could* be session-specific but it isn't right now);
2011-07-04, by wenzelm
quasi-static Isabelle_System -- reduced tendency towards "functorial style";
2011-07-04, by wenzelm
explicit class Counter;
2011-07-04, by wenzelm
merged
2011-07-04, by wenzelm
the borel probability measure is easier to handle with {0 ..< 1} (coverable by disjoint intervals {_ ..< _})
2011-07-04, by hoelzl
equalities of subsets of atLeastLessThan
2011-07-04, by hoelzl
adding documentation of the value antiquotation to the code generation manual
2011-07-03, by bulwahn
make SML/NJ happy
2011-07-03, by blanchet
install case certificate for If after code_datatype declaration for bool
2011-07-02, by haftmann
tuned typo
2011-07-02, by haftmann
pervasive Basic_Library in Scala;
2011-07-04, by wenzelm
some support for theory files within Isabelle/Scala session;
2011-07-04, by wenzelm
imitate exception ERROR of Isabelle/ML;
2011-07-04, by wenzelm
eliminated null;
2011-07-03, by wenzelm
more explicit edit_node vs. init_node;
2011-07-03, by wenzelm
tuned signature;
2011-07-03, by wenzelm
Thy_Header.read convenience;
2011-07-02, by wenzelm
some support for Session.File_Store;
2011-07-02, by wenzelm
tuned signature;
2011-07-02, by wenzelm
eliminated redundant session_ready;
2011-07-02, by wenzelm
tuned;
2011-07-02, by wenzelm
uniform finish_thy -- always Global_Theory.join_proofs, even with sequential scheduling;
2011-07-02, by wenzelm
misc tuning;
2011-07-02, by wenzelm
correction: do not assume that case const index covered all cases
2011-07-02, by haftmann
remove illegal case combinators after merge
2011-07-01, by haftmann
corrected misunderstanding what `old functions` are supposed to be
2011-07-01, by haftmann
centralized deletion of equations for constructors; corrected misunderstanding what `old functions` are supposed to be
2011-07-01, by haftmann
merged
2011-07-01, by haftmann
index cases for constructors
2011-07-01, by haftmann
cover induct's "arbitrary" more deeply
2011-07-01, by noschinl
merged;
2011-07-01, by wenzelm
enforce hard timeout on ATPs (esp. "z3_atp" on Linux) + remove obsolete failure codes
2011-07-01, by blanchet
made minimizer informative output accurate
2011-07-01, by blanchet
test a few more type encodings
2011-07-01, by blanchet
further repair "mangled_tags", now that tags are also mangled
2011-07-01, by blanchet
update documentation after "type_enc" renaming + fixed a few other out-of-date factlets
2011-07-01, by blanchet
renamed "type_sys" to "type_enc", which is more accurate
2011-07-01, by blanchet
document "simple_higher" type encoding
2011-07-01, by blanchet
cleaner handling of higher-order simple types, so that it's also possible to use first-order simple types with LEO-II and company
2011-07-01, by blanchet
mangle "ti" tags
2011-07-01, by blanchet
tuning
2011-07-01, by blanchet
clarified Thy_Syntax.element;
2011-07-01, by wenzelm
tuned layout;
2011-07-01, by wenzelm
proper @{binding} antiquotations (relevant for formal references);
2011-07-01, by wenzelm
tuned;
2011-07-01, by wenzelm
merged
2011-07-01, by wenzelm
reverted 782991e4180d: fold_fields was never used
2011-07-01, by noschinl
reverted ce00462f,b3759dce, 7a165592: unwanted generalisation
2011-07-01, by noschinl
improving actual dependencies
2011-07-01, by bulwahn
adding a minimalistic documentation of the value antiquotation in the Isar reference manual
2011-07-01, by bulwahn
adding a value antiquotation
2011-07-01, by bulwahn
more general theory header parsing;
2011-06-30, by wenzelm
back to sequential merge_data, reverting 741373421318 (NB: expensive Parser.merge_gram is already asynchronous since 3daff3cc2214);
2011-06-30, by wenzelm
merged
2011-06-30, by wenzelm
parse term in auxiliary context augmented with variable;
2011-06-30, by krauss
linarith counterexamples now provide only valuations for variables (which should restrict the number of linarith trace messages);
2011-06-29, by boehmes
prefer Isabelle path algebra;
2011-06-30, by wenzelm
proper fold order;
2011-06-30, by wenzelm
more Path operations;
2011-06-30, by wenzelm
getenv_strict in ML;
2011-06-30, by wenzelm
standardized use of Path operations;
2011-06-30, by wenzelm
tuned comments;
2011-06-30, by wenzelm
abstract algebra of file paths in Scala (cf. path.ML);
2011-06-30, by wenzelm
proper Path.print;
2011-06-30, by wenzelm
basic operations on lists and strings;
2011-06-29, by wenzelm
tuned signature;
2011-06-29, by wenzelm
simplified/unified Simplifier.mk_solver;
2011-06-29, by wenzelm
modernized some simproc setup;
2011-06-29, by wenzelm
modernized some simproc setup;
2011-06-29, by wenzelm
print Path.T with some markup;
2011-06-29, by wenzelm
HTML: render control symbols more like Isabelle/Scala/jEdit;
2011-06-29, by wenzelm
collapse map functions with identity subcoercions to identities;
2011-06-28, by traytel
reenabled accidentally-disabled automatic minimization
2011-06-28, by blanchet
tuned markup;
2011-06-28, by wenzelm
merged
2011-06-28, by paulson
tidied messy proofs
2011-06-28, by paulson
merged
2011-06-28, by bulwahn
adding timeout to quickcheck narrowing
2011-06-28, by bulwahn
simplified proofs using metis calls
2011-06-28, by paulson
merged
2011-06-28, by paulson
keyfree: The set of key-free messages (and associated theorems)
2011-06-28, by paulson
merged
2011-06-27, by wenzelm
new Datatype.info_of_constr with strict behaviour wrt. to overloaded constructors -- side effect: function package correctly identifies 0::int as a non-constructor;
2011-06-27, by krauss
added reference for MESON
2011-06-27, by blanchet
document "meson" and "metis" in HOL specific section of the Isar ref manual
2011-06-27, by blanchet
clarify minimizer output
2011-06-27, by blanchet
don't export any metastrange or other nonatomizable formulas, since these don't help proving normal things, they are somewhat broken in the ATP output, and they are atypical
2011-06-27, by blanchet
tweaked comment
2011-06-27, by blanchet
document "sound" option
2011-06-27, by blanchet
minor Sledgehammer news
2011-06-27, by blanchet
added "sound" option to force Sledgehammer to be pedantically sound
2011-06-27, by blanchet
removed "full_types" option from documentation
2011-06-27, by blanchet
document changes to Sledgehammer and "try"
2011-06-27, by blanchet
removed "full_types" option from Sledgehammer, now that virtually sound encodings are used as the default anyway
2011-06-27, by blanchet
clarify warning message to avoid confusing beginners
2011-06-27, by blanchet
remove experimental trimming feature -- it slowed down things on Linux for some reason
2011-06-27, by blanchet
filter out some tautologies using an ATP, especially for those theories that are known for producing such things
2011-06-27, by blanchet
NEWS;
2011-06-27, by wenzelm
document antiquotations are managed as theory data, with proper name space and entity markup;
2011-06-27, by wenzelm
proper checking of @{ML_antiquotation};
2011-06-27, by wenzelm
hide rather short auxiliary names, which can easily occur in user theories;
2011-06-27, by wenzelm
updated generated file;
2011-06-27, by wenzelm
ML antiquotations are managed as theory data, with proper name space and entity markup;
2011-06-27, by wenzelm
old gensym is now legacy -- global state is out of fashion, and its result is not guaranteed to be fresh;
2011-06-27, by wenzelm
parallel Syntax.parse, which is rather slow;
2011-06-27, by wenzelm
markup binding like class, which is the only special markup where Proof General (including version 4.1) allows "isar-long-id-stuff";
2011-06-27, by wenzelm
move conditional expectation to its own theory file
2011-06-27, by hoelzl
updated SMT certificates
2011-06-26, by boehmes
generalized introduction of explicit application constant: consider more functions as possible witness/instance of quantifiers than before (a constant of type T1 -> T2 -> T3 should be considered to have a rank less or equal to 1 if variables of type T2 -> T3 occur bound in a problem);
2011-06-26, by boehmes
proper tokens only if session is ready;
2011-06-25, by wenzelm
entity markup for "type", "constant";
2011-06-25, by wenzelm
clarified Markup.CLASS vs. HTML.CLASS;
2011-06-25, by wenzelm
tuned color, to avoid confusion with type variables;
2011-06-25, by wenzelm
discontinued generic XML markup -- this is for XHTML with <span/> elements;
2011-06-25, by wenzelm
type classes: entity markup instead of old-style token markup;
2011-06-25, by wenzelm
clarified Binding.pretty/print: no quotes, only markup -- Binding.str_of is rendered obsolete;
2011-06-25, by wenzelm
clarified Binding.str_of/print: show full prefix + qualifier, which is relevant for print_locale, for example;
2011-06-25, by wenzelm
produce string constant directly;
2011-06-25, by wenzelm
merged
2011-06-25, by wenzelm
While reading equations of an interpretation, already allow syntax provided by the interpretation base.
2011-06-25, by ballarin
removed very slow proof of unnamed/unused theorem from HOL/Quickcheck_Narrowing.thy (cf. 2dee03f192b7) -- can take seconds for main HOL and minutes for HOL-Proofs;
2011-06-25, by wenzelm
clarified java.ext.dirs: putting Isabelle extensions first makes it work miraculously even on Cygwin with Java in "C:\Program Files\..." (with spaces in file name);
2011-06-25, by wenzelm
CLASSPATH already converted in isabelle java wrapper;
2011-06-25, by wenzelm
removed unused/broken Isabelle.exe for now -- needs update of Admin/launch4j;
2011-06-25, by wenzelm
more robust join_results: join_work needs to be uninterruptible, otherwise the task being dequeued by join_next might be never executed/finished!
2011-06-23, by wenzelm
clarified EXCEPTIONS [] (cf. Exn.is_interrupt and Runtime.exn_message);
2011-06-23, by wenzelm
more robust concurrent builds;
2011-06-23, by wenzelm
merged
2011-06-23, by huffman
add countable_datatype method for proving countable class instances
2011-06-23, by huffman
merged;
2011-06-23, by wenzelm
instance inat :: number_semiring
2011-06-23, by huffman
added number_semiring class, plus a few new lemmas;
2011-06-23, by huffman
merged
2011-06-23, by blanchet
fiddle with remote ATP settings, based on Judgment Day
2011-06-23, by blanchet
give slightly more time to server to respond, to avoid leaving too much garbage on Geoff's servers
2011-06-23, by blanchet
Release notes should be written from the user's perspective. Don't assume the user has universal knowledge of the system.
2011-06-23, by ballarin
generalize lemmas power_number_of_even and power_number_of_odd
2011-06-22, by huffman
merged
2011-06-22, by huffman
add HOLCF/ex/Concurrency_Monad.thy, which contains resumption/state/powerdomain monad example from my PhD thesis
2011-06-22, by huffman
simplified arrangement of jars;
2011-06-23, by wenzelm
adapted to Cygwin;
2011-06-23, by wenzelm
provide Isabelle/Scala environment as Java extension, instead of user classpath
2011-06-23, by wenzelm
explicit import java.lang.System to prevent odd scope problems;
2011-06-23, by wenzelm
ensure export of initial CLASSPATH;
2011-06-23, by wenzelm
augment Java extension directories;
2011-06-23, by wenzelm
basic setup for Isabelle charset;
2011-06-23, by wenzelm
prefer actual charset over charset name;
2011-06-22, by wenzelm
clarified default ML settings;
2011-06-22, by wenzelm
lazy Isabelle_System.default supports implicit boot;
2011-06-22, by wenzelm
clarified plugin start/stop;
2011-06-22, by wenzelm
clarified init/exit procedure;
2011-06-22, by wenzelm
clarified decoded control symbols;
2011-06-22, by wenzelm
init/exit model/view synchronously within the swing thread -- EditBus.send in jedit-4.4.1 always runs there;
2011-06-22, by wenzelm
prefer STIXGeneral -- hard to tell if better or worse;
2011-06-22, by wenzelm
merged
2011-06-22, by wenzelm
export lambda-lifting code as there is potential use for it within Sledgehammer
2011-06-22, by boehmes
updated to jedit-4.4.1 and jedit_build-20110622;
2011-06-22, by wenzelm
clarified chunk.offset, chunk.length;
2011-06-22, by wenzelm
avoid fractional font metrics, which makes rendering really ugly (e.g. on Linux);
2011-06-21, by wenzelm
some arrow symbols from DejaVuSansMono for bsub/esub/bsup/esup;
2011-06-21, by wenzelm
more precise font transformations: shift sub/superscript, adjust size for user fonts;
2011-06-21, by wenzelm
don't change the way helpers are generated for the exporter's sake
2011-06-21, by blanchet
provide appropriate type system and number of fact defaults for remote ATPs
2011-06-21, by blanchet
order generated facts topologically
2011-06-21, by blanchet
peel off two or more layers in exceptional cases where the proof term refers to the proved theorems twice with the same name (e.g., "Transitive_Closure.trancl_into_trancl")
2011-06-21, by blanchet
tweaked E, SPASS, Vampire setup based on latest Judgment Day results
2011-06-21, by blanchet
remove historical bloat -- another benefit of merging Metis's and Sledgehammer's translations
2011-06-21, by blanchet
avoid double ASCII-fication
2011-06-21, by blanchet
make sure that enough type information is generated -- because the exported "lemma"s are also used as "conjecture", we can't optimize type information based on polarity
2011-06-21, by blanchet
generate type predicates for existentials/skolems, otherwise some problems might not be provable
2011-06-21, by blanchet
insert rather than append special facts to make it less likely that they're truncated away
2011-06-21, by blanchet
hidden font: full height makes cursor more visible;
2011-06-21, by wenzelm
more uniform treatment of recode_set/recode_map;
2011-06-21, by wenzelm
tuned iteration over short symbols;
2011-06-21, by wenzelm
Symbol.is_ctrl: handle decoded version as well;
2011-06-21, by wenzelm
some support for user symbol fonts;
2011-06-21, by wenzelm
removed obsolete font specification;
2011-06-20, by wenzelm
more tolerant Symbol.decode;
2011-06-20, by wenzelm
simplified/generalized ISABELLE_FONTS handling;
2011-06-20, by wenzelm
updated to jedit_build-20110620;
2011-06-20, by wenzelm
added SyntaxUtilities.StyleExtender hook, with actual functionality in Isabelle/Scala;
2011-06-20, by wenzelm
clean up SPASS FLOTTER hack
2011-06-20, by blanchet
remove automatic recovery from (some) unsound proofs, now that we use sound encodings for all the interesting provers
2011-06-20, by blanchet
only refer to facts found in TPTP file -- e.g. facts that simplify to true are excluded
2011-06-20, by blanchet
slightly better setup for E
2011-06-20, by blanchet
respect "really_all" argument, which is used by "ATP_Export"
2011-06-20, by blanchet
slightly better setup for SPASS and Vampire as more results have come in
2011-06-20, by blanchet
optimized SPASS and Vampire time slices, like E before
2011-06-20, by blanchet
optimized E's time slicing, based on latest exhaustive Judgment Day results
2011-06-20, by blanchet
deal with ATP time slices in a more flexible/robust fashion
2011-06-20, by blanchet
literal unicode in README.html allows to copy/paste from Lobo output;
2011-06-20, by wenzelm
merged;
2011-06-19, by wenzelm
explain special control symbols;
2011-06-19, by wenzelm
accept control symbols;
2011-06-19, by wenzelm
fixed silly ATP exporter bug: if the proof of lemma A relies on B and C, and the proof of B relies on C, return {B, C}, not {B}, as the set of dependencies
2011-06-19, by blanchet
recognize one more E failure message
2011-06-19, by blanchet
tweaked TPTP formula kind for typing information used in the conjecture
2011-06-19, by blanchet
more forceful message
2011-06-19, by blanchet
treat quotes as non-controllable, to reduce surprise in incremental editing;
2011-06-19, by wenzelm
abbreviations for special control symbols;
2011-06-19, by wenzelm
completion for control symbols;
2011-06-19, by wenzelm
updated to jedit_build-20110619;
2011-06-19, by wenzelm
support for bold style within text buffer;
2011-06-19, by wenzelm
tuned;
2011-06-19, by wenzelm
discontinued special treatment of \<^loc> (which was original meant as workaround for "local" syntax);
2011-06-19, by wenzelm
added glyphs 21e0..21e4, 21e6..21e9, 2759 from DejaVuSansMono;
2011-06-19, by wenzelm
names for control symbols without "^", which is relevant for completion;
2011-06-19, by wenzelm
some unicode chars for special control symbols;
2011-06-19, by wenzelm
tuned;
2011-06-19, by wenzelm
tuned markup;
2011-06-18, by wenzelm
avoid setTokenMarker fluctuation on buffer reload etc. via static isabelle_token_marker, which is installed by hijacking the jEdit ModeProvider;
2011-06-18, by wenzelm
proper gfx.setColor;
2011-06-18, by wenzelm
proper x1;
2011-06-18, by wenzelm
convenience functions;
2011-06-18, by wenzelm
more robust caret painting wrt. surrogate characters;
2011-06-18, by wenzelm
do not control malformed symbols;
2011-06-18, by wenzelm
Buffer.editSyntaxStyle: mask extended syntax styles;
2011-06-18, by wenzelm
hardwired abbreviations for standard control symbols;
2011-06-18, by wenzelm
updated to jedit_build-20110618, which is required for sub/superscript rendering;
2011-06-18, by wenzelm
basic support for extended syntax styles: sub/superscript;
2011-06-18, by wenzelm
tuned -- Map.empty serves as partial function;
2011-06-18, by wenzelm
proper place for config files (cf. 55866987a7d9);
2011-06-18, by wenzelm
tuned signature;
2011-06-18, by wenzelm
merged
2011-06-18, by wenzelm
IMP compiler with int, added reverse soundness direction
2011-06-17, by kleing
proper place for config files;
2011-06-18, by wenzelm
tuned markup;
2011-06-18, by wenzelm
highlight via foreground painter, using alpha channel;
2011-06-18, by wenzelm
tuned signature;
2011-06-18, by wenzelm
tuned text;
2011-06-18, by wenzelm
inner literal/delimiter corresponds to outer keyword/operator;
2011-06-18, by wenzelm
tuned markup;
2011-06-18, by wenzelm
more uniform treatment of "keyword" vs. "operator";
2011-06-18, by wenzelm
simplified Line_Context (again);
2011-06-18, by wenzelm
more robust treatment of partial range restriction;
2011-06-18, by wenzelm
select_markup: no filtering here -- results may be distorted anyway;
2011-06-18, by wenzelm
more explicit treatment of ranges after revert/convert, which may well distort the overall start/end positions;
2011-06-17, by wenzelm
more explicit error message;
2011-06-17, by wenzelm
merged
2011-06-17, by wenzelm
gave up an optimization that sometimes lead to unsound proofs -- in short, facts talking about a schematic type variable can encode a cardinality constraint and be consistent with HOL, e.g. "card (UNIV::?'a set) = 1 ==> ALL x y. x = y"
2011-06-16, by blanchet
added missing case in pattern matching -- solves Waldmeister "Match" exceptions that have been plaguing some users
2011-06-16, by blanchet
less
more
|
(0)
-30000
-10000
-3000
-1000
-256
+256
+1000
+3000
+10000
+30000
tip