Mercurial
Mercurial
>
repos
>
isabelle
/ graph
summary
|
shortlog
|
changelog
| graph |
tags
|
bookmarks
|
branches
|
files
|
gz
|
help
less
more
|
(0)
-30000
-10000
-3000
-1000
-120
+120
+1000
+3000
+10000
+30000
tip
Find changesets by keywords (author, files, the commit message), revision number or hash, or
revset expression
.
The revision graph only works with JavaScript-enabled browsers.
more 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
less
more
|
(0)
-30000
-10000
-3000
-1000
-120
+120
+1000
+3000
+10000
+30000
tip