Mercurial
Mercurial
>
repos
>
isabelle
/ graph
summary
|
shortlog
|
changelog
| graph |
tags
|
bookmarks
|
branches
|
files
|
gz
|
help
less
more
|
(0)
-30000
-10000
-3000
-1000
-512
+512
+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.
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
proper theory name (cf. e84f82418e09);
2010-12-02, by wenzelm
merged;
2010-12-02, by wenzelm
merged
2010-12-02, by huffman
tuned cpodef code
2010-12-01, by huffman
reformulate lemma preorder.ex_ideal, and use it for typedefs
2010-12-01, by huffman
Prove rel_interior_convex_hull_union (by Grechuck Bogdan).
2010-12-02, by hoelzl
merged
2010-12-02, by haftmann
adapted expected value to more idiomatic numeral representation
2010-12-02, by haftmann
corrected representation for code_numeral numerals
2010-12-02, by haftmann
separate term_of function for integers -- more canonical representation of negative integers
2010-12-02, by haftmann
merged
2010-12-02, by hoelzl
Use coercions in Approximation (by Dmitriy Traytel).
2010-12-02, by hoelzl
more antiquotations;
2010-12-02, by wenzelm
configuration option "show_abbrevs" supersedes print mode "no_abbrevs", with inverted meaning;
2010-12-02, by wenzelm
renamed trace_simp to simp_trace, and debug_simp to simp_debug;
2010-12-02, by wenzelm
merged
2010-12-02, by wenzelm
merged
2010-12-02, by hoelzl
generalized simple_functionD
2010-12-02, by hoelzl
Moved theorems to appropriate place.
2010-12-02, by hoelzl
Shorter definition for positive_integral.
2010-12-02, by hoelzl
Move SUP_commute, SUP_less_iff to HOL image;
2010-12-02, by hoelzl
Generalized simple_functionD and less_SUP_iff.
2010-12-01, by hoelzl
Tuned setup for borel_measurable with min, max and psuminf.
2010-12-01, by hoelzl
Replace algebra_eqI by algebra.equality;
2010-12-01, by hoelzl
give the Isabelle proof the benefice of the doubt when the Isabelle theorem has fewer literals than the Metis one -- this makes a difference on lemma "Let (x::'a, y::'a) (inv_image (r::'b * 'b => bool) (f::'a => 'b)) = ((f x, f y) : r)" apply (metis in_inv_image mem_def)
2010-12-02, by blanchet
merged
2010-12-02, by wenzelm
coercions
2010-12-02, by nipkow
merged
2010-12-01, by nipkow
moved activation of coercion inference into RealDef and declared function real a coercion.
2010-12-01, by nipkow
Corrected IsaMakefile
2010-12-01, by hoelzl
merged
2010-12-01, by hoelzl
Updated NEWS
2010-12-01, by hoelzl
More correct make dependencies for HOL-Multivariate_Analysis and HOL-Probability.
2010-12-01, by hoelzl
Support product spaces on sigma finite measures.
2010-12-01, by hoelzl
merged
2010-12-01, by haftmann
use type constructor as name for variable
2010-12-01, by haftmann
optional explicit prefix for type mapper theorems
2010-12-01, by haftmann
file for package tool type_mapper carries the same name as its Isar command
2010-12-01, by haftmann
merged
2010-12-01, by huffman
domain package generates non-authentic syntax rules for parsing only
2010-12-01, by huffman
builtin time bounds (again);
2010-12-02, by wenzelm
tuned;
2010-12-02, by wenzelm
more abstract handling of Time properties;
2010-12-01, by wenzelm
store tooltip-dismiss-delay as Double(seconds);
2010-12-01, by wenzelm
more abstract/uniform handling of time, preferring seconds as Double;
2010-12-01, by wenzelm
merged
2010-12-01, by wenzelm
NEWS
2010-12-01, by haftmann
just one HOLogic.mk_comp;
2010-12-01, by wenzelm
more direct use of binder_types/body_type;
2010-12-01, by wenzelm
tuned;
2010-12-01, by wenzelm
simplified HOL.eq simproc matching;
2010-12-01, by wenzelm
tuned;
2010-12-01, by wenzelm
just one Term.dest_funT;
2010-12-01, by wenzelm
activate subtyping/coercions in theory Complex_Main;
2010-12-01, by wenzelm
simplified equality on pairs of types;
2010-12-01, by wenzelm
more precise dependencies;
2010-12-01, by wenzelm
two-staged architecture for subtyping;
2010-11-29, by traytel
merged
2010-11-30, by huffman
change cpodef-generated cont_Rep rules to cont2cont format
2010-11-30, by huffman
internal domain package proofs use cont2cont simproc instead of a fixed list of cont rules
2010-11-30, by huffman
remove gratuitous semicolons from ML code
2010-11-30, by huffman
add continuity lemma for List.map
2010-11-30, by huffman
simplify predomain instances
2010-11-30, by huffman
merged
2010-11-30, by boehmes
split up Z3 models into constraints on free variables and constant definitions;
2010-11-30, by boehmes
code preprocessor setup for numerals on word type;
2010-11-30, by haftmann
merged
2010-11-30, by haftmann
adaptions to changes in Equiv_Relation.thy
2010-11-30, by haftmann
adapted fragile proof
2010-11-30, by haftmann
adaptions to changes in Equiv_Relation.thy; prefer primrec if possible
2010-11-30, by haftmann
adaptions to changes in Equiv_Relation.thy
2010-11-30, by haftmann
merged
2010-11-30, by haftmann
more systematic and compact proofs on type relation operators using natural deduction rules
2010-11-30, by haftmann
adapted proofs to slightly changed definitions of congruent(2)
2010-11-30, by haftmann
reorienting iff in Quotient_rel prevents simplifier looping;
2010-11-29, by haftmann
replaced slightly odd locale congruent2 by plain definition
2010-11-29, by haftmann
replaced slightly odd locale congruent by plain definition
2010-11-29, by haftmann
equivI has replaced equiv.intro
2010-11-29, by haftmann
moved generic definitions about (partial) equivalence relations from Quotient to Equiv_Relations;
2010-11-29, by haftmann
moved generic definitions about relations from Quotient.thy to Predicate;
2010-11-29, by haftmann
moved generic definitions about (partial) equivalence relations from Quotient to Equiv_Relations;
2010-11-29, by haftmann
simplify proof of LIMSEQ_unique
2010-11-30, by huffman
use new 'file' antiquotation for reference to Dedekind_Real.thy
2010-11-30, by huffman
merged
2010-11-30, by huffman
instance list :: (discrete_cpo) discrete_cpo;
2010-11-29, by huffman
merged
2010-11-30, by boehmes
also support higher-order rules for Z3 proof reconstruction
2010-11-29, by boehmes
merged
2010-11-29, by wenzelm
less ghc-specific pragma
2010-11-29, by haftmann
tuned
2010-11-29, by haftmann
updated generated files;
2010-11-29, by wenzelm
added document antiquotation @{file};
2010-11-29, by wenzelm
Parse.liberal_name for document antiquotations and attributes;
2010-11-28, by wenzelm
ML results: enter before printing (cf. Poly/ML SVN 1218);
2010-11-28, by wenzelm
merged
2010-11-28, by wenzelm
merged
2010-11-28, by huffman
merged
2010-11-28, by huffman
change match_bottom_simps to produce if-then-else, making more uses of bottom-patterns work with fixrec
2010-11-28, by huffman
add lemma cont2cont_if_bottom
2010-11-27, by huffman
added Parse.literal_fact with proper inner_syntax markup (source position);
2010-11-28, by wenzelm
tuned signature;
2010-11-28, by wenzelm
less frequent sidekick parsing, which is relatively slow;
2010-11-28, by wenzelm
basic setup for bundled Java runtime;
2010-11-28, by wenzelm
updated reference platforms;
2010-11-28, by wenzelm
merged
2010-11-28, by wenzelm
merged
2010-11-28, by nipkow
gave more standard finite set rules simp and intro attribute
2010-11-28, by nipkow
more permissive Isabelle_System.mkdir;
2010-11-28, by wenzelm
added 'syntax_declaration' command;
2010-11-28, by wenzelm
more conventional exception propagation -- taking into account Simple_Thread.fork wrapping;
2010-11-28, by wenzelm
superficial tuning;
2010-11-28, by wenzelm
updated versions;
2010-11-28, by wenzelm
recovered Isabelle2009-2 NEWS -- published part is read-only;
2010-11-28, by wenzelm
follow-up to HOLCF move (cf. 0437dbc127b3, 04d44a20fccf);
2010-11-28, by wenzelm
removed HOLCF for now as explicit component
2010-11-28, by krauss
fix cut-and-paste errors for HOLCF entries in IsaMakefile
2010-11-27, by huffman
update web description of HOLCF;
2010-11-27, by huffman
remove HOLCF from build script, since it no longer works
2010-11-27, by huffman
moved directory src/HOLCF to src/HOL/HOLCF;
2010-11-27, by huffman
merged
2010-11-27, by huffman
rename Pcpodef.thy to Cpodef.thy;
2010-11-27, by huffman
renamed several HOLCF theorems (listed in NEWS)
2010-11-27, by huffman
rename cpodef theorems: lub_foo -> is_lub_foo, thelub_foo -> lub_foo
2010-11-27, by huffman
rename rep_contlub lemmas to rep_lub
2010-11-27, by huffman
rename function 'match_UU' to 'match_bottom'
2010-11-27, by huffman
rename function 'strict' to 'seq', which is its name in Haskell
2010-11-27, by huffman
merged
2010-11-27, by haftmann
merged
2010-11-27, by haftmann
typscheme with signatures is inappropriate when building empty certificate;
2010-11-27, by haftmann
merged
2010-11-27, by haftmann
merged
2010-11-27, by haftmann
corrected: use canonical variables of type scheme uniformly
2010-11-27, by haftmann
tuned
2010-11-27, by haftmann
merged
2010-11-26, by haftmann
consider sort constraints for datatype constructors when constructing the empty equation certificate;
2010-11-26, by haftmann
tuned example
2010-11-26, by haftmann
merged
2010-11-27, by wenzelm
updated generated documents
2010-11-27, by haftmann
added equation for Queue;
2010-11-27, by haftmann
added evaluation section
2010-11-27, by haftmann
tuned formatting;
2010-11-27, by haftmann
added label
2010-11-27, by haftmann
more thorough process termination (cf. Scala version);
2010-11-27, by wenzelm
prefer Isabelle/ML concurrency elements;
2010-11-27, by wenzelm
removed bash from ML system bootstrap, and past the Secure ML barrier;
2010-11-27, by wenzelm
more proper int wrappers;
2010-11-27, by wenzelm
explicit check for requirement;
2010-11-27, by wenzelm
more basic Isabelle_System.mkdir;
2010-11-27, by wenzelm
tuned;
2010-11-27, by wenzelm
more explicit Isabelle_System operations;
2010-11-27, by wenzelm
prefer Synchronized.var over CRITICAL/Unsynchronized.ref;
2010-11-27, by wenzelm
moved file identification to thy_load.ML (where it is actually used);
2010-11-27, by wenzelm
removed some old settings;
2010-11-27, by wenzelm
recovered global "Isabelle" symlink for isatest (cf. 7f745e4b7cce);
2010-11-27, by wenzelm
merged
2010-11-26, by huffman
remove map function names from domain package theory data
2010-11-26, by huffman
isar-style proof for lemma contI2
2010-11-26, by huffman
remove case combinator for fixrec match type
2010-11-26, by huffman
declare more simp rules for powerdomains
2010-11-26, by huffman
merged;
2010-11-27, by wenzelm
merged
2010-11-26, by haftmann
strict forall2
2010-11-26, by haftmann
nbe decides equality of abstractions by extensionality
2010-11-26, by haftmann
eliminated some generated comments;
2010-11-26, by wenzelm
merged
2010-11-26, by wenzelm
merged
2010-11-26, by haftmann
keep type variable arguments of datatype constructors in bookkeeping
2010-11-26, by haftmann
document changes in Nitpick and MESON/Metis
2010-11-26, by blanchet
renamed "trace_me{son,tis}" and "verbose_metis" to have the name of the tool first
2010-11-26, by blanchet
put facts found by SMT solver in alphabetical order and omit chained facts, as was done already for ATP proofs
2010-11-26, by blanchet
make two copies (!) of Library.UnequalLengths coincide with ListPair.UnequalLengths;
2010-11-26, by wenzelm
just one version of fold_rev2;
2010-11-26, by wenzelm
explicit use of unprefix;
2010-11-26, by wenzelm
keep private things private, without comments;
2010-11-26, by wenzelm
eliminated some clones of eq_list;
2010-11-26, by wenzelm
merged
2010-11-26, by nipkow
new lemma
2010-11-26, by nipkow
lemma trans_sym allows single-step "normalization" in Isar, e.g. via moreover/ultimately;
2010-11-26, by wenzelm
prefer non-classical eliminations in Pure reasoning, notably "rule" steps;
2010-11-26, by wenzelm
discontinued global "Isabelle" symlink, to make each distribution even more self-contained;
2010-11-26, by wenzelm
more correct spelling;
2010-11-26, by wenzelm
globbing constant expressions use more idiomatic underscore rather than star
2010-11-26, by haftmann
globbing constant expressions use more idiomatic underscore rather than star;
2010-11-26, by haftmann
datatype constructor glob for code_reflect
2010-11-26, by haftmann
merged
2010-11-26, by haftmann
merged
2010-11-26, by haftmann
merged
2010-11-25, by haftmann
toplevel deresolving for flat module name space
2010-11-25, by haftmann
merged
2010-11-26, by hoelzl
Move some missing lemmas from Andrei Popescus 'Ordinals and Cardinals' AFP entry to the HOL-image.
2010-11-23, by hoelzl
Replace surj by abbreviation; remove surj_on.
2010-11-22, by hoelzl
adjust Sledgehammer/SMT fudge factor
2010-11-26, by blanchet
clarified Par_List.managed_results, with explicit propagation of outermost physical interrupt to forked futures (e.g. to make timeout apply here as expected and prevent zombies);
2010-11-25, by wenzelm
merge
2010-11-25, by blanchet
cosmetics
2010-11-25, by blanchet
eta-reduce on the fly to prevent an exception
2010-11-25, by blanchet
merged
2010-11-25, by nipkow
Added the simplest finite Ramsey theorem
2010-11-25, by nipkow
reverted c059d550afec -- the triviality check had apparently nothing to do with spontaneous Interrupt exceptions
2010-11-25, by blanchet
set Metis option on correct context, lest it be ignored
2010-11-25, by blanchet
make "debug" mode of Sledgehammer/SMT more liberal
2010-11-25, by blanchet
fix check for builtinness of 0 and 1 -- these aren't functions
2010-11-25, by blanchet
added "no_atp" for fact that confuses the SMT normalizer and that doesn't help ATPs anyway
2010-11-25, by blanchet
document requirement on theory import
2010-11-24, by blanchet
corrected abd4e7358847 where SOMEthing went utterly wrong
2010-11-24, by haftmann
merged
2010-11-24, by boehmes
swap names for built-in tester functions (to better reflect the intuition of what they do);
2010-11-24, by boehmes
instantiate elimination rules (reduces number of quantified variables, and makes such theorems better amenable for SMT solvers)
2010-11-24, by boehmes
more precise error handling in Sledgehammer/SMT for Z3 and remote SMT provers
2010-11-24, by blanchet
removing Enum.in_enum from the claset
2010-11-24, by bulwahn
merged
2010-11-24, by boehmes
be more precise: only treat constant 'distinct' applied to an explicit list as built-in
2010-11-24, by boehmes
be more liberal in reconstructing congruences from Z3 (sometimes the symmetric version of a premise is needed)
2010-11-24, by boehmes
announcing some latest change (d40b347d5b0b)
2010-11-24, by bulwahn
merged
2010-11-23, by blanchet
more precise characterization of built-in constants "number_of", "0", and "1"
2010-11-23, by blanchet
merged
2010-11-23, by haftmann
merged
2010-11-22, by haftmann
adhere established Collect/mem convention more closely
2010-11-22, by haftmann
merged
2010-11-22, by haftmann
replaced misleading Fset/fset name -- these do not stand for finite sets
2010-11-22, by haftmann
renamed slightly ambivalent crel to effect
2010-11-22, by haftmann
disable triviality checking -- it might be the source of the spurious Interrupt exceptions that make it almost impossible to run Judgement Day
2010-11-23, by blanchet
more precise error handling for Z3;
2010-11-23, by blanchet
use "Thm.transfer" in Sledgehammer to prevent theory merger issues in "SMT_Solver.smt_filter" later on
2010-11-23, by blanchet
make Mirabelle take into consideration whether the SMT solver proof should be reconstructed with Metis or SMT
2010-11-23, by blanchet
try Metis to reconstruct SMT proofs, to increase success rate and reduce dependency on (often remote) SMT solvers or certificates
2010-11-23, by blanchet
added "verbose" option to Metis to shut up its warnings if necessary
2010-11-23, by blanchet
added support for quantifier weight annotations
2010-11-22, by boehmes
share and use more utility functions;
2010-11-22, by boehmes
added prove reconstruction for injective functions;
2010-11-22, by boehmes
generous timeout gives more breath in parallel run on less luxury machines
2010-11-22, by haftmann
adding setup for exhaustive testing in example file
2010-11-22, by bulwahn
hiding enum
2010-11-22, by bulwahn
adapting example in Predicate_Compile_Examples
2010-11-22, by bulwahn
hiding the constants
2010-11-22, by bulwahn
improving function is_iterable in quickcheck
2010-11-22, by bulwahn
adding temporary options to the quickcheck examples
2010-11-22, by bulwahn
adapting the quickcheck examples
2010-11-22, by bulwahn
adding AFP tests to Mutabelle_Extra; adopting mutabelle to recent quickcheck changes; filtering strange mutants; adding solvers to mutabelle; restructuring mutabelle
2010-11-22, by bulwahn
adding code equations for EX1 on finite types
2010-11-22, by bulwahn
adding code equation for function equality; adding some instantiations for the finite types
2010-11-22, by bulwahn
adding Enum to HOL-Main image and removing it from HOL-Library
2010-11-22, by bulwahn
moving Enum theory from HOL/Library to HOL
2010-11-22, by bulwahn
splitting test_goal function in two functions; exporting new configurations in quickcheck; iterations depend on generator_name in quickcheck
2010-11-22, by bulwahn
adding prototype for finite_type instantiations
2010-11-22, by bulwahn
adding option finite_types to quickcheck
2010-11-22, by bulwahn
adding test cases for smallcheck and adding examples where exhaustive testing is more successful
2010-11-22, by bulwahn
changed old-style quickcheck configurations to new Config.T configurations
2010-11-22, by bulwahn
adding temporary function test_test_small to Quickcheck
2010-11-22, by bulwahn
added useful function map_context_result to signature
2010-11-22, by bulwahn
moving the error handling to the right scope in smallvalue_generators
2010-11-22, by bulwahn
removing clone from function package and using the clean interface from Function_Relation instead
2010-11-22, by bulwahn
adding function generation to SmallCheck; activating exhaustive search space testing
2010-11-22, by bulwahn
adding dummy definition for Code_Evaluation.Abs and hiding constants App less strict
2010-11-22, by bulwahn
generalized ensure_random_datatype to ensure_sort_datatype
2010-11-22, by bulwahn
renaming quickcheck generator code to random
2010-11-22, by bulwahn
ported sledgehammer_tactic to current development version
2010-11-22, by bulwahn
adding dependencies to IsaMakefile; adding sledgehammer_tactic in Mirabelle_Test
2010-11-22, by bulwahn
adding files to use sledgehammer as a tactic for non-interactive use
2010-11-22, by bulwahn
adding birthday paradoxon from some abandoned drawer
2010-11-22, by bulwahn
adding extensional function spaces to the FuncSet library theory
2010-11-22, by bulwahn
tuned
2010-11-22, by haftmann
tuned
2010-11-22, by haftmann
updated explode vs. raw_explode;
2010-11-20, by wenzelm
renamed raw "explode" function to "raw_explode" to emphasize its meaning;
2010-11-20, by wenzelm
total Symbol.explode (cf. 1050315f6ee2);
2010-11-19, by wenzelm
do not export Thy_Load.required, to avoid confusion about the interface;
2010-11-19, by wenzelm
merged
2010-11-19, by huffman
declare adm_chfin [simp]
2010-11-17, by huffman
add lemma cont_fun; remove unused lemma monofun_app
2010-11-17, by huffman
accumulated NEWS updates for HOLCF
2010-11-17, by huffman
section -> subsection
2010-11-17, by huffman
add lemma adm_prod_case
2010-11-17, by huffman
merged
2010-11-19, by paulson
First-order pattern matching: catch a rogue exception (differing numbers of arguments)
2010-11-19, by paulson
eval simp rules for predicate type, simplify primitive proofs
2010-11-19, by haftmann
generalized type
2010-11-19, by haftmann
made smlnj happy
2010-11-19, by haftmann
merged
2010-11-19, by haftmann
proper qualification needed due to shadowing on theory merge
2010-11-18, by haftmann
more appropriate name for property
2010-11-18, by haftmann
mapper for sum type
2010-11-18, by haftmann
mapper for option type
2010-11-18, by haftmann
mapper for list type; map_pair replaces prod_fun
2010-11-18, by haftmann
map_pair replaces prod_fun
2010-11-18, by haftmann
mapper for mulitset type
2010-11-18, by haftmann
mapper for mapping type
2010-11-18, by haftmann
mapper for fset type
2010-11-18, by haftmann
mapper for dlist type
2010-11-18, by haftmann
map_fun combinator in theory Fun
2010-11-18, by haftmann
some updates after 2 years of Mercurial usage;
2010-11-18, by wenzelm
mention Sledgehammer with SMT
2010-11-18, by blanchet
enabled SMT solver in Sledgehammer by default
2010-11-18, by blanchet
merged
2010-11-18, by haftmann
keep variables bound
2010-11-18, by haftmann
remove "Time limit reached" as potential error, because this is sometimes generated for individual slices and not for the entire problem
2010-11-18, by blanchet
merged
2010-11-17, by haftmann
infer variances of user-given mapper operation; proper thm storing
2010-11-17, by haftmann
code eqn for slice was missing; redefined splice with fun
2010-11-17, by nipkow
move strict function type into main HOLCF; instance cfun :: (predomain, domain) domain
2010-11-17, by huffman
merged
2010-11-17, by huffman
typedef (open) unit
2010-11-16, by huffman
add bind_bind rules for powerdomains
2010-11-16, by huffman
merged
2010-11-17, by wenzelm
emerging Isar command interface
2010-11-17, by haftmann
fixed typo
2010-11-17, by haftmann
updated keywords
2010-11-17, by haftmann
ML signature interface
2010-11-17, by haftmann
stub for Isar command interface
2010-11-17, by haftmann
module for functorial mappers
2010-11-17, by haftmann
merged
2010-11-17, by wenzelm
require the b2i file ending in the boogie_open command (for consistency with the theory header)
2010-11-17, by boehmes
use the const antiquotation for constants (this checks that the constant is declared, whereas the more general term antiquotation treats undeclared names as free variable)
2010-11-17, by boehmes
keep input and output files used to communicate with the SMT solver (for debugging purposes mainly)
2010-11-17, by boehmes
add lemmas about powerdomains
2010-11-16, by huffman
declare {upper,lower,convex}_pd_induct as default induction rules
2010-11-16, by huffman
rename 'repdef' to 'domaindef'
2010-11-16, by huffman
refrain from opening Scratch.thy by default, to avoid bombing the editor with old/long theory text;
2010-11-17, by wenzelm
less parentheses, cf. Session.welcome;
2010-11-17, by wenzelm
avoid spam;
2010-11-16, by wenzelm
more robust determination of java executable;
2010-11-16, by wenzelm
init_component: require absolute path (when invoked by user scripts);
2010-11-16, by wenzelm
more explicit explanation of init_component shell function;
2010-11-16, by wenzelm
paranoia export of CLASSPATH, just in case the initial status via allexport is lost due to other scripts;
2010-11-16, by wenzelm
tuned message;
2010-11-16, by wenzelm
post raw messages last, to ensure that result has been handled by session actor already (e.g. to avoid race between Session.session_actor and Session_Dockable.main_actor);
2010-11-16, by wenzelm
more reasonably defaults for typical laptops (2 GB RAM, 2 cores);
2010-11-16, by wenzelm
added forall2 predicate lifter
2010-11-16, by haftmann
merged
2010-11-15, by wenzelm
merged
2010-11-15, by boehmes
renamed SMT failure: Abnormal_Termination is indeed more appropriate than Solver_Crashed
2010-11-15, by boehmes
honour timeouts which are not rounded to full seconds
2010-11-15, by boehmes
better error message
2010-11-15, by blanchet
better error message
2010-11-15, by blanchet
merged
2010-11-15, by wenzelm
cosmetics
2010-11-15, by blanchet
interpret SMT_Failure.Solver_Crashed correctly
2010-11-15, by blanchet
turn on Sledgehammer verbosity so we can track down crashes
2010-11-15, by blanchet
pick up SMT solver crashes and report them to the user/Mirabelle if desired
2010-11-15, by blanchet
merged
2010-11-15, by boehmes
only replace unknowns of type nat with known integer numbers, don't alias unknown values in Z3's counterexamples with known integers
2010-11-15, by boehmes
trace more solver output before raising an exception due to a non-zero return code (avoids truncating potential counterexamples produced by Z3)
2010-11-15, by boehmes
merged
2010-11-15, by bulwahn
ignoring the constant STR in the predicate compiler
2010-11-15, by bulwahn
non-executable source files;
2010-11-15, by wenzelm
eliminated old-style sed in favour of builtin regex matching;
2010-11-15, by wenzelm
more robust treatment of spaces in file names;
2010-11-15, by wenzelm
tuned error messages;
2010-11-15, by wenzelm
merged
2010-11-15, by wenzelm
re-generalized type of option_rel and sum_rel (accident from 2989f9f3aa10)
2010-11-15, by haftmann
re-generalized type of prod_rel (accident from 2989f9f3aa10)
2010-11-15, by haftmann
formal dependency on b2i files
2010-11-15, by boehmes
merged
2010-11-14, by boehmes
check the return code of the SMT solver and raise an exception if the prover failed
2010-11-12, by boehmes
updated README;
2010-11-14, by wenzelm
tuned;
2010-11-14, by wenzelm
cover 'write' as primitive proof command;
2010-11-14, by wenzelm
clarified interact/print state: proof commands are treated as in TTY mode to get full response;
2010-11-14, by wenzelm
somewhat adhoc replacement for 'thus' and 'hence';
2010-11-13, by wenzelm
always print state of proof commands (notably "qed" etc.);
2010-11-13, by wenzelm
simplified message: malformed symbols are fully internalized, i.e. can be printed without crashing;
2010-11-13, by wenzelm
tuned message;
2010-11-13, by wenzelm
proper escape in regex;
2010-11-13, by wenzelm
report malformed symbols;
2010-11-13, by wenzelm
qualified Symbol_Pos.symbol;
2010-11-13, by wenzelm
total Symbol.source;
2010-11-13, by wenzelm
eliminated slightly odd pervasive Symbol_Pos.symbol;
2010-11-13, by wenzelm
treat Unicode "replacement character" (i.e. decoding error) is malformed;
2010-11-13, by wenzelm
simplified/robustified treatment of malformed symbols, which are now fully internalized (total Symbol.explode etc.);
2010-11-13, by wenzelm
tuned;
2010-11-13, by wenzelm
back to quick_and_dirty, which is still practically important since the scheduler does not jump over subproofs;
2010-11-13, by wenzelm
await_cancellation in the main thread, independently of the execution futures, which might get interrupted or be absent after node deletetion;
2010-11-13, by wenzelm
updated README;
2010-11-13, by wenzelm
defensive defaults for more robust experience for new users;
2010-11-12, by wenzelm
merged
2010-11-12, by wenzelm
preliminary support for newer versions of Z3
2010-11-12, by boehmes
turned SMT counterexamples into verbose messages (they had been swallowed before, following the state of smt_trace -- which is off by default), because they might be useful for the user
2010-11-12, by boehmes
let the theory formally depend on the Boogie output
2010-11-12, by boehmes
look for certificates relative to the theory
2010-11-12, by boehmes
dropped numerals from monomorphization blacklist (only particular numerals are builtin, all other numerals should be treated uninterpreted), this blacklist should contain only truely polymorphic builtin constants supported by SMT
2010-11-12, by boehmes
merged
2010-11-12, by huffman
update Theory.requires with new theory name
2010-11-12, by huffman
tuned signatures;
2010-11-12, by wenzelm
never open Unsynchronized;
2010-11-12, by wenzelm
less
more
|
(0)
-30000
-10000
-3000
-1000
-512
+512
+1000
+3000
+10000
+30000
tip