Mercurial
Mercurial
>
repos
>
isabelle
/ graph
summary
|
shortlog
|
changelog
| graph |
tags
|
bookmarks
|
branches
|
files
|
gz
|
help
less
more
|
(0)
-30000
-10000
-3000
-1000
-480
+480
+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.
misc tuning for release;
2011-01-15, by wenzelm
normalize Z3 models: assignments to free variables should ideally not refer to other free variables
2011-01-15, by boehmes
Also added SPARK to test and clean targets.
2011-01-15, by berghofe
merged
2011-01-15, by berghofe
Added entry for HOL-SPARK
2011-01-15, by berghofe
Added HOL-SPARK and removed old_primrec.ML
2011-01-15, by berghofe
unused_thms no longer compares propositions, since this is no longer needed
2011-01-15, by berghofe
Include HOL-SPARK keywords
2011-01-15, by berghofe
Include HOL-SPARK
2011-01-15, by berghofe
Finally removed old primrec package, since Primrec.add_primrec_global
2011-01-15, by berghofe
Added new SPARK verification environment.
2011-01-15, by berghofe
remove presently unused Isabelle application for official releases;
2011-01-15, by wenzelm
hardwired default for proof-shell-quit-timeout (PG 4.1 provides rather low value);
2011-01-15, by wenzelm
treat HOLCF as HOL library session, not as "logic";
2011-01-15, by wenzelm
increased startup-timeout to accommodate slow systems (especially Windows/Cygwin);
2011-01-15, by wenzelm
bundle main HOL image only, to save about 300 MB disk space;
2011-01-14, by wenzelm
updated for release;
2011-01-14, by wenzelm
adjusted mira configuration
2011-01-14, by haftmann
merged
2011-01-14, by wenzelm
global "prems" is legacy feature;
2011-01-14, by wenzelm
tuned markup;
2011-01-14, by wenzelm
eliminated global prems;
2011-01-14, by wenzelm
more precise import;
2011-01-14, by wenzelm
Thy_Load.begin_theory: maintain source specification of imports;
2011-01-14, by wenzelm
merged
2011-01-14, by hoelzl
integral on lebesgue measure is extension of integral on borel measure
2011-01-14, by hoelzl
tuned formalization of subalgebra
2011-01-14, by hoelzl
introduced integral syntax
2011-01-14, by hoelzl
tuned theorem order
2011-01-14, by hoelzl
configuration file for mira
2011-01-14, by haftmann
eliminated global prems;
2011-01-13, by wenzelm
more precise pretty printing -- to accomodate Scala message layout;
2011-01-13, by wenzelm
less verbosity -- avoid slightly odd tracing information on warning channel;
2011-01-13, by wenzelm
updated Isabelle/jEdit limitations and workarounds;
2011-01-13, by wenzelm
full theory path enables loading parents via master directory and keeps files strictly separate;
2011-01-13, by wenzelm
Toplevel.init_theory: maintain optional master directory, to allow bypassing global Thy_Load.master_path;
2011-01-13, by wenzelm
clarified split_thy_path;
2011-01-13, by wenzelm
less verbosity;
2011-01-13, by wenzelm
proper 'domain' class instance for 'a defl, with deflation combinator
2011-01-12, by huffman
documented Option.bind
2011-01-12, by krauss
CONTRIBUTORS
2011-01-12, by krauss
updated keywords;
2011-01-12, by wenzelm
eliminated global prems;
2011-01-12, by wenzelm
eliminated global prems;
2011-01-12, by wenzelm
updated to ProofGeneral-4.x;
2011-01-12, by wenzelm
eliminated global prems;
2011-01-12, by wenzelm
tuned proof;
2011-01-12, by wenzelm
eliminated global prems;
2011-01-12, by wenzelm
compile;
2011-01-12, by wenzelm
more FIXMEs concerning bad catch-all exception handlers;
2011-01-12, by wenzelm
eliminated obsolete print_sign_exn_unit;
2011-01-12, by wenzelm
reraise interrupts as usual;
2011-01-12, by wenzelm
avoid catch-all exception handler, presumably TERM was meant here;
2011-01-12, by wenzelm
disabled experimental treatment of replacement text for now, which leads to odd spacing and strange effects on non-poppler viewers;
2011-01-12, by wenzelm
observe line length limit;
2011-01-12, by wenzelm
smart_string_of_real: print integer values without fractional part;
2011-01-12, by wenzelm
tuned (cf. 2fe62d602681);
2011-01-11, by wenzelm
added dist/jedit symlink for convenience;
2011-01-11, by wenzelm
record versions of both jEdit and Isabelle;
2011-01-11, by wenzelm
updated to Isabelle2011;
2011-01-11, by wenzelm
isabelle version -i;
2011-01-11, by wenzelm
NEWS
2011-01-11, by haftmann
NEWS
2011-01-11, by bulwahn
eliminated duplication
2011-01-11, by krauss
merged
2011-01-11, by wenzelm
tuned text
2011-01-11, by haftmann
"enriched_type" replaces less specific "type_lifting"
2011-01-11, by haftmann
clarified notion Position.is_reported;
2011-01-11, by wenzelm
refined report_parse_tree: reverse reports happen to produce proper type information for inlined @{term}, @{typ} etc.;
2011-01-10, by wenzelm
refined ML_Lex.flatten: ensure proper separation of tokens;
2011-01-10, by wenzelm
ML compiler: more careful treatment of input tokens -- trailing space ensures proper separation and end position (cf. 82c1e348bc18, 08240feb69c7);
2011-01-10, by wenzelm
use just one data slot to VC-related information
2011-01-10, by boehmes
be more precise: also merge option values
2011-01-10, by boehmes
only print warning in a visible context (previously, the warning was printed more than once)
2011-01-10, by boehmes
dropped superfluous error message
2011-01-10, by boehmes
removed obsolete make target (now in doc-src, cf. 28b487cd9e15)
2011-01-10, by krauss
updated for polyml-5.4.0;
2011-01-10, by wenzelm
made SML/NJ happy;
2011-01-10, by wenzelm
added merge_options convenience;
2011-01-10, by wenzelm
tuned string_of_int to avoid allocation for small integers;
2011-01-10, by wenzelm
eliminated Int.toString;
2011-01-10, by wenzelm
eliminated obsolete LargeInt -- Int is unbounded;
2011-01-10, by wenzelm
standardized split_last/last_elem towards List.last;
2011-01-10, by wenzelm
removing dead code; tuned
2011-01-10, by bulwahn
made SML/NJ happy
2011-01-10, by bulwahn
reverted 08240feb69c7 -- breaks positions of reports;
2011-01-09, by wenzelm
ML_trace: observe context visibility flag (import for Latex mode, for example);
2011-01-09, by wenzelm
more direct treatment of Position.end_offset;
2011-01-09, by wenzelm
discontinued unused end_line, end_column;
2011-01-09, by wenzelm
more scalable HTML.output_width;
2011-01-09, by wenzelm
refined comment (again);
2011-01-09, by wenzelm
merged
2011-01-08, by huffman
use proper syntactic types for 'syntax' commands
2011-01-08, by huffman
make print translation for Abs_cfun consistent with other binders: prevent eta-contraction, but don't force eta-expansion
2011-01-08, by huffman
use full path for library imports
2011-01-08, by huffman
types -> type_synonym
2011-01-08, by huffman
updated NEOS_SERVER, which is now provided via settings;
2011-01-08, by wenzelm
renamed Sum_Of_Squares to Sum_of_Squares;
2011-01-08, by wenzelm
Ord_List.merge convenience;
2011-01-08, by wenzelm
misc tuning and comments based on review of Theory_Data, Proof_Data, Generic_Data usage;
2011-01-08, by wenzelm
modernized structure Prop_Logic;
2011-01-08, by wenzelm
added Context_Position.is_visible_proof, which treats a global theory as invisible (unlike the default);
2011-01-08, by wenzelm
tuned;
2011-01-08, by wenzelm
tuned;
2011-01-08, by wenzelm
tuned headers;
2011-01-08, by wenzelm
merged
2011-01-07, by wenzelm
adding example theory for list comprehension to set comprehension simproc
2011-01-07, by bulwahn
adopting proofs due to new list comprehension to set comprehension simproc
2011-01-07, by bulwahn
adding simproc to rewrite list comprehensions to set comprehensions; adopting proofs
2011-01-07, by bulwahn
tuned text
2011-01-07, by boehmes
merged
2011-01-07, by bulwahn
removing obselete Id comments from HOL/ex theories
2011-01-07, by bulwahn
added hints about licensing restrictions and how to enable Z3
2011-01-07, by boehmes
tuned
2011-01-07, by boehmes
eliminated hard tabs;
2011-01-07, by wenzelm
allow spaces in $SPASS_HOME value;
2011-01-07, by wenzelm
tuned;
2011-01-07, by wenzelm
eliminated alias;
2011-01-07, by wenzelm
do not open ML structures;
2011-01-07, by wenzelm
more standard package setup;
2011-01-07, by wenzelm
do not open ML structures;
2011-01-07, by wenzelm
updated scala;
2011-01-07, by wenzelm
do not open ML structures;
2011-01-07, by wenzelm
do not open Codegen;
2011-01-07, by wenzelm
tuned whitespace, indentation, comments;
2011-01-07, by wenzelm
updated for release;
2011-01-07, by wenzelm
tuned;
2011-01-07, by wenzelm
more precise parentheses and indentation;
2011-01-07, by wenzelm
comments;
2011-01-07, by wenzelm
updated for 2011;
2011-01-07, by wenzelm
shortened the warning about uninstalled SMT solvers (the additional hint might get obsolete without further notice)
2011-01-07, by boehmes
tuned NEWS
2011-01-07, by krauss
avoid ML structure aliases (especially single-letter abbreviations)
2011-01-07, by boehmes
made SML/NJ happy
2011-01-07, by boehmes
rename constant u_defl to u_liftdefl;
2011-01-06, by huffman
rename constant pdefl to liftdefl_of
2011-01-06, by huffman
Diagnostic command to show locale dependencies.
2011-01-06, by ballarin
Documentation for 'interpret' and 'sublocale' with mixins.
2011-01-06, by ballarin
Abelian group facts obtained from group facts via interpretation (sublocale).
2011-01-06, by ballarin
differentiate between local and remote SMT solvers (e.g., "z3" vs. "remote_z3");
2011-01-06, by boehmes
remove various lemmas redundant with lub_eq_bottom_iff
2011-01-04, by huffman
change some lemma names containing 'UU' to 'bottom'
2011-01-04, by huffman
renamed constant 'UU' to 'bottom', keeping 'UU' as alternative input syntax;
2011-01-04, by huffman
merged
2011-01-03, by boehmes
updated SMT certificates
2011-01-03, by boehmes
re-implemented support for datatypes (including records and typedefs);
2011-01-03, by boehmes
tuned whitespace
2011-01-03, by haftmann
do not open structure Codegen;
2010-12-31, by wenzelm
do not open auxiliary ML structures;
2010-12-30, by wenzelm
uniform treatment of type vs. term environment (cf. b654fa27fbc4);
2010-12-30, by wenzelm
uniform treatment of typ_match and raw_match (cf. b654fa27fbc4);
2010-12-30, by wenzelm
tuned isatest settings;
2010-12-30, by wenzelm
merged
2010-12-29, by wenzelm
more robust decomposition of simultaneous goals
2010-12-29, by krauss
function (default) is legacy feature
2010-12-29, by krauss
more scalable Symbol_Pos.explode;
2010-12-29, by wenzelm
tuned ML toplevel pp for type string: observe depth limit;
2010-12-29, by wenzelm
theory loader: implicit load path is considered legacy;
2010-12-29, by wenzelm
explicit file specifications -- avoid secondary load path;
2010-12-29, by wenzelm
check_file: secondary load path is legacy feature;
2010-12-29, by wenzelm
share_common_data dummy;
2010-12-29, by wenzelm
made SML/NJ happy;
2010-12-29, by wenzelm
made SML/NJ happy;
2010-12-29, by wenzelm
tuned comments;
2010-12-29, by wenzelm
made SML/NJ happy;
2010-12-29, by wenzelm
made SML/NJ happy;
2010-12-28, by wenzelm
function (tailrec) is a legacy feature
2010-12-27, by krauss
dropped duplicate unused lemmas;
2010-12-25, by krauss
partial_function (tailrec) replaces function (tailrec);
2010-12-25, by krauss
remove lemma ideal_completion.principal_induct2, use principal_induct twice instead
2010-12-24, by huffman
NEWS updates for HOLCF
2010-12-23, by huffman
replaced separate lemmas seq{1,2,3} with seq_simps
2010-12-23, by huffman
changed syntax of powerdomain binary union operators
2010-12-23, by huffman
tuned order of NEWS
2010-12-23, by haftmann
NEWS
2010-12-23, by haftmann
documentation stub on type_lifting
2010-12-23, by haftmann
tuned comments and line breaks
2010-12-23, by haftmann
rename function ideal_completion.basis_fun to ideal_completion.extension
2010-12-22, by huffman
fix another proof script broken by a35af5180c01
2010-12-22, by huffman
fix proof script broken by a35af5180c01
2010-12-22, by huffman
merged
2010-12-22, by haftmann
full localization with possibly multiple entries;
2010-12-22, by haftmann
tool-compliant mapper declaration
2010-12-22, by haftmann
more proof contexts; formal declaration
2010-12-22, by haftmann
mapper is arbitrary term, not only constant;
2010-12-22, by haftmann
tuned comment
2010-12-22, by haftmann
merged
2010-12-22, by wenzelm
made SML/NJ happy
2010-12-22, by blanchet
check JVM later, to avoid potential conflict with jEdit splash screen;
2010-12-22, by wenzelm
explicit JVM check on startup;
2010-12-22, by wenzelm
more explicit jvm_name;
2010-12-22, by wenzelm
isabelle java: prefer -server here;
2010-12-22, by wenzelm
configuration option "rule_trace";
2010-12-21, by wenzelm
configuration option "syntax_branching_level";
2010-12-21, by wenzelm
configuration option "syntax_ast_trace" and "syntax_ast_stat";
2010-12-21, by wenzelm
more robust ML antiquotations -- allow original tokens without adjacent whitespace;
2010-12-21, by wenzelm
configuration option "ML_trace";
2010-12-21, by wenzelm
merged
2010-12-21, by haftmann
id_const replaces mk_id
2010-12-21, by haftmann
tuned type_lifting declarations
2010-12-21, by haftmann
prove more algebraic version of functorial properties; retain old properties for convenience
2010-12-21, by haftmann
declare more simp rules, rewrite proofs in Isar-style
2010-12-21, by huffman
merged
2010-12-21, by hoelzl
use DERIV_intros
2010-12-21, by hoelzl
generalized monoseq, decseq and incseq; simplified proof for seq_monosub
2010-12-21, by hoelzl
merged
2010-12-21, by haftmann
proper static closures
2010-12-21, by haftmann
tuned names
2010-12-21, by haftmann
renamed mk_id to the more canonical id_const
2010-12-21, by haftmann
merged
2010-12-21, by blanchet
better parsing of options, in case the value has '='
2010-12-21, by blanchet
show the relation
2010-12-21, by blanchet
merged
2010-12-21, by blanchet
renamed "sledgehammer_tactic.ML" to "sledgehammer_tactics.ML" (cf. module name);
2010-12-21, by blanchet
added "sledgehammer_tac" as possible reconstructor in Mirabelle
2010-12-21, by blanchet
merged
2010-12-21, by wenzelm
merged
2010-12-21, by boehmes
also provide a view on arguments for "external" built-in symbols (similar to "internal" (real) built-in symbols)
2010-12-21, by boehmes
Enabled non fully polymorphic map functions in subtyping
2010-12-21, by traytel
make SML/NJ and Poly/ML agree on the type of "before";
2010-12-21, by wenzelm
only depend on exisiting statements
2010-12-21, by haftmann
merged
2010-12-21, by haftmann
evaluator separating static and dynamic operations
2010-12-21, by haftmann
tuned naming
2010-12-21, by haftmann
evaluator separating static and dynamic operations
2010-12-21, by haftmann
canonical handling of theory context argument
2010-12-21, by haftmann
merged
2010-12-21, by haftmann
evaluator separating static and dynamic operations
2010-12-21, by haftmann
program is separate argument to serializer
2010-12-21, by haftmann
more explicit structure for serializer invocation
2010-12-21, by haftmann
merged
2010-12-21, by nipkow
tuned proof
2010-12-21, by nipkow
HOLogic.mk_id
2010-12-21, by haftmann
avoid weird symbols in path
2010-12-21, by blanchet
mechanism to keep SMT input and output files around in Mirabelle
2010-12-21, by blanchet
proper handling of the arguments of SMT builtins -- for numerals, ignore the arguments (Pls, Bit0, Bit1, ..), for functions, consider them;
2010-12-21, by blanchet
added "smt_triggers" option to experiment with triggers in Sledgehammer;
2010-12-21, by blanchet
enable E weight generation with unofficial latest version of E (tentatively called E 1.2B) -- backed by Judgment Day
2010-12-21, by blanchet
Cygwin: Poly/ML 5.4.0 requires libgmp3;
2010-12-20, by wenzelm
updated to polyml-5.4.0;
2010-12-20, by wenzelm
tuned;
2010-12-20, by wenzelm
updated for Poly/ML 5.4.0;
2010-12-20, by wenzelm
merged
2010-12-20, by boehmes
avoid ML structure aliases (especially single-letter abbreviations)
2010-12-20, by boehmes
added an additional beta reduction: unfolding of special quantifiers might leave terms unnormalized wrt to beta reductions
2010-12-20, by boehmes
merged
2010-12-20, by huffman
configure domain package to work with HOL option type
2010-12-20, by huffman
make internal proofs for deflation and isodefl theorems more robust, by avoiding calls to the simplifier for beta-reduction
2010-12-20, by huffman
simplify proofs
2010-12-20, by huffman
beta-reduction simproc uses lemma Abs_cfun_inverse2 instead of beta_cfun, to be more robust against eta-contraction
2010-12-20, by huffman
configure domain package to work with HOL sum type
2010-12-20, by huffman
replace list_map function with an abbreviation
2010-12-20, by huffman
merged
2010-12-20, by blanchet
run SPASS and Vampire in SOS mode only if >= 50 facts are passed -- otherwise we are probably minimizing and then it's better if the prover is run only once with a full strategy
2010-12-20, by blanchet
disable feature that was enabled by mistake
2010-12-20, by blanchet
make exceptions more transparent in "debug" mode
2010-12-20, by blanchet
remove spurious line
2010-12-20, by blanchet
use the options provided by Stephan Schulz -- much better
2010-12-20, by blanchet
optionally supply constant weights to E -- turned off by default until properly parameterized
2010-12-20, by blanchet
merged
2010-12-20, by haftmann
type_lifting for predicates
2010-12-20, by haftmann
proper identifiers for consts and types;
2010-12-20, by wenzelm
some attempts to fit diagnostic output into regular TTY (75-80 characters per line);
2010-12-20, by wenzelm
tuned/clarified some component settings;
2010-12-20, by wenzelm
slightly more standard Isabelle_System.with_tmp_file/with_tmp_dir (cf. Scala version);
2010-12-20, by wenzelm
purged some comments (Locale_Test is already clean thanks to configuration options);
2010-12-20, by wenzelm
actually enable show_hyps option, unlike local_setup in 6da953d30f48 which merely affects the (temporary) auxiliary context;
2010-12-20, by wenzelm
merged
2010-12-20, by boehmes
updated SMT certificates
2010-12-20, by boehmes
re-introduced support for nonlinear multiplication in Z3 (overriding the built-in linear multiplication of the SMT-LIB class of solvers)
2010-12-20, by boehmes
derived SMT solver classes override inherited properties (properties of derived classes have a higher priority than properties of base classes)
2010-12-20, by boehmes
perform monomorphization during normalization: schematic numerals might be monomorphized into built-in numerals and then numeral normalization is required
2010-12-20, by boehmes
merge
2010-12-20, by haftmann
more convenient order of type variables
2010-12-17, by haftmann
rename function cprod_map to prod_map
2010-12-19, by huffman
switch to transparent ascription, to avoid warning messages
2010-12-19, by huffman
types -> type_synonym
2010-12-19, by huffman
fix typo
2010-12-19, by huffman
merged
2010-12-19, by huffman
use deflations over type 'udom u' to represent predomains;
2010-12-19, by huffman
add lemma u_map_oo
2010-12-19, by huffman
replace foo_approx functions with foo_emb, foo_prj functions for universal domain embeddings
2010-12-19, by huffman
minimize imports; move domain class instances for powerdomain types into Powerdomains.thy
2010-12-19, by huffman
powerdomain theories require class 'bifinite' instead of 'domain'
2010-12-19, by huffman
type 'defl' takes a type parameter again (cf. b525988432e9)
2010-12-19, by huffman
reintroduce 'bifinite' class, now with existentially-quantified approx function (cf. b525988432e9)
2010-12-19, by huffman
renamed Bifinite.thy to Representable.thy
2010-12-19, by huffman
renamed CompactBasis.thy to Compact_Basis.thy
2010-12-17, by huffman
merged
2010-12-19, by boehmes
updated SMT certificates
2010-12-19, by boehmes
removed odd decoration of built-in symbols as Vars (instead provide built-in desctructor functions along with their inverse functions);
2010-12-19, by boehmes
only linear occurrences of multiplication are treated as built-in (SMT solvers only support linear arithmetic in general);
2010-12-19, by boehmes
escape backticks in altstrings
2010-12-19, by blanchet
added a timestamp to Nitpick in verbose mode for debugging purposes;
2010-12-19, by blanchet
reduce the minimizer slack and add verbose information
2010-12-19, by blanchet
two layers of timeouts seem to be less reliable than a single layer
2010-12-18, by blanchet
move relevance filter into hard timeout
2010-12-18, by blanchet
handle timeouts in Mirabelle more gracefully
2010-12-18, by blanchet
made the relevance filter treat unatomizable facts like "atomize_all" properly (these result in problems that get E spinning seemingly forever);
2010-12-18, by blanchet
Add mixins to locale dependencies.
2010-12-18, by ballarin
Enable show_hyps, which appears to be set in batch mode but in an interactive session.
2010-12-18, by ballarin
Add mixins to sublocale command.
2010-12-18, by ballarin
tuning
2010-12-18, by blanchet
higher hard timeout
2010-12-18, by blanchet
lower threshold where the binary algorithm kick in and use the same value for automatic minimization
2010-12-18, by blanchet
compile
2010-12-18, by blanchet
let each prover minimizes its own stuff (rather than taking the first prover of the list to minimize every prover's stuff)
2010-12-18, by blanchet
use minimizing prover in Mirabelle
2010-12-18, by blanchet
renamed function to run prover with minimizer and changed signature to clarify its semantics and make it a drop in replacement for "get_prover"
2010-12-18, by blanchet
factored out running a prover with (optionally) an implicit minimizer phrase
2010-12-18, by blanchet
merged;
2010-12-17, by wenzelm
remove option that doesn't work in Mirabelle anyway (Mirabelle uses Sledgehammer_Provers, not Sledgehammer_Run)
2010-12-17, by blanchet
more precise error messages in "verbose" (or "debug") mode, following this morning's permission debacle
2010-12-17, by blanchet
convenient syntax for setting provers -- useful for debugging, not for general consumption and hence not documented
2010-12-17, by blanchet
merged
2010-12-17, by blanchet
put the SMT weights back where they belong, so that they're also used by Mirabelle
2010-12-17, by blanchet
added debugging option to find out how good the relevance filter was at identifying relevant facts
2010-12-17, by blanchet
extra checking of name bindings for classes, types, consts;
2010-12-17, by wenzelm
more explicit references to structure Raw_Simplifier;
2010-12-17, by wenzelm
merged
2010-12-17, by wenzelm
merged
2010-12-17, by wenzelm
merged
2010-12-17, by wenzelm
Command 'type_synonym' (with single argument) supersedes 'types' (legacy feature);
2010-12-17, by wenzelm
dropped slightly odd Conv.tap_thy
2010-12-17, by haftmann
avoid slightly odd Conv.tap_thy
2010-12-17, by haftmann
allocate intermediate directories in module hierarchy
2010-12-17, by haftmann
export experimental options
2010-12-17, by blanchet
merged
2010-12-17, by blanchet
compile
2010-12-17, by blanchet
run the SMT relevance filter only once, then run the normalization/monomorphization code once _per class_ of SMT solvers
2010-12-17, by blanchet
make timeout part of the SMT filter's tail
2010-12-17, by blanchet
merge
2010-12-17, by blanchet
split "smt_filter" into head and tail
2010-12-17, by blanchet
fewer facts to SInE-E
2010-12-17, by blanchet
Z3 sometimes reports two errors, with the first one referring to line 1 for some strange reason -- but it makes no sense to kill line 1, so we traverse the errors in reverse and consider only the last error
2010-12-17, by blanchet
trap one more Z3 error
2010-12-17, by blanchet
fixed the command-line syntax for setting Yices' random seed
2010-12-17, by boehmes
merged
2010-12-17, by boehmes
updated SMT certificates
2010-12-17, by boehmes
fixed lambda-lifting: shift indices of bound variables correctly (after locking the required bound variables) and apply bound variables to the new function symbol in the right order;
2010-12-17, by boehmes
adding exhaustive tester instances for numeric types: code_numeral, nat, rat and real
2010-12-17, by bulwahn
updated generated file;
2010-12-17, by wenzelm
replaced command 'nonterminals' by slightly modernized version 'nonterminal';
2010-12-17, by wenzelm
renamed structure MetaSimplifier to raw_Simplifer, to emphasize its meaning;
2010-12-17, by wenzelm
tuned signature;
2010-12-17, by wenzelm
clarified exports of structure Simplifier;
2010-12-17, by wenzelm
refer to regular structure Simplifier;
2010-12-17, by wenzelm
tuned;
2010-12-17, by wenzelm
updated SMT certificates
2010-12-17, by boehmes
more precise/correct SMT error handling
2010-12-17, by blanchet
fixed off-by-one and return proper error code -- never underestimate the number of oddities in Perl
2010-12-17, by blanchet
discriminate SMT errors a bit better
2010-12-16, by blanchet
keep track of errors in Z3 input file for debugging purposes
2010-12-16, by blanchet
better propagation of stdout in case of failure + comply with strict/warnings
2010-12-16, by blanchet
merge
2010-12-16, by blanchet
cleaner handling of temporary files
2010-12-16, by blanchet
merged
2010-12-16, by paulson
made sml/nj happy
2010-12-16, by paulson
added self-correcting wrapper for Z3 -- see comment in the file for details
2010-12-16, by blanchet
impose a limit on the breadth of monomorphization (in addition to on the depth) to prevent an explosion of the number of monomorphic instances
2010-12-16, by blanchet
no need to do a super-duper atomization if Metis fails afterwards anyway
2010-12-16, by blanchet
removed unused variable
2010-12-16, by blanchet
robustly handle SMT exceptions in Sledgehammer
2010-12-16, by blanchet
make "debug" imply "blocking", since in blocking mode the exceptions flow through and are more instructive
2010-12-16, by blanchet
reintroduce the higher penalty for skolems
2010-12-16, by blanchet
tuning
2010-12-16, by blanchet
comment tuning
2010-12-16, by blanchet
get rid of experimental feature of term patterns in relevance filter -- doesn't work well unless we take into consideration the equality theory entailed by the relevant facts
2010-12-16, by blanchet
fixed more issues with the Vampire output parser, and added support for Vampire's TSTP output (--proof tptp)
2010-12-16, by blanchet
make it more likely that induction rules are picked up by Sledgehammer
2010-12-16, by blanchet
generalize the Vampire parser some more to cope with things like "{2, 3\}" seen in some proofs
2010-12-16, by blanchet
add the current theory's constant to the goal to make theorems from the current theory more relevant on the first iteration already
2010-12-16, by blanchet
instantiate induction rules automatically
2010-12-16, by blanchet
merged
2010-12-16, by boehmes
fix lambda-lifting: take level of bound variables into account and also apply bound variables from outer scope
2010-12-16, by boehmes
fixed introduction of explicit application function: bound variables always need explicit application if they are applied to some term
2010-12-16, by boehmes
fixed eta-expansion: introduce a couple of abstractions at once
2010-12-16, by boehmes
merged
2010-12-16, by paulson
made sml/nj happy
2010-12-16, by paulson
removing file refute_isar.ML that was missed in 4006f5c3f421
2010-12-16, by bulwahn
added nitpick to mutabelle script
2010-12-16, by bulwahn
reactivating nitpick in Mutabelle
2010-12-16, by bulwahn
more appropriate closures for static evaluation
2010-12-16, by haftmann
more uniform naming
2010-12-16, by haftmann
merged
2010-12-16, by haftmann
merged
2010-12-15, by haftmann
updated generated files
2010-12-15, by haftmann
simplified evaluation function names
2010-12-15, by haftmann
turned simp_trace_depth_limit into a configuration option
2010-12-16, by boehmes
add notsqsubseteq syntax
2010-12-15, by huffman
show: display goal refinement rule as "state", to avoid odd Output.urgent_message and make its association with the goal more explicit;
2010-12-15, by wenzelm
make sure errors generated in a thread don't vanish in cyberspace (e.g., when invoking Sledgehammer with unknown facts)
2010-12-15, by blanchet
merged
2010-12-15, by bulwahn
adding postprocessing for maps in term construction of quickcheck; fixed check_all_option definition
2010-12-15, by bulwahn
added enum_term_of to correct present nested functions
2010-12-15, by bulwahn
adding postprocessing for sets in term construction of quickcheck
2010-12-15, by bulwahn
merged
2010-12-15, by boehmes
fixed trigger inference: testing if a theorem already has a trigger was too strict;
2010-12-15, by boehmes
fixed checking and translation of weights (previously, weights occurring in terms were rejected, and weight numbers were unintended translated into Vars)
2010-12-15, by boehmes
the functions term_of and prop_of are also needed in earlier stages, not only for Z3 proof reconstruction, so they really belong in SMT_Utils
2010-12-15, by boehmes
facilitate debugging
2010-12-15, by blanchet
merged
2010-12-15, by wenzelm
clean up fudge factors a little bit
2010-12-15, by blanchet
added weights to SMT problems
2010-12-15, by blanchet
move facts supplied with "add:" to the front, so that they get a better weight (SMT)
2010-12-15, by blanchet
beautify MacLaurin proofs; make better use of DERIV_intros
2010-12-15, by hoelzl
workaround for bug in weight handling -- sometimes numerals got replaced by Vars and this confused the weight extractor
2010-12-15, by blanchet
avoid ML structure aliases (especially single-letter abbreviations);
2010-12-15, by wenzelm
eliminated dead code;
2010-12-15, by wenzelm
more correct ML snippets that are unchecked;
2010-12-15, by wenzelm
merged
2010-12-15, by paulson
Added two theorems about the concept of range. Tidied up the comments.
2010-12-15, by paulson
honor "overlord" option for SMT solvers as well and don't pass "ext" to them
2010-12-15, by blanchet
make Sledgehammer's relevance filter include the "ext" rule when appropriate
2010-12-15, by blanchet
tuning
2010-12-15, by blanchet
tuning
2010-12-15, by blanchet
added support for "type_sys" option to Mirabelle
2010-12-15, by blanchet
honor "metisFT" in Mirabelle
2010-12-15, by blanchet
make "full_types" take precedence over "type_sys"
2010-12-15, by blanchet
crank up Metis's timeout for SMT solvers, since users love Metis
2010-12-15, by blanchet
generate a "using [[smt_solver = ...]]" command if a proof is found by another SMT solver than the current one, to ensure it's also used for reconstruction
2010-12-15, by blanchet
make sure first-order occurrences of "False" and "True" are handled correctly -- this broke when adding proper support for higher-order occurrences
2010-12-15, by blanchet
consider "finite" overloaded in "precise_overloaded_args" mode
2010-12-15, by blanchet
added timeout max for remote server invocation
2010-12-15, by blanchet
fix translation of higher-order equality ("fequal") if "precise_overloaded_args" is "true"
2010-12-15, by blanchet
fix Vampire parsing problem
2010-12-15, by blanchet
improve partially tagged encoding by adding a helper fact that coalesces consecutive "ti" tags
2010-12-15, by blanchet
example tuning
2010-12-15, by blanchet
remove at most one double negation -- any other double negations are part of some higher-order reasoning and should be left alone, cf. "HO_Reas.thy"
2010-12-15, by blanchet
weaken the "expect" flag so that it doesn't trigger errors if a prover is not installed
2010-12-15, by blanchet
added example to exercise higher-order reasoning with Sledgehammer and Metis
2010-12-15, by blanchet
added Sledgehammer support for higher-order propositional reasoning
2010-12-15, by blanchet
add Metis support for higher-order propositional reasoning
2010-12-15, by blanchet
implemented partially-typed "tags" type encoding
2010-12-15, by blanchet
implemented "no_types" encoding, which is too unsound to be useful but can come in handy for evaluations
2010-12-15, by blanchet
implemented new type system encoding "overload_args", which is more lightweight than "const_args" (the unsound default) and hopefully almost as sound
2010-12-15, by blanchet
tuning: unused var
2010-12-15, by blanchet
added "type_sys" option to Sledgehammer
2010-12-15, by blanchet
merged
2010-12-15, by boehmes
updated SMT certificates
2010-12-15, by boehmes
fixed proof reconstruction for lambda-lifted problems (which broke when the lambda-lifting code was changed to operate on terms instead of on theorems)
2010-12-15, by boehmes
adapted the Z3 proof parser to recent changes in Z3's proof format;
2010-12-15, by boehmes
also show function definitions for higher-order free variables in Z3 models
2010-12-15, by boehmes
always add pair rules and function update rules automatically (Boogie provides pairs and function update as built-in concepts and does not generate background axioms for them)
2010-12-15, by boehmes
re-implemented eta-expansion, lambda-lifting, and explicit application on terms (exploiting the control over the term structure);
2010-12-15, by boehmes
re-ordered SMT normalization code (eta-normalization, lambda abstractions and partial functions will be dealt with on the term level);
2010-12-15, by boehmes
added option to enable trigger inference;
2010-12-15, by boehmes
moved SMT classes and dictionary functions to SMT_Utils
2010-12-15, by boehmes
tuned
2010-12-15, by boehmes
rewrite Z3 model equations one-by-one (the previous approach led to loss of information)
2010-12-15, by boehmes
added option to modify the random seed of SMT solvers
2010-12-15, by boehmes
adding an Isar version of the MacLaurin theorem from some students' work in 2005
2010-12-15, by bulwahn
Admin/contributed_components tries to formalize compatibility with external components (for use e.g. by testing tools), guessing from the content of TUM contrib_devel directory
2010-12-14, by krauss
separated dictionary weakning into separate type
2010-12-13, by haftmann
eliminated dest_all_all_ctx
2010-12-13, by krauss
private term variant of Variable.focus
2010-12-13, by krauss
adding an executable THE operator on finite types
2010-12-13, by bulwahn
tuned headers
2010-12-12, by krauss
added signature;
2010-12-12, by krauss
add HOLCF library theories with cpo/predomain instances for HOL types
2010-12-11, by huffman
xsymbol notation for powerdomain types
2010-12-11, by huffman
new powerdomain lemmas
2010-12-11, by huffman
made smlnj happy
2010-12-11, by krauss
merged
2010-12-10, by haftmann
moved most fundamental lemmas upwards
2010-12-10, by haftmann
setting finite_type_size to 1 in mutabelle_extra
2010-12-10, by bulwahn
adding check_all instances for a few more finite types in smallcheck
2010-12-10, by bulwahn
removing unneccassary sort constraints
2010-12-10, by bulwahn
made smlnj happy
2010-12-10, by krauss
merged
2010-12-09, by haftmann
tuned names
2010-12-09, by haftmann
dictionary constants must permit explicit weakening of classes;
2010-12-09, by haftmann
tracing of term to be evaluated
2010-12-09, by haftmann
merged
2010-12-09, by hoelzl
use SUPR_ and INFI_apply instead of SUPR_, INFI_fun_expand
2010-12-08, by hoelzl
integral over setprod
2010-12-08, by hoelzl
cleanup bijectivity btw. product spaces and pairs
2010-12-08, by hoelzl
compile
2010-12-09, by blanchet
lower fudge factor
2010-12-08, by blanchet
reword error message
2010-12-08, by blanchet
less
more
|
(0)
-30000
-10000
-3000
-1000
-480
+480
+1000
+3000
+10000
+30000
tip