wenzelm [Sat, 27 Mar 2010 14:10:37 +0100] rev 35984
eliminated old-style Theory.add_defs_i;
boehmes [Sat, 27 Mar 2010 02:10:00 +0100] rev 35983
slightly more general simproc (avoids errors of linarith)
boehmes [Sat, 27 Mar 2010 00:08:39 +0100] rev 35982
merged
boehmes [Fri, 26 Mar 2010 23:58:27 +0100] rev 35981
updated SMT certificates
boehmes [Fri, 26 Mar 2010 23:57:35 +0100] rev 35980
made renamings stable under name changes in the original problem (uninterpreted names are irrelevant to the SMT solver, and caching of SMT certificates relies on irrelevancy of renamings)
boehmes [Fri, 26 Mar 2010 23:46:22 +0100] rev 35979
replaced references 'trace_simp' and 'debug_simp' by configuration options stored in the context
wenzelm [Fri, 26 Mar 2010 20:30:03 +0100] rev 35978
merged
hoelzl [Fri, 26 Mar 2010 18:03:01 +0100] rev 35977
Added finite measure space.
wenzelm [Fri, 26 Mar 2010 20:30:05 +0100] rev 35976
tuned white space;
wenzelm [Fri, 26 Mar 2010 20:28:15 +0100] rev 35975
more efficient merge_algebra for important special cases -- tricky due to required completion if class algebra changes;
wenzelm [Fri, 26 Mar 2010 17:59:11 +0100] rev 35974
low-level tuning for join/merge: ignore identical versions (SUBTLE CHANGE IN SEMANTICS);
wenzelm [Thu, 25 Mar 2010 23:18:42 +0100] rev 35973
merged
blanchet [Thu, 25 Mar 2010 17:56:31 +0100] rev 35972
merged
blanchet [Thu, 25 Mar 2010 17:55:55 +0100] rev 35971
make Mirabelle happy again
blanchet [Wed, 24 Mar 2010 14:51:36 +0100] rev 35970
revert debugging output that shouldn't have been submitted in the first place
blanchet [Wed, 24 Mar 2010 14:49:32 +0100] rev 35969
added support for Sledgehammer parameters;
this change goes hand in hand with f8c738abaed8
blanchet [Wed, 24 Mar 2010 14:43:35 +0100] rev 35968
simplify Nitpick parameter parsing code a little bit + make compile
blanchet [Wed, 24 Mar 2010 12:31:37 +0100] rev 35967
add new file "sledgehammer_util.ML" to setup
blanchet [Wed, 24 Mar 2010 12:30:33 +0100] rev 35966
honor the newly introduced Sledgehammer parameters and fixed the parsing;
e.g. the prover "e_isar" (formely "e_full") is gone, instead do sledgehammer [atps = e, isar_proof] to get the same effect
blanchet [Tue, 23 Mar 2010 14:43:22 +0100] rev 35965
added a syntax for specifying facts to Sledgehammer;
e.g., sledgehammer (add: foo del: bar)
which tells the relevance filter to include "foo" but omit "bar".
blanchet [Tue, 23 Mar 2010 11:40:46 +0100] rev 35964
leverage code now in Sledgehammer
blanchet [Tue, 23 Mar 2010 11:39:21 +0100] rev 35963
added options to Sledgehammer;
syntax: sledgehammer [options] goal_no, where "[options]" and "goal_no" are optional
blanchet [Mon, 22 Mar 2010 15:23:18 +0100] rev 35962
make "sledgehammer" and "atp_minimize" improper commands
wenzelm [Thu, 25 Mar 2010 21:27:04 +0100] rev 35961
Sorts.of_sort_derivation: do not use slow Graph.irreducible_paths here, which not always needed (SUBTLE CHANGE IN SEMANTICS);
officially export weaken as Sorts.classrel_derivation;
tuned comments;
wenzelm [Thu, 25 Mar 2010 21:14:15 +0100] rev 35960
removed unused AxClass.of_sort derivation;
wenzelm [Wed, 24 Mar 2010 22:30:33 +0100] rev 35959
more precise dependencies;
wenzelm [Wed, 24 Mar 2010 22:08:03 +0100] rev 35958
merged
bulwahn [Wed, 24 Mar 2010 17:41:25 +0100] rev 35957
merged
bulwahn [Wed, 24 Mar 2010 17:40:44 +0100] rev 35956
removed predicate_compile_core.ML from HOL-ex session
bulwahn [Wed, 24 Mar 2010 17:40:44 +0100] rev 35955
added predicate compiler quickcheck examples to new session Predicate_Compile_Examples
bulwahn [Wed, 24 Mar 2010 17:40:44 +0100] rev 35954
adopting examples to Library move
bulwahn [Wed, 24 Mar 2010 17:40:43 +0100] rev 35953
moved further predicate compile files to HOL-Library
bulwahn [Wed, 24 Mar 2010 17:40:43 +0100] rev 35952
added simple setup for arithmetic on natural numbers
bulwahn [Wed, 24 Mar 2010 17:40:43 +0100] rev 35951
removing uncommented examples in setup theory of predicate compile quickcheck
bulwahn [Wed, 24 Mar 2010 17:40:43 +0100] rev 35950
moved examples for the predicate compiler into its own session Predicate_Compile_Examples to slenderise the HOL-ex session
wenzelm [Wed, 24 Mar 2010 21:55:30 +0100] rev 35949
slightly more logical bootstrap order -- also helps to sort out proof terms extension;
huffman [Wed, 24 Mar 2010 07:50:21 -0700] rev 35948
remove ancient continuity tactic
boehmes [Wed, 24 Mar 2010 15:21:42 +0100] rev 35947
removed Cache_IO component
boehmes [Wed, 24 Mar 2010 14:08:07 +0100] rev 35946
updated SMT certificates
boehmes [Wed, 24 Mar 2010 14:03:52 +0100] rev 35945
inhibit invokation of external SMT solver
boehmes [Wed, 24 Mar 2010 12:30:21 +0100] rev 35944
more precise dependencies
boehmes [Wed, 24 Mar 2010 09:44:47 +0100] rev 35943
cache_io is now just a single ML file instead of a component
boehmes [Wed, 24 Mar 2010 09:43:34 +0100] rev 35942
use internal SHA1 digest implementation for generating hash keys
boehmes [Wed, 24 Mar 2010 08:22:43 +0100] rev 35941
remove component Cache_IO (external dependency on MD5 will be replaced by internal SHA1 digest implementation)
huffman [Tue, 23 Mar 2010 19:03:05 -0700] rev 35940
merged
huffman [Tue, 23 Mar 2010 13:42:12 -0700] rev 35939
minimize dependencies
huffman [Tue, 23 Mar 2010 12:20:27 -0700] rev 35938
sublocale comm_monoid_add < setprod --> sublocale comm_monoid_mult < setprod
boehmes [Tue, 23 Mar 2010 22:43:53 +0100] rev 35937
use ml_platform instead of ml_system to distinguish library names
boehmes [Tue, 23 Mar 2010 20:46:47 +0100] rev 35936
merged
boehmes [Tue, 23 Mar 2010 20:46:08 +0100] rev 35935
use LONG rather than INT to represent the C datatype size_t
wenzelm [Tue, 23 Mar 2010 19:35:33 +0100] rev 35934
merged
huffman [Tue, 23 Mar 2010 10:07:39 -0700] rev 35933
remove continuous let-binding function CLet; add cont2cont rule ordinary Let
huffman [Tue, 23 Mar 2010 09:39:21 -0700] rev 35932
move letrec stuff to new file HOLCF/ex/Letrec.thy
wenzelm [Tue, 23 Mar 2010 19:35:03 +0100] rev 35931
more accurate dependencies;
wenzelm [Tue, 23 Mar 2010 17:26:41 +0100] rev 35930
even less ambitious isatest for smlnj;
hoelzl [Tue, 23 Mar 2010 16:18:44 +0100] rev 35929
Unhide measure_space.positive defined in Caratheodory.
hoelzl [Tue, 23 Mar 2010 16:17:41 +0100] rev 35928
Generate image for HOL-Probability
wenzelm [Tue, 23 Mar 2010 12:29:41 +0100] rev 35927
updated Thm.add_axiom/add_def;
huffman [Mon, 22 Mar 2010 23:34:23 -0700] rev 35926
completely remove constants cpair, cfst, csnd
huffman [Mon, 22 Mar 2010 23:33:23 -0700] rev 35925
use Pair instead of cpair in Fixrec_ex.thy
huffman [Mon, 22 Mar 2010 23:33:02 -0700] rev 35924
use Pair instead of cpair
huffman [Mon, 22 Mar 2010 23:02:43 -0700] rev 35923
define CLetrec using Pair, fst, snd instead of cpair, cfst, csnd
huffman [Mon, 22 Mar 2010 22:55:26 -0700] rev 35922
define csplit using fst, snd
huffman [Mon, 22 Mar 2010 22:43:21 -0700] rev 35921
convert lemma fix_cprod to use Pair, fst, snd
huffman [Mon, 22 Mar 2010 22:42:34 -0700] rev 35920
remove unused syntax for as_pat, lazy_pat
huffman [Mon, 22 Mar 2010 22:41:41 -0700] rev 35919
add lemmas fst_monofun, snd_monofun
huffman [Mon, 22 Mar 2010 21:37:48 -0700] rev 35918
use Pair instead of cpair
huffman [Mon, 22 Mar 2010 21:33:31 -0700] rev 35917
use fixrec_simp instead of fixpat
huffman [Mon, 22 Mar 2010 21:31:32 -0700] rev 35916
use Pair, fst, snd instead of cpair, cfst, csnd
huffman [Mon, 22 Mar 2010 21:11:54 -0700] rev 35915
remove admw predicate
huffman [Mon, 22 Mar 2010 20:54:52 -0700] rev 35914
remove contlub predicate
huffman [Mon, 22 Mar 2010 16:02:51 -0700] rev 35913
merged
huffman [Mon, 22 Mar 2010 15:53:25 -0700] rev 35912
error -> raise Fail
wenzelm [Mon, 22 Mar 2010 23:48:27 +0100] rev 35911
merged
wenzelm [Mon, 22 Mar 2010 23:20:55 +0100] rev 35910
merged
wenzelm [Mon, 22 Mar 2010 22:56:46 +0100] rev 35909
merged
huffman [Mon, 22 Mar 2010 15:45:54 -0700] rev 35908
remove unused adm_tac.ML
huffman [Mon, 22 Mar 2010 15:42:07 -0700] rev 35907
avoid dependence on adm_tac solver
huffman [Mon, 22 Mar 2010 15:23:16 -0700] rev 35906
remove obsolete holcf_logic.ML
huffman [Mon, 22 Mar 2010 15:05:20 -0700] rev 35905
fix ML warning in domain_library.ML
huffman [Mon, 22 Mar 2010 14:58:21 -0700] rev 35904
fix ML warnings in repdef.ML
huffman [Mon, 22 Mar 2010 14:44:37 -0700] rev 35903
fix ML warnings in fixrec.ML
huffman [Mon, 22 Mar 2010 14:11:13 -0700] rev 35902
fix ML warnings in pcpodef.ML
huffman [Mon, 22 Mar 2010 13:27:35 -0700] rev 35901
fix LaTeX overfull hbox warnings in HOLCF document
huffman [Mon, 22 Mar 2010 12:52:51 -0700] rev 35900
remove LaTeX hyperref warnings by avoiding antiquotations within section headings
wenzelm [Mon, 22 Mar 2010 20:59:22 +0100] rev 35899
explicit Simplifier.global_context;
wenzelm [Mon, 22 Mar 2010 20:58:52 +0100] rev 35898
recovered header;
wenzelm [Mon, 22 Mar 2010 19:29:11 +0100] rev 35897
eliminated old-style Drule.add_axiom in favour of Specification.axiom, with explicit Drule.export_without_context to imitate the old behaviour;
wenzelm [Mon, 22 Mar 2010 19:26:12 +0100] rev 35896
inlined version of old-style Drule.add_axioms -- Specification.axiom is not bootstrapped yet;
wenzelm [Mon, 22 Mar 2010 19:25:14 +0100] rev 35895
use Specification.axiom, together with Drule.export_without_context that was implicit in the former PureThy.add_axioms (cf. f81557a124d5);
wenzelm [Mon, 22 Mar 2010 19:23:03 +0100] rev 35894
added Specification.axiom convenience;
blanchet [Mon, 22 Mar 2010 15:07:07 +0100] rev 35893
detect OFCLASS() axioms in Nitpick;
this is necessary now that "Thy.all_axioms_of" returns such axiom (starting with change 46cfc4b8112e)
bulwahn [Mon, 22 Mar 2010 13:48:15 +0100] rev 35892
merged
bulwahn [Mon, 22 Mar 2010 08:30:13 +0100] rev 35891
contextifying the compilation of the predicate compiler
bulwahn [Mon, 22 Mar 2010 08:30:13 +0100] rev 35890
removed unused Predicate_Compile_Set
bulwahn [Mon, 22 Mar 2010 08:30:13 +0100] rev 35889
avoiding fishing for split_asm rule in the predicate compiler