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.
tuned subsubsection names in Quickcheck_Narrowing
2011-03-14, by bulwahn
tuned exhaustive generator compilation; added narrowing generator compilation; removed exec as does not work properly here (reverting changeset 994d088fbfbc)
2011-03-14, by bulwahn
correcting names in Narrowing_Engine and example theory for Quickcheck_Narrowing
2011-03-14, by bulwahn
renaming series and serial to narrowing in Quickcheck_Narrowing
2011-03-14, by bulwahn
eliminated Bali.thy which takes quite long to merge and does not parallelize so well -- essentially reverting 9b19cbb0af28;
2011-03-13, by wenzelm
tuned headers;
2011-03-13, by wenzelm
eliminated hard tabs;
2011-03-13, by wenzelm
less ambitious isatest;
2011-03-13, by wenzelm
modernized imports (untested!?);
2011-03-13, by wenzelm
files are identified via SHA1 digests -- discontinued ISABELLE_FILE_IDENT;
2011-03-13, by wenzelm
explicit type SHA1.digest;
2011-03-13, by wenzelm
slightly more robust bash exec, which fails on empty executable;
2011-03-13, by wenzelm
cleanup of former settings GHC_PATH, EXEC_GHC, EXEC_OCAML, EXEC_SWIPL, EXEC_YAP -- discontinued implicit detection;
2011-03-13, by wenzelm
some cleanup of old-style settings;
2011-03-13, by wenzelm
clarified ISABELLE_CSDP setting (formerly CSDP_EXE);
2011-03-13, by wenzelm
more conventional Mutabelle settings -- similar to Mirabelle;
2011-03-13, by wenzelm
more basic use of Path.position/File.read;
2011-03-13, by wenzelm
prefer qualified ISABELLE_NEOS_SERVER;
2011-03-13, by wenzelm
proper File.shell_path;
2011-03-13, by wenzelm
more conventional variable name;
2011-03-13, by wenzelm
Path.print is the official way to show file-system paths to users -- note that Path.implode often indicates violation of the abstract datatype;
2011-03-13, by wenzelm
fixed document;
2011-03-13, by wenzelm
isatest: test more external code;
2011-03-13, by wenzelm
tuned headers;
2011-03-13, by wenzelm
allow spaces in executable names;
2011-03-13, by wenzelm
tuned;
2011-03-13, by wenzelm
tuned headers;
2011-03-13, by wenzelm
adapting example file to renaming of the quickcheck tester
2011-03-11, by bulwahn
renaming tester from lazy_exhaustive to narrowing
2011-03-11, by bulwahn
minor corrections for renaming; moved postprocessing of terms to Quickcheck_Common
2011-03-11, by bulwahn
renaming example file correctly
2011-03-11, by bulwahn
adapting Main file generation for Quickcheck_Narrowing
2011-03-11, by bulwahn
adapting Quickcheck_Narrowing and example file to new names
2011-03-11, by bulwahn
renaming LSC_Examples theory to Quickcheck_Narrowing
2011-03-11, by bulwahn
renaming lazysmallcheck ML file to Quickcheck_Narrowing
2011-03-11, by bulwahn
renaming LSC to Quickcheck_Narrowing
2011-03-11, by bulwahn
adaptions in generators using the common functions
2011-03-11, by bulwahn
adding file quickcheck_common to carry common functions of all quickcheck generators
2011-03-11, by bulwahn
adapting record package to renaming of quickcheck's structures
2011-03-11, by bulwahn
moving and renaming lazysmallcheck to narrowing which reflects the characteristical behaviour better
2011-03-11, by bulwahn
correcting dependencies in IsaMakefile
2011-03-11, by bulwahn
renaming signatures and structures; correcting header
2011-03-11, by bulwahn
adapting Quickcheck theory after moving ML files
2011-03-11, by bulwahn
moving quickcheck_generators.ML to Quickcheck directory and renaming it random_generators.ML
2011-03-11, by bulwahn
moving exhaustive_generators.ML to Quickcheck directory
2011-03-11, by bulwahn
correcting dependencies after renaming
2011-03-11, by bulwahn
replacing naming of small by exhaustive
2011-03-11, by bulwahn
renaming smallvalue_generators.ML to exhaustive_generators.ML
2011-03-11, by bulwahn
renaming constants in Quickcheck_Exhaustive theory
2011-03-11, by bulwahn
renaming Smallcheck to Quickcheck_Exhaustive
2011-03-11, by bulwahn
only testing theory LSC_Examples when GHC is installed on the machine
2011-03-11, by bulwahn
increasing timeout of example for counterexample generation
2011-03-11, by bulwahn
adding termination proofs to series functions in LSC; commenting out momentarily unused term refinement functions in LSC
2011-03-11, by bulwahn
adding lazysmallcheck example theory to HOL-ex session
2011-03-11, by bulwahn
adding serial instance of finite_4 in lazysmallcheck; changing code equations for implies
2011-03-11, by bulwahn
replacing strings in generated Code resolves the changing names of Typerep in lazysmallcheck prototype
2011-03-11, by 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
2011-03-11, by bulwahn
adding an example theory for Lazysmallcheck prototype
2011-03-11, by bulwahn
adding Lazysmallcheck prototype to HOL-Library
2011-03-11, by bulwahn
adding files for prototype of lazysmallcheck
2011-03-11, by bulwahn
removing debug message in quickcheck's postprocessor
2011-03-11, by bulwahn
fixing postprocessing; adding a configuration to enable and disable pretty presentation of quickcheck's counterexample
2011-03-11, by bulwahn
renaming dest_plain_fun to dest_fun_upds and adding handling of undefined for postprocessing of quickcheck
2011-03-11, by bulwahn
improving term postprocessing for counterexample presentation in quickcheck
2011-03-11, by bulwahn
tuned
2011-03-11, by bulwahn
finished and tested Z3 proof reconstruction for injective functions;
2011-03-09, by boehmes
improved formula for specialization, to prevent needless specializations -- and removed dead code
2011-03-09, by blanchet
perform no arity check in debug mode so that we get to see the Kodkod problem
2011-03-09, by blanchet
spark_end now joins proofs of VCs before writing *.prv file.
2011-03-04, by berghofe
clarified
2011-03-04, by krauss
produce helpful mira summary for more errors
2011-03-04, by krauss
eliminated prems;
2011-03-04, by wenzelm
eliminated UNITY_Examples.thy which takes quite long to merge and does not parallelize so well -- essentially reverting 3dec57ec3473;
2011-03-03, by wenzelm
tuned proofs -- eliminated prems;
2011-03-03, by wenzelm
merged
2011-03-03, by wenzelm
merged
2011-03-03, by blanchet
don't forget to look for constants appearing only in "need" option -- otherwise we get exceptions in "the_name" later on
2011-03-03, by blanchet
simplified Thy_Info.check_file -- discontinued load path;
2011-03-03, by wenzelm
discontinued legacy load path;
2011-03-03, by wenzelm
re-interpret ProofGeneralPgip.changecwd as Thy_Load.set_master_path, presuming that this is close to the intended semantics;
2011-03-03, by wenzelm
modernized imports;
2011-03-03, by wenzelm
observe standard header format;
2011-03-03, by wenzelm
removed spurious 'unused_thms' (cf. 1a65b780bd56);
2011-03-03, by wenzelm
isatest cygwin-poly-e: new memory management of polyml-svn could be more stable;
2011-03-03, by wenzelm
merged
2011-03-03, by berghofe
merged
2011-03-03, by berghofe
- Made sure that sort_defs is aware of constants introduced by add_type_def
2011-03-03, by berghofe
mention new Nitpick options
2011-03-03, by blanchet
simplify "need" option's syntax
2011-03-03, by blanchet
renamed "preconstr" option "need"
2011-03-03, by blanchet
finally remove upper_bound_finite_set
2011-03-03, by hoelzl
separate settings for afp test
2011-03-03, by kleing
added missing spaces in output
2011-03-02, by blanchet
lower threshold for implicitly using "nitpick_simp" for predicate definitions when "total_consts" is on
2011-03-02, by blanchet
unfold definitions in "preconstrs" option
2011-03-02, by blanchet
robust handling of types occurring in "eval" and "preconstr" options but not in the goal
2011-03-02, by blanchet
make "preconstr" option more robust -- shouldn't throw exceptions
2011-03-02, by blanchet
merged
2011-03-01, by paulson
merged
2011-02-28, by paulson
declare ext [intro]: Extensionality now available by default
2011-02-28, by paulson
merged
2011-02-28, by boehmes
removed dependency on Dense_Linear_Order
2011-02-28, by boehmes
adding function Quickcheck.test_terms to provide checking a batch of terms
2011-02-28, by bulwahn
adding a function to compile a batch of terms for quickcheck with one code generation invocation
2011-02-28, by bulwahn
improved "is_special_eligible_arg" further, by approximating the cardinality of the argument (as is done quite successfully elsewhere)
2011-02-28, by blanchet
made "fixed_is_special_eligible_arg" smarter w.r.t. pairs, and fixed previous unintended behavior because "andalso" ties more tightly than "orelse"
2011-02-28, by blanchet
if "total_consts" is set, report cex's as quasi-genuine
2011-02-28, by blanchet
document new "total_consts" option
2011-02-28, by blanchet
added "total_consts" option
2011-02-28, by blanchet
added a few lemmas by Andreas Lochbihler
2011-02-26, by nipkow
Corrected HOLCF/FOCUS dependency
2011-02-26, by nipkow
Added material by David Trachtenherz
2011-02-26, by nipkow
corrected HOLCF dependency on Nat_Infinity
2011-02-26, by nipkow
got rid of lemma upper_bound_finite_set
2011-02-25, by nipkow
merged
2011-02-25, by nipkow
Some cleaning up
2011-02-25, by nipkow
updated generated files
2011-02-25, by krauss
fixed manual (rule no longer exists)
2011-02-25, by krauss
removed support for tail-recursion from function package (now implemented by partial_function)
2011-02-25, by krauss
reactivate time measurement (partly reverting c27b0b37041a);
2011-02-25, by krauss
less
more
|
(0)
-30000
-10000
-3000
-1000
-120
+120
+1000
+3000
+10000
+30000
tip