hoelzl [Mon, 14 Mar 2011 14:37:46 +0100] rev 41979
lemmas about addition, SUP on countable sets and infinite sums for extreal
hoelzl [Mon, 14 Mar 2011 14:37:45 +0100] rev 41978
add infinite sums and power on extreal
hoelzl [Mon, 14 Mar 2011 14:37:44 +0100] rev 41977
introduce setsum on extreal
hoelzl [Mon, 14 Mar 2011 14:37:42 +0100] rev 41976
use abs_extreal
hoelzl [Mon, 14 Mar 2011 14:37:41 +0100] rev 41975
simplified definition of open_extreal
hoelzl [Mon, 14 Mar 2011 14:37:40 +0100] rev 41974
use case_product for extrel[2,3]_cases
hoelzl [Mon, 14 Mar 2011 14:37:39 +0100] rev 41973
add Extended_Reals from AFP/Lower_Semicontinuous
hoelzl [Mon, 14 Mar 2011 14:37:37 +0100] rev 41972
add lemmas for monotone sequences
hoelzl [Mon, 14 Mar 2011 14:37:36 +0100] rev 41971
add lemmas for SUP and INF
hoelzl [Mon, 14 Mar 2011 14:37:35 +0100] rev 41970
generalize infinite sums
hoelzl [Mon, 14 Mar 2011 14:37:33 +0100] rev 41969
moved t2_spaces to HOL image
wenzelm [Mon, 14 Mar 2011 15:17:10 +0100] rev 41968
example settings for ISABELLE_GHC, ISABELLE_OCAML, ISABELLE_SWIPL;
wenzelm [Mon, 14 Mar 2011 15:13:00 +0100] rev 41967
isatest: fresh copy of settings avoids odd cumulative environment;
bulwahn [Mon, 14 Mar 2011 12:34:12 +0100] rev 41966
tuned exhaustive_generators
bulwahn [Mon, 14 Mar 2011 12:34:11 +0100] rev 41965
removing definition of cons0; hiding constants in Quickcheck_Narrowing
bulwahn [Mon, 14 Mar 2011 12:34:10 +0100] rev 41964
tuned subsubsection names in Quickcheck_Narrowing
bulwahn [Mon, 14 Mar 2011 12:34:10 +0100] rev 41963
tuned exhaustive generator compilation; added narrowing generator compilation; removed exec as does not work properly here (reverting changeset 994d088fbfbc)
bulwahn [Mon, 14 Mar 2011 12:34:09 +0100] rev 41962
correcting names in Narrowing_Engine and example theory for Quickcheck_Narrowing
bulwahn [Mon, 14 Mar 2011 12:34:08 +0100] rev 41961
renaming series and serial to narrowing in Quickcheck_Narrowing
wenzelm [Sun, 13 Mar 2011 23:12:38 +0100] rev 41960
eliminated Bali.thy which takes quite long to merge and does not parallelize so well -- essentially reverting 9b19cbb0af28;
wenzelm [Sun, 13 Mar 2011 22:55:50 +0100] rev 41959
tuned headers;
wenzelm [Sun, 13 Mar 2011 22:24:10 +0100] rev 41958
eliminated hard tabs;
wenzelm [Sun, 13 Mar 2011 21:41:44 +0100] rev 41957
less ambitious isatest;
wenzelm [Sun, 13 Mar 2011 21:21:48 +0100] rev 41956
modernized imports (untested!?);
wenzelm [Sun, 13 Mar 2011 20:56:00 +0100] rev 41955
files are identified via SHA1 digests -- discontinued ISABELLE_FILE_IDENT;
wenzelm [Sun, 13 Mar 2011 20:21:24 +0100] rev 41954
explicit type SHA1.digest;
wenzelm [Sun, 13 Mar 2011 19:27:39 +0100] rev 41953
slightly more robust bash exec, which fails on empty executable;
wenzelm [Sun, 13 Mar 2011 19:16:19 +0100] rev 41952
cleanup of former settings GHC_PATH, EXEC_GHC, EXEC_OCAML, EXEC_SWIPL, EXEC_YAP -- discontinued implicit detection;
determine swipl_version at runtime;
wenzelm [Sun, 13 Mar 2011 17:35:35 +0100] rev 41951
some cleanup of old-style settings;
wenzelm [Sun, 13 Mar 2011 17:28:14 +0100] rev 41950
clarified ISABELLE_CSDP setting (formerly CSDP_EXE);
wenzelm [Sun, 13 Mar 2011 16:52:59 +0100] rev 41949
more conventional Mutabelle settings -- similar to Mirabelle;
wenzelm [Sun, 13 Mar 2011 16:38:54 +0100] rev 41948
more basic use of Path.position/File.read;
wenzelm [Sun, 13 Mar 2011 16:38:14 +0100] rev 41947
prefer qualified ISABELLE_NEOS_SERVER;
wenzelm [Sun, 13 Mar 2011 16:30:02 +0100] rev 41946
proper File.shell_path;
wenzelm [Sun, 13 Mar 2011 16:14:14 +0100] rev 41945
more conventional variable name;
wenzelm [Sun, 13 Mar 2011 16:01:00 +0100] rev 41944
Path.print is the official way to show file-system paths to users -- note that Path.implode often indicates violation of the abstract datatype;
wenzelm [Sun, 13 Mar 2011 15:16:37 +0100] rev 41943
fixed document;
wenzelm [Sun, 13 Mar 2011 15:13:53 +0100] rev 41942
isatest: test more external code;
wenzelm [Sun, 13 Mar 2011 15:10:00 +0100] rev 41941
tuned headers;
wenzelm [Sun, 13 Mar 2011 14:51:38 +0100] rev 41940
allow spaces in executable names;
simplified generated bash scripts;
wenzelm [Sun, 13 Mar 2011 13:57:20 +0100] rev 41939
tuned;
wenzelm [Sun, 13 Mar 2011 13:53:54 +0100] rev 41938
tuned headers;
bulwahn [Fri, 11 Mar 2011 15:21:13 +0100] rev 41937
adapting example file to renaming of the quickcheck tester
bulwahn [Fri, 11 Mar 2011 15:21:13 +0100] rev 41936
renaming tester from lazy_exhaustive to narrowing
bulwahn [Fri, 11 Mar 2011 15:21:13 +0100] rev 41935
minor corrections for renaming; moved postprocessing of terms to Quickcheck_Common
bulwahn [Fri, 11 Mar 2011 15:21:13 +0100] rev 41934
renaming example file correctly
bulwahn [Fri, 11 Mar 2011 15:21:13 +0100] rev 41933
adapting Main file generation for Quickcheck_Narrowing
bulwahn [Fri, 11 Mar 2011 15:21:13 +0100] rev 41932
adapting Quickcheck_Narrowing and example file to new names
bulwahn [Fri, 11 Mar 2011 15:21:13 +0100] rev 41931
renaming LSC_Examples theory to Quickcheck_Narrowing
bulwahn [Fri, 11 Mar 2011 15:21:13 +0100] rev 41930
renaming lazysmallcheck ML file to Quickcheck_Narrowing
bulwahn [Fri, 11 Mar 2011 15:21:13 +0100] rev 41929
renaming LSC to Quickcheck_Narrowing
bulwahn [Fri, 11 Mar 2011 15:21:13 +0100] rev 41928
adaptions in generators using the common functions
bulwahn [Fri, 11 Mar 2011 15:21:13 +0100] rev 41927
adding file quickcheck_common to carry common functions of all quickcheck generators
bulwahn [Fri, 11 Mar 2011 15:21:13 +0100] rev 41926
adapting record package to renaming of quickcheck's structures
bulwahn [Fri, 11 Mar 2011 15:21:13 +0100] rev 41925
moving and renaming lazysmallcheck to narrowing which reflects the characteristical behaviour better
bulwahn [Fri, 11 Mar 2011 15:21:13 +0100] rev 41924
correcting dependencies in IsaMakefile
bulwahn [Fri, 11 Mar 2011 15:21:13 +0100] rev 41923
renaming signatures and structures; correcting header
bulwahn [Fri, 11 Mar 2011 15:21:13 +0100] rev 41922
adapting Quickcheck theory after moving ML files
bulwahn [Fri, 11 Mar 2011 15:21:13 +0100] rev 41921
moving quickcheck_generators.ML to Quickcheck directory and renaming it random_generators.ML
bulwahn [Fri, 11 Mar 2011 15:21:13 +0100] rev 41920
moving exhaustive_generators.ML to Quickcheck directory
bulwahn [Fri, 11 Mar 2011 15:21:13 +0100] rev 41919
correcting dependencies after renaming
bulwahn [Fri, 11 Mar 2011 15:21:13 +0100] rev 41918
replacing naming of small by exhaustive
bulwahn [Fri, 11 Mar 2011 15:21:13 +0100] rev 41917
renaming smallvalue_generators.ML to exhaustive_generators.ML
bulwahn [Fri, 11 Mar 2011 15:21:13 +0100] rev 41916
renaming constants in Quickcheck_Exhaustive theory
bulwahn [Fri, 11 Mar 2011 15:21:12 +0100] rev 41915
renaming Smallcheck to Quickcheck_Exhaustive
bulwahn [Fri, 11 Mar 2011 10:37:45 +0100] rev 41914
only testing theory LSC_Examples when GHC is installed on the machine
bulwahn [Fri, 11 Mar 2011 10:37:43 +0100] rev 41913
increasing timeout of example for counterexample generation
bulwahn [Fri, 11 Mar 2011 10:37:42 +0100] rev 41912
adding termination proofs to series functions in LSC; commenting out momentarily unused term refinement functions in LSC
bulwahn [Fri, 11 Mar 2011 10:37:41 +0100] rev 41911
adding lazysmallcheck example theory to HOL-ex session
bulwahn [Fri, 11 Mar 2011 10:37:40 +0100] rev 41910
adding serial instance of finite_4 in lazysmallcheck; changing code equations for implies
bulwahn [Fri, 11 Mar 2011 10:37:38 +0100] rev 41909
replacing strings in generated Code resolves the changing names of Typerep in lazysmallcheck prototype
bulwahn [Fri, 11 Mar 2011 10:37:37 +0100] rev 41908
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
bulwahn [Fri, 11 Mar 2011 10:37:37 +0100] rev 41907
adding an example theory for Lazysmallcheck prototype
bulwahn [Fri, 11 Mar 2011 10:37:36 +0100] rev 41906
adding Lazysmallcheck prototype to HOL-Library
bulwahn [Fri, 11 Mar 2011 10:37:35 +0100] rev 41905
adding files for prototype of lazysmallcheck
bulwahn [Fri, 11 Mar 2011 08:58:29 +0100] rev 41904
removing debug message in quickcheck's postprocessor
bulwahn [Fri, 11 Mar 2011 08:13:00 +0100] rev 41903
fixing postprocessing; adding a configuration to enable and disable pretty presentation of quickcheck's counterexample
bulwahn [Fri, 11 Mar 2011 08:12:59 +0100] rev 41902
renaming dest_plain_fun to dest_fun_upds and adding handling of undefined for postprocessing of quickcheck
bulwahn [Fri, 11 Mar 2011 08:12:58 +0100] rev 41901
improving term postprocessing for counterexample presentation in quickcheck
bulwahn [Fri, 11 Mar 2011 08:12:55 +0100] rev 41900
tuned
boehmes [Wed, 09 Mar 2011 21:40:38 +0100] rev 41899
finished and tested Z3 proof reconstruction for injective functions;
only treat variables as atomic, and especially abstract constants (Isabelle's interpretation of these constants is most likely not known to Z3 and thus irrelevant for the proof)
blanchet [Wed, 09 Mar 2011 10:28:01 +0100] rev 41898
improved formula for specialization, to prevent needless specializations -- and removed dead code
blanchet [Wed, 09 Mar 2011 10:25:29 +0100] rev 41897
perform no arity check in debug mode so that we get to see the Kodkod problem
berghofe [Fri, 04 Mar 2011 17:39:30 +0100] rev 41896
spark_end now joins proofs of VCs before writing *.prv file.
krauss [Fri, 04 Mar 2011 11:43:20 +0100] rev 41895
clarified
krauss [Fri, 04 Mar 2011 11:52:54 +0100] rev 41894
produce helpful mira summary for more errors
wenzelm [Fri, 04 Mar 2011 00:09:47 +0100] rev 41893
eliminated prems;
wenzelm [Thu, 03 Mar 2011 22:06:15 +0100] rev 41892
eliminated UNITY_Examples.thy which takes quite long to merge and does not parallelize so well -- essentially reverting 3dec57ec3473;
wenzelm [Thu, 03 Mar 2011 21:43:06 +0100] rev 41891
tuned proofs -- eliminated prems;
wenzelm [Thu, 03 Mar 2011 18:43:15 +0100] rev 41890
merged
blanchet [Thu, 03 Mar 2011 14:38:31 +0100] rev 41889
merged
blanchet [Thu, 03 Mar 2011 14:25:15 +0100] rev 41888
don't forget to look for constants appearing only in "need" option -- otherwise we get exceptions in "the_name" later on
wenzelm [Thu, 03 Mar 2011 18:42:12 +0100] rev 41887
simplified Thy_Info.check_file -- discontinued load path;
wenzelm [Thu, 03 Mar 2011 18:10:28 +0100] rev 41886
discontinued legacy load path;
wenzelm [Thu, 03 Mar 2011 15:56:17 +0100] rev 41885
re-interpret ProofGeneralPgip.changecwd as Thy_Load.set_master_path, presuming that this is close to the intended semantics;
wenzelm [Thu, 03 Mar 2011 15:46:02 +0100] rev 41884
modernized imports;
wenzelm [Thu, 03 Mar 2011 15:36:54 +0100] rev 41883
observe standard header format;
wenzelm [Thu, 03 Mar 2011 15:19:20 +0100] rev 41882
removed spurious 'unused_thms' (cf. 1a65b780bd56);
wenzelm [Thu, 03 Mar 2011 15:18:05 +0100] rev 41881
isatest cygwin-poly-e: new memory management of polyml-svn could be more stable;
berghofe [Thu, 03 Mar 2011 11:36:10 +0100] rev 41880
merged
berghofe [Thu, 03 Mar 2011 11:15:50 +0100] rev 41879
merged
berghofe [Thu, 03 Mar 2011 11:01:42 +0100] rev 41878
- Made sure that sort_defs is aware of constants introduced by add_type_def
- add_def now compares Isabelle types rather than SPARK types to ensure that
type abbreviations are taken into account
blanchet [Thu, 03 Mar 2011 11:20:48 +0100] rev 41877
mention new Nitpick options
blanchet [Thu, 03 Mar 2011 11:20:48 +0100] rev 41876
simplify "need" option's syntax
blanchet [Thu, 03 Mar 2011 11:20:48 +0100] rev 41875
renamed "preconstr" option "need"
hoelzl [Thu, 03 Mar 2011 10:55:41 +0100] rev 41874
finally remove upper_bound_finite_set
kleing [Thu, 03 Mar 2011 15:59:44 +1100] rev 41873
separate settings for afp test
blanchet [Wed, 02 Mar 2011 15:51:22 +0100] rev 41872
added missing spaces in output
blanchet [Wed, 02 Mar 2011 14:50:16 +0100] rev 41871
lower threshold for implicitly using "nitpick_simp" for predicate definitions when "total_consts" is on
blanchet [Wed, 02 Mar 2011 13:09:57 +0100] rev 41870
unfold definitions in "preconstrs" option
blanchet [Wed, 02 Mar 2011 13:09:57 +0100] rev 41869
robust handling of types occurring in "eval" and "preconstr" options but not in the goal
blanchet [Wed, 02 Mar 2011 13:09:57 +0100] rev 41868
make "preconstr" option more robust -- shouldn't throw exceptions
paulson [Tue, 01 Mar 2011 10:40:14 +0000] rev 41867
merged
paulson [Mon, 28 Feb 2011 15:06:55 +0000] rev 41866
merged
paulson [Mon, 28 Feb 2011 15:06:36 +0000] rev 41865
declare ext [intro]: Extensionality now available by default
boehmes [Mon, 28 Feb 2011 22:12:09 +0100] rev 41864
merged
boehmes [Mon, 28 Feb 2011 22:10:57 +0100] rev 41863
removed dependency on Dense_Linear_Order
bulwahn [Mon, 28 Feb 2011 19:06:24 +0100] rev 41862
adding function Quickcheck.test_terms to provide checking a batch of terms
bulwahn [Mon, 28 Feb 2011 19:06:23 +0100] rev 41861
adding a function to compile a batch of terms for quickcheck with one code generation invocation
blanchet [Mon, 28 Feb 2011 17:53:10 +0100] rev 41860
improved "is_special_eligible_arg" further, by approximating the cardinality of the argument (as is done quite successfully elsewhere)
blanchet [Mon, 28 Feb 2011 17:53:10 +0100] rev 41859
made "fixed_is_special_eligible_arg" smarter w.r.t. pairs, and fixed previous unintended behavior because "andalso" ties more tightly than "orelse"
blanchet [Mon, 28 Feb 2011 17:53:10 +0100] rev 41858
if "total_consts" is set, report cex's as quasi-genuine
blanchet [Mon, 28 Feb 2011 17:53:10 +0100] rev 41857
document new "total_consts" option
blanchet [Mon, 28 Feb 2011 17:53:10 +0100] rev 41856
added "total_consts" option
nipkow [Sat, 26 Feb 2011 20:40:45 +0100] rev 41855
added a few lemmas by Andreas Lochbihler
nipkow [Sat, 26 Feb 2011 20:16:44 +0100] rev 41854
Corrected HOLCF/FOCUS dependency
nipkow [Sat, 26 Feb 2011 17:44:42 +0100] rev 41853
Added material by David Trachtenherz
nipkow [Sat, 26 Feb 2011 16:16:36 +0100] rev 41852
corrected HOLCF dependency on Nat_Infinity
nipkow [Fri, 25 Feb 2011 22:07:56 +0100] rev 41851
got rid of lemma upper_bound_finite_set
nipkow [Fri, 25 Feb 2011 20:08:00 +0100] rev 41850
merged
nipkow [Fri, 25 Feb 2011 20:07:48 +0100] rev 41849
Some cleaning up
krauss [Fri, 25 Feb 2011 17:11:24 +0100] rev 41848
updated generated files
krauss [Fri, 25 Feb 2011 17:11:05 +0100] rev 41847
fixed manual (rule no longer exists)
krauss [Fri, 25 Feb 2011 16:59:48 +0100] rev 41846
removed support for tail-recursion from function package (now implemented by partial_function)
krauss [Fri, 25 Feb 2011 16:57:44 +0100] rev 41845
reactivate time measurement (partly reverting c27b0b37041a);
export pretty_theorem, to display both internal or external facts
krauss [Fri, 25 Feb 2011 16:57:43 +0100] rev 41844
generalize find_theorems filters to work on raw propositions, too
nipkow [Fri, 25 Feb 2011 14:25:52 +0100] rev 41843
merged
nipkow [Fri, 25 Feb 2011 14:25:41 +0100] rev 41842
added simp lemma nth_Cons_pos to List
noschinl [Fri, 25 Feb 2011 12:16:18 +0100] rev 41841
Refactor find_theorems to provide a more general filter_facts method
krauss [Fri, 25 Feb 2011 08:46:52 +0100] rev 41840
removed dead code/unused exports/speculative generality
krauss [Thu, 24 Feb 2011 21:54:28 +0100] rev 41839
recdef -> fun(ction)
krauss [Thu, 24 Feb 2011 20:52:05 +0100] rev 41838
removed unused lemma
krauss [Thu, 24 Feb 2011 17:54:36 +0100] rev 41837
recdef -> fun(ction);
tuned
krauss [Thu, 24 Feb 2011 17:38:05 +0100] rev 41836
eliminated clones of List.upto
noschinl [Wed, 23 Feb 2011 17:40:28 +0100] rev 41835
fix non-exhaustive pattern match in find_theorems
hoelzl [Wed, 23 Feb 2011 11:42:01 +0100] rev 41834
merged
hoelzl [Wed, 23 Feb 2011 11:40:18 +0100] rev 41833
add lemma KL_divergence_vimage, mutual_information_generic
hoelzl [Wed, 23 Feb 2011 11:40:17 +0100] rev 41832
add lemma RN_deriv_vimage
hoelzl [Wed, 23 Feb 2011 11:40:12 +0100] rev 41831
use measure_preserving in ..._vimage lemmas
hoelzl [Wed, 23 Feb 2011 11:33:45 +0100] rev 41830
log is borel measurable
hoelzl [Tue, 22 Feb 2011 16:07:23 +0100] rev 41829
add name continuous_isCont to unnamed lemma
noschinl [Wed, 23 Feb 2011 11:23:26 +0100] rev 41828
add example for case_product usage
noschinl [Wed, 23 Feb 2011 11:23:26 +0100] rev 41827
setup case_product attribute in HOL and FOL
noschinl [Wed, 08 Dec 2010 18:18:36 +0100] rev 41826
introduce attribute case_prod for combining case rules
* * *
[PATCH 1/9] Make tac independent of consumes
From 1a53ef4c070f924ff8e69529b0c1b13fa2844722 Mon Sep 17 00:00:00 2001
---
case_product.ML | 11 ++++++-----
1 files changed, 6 insertions(+), 5 deletions(-)
* * *
[PATCH 2/9] Replace MRS by OF
From da55d08ae287bfdc18dec554067b45a3e298c243 Mon Sep 17 00:00:00 2001
---
case_product.ML | 4 ++--
1 files changed, 2 insertions(+), 2 deletions(-)
* * *
[PATCH 3/9] Clean up tactic
From d26d50caaa3526c8c0625d7395467c6914f1a8d9 Mon Sep 17 00:00:00 2001
---
case_product.ML | 13 +++++--------
1 files changed, 5 insertions(+), 8 deletions(-)
* * *
[PATCH 4/9] Move out get_consumes a bit more
From 6ed5415f29cc43cea30c216edb1e74ec6c0f6c33 Mon Sep 17 00:00:00 2001
---
case_product.ML | 4 +++-
1 files changed, 3 insertions(+), 1 deletions(-)
* * *
[PATCH 5/9] Clean up tactic
From d301cfe6377e9f7db74b190fb085e0e66eeadfb5 Mon Sep 17 00:00:00 2001
---
case_product.ML | 3 +--
1 files changed, 1 insertions(+), 2 deletions(-)
* * *
[PATCH 6/9] Cleanup build_concl_prems
From c30889e131e74a92caac5b1e6d3d816890406ca7 Mon Sep 17 00:00:00 2001
---
case_product.ML | 18 ++++++++----------
1 files changed, 8 insertions(+), 10 deletions(-)
* * *
[PATCH 7/9] Split logic & annotation a bit
From e065606118308c96e013fad72ab9ad89b5a4b945 Mon Sep 17 00:00:00 2001
---
case_product.ML | 26 ++++++++++++++++++--------
1 files changed, 18 insertions(+), 8 deletions(-)
* * *
[PATCH 8/9] Remove dependency on consumes attribute
From e2a4de044481586d6127bbabd0ef48d0e3ab57c0 Mon Sep 17 00:00:00 2001
---
case_product.ML | 46 ++++++++++++++++++++++------------------------
1 files changed, 22 insertions(+), 24 deletions(-)
* * *
[PATCH 9/9] whitespace
From 59f5036bd8f825da4a362970292a34ec06c0f1a2 Mon Sep 17 00:00:00 2001
---
case_product.ML | 2 +-
1 files changed, 1 insertions(+), 1 deletions(-)
blanchet [Wed, 23 Feb 2011 11:18:10 +0100] rev 41825
merged
blanchet [Wed, 23 Feb 2011 11:17:48 +0100] rev 41824
remove confusing message
krauss [Wed, 23 Feb 2011 11:16:56 +0100] rev 41823
eliminated remdps in favor of List.remdups
krauss [Wed, 23 Feb 2011 11:15:06 +0100] rev 41822
recdef -> fun
krauss [Wed, 23 Feb 2011 10:48:57 +0100] rev 41821
recdef -> fun
wenzelm [Tue, 22 Feb 2011 21:54:56 +0100] rev 41820
updated generated file;
wenzelm [Tue, 22 Feb 2011 19:44:15 +0100] rev 41819
scale parallel_proofs_threshold with max_threads_value to improve saturation of cores;
wenzelm [Tue, 22 Feb 2011 17:06:14 +0100] rev 41818
modernized specifications;
krauss [Tue, 22 Feb 2011 16:47:18 +0100] rev 41817
dropped obsolete FIXMEs
wenzelm [Mon, 21 Feb 2011 23:54:53 +0100] rev 41816
merged, resolving spurious conflicts and giving up Reflected_Multivariate_Polynomial.thy from ab5d2d81f9fb;
krauss [Mon, 21 Feb 2011 23:14:36 +0100] rev 41815
eliminated global prems
krauss [Mon, 21 Feb 2011 23:14:36 +0100] rev 41814
modernized specification; curried
krauss [Mon, 21 Feb 2011 23:14:36 +0100] rev 41813
recdef -> fun; curried
krauss [Mon, 21 Feb 2011 23:14:36 +0100] rev 41812
recdef -> fun; curried
krauss [Mon, 21 Feb 2011 23:14:36 +0100] rev 41811
strengthened polymul.induct
krauss [Mon, 21 Feb 2011 23:14:36 +0100] rev 41810
dropped stupid name
krauss [Mon, 21 Feb 2011 23:14:36 +0100] rev 41809
removed duplicate declarations
krauss [Mon, 21 Feb 2011 23:14:36 +0100] rev 41808
recdef -> function
wenzelm [Mon, 21 Feb 2011 23:47:19 +0100] rev 41807
tuned proofs -- eliminated prems;
blanchet [Mon, 21 Feb 2011 18:29:47 +0100] rev 41806
merged
blanchet [Mon, 21 Feb 2011 18:28:28 +0100] rev 41805
adjust example
blanchet [Mon, 21 Feb 2011 18:02:14 +0100] rev 41804
document new "preconstr" option
blanchet [Mon, 21 Feb 2011 17:36:32 +0100] rev 41803
more work on "fix_datatype_vals" optimization (renamed "preconstruct")
blanchet [Mon, 21 Feb 2011 16:33:21 +0100] rev 41802
more work on "fix_datatype_vals"
blanchet [Mon, 21 Feb 2011 15:45:44 +0100] rev 41801
first steps in implementing "fix_datatype_vals" optimization
blanchet [Mon, 21 Feb 2011 14:02:07 +0100] rev 41800
better fudge factors for CVC3 and Yices based on Judgment Day
blanchet [Mon, 21 Feb 2011 13:59:44 +0100] rev 41799
exit code 127 can mean many things -- not just (and probably not) Perl missing
wenzelm [Mon, 21 Feb 2011 17:43:23 +0100] rev 41798
modernized specifications;
blanchet [Mon, 21 Feb 2011 11:50:38 +0100] rev 41797
rename Nitpick's (internal) auxiliary lemmas
blanchet [Mon, 21 Feb 2011 11:50:38 +0100] rev 41796
updated docs w.r.t. "nitpick_unfold" attribute
blanchet [Mon, 21 Feb 2011 11:50:38 +0100] rev 41795
improve optimization
blanchet [Mon, 21 Feb 2011 11:50:37 +0100] rev 41794
updated docs
blanchet [Mon, 21 Feb 2011 11:50:31 +0100] rev 41793
tweaked Nitpick based on C++ memory model example
blanchet [Mon, 21 Feb 2011 10:44:19 +0100] rev 41792
renamed "nitpick\_def" to "nitpick_unfold" to reflect its new semantics
blanchet [Mon, 21 Feb 2011 10:42:29 +0100] rev 41791
always unfold constant defitions marked with "nitpick_def" -- to prevent unfolding, there's already "nitpick_simp"
blanchet [Mon, 21 Feb 2011 10:31:48 +0100] rev 41790
give more weight to Frees than to Consts in relevance filter
blanchet [Mon, 21 Feb 2011 10:29:13 +0100] rev 41789
don't distinguish between "fixes" and other free variables -- this confuses users
blanchet [Mon, 21 Feb 2011 10:29:00 +0100] rev 41788
added a timeout around SMT preprocessing (notably monomorphization)
blanchet [Mon, 21 Feb 2011 10:03:48 +0100] rev 41787
comments to find fudge factors easily
boehmes [Mon, 21 Feb 2011 09:19:44 +0100] rev 41786
added test cases with quantifier occurring in first-order term positions
boehmes [Mon, 21 Feb 2011 09:14:48 +0100] rev 41785
wrap occurrences of quantifiers in first-order terms (i.e., outside first-order formulas) in If-expressions
haftmann [Sat, 19 Feb 2011 08:47:46 +0100] rev 41784
dropped redundancy
haftmann [Sat, 19 Feb 2011 08:39:05 +0100] rev 41783
merged
haftmann [Thu, 17 Feb 2011 09:31:29 +0100] rev 41782
added is_IAbs; tuned brackets and comments
haftmann [Thu, 17 Feb 2011 09:31:29 +0100] rev 41781
more idiomatic printing of let cascades and type variable constraints
wenzelm [Fri, 18 Feb 2011 17:05:19 +0100] rev 41780
merged
wenzelm [Fri, 18 Feb 2011 17:03:30 +0100] rev 41779
modernized specifications;
wenzelm [Fri, 18 Feb 2011 16:36:42 +0100] rev 41778
modernized specifications;
wenzelm [Fri, 18 Feb 2011 16:22:27 +0100] rev 41777
more precise headers;
wenzelm [Fri, 18 Feb 2011 16:11:58 +0100] rev 41776
less verbose tracing;
wenzelm [Fri, 18 Feb 2011 16:07:32 +0100] rev 41775
standardized headers;
wenzelm [Fri, 18 Feb 2011 15:46:13 +0100] rev 41774
modernized specifications;
blanchet [Fri, 18 Feb 2011 16:30:44 +0100] rev 41773
gracious timeout in "blocking" mode
blanchet [Fri, 18 Feb 2011 16:19:08 +0100] rev 41772
make Nitpick's timeout mechanism somewhat more reliable/friendly;
avoid producing warnings when invoked in "auto" mode
blanchet [Fri, 18 Feb 2011 15:44:52 +0100] rev 41771
better fudge factors for Sledgehammer
blanchet [Fri, 18 Feb 2011 15:17:39 +0100] rev 41770
adjust fudge factors
blanchet [Fri, 18 Feb 2011 12:32:55 +0100] rev 41769
extended ATP problem syntax to support other applications than Sledgehammer, e.g. experiments with ATPs
blanchet [Thu, 17 Feb 2011 12:14:47 +0100] rev 41768
export more functionality of Sledgehammer to applications (for experiments)
blanchet [Wed, 16 Feb 2011 19:07:53 +0100] rev 41767
export useful function (needed in a Sledgehammer-related experiment)
blanchet [Tue, 15 Feb 2011 18:32:58 +0100] rev 41766
make experimental "Z3 ATP" work on Linux as well
blanchet [Tue, 15 Feb 2011 10:03:10 +0100] rev 41765
adjusted fudge factors (based on Judgment Day runs)
nipkow [Mon, 14 Feb 2011 18:28:36 +0100] rev 41764
generalized termination lemmas
krauss [Mon, 14 Feb 2011 15:27:23 +0100] rev 41763
strengthened induction rule;
clarified some proofs
boehmes [Mon, 14 Feb 2011 12:25:26 +0100] rev 41762
limit the number of generated SMT monomorphization instances (in addition to the existing monomorphization limit which does not prevent seemingly infinite loops);
updated SMT certificate
boehmes [Mon, 14 Feb 2011 10:40:43 +0100] rev 41761
more explicit errors to inform users about problems related to SMT solvers;
fall back to remote SMT solver (if local version does not exist);
extend the Z3 proof parser to accommodate for slight changes introduced by Z3 2.18
wenzelm [Sun, 13 Feb 2011 17:45:21 +0100] rev 41760
more explicit exit due to failed etc/settings -- normally return code 0=true and 1=false could be tolerated, but bash syntax errors also return 1;
wenzelm [Sun, 13 Feb 2011 17:29:44 +0100] rev 41759
eliminated somewhat obsolete warning -- former "$HOME/Isabelle" vs. "$HOME/isabelle" no longer exist;
wenzelm [Sun, 13 Feb 2011 17:19:43 +0100] rev 41758
tuned;
nipkow [Sun, 13 Feb 2011 08:47:36 +0100] rev 41757
more pretty set comprehension sugar
bulwahn [Fri, 11 Feb 2011 15:31:19 +0100] rev 41756
merged
bulwahn [Fri, 11 Feb 2011 11:47:44 +0100] rev 41755
adjusting HOL-Mutabelle to changes in quickcheck
bulwahn [Fri, 11 Feb 2011 11:47:43 +0100] rev 41754
quickcheck can be invoked with its internal timelimit or without
bulwahn [Fri, 11 Feb 2011 11:47:42 +0100] rev 41753
quickcheck invokes TimeLimit.timeLimit only in one separate function
blanchet [Fri, 11 Feb 2011 11:54:24 +0100] rev 41752
added option to Mirabelle Sledgehammer
haftmann [Thu, 10 Feb 2011 18:44:39 +0100] rev 41751
merged
haftmann [Thu, 10 Feb 2011 10:32:12 +0100] rev 41750
reverted cs. 0a3fa8fbcdc5 -- motivation is unreconstructable, produces confusion in user space
blanchet [Thu, 10 Feb 2011 17:18:52 +0100] rev 41749
tuning
blanchet [Thu, 10 Feb 2011 17:17:31 +0100] rev 41748
fix handling of "fequal" in generated ATP problems -- the bug was visible if "explicit_apply" was on and "singleton_conv" is one of the facts being translated, as it resulted in an arity error in the ATP (e.g., E)
blanchet [Thu, 10 Feb 2011 16:38:12 +0100] rev 41747
fix path to etc/settings and etc/components in doc
blanchet [Thu, 10 Feb 2011 16:15:43 +0100] rev 41746
run all provers in blocking mode, even if a proof was already found -- this behavior is less confusing to the user
blanchet [Thu, 10 Feb 2011 16:05:33 +0100] rev 41745
remove pointless clutter
blanchet [Thu, 10 Feb 2011 10:09:38 +0100] rev 41744
make minimizer verbose
blanchet [Wed, 09 Feb 2011 17:18:58 +0100] rev 41743
tuning
blanchet [Wed, 09 Feb 2011 17:18:58 +0100] rev 41742
automatically minimize Z3-as-an-ATP proofs (cf. CVC3 and Yices)
blanchet [Wed, 09 Feb 2011 17:18:58 +0100] rev 41741
renamed field
blanchet [Wed, 09 Feb 2011 17:18:58 +0100] rev 41740
added "Z3 as an ATP" support to Sledgehammer locally