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.
adding size as static argument in quickcheck_narrowing compilation
2011-03-18, by bulwahn
modernized specifications;
2011-03-20, by wenzelm
dropped unused structure aliases;
2011-03-20, by wenzelm
tuned;
2011-03-20, by wenzelm
NEWS: structure Timing provides various operations for timing;
2011-03-20, by wenzelm
simplified various cpu_time clones (!): eliminated odd Exn.capture/Exn.release (no need to "stop" timing);
2011-03-20, by wenzelm
pure Timing.timing, without any exception handling;
2011-03-20, by wenzelm
structure Timing: covers former start_timing/end_timing and Output.timeit etc;
2011-03-20, by wenzelm
pervasive cond_timeit;
2011-03-20, by wenzelm
eliminated dead code;
2011-03-20, by wenzelm
parallel preparation of document variants, within separate directories;
2011-03-20, by wenzelm
Present.init/finish/no_document are not thread-safe -- eliminated futile CRITICAL sections;
2011-03-20, by wenzelm
eliminated redundant doc_prefix1;
2011-03-20, by wenzelm
renamed doc_prefix2 to dump_prefix;
2011-03-20, by wenzelm
tuned;
2011-03-20, by wenzelm
tuned terminology for document variants;
2011-03-20, by wenzelm
replaced File.check by specific File.check_file, File.check_dir;
2011-03-20, by wenzelm
tuned;
2011-03-20, by wenzelm
preencode value of "need" selectors in Kodkod bounds as an optimization
2011-03-19, by blanchet
ignore "need" axioms for "nat"-like types
2011-03-19, by blanchet
added "simp:", "intro:", and "elim:" to "try" command
2011-03-18, by blanchet
optimize Kodkod axioms further w.r.t. "need" option
2011-03-18, by blanchet
optimize Kodkod bounds of nat-like datatypes
2011-03-18, by blanchet
more optimizations of bounds for "need"
2011-03-18, by blanchet
optimize Kodkod bounds when "need" is specified
2011-03-18, by blanchet
always destroy constructor patterns, since this seems to be always useful
2011-03-18, by blanchet
reintroduced "show_skolems" option -- useful when too many Skolems are displayed
2011-03-17, by blanchet
reword Nitpick's wording concerning potential counterexamples
2011-03-17, by blanchet
prevent an exception if "card" is empty (e.g., "nitpick [card]")
2011-03-17, by blanchet
add option to function to keep trivial ATP formulas, needed for some experiments
2011-03-17, by blanchet
add option to relevance filter's "all_facts" function to really get all facts (needed for some experiments)
2011-03-17, by blanchet
tuned lemma
2011-03-17, by nipkow
added lemmas
2011-03-16, by nipkow
added lemma
2011-03-15, by nipkow
support non-ground "need" values
2011-03-15, by blanchet
recover Isabelle symlink for public distribution, notably website;
2011-03-15, by wenzelm
standardized headers;
2011-03-14, by wenzelm
merged
2011-03-14, by hoelzl
reworked Probability theory: measures are not type restricted to positive extended reals
2011-03-14, by hoelzl
split Extended_Reals into parts for Library and Multivariate_Analysis
2011-03-14, by hoelzl
lemmas about addition, SUP on countable sets and infinite sums for extreal
2011-03-14, by hoelzl
add infinite sums and power on extreal
2011-03-14, by hoelzl
introduce setsum on extreal
2011-03-14, by hoelzl
use abs_extreal
2011-03-14, by hoelzl
simplified definition of open_extreal
2011-03-14, by hoelzl
use case_product for extrel[2,3]_cases
2011-03-14, by hoelzl
add Extended_Reals from AFP/Lower_Semicontinuous
2011-03-14, by hoelzl
add lemmas for monotone sequences
2011-03-14, by hoelzl
add lemmas for SUP and INF
2011-03-14, by hoelzl
generalize infinite sums
2011-03-14, by hoelzl
moved t2_spaces to HOL image
2011-03-14, by hoelzl
example settings for ISABELLE_GHC, ISABELLE_OCAML, ISABELLE_SWIPL;
2011-03-14, by wenzelm
isatest: fresh copy of settings avoids odd cumulative environment;
2011-03-14, by wenzelm
tuned exhaustive_generators
2011-03-14, by bulwahn
removing definition of cons0; hiding constants in Quickcheck_Narrowing
2011-03-14, by bulwahn
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
less
more
|
(0)
-30000
-10000
-3000
-1000
-120
+120
+1000
+3000
+10000
+30000
tip