Mercurial
Mercurial
>
repos
>
isabelle
/ graph
summary
|
shortlog
|
changelog
| graph |
tags
|
bookmarks
|
branches
|
files
|
gz
|
help
less
more
|
(0)
-30000
-10000
-3000
-1000
-240
+240
+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.
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
implicitly call the minimizer for SMT solvers that don't return an unsat core
2010-12-08, by blanchet
renamings
2010-12-08, by blanchet
moved function to later module
2010-12-08, by blanchet
clarified terminology
2010-12-08, by blanchet
split "Sledgehammer" module into two parts, to resolve forthcoming dependency problems
2010-12-08, by blanchet
if only finite types and no real datatypes occur in the quantifiers only enumerate cardinality not size in quickcheck
2010-12-08, by bulwahn
adding a smarter enumeration scheme for finite functions
2010-12-08, by bulwahn
merged
2010-12-08, by haftmann
work around problems with eta-expansion of equations
2010-12-08, by haftmann
bot comes before top, inf before sup etc.
2010-12-08, by haftmann
tuned
2010-12-08, by haftmann
nice syntax for lattice INFI, SUPR;
2010-12-08, by haftmann
NEWS
2010-12-08, by haftmann
adding more efficient implementations for quantifiers in Enum
2010-12-08, by bulwahn
improving the mutabelle script
2010-12-08, by bulwahn
primitive definitions of bot/top/inf/sup for bool and fun are named with canonical suffix `_def` rather than `_eq`;
2010-12-08, by haftmann
primitive definitions of bot/top/inf/sup for bool and fun are named with canonical suffix `_def` rather than `_eq`
2010-12-08, by haftmann
hide popular names R and B
2010-12-08, by haftmann
built-in numbers are also built-in terms
2010-12-08, by boehmes
be more flexible: store SMT built-in symbols in generic contexts (not in theory contexts)
2010-12-08, by boehmes
merged
2010-12-07, by haftmann
more concise case names; proved extensionality
2010-12-07, by haftmann
name filter operation just filter (c.f. List.filter and list comprehension syntax)
2010-12-07, by haftmann
tuned whitespace
2010-12-07, by haftmann
eliminated some hard tabulators (deprecated);
2010-12-07, by wenzelm
pass constant arguments to the built-in check function, cf. d2b1fc1b8e19
2010-12-07, by blanchet
merged
2010-12-07, by boehmes
updated SMT certificates
2010-12-07, by boehmes
reduced unnecessary complexity; improved documentation; tuned
2010-12-07, by boehmes
tuned
2010-12-07, by boehmes
centralized handling of built-in types and constants for bitvectors
2010-12-07, by boehmes
moved smt_word.ML into the directory of the Word library
2010-12-07, by boehmes
centralized handling of built-in types and constants;
2010-12-07, by boehmes
more aggressive unfolding of unknowns in Z3 models
2010-12-06, by boehmes
tuned
2010-12-06, by boehmes
adding a definition for refl_on which is friendly for quickcheck and nitpick
2010-12-07, by bulwahn
merged
2010-12-07, by blanchet
simplify monotonicity code after killing "fin_fun" optimization
2010-12-07, by blanchet
updated Nitpick's documentation w.r.t. finitization
2010-12-07, by blanchet
remove the "fin_fun" optimization in Nitpick -- it was always a hack and didn't help much
2010-12-07, by blanchet
give the inner timeout mechanism a chance, since it gives more precise information to the user
2010-12-07, by blanchet
updated monotonicity calculus w.r.t. set products
2010-12-07, by blanchet
removed needless optimization for image -- there might be cases that benefit from it but there are others where it is clearly evil
2010-12-07, by blanchet
added a hint when the user obviously just forgot a colon after the lemma's name
2010-12-07, by blanchet
simplified special handling of set products
2010-12-07, by blanchet
fix special handling of set products
2010-12-07, by blanchet
use heuristic to determine whether to keep or drop an existing "let" -- and drop all higher-order lets
2010-12-07, by blanchet
merged
2010-12-07, by bulwahn
testing smartly in two dimensions (cardinality and size) in quickcheck
2010-12-07, by bulwahn
load "try" after "Metis" and move "Async_Manager" back to Sledgehammer
2010-12-07, by blanchet
make SML/NJ happy
2010-12-07, by blanchet
merge
2010-12-07, by blanchet
show strings as "s_1" etc. rather than "l_1" etc.
2010-12-06, by blanchet
quiet Metis in "try"
2010-12-06, by blanchet
removed experimental equality checking of closures; acknowledge underapproximation of equality in function name
2010-12-07, by haftmann
add set-union-like syntax for powerdomain bind operators
2010-12-06, by huffman
merged
2010-12-06, by huffman
instance unit :: domain
2010-12-06, by huffman
simplify ideal completion proofs
2010-12-06, by huffman
remove unused lemmas
2010-12-06, by huffman
remove lemma cont_cfun;
2010-12-06, by huffman
rename lub_fun -> is_lub_fun, thelub_fun -> lub_fun
2010-12-06, by huffman
pcpodef no longer generates _defined lemmas, use _bottom_iff lemmas instead
2010-12-06, by huffman
cpodef no longer generates lemma is_lub_foo, since it is redundant with lub_foo
2010-12-06, by huffman
add lemmas lub_APP, lub_LAM
2010-12-06, by huffman
folding on arbitrary Lebesgue integrable functions
2010-12-06, by hoelzl
fixed spelling errors
2010-12-06, by hoelzl
move coercions to appropriate places
2010-12-06, by hoelzl
it is known as the extended reals, not the infinite reals
2010-12-03, by hoelzl
moved coercion decl. for int
2010-12-06, by nipkow
adapting copied bash code in mutabelle script
2010-12-06, by bulwahn
more correct NEWS;
2010-12-06, by wenzelm
merged
2010-12-06, by wenzelm
fix monotonicity type of None
2010-12-06, by blanchet
compile
2010-12-06, by blanchet
introduced hack to exploit the symmetry of equality in monotonicity calculus
2010-12-06, by blanchet
cleanup example
2010-12-06, by blanchet
add more flexibility to the monotonicity calculus: instead of hardcoding F-arrows, also allow G-arrows, simulating applications of the Sub rule
2010-12-06, by blanchet
fixed bug in monotonicity solution display, whereby the polarity of literals was ignored
2010-12-06, by blanchet
improve precision of forall in constancy part of the monotonicity calculus
2010-12-06, by blanchet
added some missing well-annotatedness constraints to monotonicity calculus
2010-12-06, by blanchet
more work on the monotonicity evaluation driver
2010-12-06, by blanchet
improve precision of finite functions in monotonicity calculus
2010-12-06, by blanchet
added ML code for testing entire theories for monotonicity
2010-12-06, by blanchet
use ML SAT solvers up to a certain time limit, then switch to faster solvers with a timeout -- this becomes necessary with the new, more powerful monotonicity calculus
2010-12-06, by blanchet
added examples to exercise new monotonicity code
2010-12-06, by blanchet
fixed quantifier handling of new monotonicity calculus
2010-12-06, by blanchet
tune parentheses and indentation
2010-12-06, by blanchet
proper handling of frames for connectives in monotonicity calculus
2010-12-06, by blanchet
tune indentation
2010-12-06, by blanchet
removed old baggage from monotonicity calculus -- the "calculus" option didn't really work anyway because of on-the-fly simplifications
2010-12-06, by blanchet
implemented All rules from new monotonicity calculus
2010-12-06, by blanchet
fixed bug in clause handling in monotonicity code, whereby the unsound rule False | x <--> False was used to simplify constraints
2010-12-06, by blanchet
started implementing the new monotonicity rules for application
2010-12-06, by blanchet
implemented connectives in new monotonicity calculus
2010-12-06, by blanchet
added "Neq" operator to monotonicity inference module
2010-12-06, by blanchet
started implementing connectives in new monotonicity calculus
2010-12-06, by blanchet
more work on frames in the new monotonicity calculus
2010-12-06, by blanchet
support 3 monotonicity calculi in one and fix soundness bug
2010-12-06, by blanchet
tuning
2010-12-06, by blanchet
proper handling of assignment disjunctions vs. conjunctions
2010-12-06, by blanchet
adapt monotonicity code to four annotation types
2010-12-06, by blanchet
more monotonicity tuning
2010-12-06, by blanchet
tuning
2010-12-06, by blanchet
added frame component to Gamma in monotonicity calculus
2010-12-06, by blanchet
use boolean pair to encode annotation, which may now take four values
2010-12-06, by blanchet
started generalizing monotonicity code to accommodate new calculus
2010-12-06, by blanchet
merged
2010-12-06, by blanchet
handle "max_relevant" uniformly
2010-12-06, by blanchet
honor the default max relevant facts setting from the SMT solvers in Sledgehammer
2010-12-06, by blanchet
have SMT solvers report the number of facts that they should have by default in Sledgehammer -- the information might not seem to belong there but it also belongs nowhere else, for how is Sledgehammer to know how different solvers deal with hundreds of facts?
2010-12-06, by blanchet
return all facts for CVC3 and Yices, since there is no proof parsing / unsat core extraction
2010-12-06, by blanchet
trust SMT filter's timeout -- nested timeouts seem to be at the origin of spontaneous Interrupt exceptions in some cases
2010-12-06, by blanchet
reraise interrupt exceptions
2010-12-06, by blanchet
[mq]: sledge_binary_minimizer
2010-12-06, by blanchet
correcting usage documentation in mirabelle tool
2010-12-06, by bulwahn
adding mutabelle as a component and an isabelle tool to be used in regression testing
2010-12-06, by bulwahn
commenting out sledgehammer_mtd in Mutabelle
2010-12-06, by bulwahn
removing declaration in quickcheck to really enable exhaustive testing
2010-12-06, by bulwahn
adding timeout to try invocation in mutabelle
2010-12-06, by bulwahn
adding filtering, sytactic welltyping, and sledgehammer method in mutabelle
2010-12-06, by bulwahn
replace `type_mapper` by the more adequate `type_lifting`
2010-12-06, by haftmann
moved bootstrap of type_lifting to Fun
2010-12-06, by haftmann
replace `type_mapper` by the more adequate `type_lifting`
2010-12-06, by haftmann
avoid explicit encoding -- acknowledge UTF-8 as global default and Isabelle/jEdit preference of UTF-8-Isabelle;
2010-12-06, by wenzelm
IsabelleText font: include Cyrillic, Hebrew, Arabic from DejaVu Sans 2.32;
2010-12-05, by wenzelm
command 'notepad' replaces former 'example_proof';
2010-12-05, by wenzelm
prefer 'notepad' over 'example_proof';
2010-12-05, by wenzelm
merged
2010-12-05, by haftmann
more intimate definition of fold_list / fold_once in terms of fold
2010-12-04, by haftmann
canonical fold signature
2010-12-04, by haftmann
formal notepad without any result;
2010-12-04, by wenzelm
added Syntax.default_root;
2010-12-04, by wenzelm
eliminated obsolete Token.Malformed -- subsumed by Token.Error;
2010-12-04, by wenzelm
tuned @{datatype} using Syntax.pretty_priority (NB: postfix type application yields Syntax.max_pri, so arguments in prefix application require higher priority);
2010-12-04, by wenzelm
added Syntax.pretty_priority;
2010-12-04, by wenzelm
merged
2010-12-03, by haftmann
conventional point-free characterization of rsp_fold
2010-12-03, by haftmann
replaced memb by existing List.member
2010-12-03, by haftmann
explicit type constraint;
2010-12-03, by haftmann
tuned proposition
2010-12-03, by haftmann
lemma multiset_of_rev
2010-12-03, by haftmann
lemmas fold_remove1_split and fold_multiset_equiv
2010-12-03, by haftmann
minor tuning for release;
2010-12-03, by wenzelm
source files are always encoded as UTF-8;
2010-12-03, by wenzelm
eliminated fragile HTML.with_charset -- always use utf-8;
2010-12-03, by wenzelm
recoded latin1 as utf8;
2010-12-03, by wenzelm
removed old generated stuff;
2010-12-03, by wenzelm
comment;
2010-12-03, by wenzelm
update documentation
2010-12-03, by blanchet
replace "smt" prover with specific SMT solvers, e.g. "z3" -- whatever the SMT module gives us
2010-12-03, by blanchet
export more information about available SMT solvers
2010-12-03, by blanchet
setup subtyping/coercions once in HOL.thy, but enable it only later via configuration option;
2010-12-03, by wenzelm
use "fold_map" instead of "fold (fn .. => .. (ts @ [t], ..)) .."
2010-12-02, by traytel
updated generated file;
2010-12-03, by wenzelm
removed confusing comments (cf. 500171e7aa59);
2010-12-03, by wenzelm
merged
2010-12-03, by wenzelm
removed outdated lint script
2010-12-03, by haftmann
merged
2010-12-03, by blanchet
compile
2010-12-03, by blanchet
run synchronous Auto Tools in parallel
2010-12-03, by blanchet
really fixed comment (cf. 7abeb749ae99)
2010-12-03, by krauss
theorem names generated by the (rep_)datatype command now have mandatory qualifiers
2010-12-03, by huffman
eliminated unqualified accesses of datatype facts -- it seems like they all of them were unintended
2010-12-03, by krauss
NEWS
2010-12-03, by bulwahn
only instantiate type variable if there exists some in quickcheck
2010-12-03, by bulwahn
fixing comment in library
2010-12-03, by bulwahn
adapting predicate_compile_quickcheck
2010-12-03, by bulwahn
adding a nice definition of Id_on for quickcheck and nitpick
2010-12-03, by bulwahn
adding code equation for finiteness of finite types
2010-12-03, by bulwahn
improving sledgehammer_tactic and adding relevance filtering to the tactic
2010-12-03, by bulwahn
adapting mutabelle
2010-12-03, by bulwahn
adapting SML_Quickcheck to recent changes
2010-12-03, by bulwahn
explaining quickcheck testers in the documentation
2010-12-03, by bulwahn
adapting quickcheck examples
2010-12-03, by bulwahn
improving presentation of quickcheck reports
2010-12-03, by bulwahn
declaring quickcheck testers as default after their setup
2010-12-03, by bulwahn
activating construction of exhaustive testing combinators
2010-12-03, by bulwahn
renamed generator into exhaustive
2010-12-03, by bulwahn
checking if parameter is name of a tester which allows e.g. quickcheck[random]
2010-12-03, by bulwahn
moving iteration of tests to the testers in quickcheck
2010-12-03, by bulwahn
removed dead test_term_small function in quickcheck
2010-12-03, by bulwahn
renamed parameter from generator to tester; quickcheck only applies one tester on invocation
2010-12-03, by bulwahn
adding configuration quickcheck_tester
2010-12-03, by bulwahn
adding smart quantifiers to exhaustive testing
2010-12-03, by bulwahn
adapting mutabelle
2010-12-03, by bulwahn
only handle TimeOut exception if used interactively
2010-12-03, by bulwahn
removed interrupt handling that violates Isabelle/ML exception model
2010-12-03, by bulwahn
corrected indentation
2010-12-03, by bulwahn
tuned
2010-12-03, by bulwahn
smallvalue_generator are defined quick via oracle or sound via function package
2010-12-03, by bulwahn
adding shorter output syntax for the finite types of quickcheck
2010-12-03, by bulwahn
improving readability of Smallcheck theory; adding constant orelse to improve performance of the function package
2010-12-03, by bulwahn
changed order of lemmas to overwrite the general code equation with the nbe-specific one
2010-12-03, by bulwahn
adapt proofs to changed set_plus_image (cf. ee8d0548c148);
2010-12-03, by hoelzl
bash wrapper: terminate only in exceptional case, keep background processes running (e.g. 'thy_deps' or 'display_drafts');
2010-12-03, by wenzelm
updated latex dependencies (cf. 7d88ebdce380);
2010-12-03, by wenzelm
tuned README;
2010-12-03, by wenzelm
isabellesym.sty: eliminated dependency on latin1, to allow documents using utf8 instead;
2010-12-02, by wenzelm
less
more
|
(0)
-30000
-10000
-3000
-1000
-240
+240
+1000
+3000
+10000
+30000
tip