2011-03-11 |
bulwahn |
adding lazysmallcheck example theory to HOL-ex session
|
changeset |
files
|
2011-03-11 |
bulwahn |
adding serial instance of finite_4 in lazysmallcheck; changing code equations for implies
|
changeset |
files
|
2011-03-11 |
bulwahn |
replacing strings in generated Code resolves the changing names of Typerep in lazysmallcheck prototype
|
changeset |
files
|
2011-03-11 |
bulwahn |
changing invocation of ghc from interactive mode to compilation increases the performance of lazysmallcheck by a factor of twenty; changing Integer type to Int reduces by another 50 percent
|
changeset |
files
|
2011-03-11 |
bulwahn |
adding an example theory for Lazysmallcheck prototype
|
changeset |
files
|
2011-03-11 |
bulwahn |
adding Lazysmallcheck prototype to HOL-Library
|
changeset |
files
|
2011-03-11 |
bulwahn |
adding files for prototype of lazysmallcheck
|
changeset |
files
|
2011-03-11 |
bulwahn |
removing debug message in quickcheck's postprocessor
|
changeset |
files
|
2011-03-11 |
bulwahn |
fixing postprocessing; adding a configuration to enable and disable pretty presentation of quickcheck's counterexample
|
changeset |
files
|
2011-03-11 |
bulwahn |
renaming dest_plain_fun to dest_fun_upds and adding handling of undefined for postprocessing of quickcheck
|
changeset |
files
|
2011-03-11 |
bulwahn |
improving term postprocessing for counterexample presentation in quickcheck
|
changeset |
files
|
2011-03-11 |
bulwahn |
tuned
|
changeset |
files
|
2011-03-09 |
boehmes |
finished and tested Z3 proof reconstruction for injective functions;
|
changeset |
files
|
2011-03-09 |
blanchet |
improved formula for specialization, to prevent needless specializations -- and removed dead code
|
changeset |
files
|
2011-03-09 |
blanchet |
perform no arity check in debug mode so that we get to see the Kodkod problem
|
changeset |
files
|
2011-03-04 |
berghofe |
spark_end now joins proofs of VCs before writing *.prv file.
|
changeset |
files
|
2011-03-04 |
krauss |
clarified
|
changeset |
files
|
2011-03-04 |
krauss |
produce helpful mira summary for more errors
|
changeset |
files
|
2011-03-03 |
wenzelm |
eliminated prems;
|
changeset |
files
|
2011-03-03 |
wenzelm |
eliminated UNITY_Examples.thy which takes quite long to merge and does not parallelize so well -- essentially reverting 3dec57ec3473;
|
changeset |
files
|
2011-03-03 |
wenzelm |
tuned proofs -- eliminated prems;
|
changeset |
files
|
2011-03-03 |
wenzelm |
merged
|
changeset |
files
|
2011-03-03 |
blanchet |
merged
|
changeset |
files
|
2011-03-03 |
blanchet |
don't forget to look for constants appearing only in "need" option -- otherwise we get exceptions in "the_name" later on
|
changeset |
files
|
2011-03-03 |
wenzelm |
simplified Thy_Info.check_file -- discontinued load path;
|
changeset |
files
|
2011-03-03 |
wenzelm |
discontinued legacy load path;
|
changeset |
files
|
2011-03-03 |
wenzelm |
re-interpret ProofGeneralPgip.changecwd as Thy_Load.set_master_path, presuming that this is close to the intended semantics;
|
changeset |
files
|
2011-03-03 |
wenzelm |
modernized imports;
|
changeset |
files
|
2011-03-03 |
wenzelm |
observe standard header format;
|
changeset |
files
|
2011-03-03 |
wenzelm |
removed spurious 'unused_thms' (cf. 1a65b780bd56);
|
changeset |
files
|
2011-03-03 |
wenzelm |
isatest cygwin-poly-e: new memory management of polyml-svn could be more stable;
|
changeset |
files
|
2011-03-03 |
berghofe |
merged
|
changeset |
files
|
2011-03-03 |
berghofe |
merged
|
changeset |
files
|
2011-03-03 |
berghofe |
- Made sure that sort_defs is aware of constants introduced by add_type_def
|
changeset |
files
|
2011-03-03 |
blanchet |
mention new Nitpick options
|
changeset |
files
|
2011-03-03 |
blanchet |
simplify "need" option's syntax
|
changeset |
files
|
2011-03-03 |
blanchet |
renamed "preconstr" option "need"
|
changeset |
files
|
2011-03-03 |
hoelzl |
finally remove upper_bound_finite_set
|
changeset |
files
|
2011-03-03 |
kleing |
separate settings for afp test
|
changeset |
files
|
2011-03-02 |
blanchet |
added missing spaces in output
|
changeset |
files
|
2011-03-02 |
blanchet |
lower threshold for implicitly using "nitpick_simp" for predicate definitions when "total_consts" is on
|
changeset |
files
|
2011-03-02 |
blanchet |
unfold definitions in "preconstrs" option
|
changeset |
files
|
2011-03-02 |
blanchet |
robust handling of types occurring in "eval" and "preconstr" options but not in the goal
|
changeset |
files
|
2011-03-02 |
blanchet |
make "preconstr" option more robust -- shouldn't throw exceptions
|
changeset |
files
|
2011-03-01 |
paulson |
merged
|
changeset |
files
|
2011-02-28 |
paulson |
merged
|
changeset |
files
|
2011-02-28 |
paulson |
declare ext [intro]: Extensionality now available by default
|
changeset |
files
|
2011-02-28 |
boehmes |
merged
|
changeset |
files
|
2011-02-28 |
boehmes |
removed dependency on Dense_Linear_Order
|
changeset |
files
|
2011-02-28 |
bulwahn |
adding function Quickcheck.test_terms to provide checking a batch of terms
|
changeset |
files
|
2011-02-28 |
bulwahn |
adding a function to compile a batch of terms for quickcheck with one code generation invocation
|
changeset |
files
|
2011-02-28 |
blanchet |
improved "is_special_eligible_arg" further, by approximating the cardinality of the argument (as is done quite successfully elsewhere)
|
changeset |
files
|
2011-02-28 |
blanchet |
made "fixed_is_special_eligible_arg" smarter w.r.t. pairs, and fixed previous unintended behavior because "andalso" ties more tightly than "orelse"
|
changeset |
files
|
2011-02-28 |
blanchet |
if "total_consts" is set, report cex's as quasi-genuine
|
changeset |
files
|
2011-02-28 |
blanchet |
document new "total_consts" option
|
changeset |
files
|
2011-02-28 |
blanchet |
added "total_consts" option
|
changeset |
files
|
2011-02-26 |
nipkow |
added a few lemmas by Andreas Lochbihler
|
changeset |
files
|
2011-02-26 |
nipkow |
Corrected HOLCF/FOCUS dependency
|
changeset |
files
|
2011-02-26 |
nipkow |
Added material by David Trachtenherz
|
changeset |
files
|
2011-02-26 |
nipkow |
corrected HOLCF dependency on Nat_Infinity
|
changeset |
files
|