2010-03-29 prefer recursive calls before others in the mode inference
bulwahn [Mon, 29 Mar 2010 17:30:46 +0200] rev 36028
prefer recursive calls before others in the mode inference
2010-03-29 added statistics to values command for random generation
bulwahn [Mon, 29 Mar 2010 17:30:45 +0200] rev 36027
added statistics to values command for random generation
2010-03-29 adopting Predicate_Compile_Quickcheck
bulwahn [Mon, 29 Mar 2010 17:30:43 +0200] rev 36026
adopting Predicate_Compile_Quickcheck
2010-03-29 made quickcheck generic with respect to which compilation; added random compilation to quickcheck
bulwahn [Mon, 29 Mar 2010 17:30:43 +0200] rev 36025
made quickcheck generic with respect to which compilation; added random compilation to quickcheck
2010-03-29 removed yieldn in Lazy_Sequence and put in the ML structure; corrects behaviour of values command
bulwahn [Mon, 29 Mar 2010 17:30:41 +0200] rev 36024
removed yieldn in Lazy_Sequence and put in the ML structure; corrects behaviour of values command
2010-03-29 adding a hook for experiments in the predicate compilation process
bulwahn [Mon, 29 Mar 2010 17:30:40 +0200] rev 36023
adding a hook for experiments in the predicate compilation process
2010-03-29 removing simple equalities in introduction rules in the predicate compiler
bulwahn [Mon, 29 Mar 2010 17:30:40 +0200] rev 36022
removing simple equalities in introduction rules in the predicate compiler
2010-03-29 adopting Predicate_Compile
bulwahn [Mon, 29 Mar 2010 17:30:39 +0200] rev 36021
adopting Predicate_Compile
2010-03-29 adding values command for new monad; added new random monad compilation to predicate_compile_quickcheck
bulwahn [Mon, 29 Mar 2010 17:30:38 +0200] rev 36020
adding values command for new monad; added new random monad compilation to predicate_compile_quickcheck
2010-03-29 generalizing the compilation process of the predicate compiler
bulwahn [Mon, 29 Mar 2010 17:30:36 +0200] rev 36019
generalizing the compilation process of the predicate compiler
2010-03-29 added new compilation to predicate_compiler
bulwahn [Mon, 29 Mar 2010 17:30:36 +0200] rev 36018
added new compilation to predicate_compiler
2010-03-29 adding new depth-limited and new random monad for the predicate compiler
bulwahn [Mon, 29 Mar 2010 17:30:34 +0200] rev 36017
adding new depth-limited and new random monad for the predicate compiler
2010-03-29 recovered StringBuilder functionality after subtle change of + and ++ in Scala 2.8.0 Beta 1;
wenzelm [Tue, 30 Mar 2010 00:47:52 +0200] rev 36016
recovered StringBuilder functionality after subtle change of + and ++ in Scala 2.8.0 Beta 1;
2010-03-29 adapted to Scala 2.8.0 Beta 1;
wenzelm [Tue, 30 Mar 2010 00:13:27 +0200] rev 36015
adapted to Scala 2.8.0 Beta 1;
2010-03-29 auto update by Netbeans 6.8;
wenzelm [Tue, 30 Mar 2010 00:12:42 +0200] rev 36014
auto update by Netbeans 6.8;
2010-03-29 adapted to Netbeans 6.8 and Scala for Netbeans 6.8v1.1;
wenzelm [Tue, 30 Mar 2010 00:11:41 +0200] rev 36013
adapted to Netbeans 6.8 and Scala for Netbeans 6.8v1.1;
2010-03-29 replaced some deprecated methods;
wenzelm [Mon, 29 Mar 2010 22:55:57 +0200] rev 36012
replaced some deprecated methods;
2010-03-29 adapted to Scala 2.8.0 Beta1 -- with notable changes to scala.collection;
wenzelm [Mon, 29 Mar 2010 22:43:56 +0200] rev 36011
adapted to Scala 2.8.0 Beta1 -- with notable changes to scala.collection;
2010-03-29 merged
huffman [Mon, 29 Mar 2010 01:07:01 -0700] rev 36010
merged
2010-03-28 use lattice theorems to prove set theorems
huffman [Sun, 28 Mar 2010 12:50:38 -0700] rev 36009
use lattice theorems to prove set theorems
2010-03-28 add/change some lemmas about lattices
huffman [Sun, 28 Mar 2010 12:49:14 -0700] rev 36008
add/change some lemmas about lattices
2010-03-28 cleaned up some proofs
huffman [Sun, 28 Mar 2010 10:34:02 -0700] rev 36007
cleaned up some proofs
2010-03-29 the configuration option 'trace_simp' now uses the reference of the ProofGeneral settings menu as (dynamic) default value
boehmes [Mon, 29 Mar 2010 09:06:34 +0200] rev 36006
the configuration option 'trace_simp' now uses the reference of the ProofGeneral settings menu as (dynamic) default value
2010-03-28 merged
wenzelm [Sun, 28 Mar 2010 19:34:08 +0200] rev 36005
merged
2010-03-28 implicit checkpoint in Local_Theory.theory as well -- no longer export Local_Theory.checkpoint;
wenzelm [Sun, 28 Mar 2010 19:20:52 +0200] rev 36004
implicit checkpoint in Local_Theory.theory as well -- no longer export Local_Theory.checkpoint;
2010-03-28 make SML/NJ happy
blanchet [Sun, 28 Mar 2010 18:39:27 +0200] rev 36003
make SML/NJ happy
2010-03-28 pass raw Context.generic, to avoid wasteful Context.proof_of -- Config.get_thy is often used in performance critical spots like unify.ML;
wenzelm [Sun, 28 Mar 2010 17:43:09 +0200] rev 36002
pass raw Context.generic, to avoid wasteful Context.proof_of -- Config.get_thy is often used in performance critical spots like unify.ML;
2010-03-28 static defaults for configuration options;
wenzelm [Sun, 28 Mar 2010 16:59:06 +0200] rev 36001
static defaults for configuration options;
2010-03-28 configuration options admit dynamic default values;
wenzelm [Sun, 28 Mar 2010 16:13:29 +0200] rev 36000
configuration options admit dynamic default values;
2010-03-28 tuned;
wenzelm [Sun, 28 Mar 2010 16:29:51 +0200] rev 35999
tuned;
2010-03-28 do not export Attrib.register_config, to make it harder to use low-level Config.declare after the bootstrap phase;
wenzelm [Sun, 28 Mar 2010 15:38:07 +0200] rev 35998
do not export Attrib.register_config, to make it harder to use low-level Config.declare after the bootstrap phase;
2010-03-28 use regular Attrib.config instead of low-level Config.declare/Attrib.register_config;
wenzelm [Sun, 28 Mar 2010 15:13:19 +0200] rev 35997
use regular Attrib.config instead of low-level Config.declare/Attrib.register_config;
2010-03-27 merged
wenzelm [Sat, 27 Mar 2010 21:46:10 +0100] rev 35996
merged
2010-03-27 re-introduce reference to control simplifier tracing (needed for ProofGeneral settings menu) (cf. 12bb31230550)
boehmes [Sat, 27 Mar 2010 21:34:28 +0100] rev 35995
re-introduce reference to control simplifier tracing (needed for ProofGeneral settings menu) (cf. 12bb31230550)
2010-03-27 Typedef.info: separate global and local part, only the latter is transformed by morphisms;
wenzelm [Sat, 27 Mar 2010 21:38:38 +0100] rev 35994
Typedef.info: separate global and local part, only the latter is transformed by morphisms;
2010-03-27 merged
nipkow [Sat, 27 Mar 2010 18:43:11 +0100] rev 35993
merged
2010-03-27 added reference to Trace Simp Depth.
nipkow [Sat, 27 Mar 2010 18:42:27 +0100] rev 35992
added reference to Trace Simp Depth.
2010-03-27 merged
wenzelm [Sat, 27 Mar 2010 18:12:02 +0100] rev 35991
merged
2010-03-27 Automated lifting can be restricted to specific quotient types
Cezary Kaliszyk <kaliszyk@in.tum.de> [Sat, 27 Mar 2010 14:48:46 +0100] rev 35990
Automated lifting can be restricted to specific quotient types
2010-03-27 moved Primitive_Defs.mk_defpair to OldGoals.mk_defpair;
wenzelm [Sat, 27 Mar 2010 18:07:21 +0100] rev 35989
moved Primitive_Defs.mk_defpair to OldGoals.mk_defpair;
2010-03-27 disallow premises in primitive Theory.add_def -- handle in Thm.add_def;
wenzelm [Sat, 27 Mar 2010 17:36:32 +0100] rev 35988
disallow premises in primitive Theory.add_def -- handle in Thm.add_def; eliminated obsolete Sign.cert_def; misc tuning and clarification;
2010-03-27 disallow sort constraints in primitive Theory.add_axiom/add_def -- handled in Thm.add_axiom/add_def;
wenzelm [Sat, 27 Mar 2010 16:01:45 +0100] rev 35987
disallow sort constraints in primitive Theory.add_axiom/add_def -- handled in Thm.add_axiom/add_def;
2010-03-27 added Term.fold_atyps_sorts convenience;
wenzelm [Sat, 27 Mar 2010 15:47:57 +0100] rev 35986
added Term.fold_atyps_sorts convenience;
2010-03-27 moved Drule.forall_intr_frees to Thm.forall_intr_frees (in more_thm.ML, which is loaded before pure_thy.ML);
wenzelm [Sat, 27 Mar 2010 15:20:31 +0100] rev 35985
moved Drule.forall_intr_frees to Thm.forall_intr_frees (in more_thm.ML, which is loaded before pure_thy.ML); discontinued old-style Theory.add_defs(_i) in favour of more basic Theory.add_def; modernized PureThy.add_defs etc. -- refer to high-level Thm.add_def;
2010-03-27 eliminated old-style Theory.add_defs_i;
wenzelm [Sat, 27 Mar 2010 14:10:37 +0100] rev 35984
eliminated old-style Theory.add_defs_i;
2010-03-27 slightly more general simproc (avoids errors of linarith)
boehmes [Sat, 27 Mar 2010 02:10:00 +0100] rev 35983
slightly more general simproc (avoids errors of linarith)
2010-03-26 merged
boehmes [Sat, 27 Mar 2010 00:08:39 +0100] rev 35982
merged
2010-03-26 updated SMT certificates
boehmes [Fri, 26 Mar 2010 23:58:27 +0100] rev 35981
updated SMT certificates
2010-03-26 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: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)
2010-03-26 replaced references 'trace_simp' and 'debug_simp' by configuration options stored in the context
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
2010-03-26 merged
wenzelm [Fri, 26 Mar 2010 20:30:03 +0100] rev 35978
merged
2010-03-26 Added finite measure space.
hoelzl [Fri, 26 Mar 2010 18:03:01 +0100] rev 35977
Added finite measure space.
2010-03-26 tuned white space;
wenzelm [Fri, 26 Mar 2010 20:30:05 +0100] rev 35976
tuned white space;
2010-03-26 more efficient merge_algebra for important special cases -- tricky due to required completion if class algebra changes;
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;
2010-03-26 low-level tuning for join/merge: ignore identical versions (SUBTLE CHANGE IN SEMANTICS);
wenzelm [Fri, 26 Mar 2010 17:59:11 +0100] rev 35974
low-level tuning for join/merge: ignore identical versions (SUBTLE CHANGE IN SEMANTICS);
2010-03-25 merged
wenzelm [Thu, 25 Mar 2010 23:18:42 +0100] rev 35973
merged
2010-03-25 merged
blanchet [Thu, 25 Mar 2010 17:56:31 +0100] rev 35972
merged
2010-03-25 make Mirabelle happy again
blanchet [Thu, 25 Mar 2010 17:55:55 +0100] rev 35971
make Mirabelle happy again
2010-03-24 revert debugging output that shouldn't have been submitted in the first place
blanchet [Wed, 24 Mar 2010 14:51:36 +0100] rev 35970
revert debugging output that shouldn't have been submitted in the first place
2010-03-24 added support for Sledgehammer parameters;
blanchet [Wed, 24 Mar 2010 14:49:32 +0100] rev 35969
added support for Sledgehammer parameters; this change goes hand in hand with f8c738abaed8
2010-03-24 simplify Nitpick parameter parsing code a little bit + make compile
blanchet [Wed, 24 Mar 2010 14:43:35 +0100] rev 35968
simplify Nitpick parameter parsing code a little bit + make compile
2010-03-24 add new file "sledgehammer_util.ML" to setup
blanchet [Wed, 24 Mar 2010 12:31:37 +0100] rev 35967
add new file "sledgehammer_util.ML" to setup
2010-03-24 honor the newly introduced Sledgehammer parameters and fixed the parsing;
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
2010-03-23 added a syntax for specifying facts to Sledgehammer;
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".
2010-03-23 leverage code now in Sledgehammer
blanchet [Tue, 23 Mar 2010 11:40:46 +0100] rev 35964
leverage code now in Sledgehammer
2010-03-23 added options to 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
2010-03-22 make "sledgehammer" and "atp_minimize" improper commands
blanchet [Mon, 22 Mar 2010 15:23:18 +0100] rev 35962
make "sledgehammer" and "atp_minimize" improper commands
2010-03-25 Sorts.of_sort_derivation: do not use slow Graph.irreducible_paths here, which not always needed (SUBTLE CHANGE IN SEMANTICS);
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;
2010-03-25 removed unused AxClass.of_sort derivation;
wenzelm [Thu, 25 Mar 2010 21:14:15 +0100] rev 35960
removed unused AxClass.of_sort derivation;
2010-03-24 more precise dependencies;
wenzelm [Wed, 24 Mar 2010 22:30:33 +0100] rev 35959
more precise dependencies;
2010-03-24 merged
wenzelm [Wed, 24 Mar 2010 22:08:03 +0100] rev 35958
merged
2010-03-24 merged
bulwahn [Wed, 24 Mar 2010 17:41:25 +0100] rev 35957
merged
2010-03-24 removed predicate_compile_core.ML from HOL-ex session
bulwahn [Wed, 24 Mar 2010 17:40:44 +0100] rev 35956
removed predicate_compile_core.ML from HOL-ex session
2010-03-24 added predicate compiler quickcheck examples to new session Predicate_Compile_Examples
bulwahn [Wed, 24 Mar 2010 17:40:44 +0100] rev 35955
added predicate compiler quickcheck examples to new session Predicate_Compile_Examples
2010-03-24 adopting examples to Library move
bulwahn [Wed, 24 Mar 2010 17:40:44 +0100] rev 35954
adopting examples to Library move
2010-03-24 moved further predicate compile files to HOL-Library
bulwahn [Wed, 24 Mar 2010 17:40:43 +0100] rev 35953
moved further predicate compile files to HOL-Library
2010-03-24 added simple setup for arithmetic on natural numbers
bulwahn [Wed, 24 Mar 2010 17:40:43 +0100] rev 35952
added simple setup for arithmetic on natural numbers
2010-03-24 removing uncommented examples in setup theory of predicate compile quickcheck
bulwahn [Wed, 24 Mar 2010 17:40:43 +0100] rev 35951
removing uncommented examples in setup theory of predicate compile quickcheck
2010-03-24 moved examples for the predicate compiler into its own session Predicate_Compile_Examples to slenderise the HOL-ex session
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
2010-03-24 slightly more logical bootstrap order -- also helps to sort out proof terms extension;
wenzelm [Wed, 24 Mar 2010 21:55:30 +0100] rev 35949
slightly more logical bootstrap order -- also helps to sort out proof terms extension;
2010-03-24 remove ancient continuity tactic
huffman [Wed, 24 Mar 2010 07:50:21 -0700] rev 35948
remove ancient continuity tactic
2010-03-24 removed Cache_IO component
boehmes [Wed, 24 Mar 2010 15:21:42 +0100] rev 35947
removed Cache_IO component
2010-03-24 updated SMT certificates
boehmes [Wed, 24 Mar 2010 14:08:07 +0100] rev 35946
updated SMT certificates
2010-03-24 inhibit invokation of external SMT solver
boehmes [Wed, 24 Mar 2010 14:03:52 +0100] rev 35945
inhibit invokation of external SMT solver
2010-03-24 more precise dependencies
boehmes [Wed, 24 Mar 2010 12:30:21 +0100] rev 35944
more precise dependencies
2010-03-24 cache_io is now just a single ML file instead of a component
boehmes [Wed, 24 Mar 2010 09:44:47 +0100] rev 35943
cache_io is now just a single ML file instead of a component
2010-03-24 use internal SHA1 digest implementation for generating hash keys
boehmes [Wed, 24 Mar 2010 09:43:34 +0100] rev 35942
use internal SHA1 digest implementation for generating hash keys
2010-03-24 remove component Cache_IO (external dependency on MD5 will be replaced by internal SHA1 digest implementation)
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)
2010-03-24 merged
huffman [Tue, 23 Mar 2010 19:03:05 -0700] rev 35940
merged
2010-03-23 minimize dependencies
huffman [Tue, 23 Mar 2010 13:42:12 -0700] rev 35939
minimize dependencies
2010-03-23 sublocale comm_monoid_add < setprod --> sublocale comm_monoid_mult < setprod
huffman [Tue, 23 Mar 2010 12:20:27 -0700] rev 35938
sublocale comm_monoid_add < setprod --> sublocale comm_monoid_mult < setprod
2010-03-23 use ml_platform instead of ml_system to distinguish library names
boehmes [Tue, 23 Mar 2010 22:43:53 +0100] rev 35937
use ml_platform instead of ml_system to distinguish library names
2010-03-23 merged
boehmes [Tue, 23 Mar 2010 20:46:47 +0100] rev 35936
merged
2010-03-23 use LONG rather than INT to represent the C datatype size_t
boehmes [Tue, 23 Mar 2010 20:46:08 +0100] rev 35935
use LONG rather than INT to represent the C datatype size_t
2010-03-23 merged
wenzelm [Tue, 23 Mar 2010 19:35:33 +0100] rev 35934
merged
2010-03-23 remove continuous let-binding function CLet; add cont2cont rule ordinary Let
huffman [Tue, 23 Mar 2010 10:07:39 -0700] rev 35933
remove continuous let-binding function CLet; add cont2cont rule ordinary Let
2010-03-23 move letrec stuff to new file HOLCF/ex/Letrec.thy
huffman [Tue, 23 Mar 2010 09:39:21 -0700] rev 35932
move letrec stuff to new file HOLCF/ex/Letrec.thy
2010-03-23 more accurate dependencies;
wenzelm [Tue, 23 Mar 2010 19:35:03 +0100] rev 35931
more accurate dependencies;
2010-03-23 even less ambitious isatest for smlnj;
wenzelm [Tue, 23 Mar 2010 17:26:41 +0100] rev 35930
even less ambitious isatest for smlnj;
2010-03-23 Unhide measure_space.positive defined in Caratheodory.
hoelzl [Tue, 23 Mar 2010 16:18:44 +0100] rev 35929
Unhide measure_space.positive defined in Caratheodory.
2010-03-23 Generate image for HOL-Probability
hoelzl [Tue, 23 Mar 2010 16:17:41 +0100] rev 35928
Generate image for HOL-Probability
2010-03-23 updated Thm.add_axiom/add_def;
wenzelm [Tue, 23 Mar 2010 12:29:41 +0100] rev 35927
updated Thm.add_axiom/add_def;
2010-03-23 completely remove constants cpair, cfst, csnd
huffman [Mon, 22 Mar 2010 23:34:23 -0700] rev 35926
completely remove constants cpair, cfst, csnd
2010-03-23 use Pair instead of cpair in Fixrec_ex.thy
huffman [Mon, 22 Mar 2010 23:33:23 -0700] rev 35925
use Pair instead of cpair in Fixrec_ex.thy
2010-03-23 use Pair instead of cpair
huffman [Mon, 22 Mar 2010 23:33:02 -0700] rev 35924
use Pair instead of cpair
2010-03-23 define CLetrec using Pair, fst, snd instead of cpair, cfst, csnd
huffman [Mon, 22 Mar 2010 23:02:43 -0700] rev 35923
define CLetrec using Pair, fst, snd instead of cpair, cfst, csnd
2010-03-23 define csplit using fst, snd
huffman [Mon, 22 Mar 2010 22:55:26 -0700] rev 35922
define csplit using fst, snd
2010-03-23 convert lemma fix_cprod to use Pair, fst, snd
huffman [Mon, 22 Mar 2010 22:43:21 -0700] rev 35921
convert lemma fix_cprod to use Pair, fst, snd
2010-03-23 remove unused syntax for as_pat, lazy_pat
huffman [Mon, 22 Mar 2010 22:42:34 -0700] rev 35920
remove unused syntax for as_pat, lazy_pat
2010-03-23 add lemmas fst_monofun, snd_monofun
huffman [Mon, 22 Mar 2010 22:41:41 -0700] rev 35919
add lemmas fst_monofun, snd_monofun
2010-03-23 use Pair instead of cpair
huffman [Mon, 22 Mar 2010 21:37:48 -0700] rev 35918
use Pair instead of cpair
2010-03-23 use fixrec_simp instead of fixpat
huffman [Mon, 22 Mar 2010 21:33:31 -0700] rev 35917
use fixrec_simp instead of fixpat
2010-03-23 use Pair, fst, snd instead of cpair, cfst, csnd
huffman [Mon, 22 Mar 2010 21:31:32 -0700] rev 35916
use Pair, fst, snd instead of cpair, cfst, csnd
2010-03-23 remove admw predicate
huffman [Mon, 22 Mar 2010 21:11:54 -0700] rev 35915
remove admw predicate
2010-03-23 remove contlub predicate
huffman [Mon, 22 Mar 2010 20:54:52 -0700] rev 35914
remove contlub predicate
2010-03-22 merged
huffman [Mon, 22 Mar 2010 16:02:51 -0700] rev 35913
merged
2010-03-22 error -> raise Fail
huffman [Mon, 22 Mar 2010 15:53:25 -0700] rev 35912
error -> raise Fail
2010-03-22 merged
wenzelm [Mon, 22 Mar 2010 23:48:27 +0100] rev 35911
merged
2010-03-22 merged
wenzelm [Mon, 22 Mar 2010 23:20:55 +0100] rev 35910
merged
2010-03-22 merged
wenzelm [Mon, 22 Mar 2010 22:56:46 +0100] rev 35909
merged
2010-03-22 remove unused adm_tac.ML
huffman [Mon, 22 Mar 2010 15:45:54 -0700] rev 35908
remove unused adm_tac.ML
2010-03-22 avoid dependence on adm_tac solver
huffman [Mon, 22 Mar 2010 15:42:07 -0700] rev 35907
avoid dependence on adm_tac solver
2010-03-22 remove obsolete holcf_logic.ML
huffman [Mon, 22 Mar 2010 15:23:16 -0700] rev 35906
remove obsolete holcf_logic.ML
2010-03-22 fix ML warning in domain_library.ML
huffman [Mon, 22 Mar 2010 15:05:20 -0700] rev 35905
fix ML warning in domain_library.ML
2010-03-22 fix ML warnings in repdef.ML
huffman [Mon, 22 Mar 2010 14:58:21 -0700] rev 35904
fix ML warnings in repdef.ML
2010-03-22 fix ML warnings in fixrec.ML
huffman [Mon, 22 Mar 2010 14:44:37 -0700] rev 35903
fix ML warnings in fixrec.ML
2010-03-22 fix ML warnings in pcpodef.ML
huffman [Mon, 22 Mar 2010 14:11:13 -0700] rev 35902
fix ML warnings in pcpodef.ML
2010-03-22 fix LaTeX overfull hbox warnings in HOLCF document
huffman [Mon, 22 Mar 2010 13:27:35 -0700] rev 35901
fix LaTeX overfull hbox warnings in HOLCF document
2010-03-22 remove LaTeX hyperref warnings by avoiding antiquotations within section headings
huffman [Mon, 22 Mar 2010 12:52:51 -0700] rev 35900
remove LaTeX hyperref warnings by avoiding antiquotations within section headings
2010-03-22 explicit Simplifier.global_context;
wenzelm [Mon, 22 Mar 2010 20:59:22 +0100] rev 35899
explicit Simplifier.global_context;
2010-03-22 recovered header;
wenzelm [Mon, 22 Mar 2010 20:58:52 +0100] rev 35898
recovered header;
2010-03-22 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: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;
2010-03-22 inlined version of old-style Drule.add_axioms -- Specification.axiom is not bootstrapped yet;
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;
2010-03-22 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: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);
2010-03-22 added Specification.axiom convenience;
wenzelm [Mon, 22 Mar 2010 19:23:03 +0100] rev 35894
added Specification.axiom convenience;
2010-03-22 detect OFCLASS() axioms in Nitpick;
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)
2010-03-22 merged
bulwahn [Mon, 22 Mar 2010 13:48:15 +0100] rev 35892
merged
2010-03-22 contextifying the compilation of the predicate compiler
bulwahn [Mon, 22 Mar 2010 08:30:13 +0100] rev 35891
contextifying the compilation of the predicate compiler
2010-03-22 removed unused Predicate_Compile_Set
bulwahn [Mon, 22 Mar 2010 08:30:13 +0100] rev 35890
removed unused Predicate_Compile_Set
2010-03-22 avoiding fishing for split_asm rule in the predicate compiler
bulwahn [Mon, 22 Mar 2010 08:30:13 +0100] rev 35889
avoiding fishing for split_asm rule in the predicate compiler
2010-03-22 contextifying the proof procedure in the predicate compiler
bulwahn [Mon, 22 Mar 2010 08:30:13 +0100] rev 35888
contextifying the proof procedure in the predicate compiler
2010-03-22 making flat triples to nested tuple to remove general triple functions
bulwahn [Mon, 22 Mar 2010 08:30:13 +0100] rev 35887
making flat triples to nested tuple to remove general triple functions
2010-03-22 reduced the debug output functions from 2 to 1
bulwahn [Mon, 22 Mar 2010 08:30:13 +0100] rev 35886
reduced the debug output functions from 2 to 1
2010-03-22 some improvements thanks to Makarius source code review
bulwahn [Mon, 22 Mar 2010 08:30:13 +0100] rev 35885
some improvements thanks to Makarius source code review
2010-03-22 adding proof procedure for cases rule with tuples; adding introduction rule for negated premises; improving proof procedure with negated premises
bulwahn [Mon, 22 Mar 2010 08:30:13 +0100] rev 35884
adding proof procedure for cases rule with tuples; adding introduction rule for negated premises; improving proof procedure with negated premises
2010-03-22 enabling a previously broken example of the predicate compiler again
bulwahn [Mon, 22 Mar 2010 08:30:13 +0100] rev 35883
enabling a previously broken example of the predicate compiler again
2010-03-22 improving handling of case expressions in predicate rewriting
bulwahn [Mon, 22 Mar 2010 08:30:13 +0100] rev 35882
improving handling of case expressions in predicate rewriting
2010-03-22 adding depth_limited_random compilation to predicate compiler
bulwahn [Mon, 22 Mar 2010 08:30:13 +0100] rev 35881
adding depth_limited_random compilation to predicate compiler
2010-03-22 a new simpler random compilation for the predicate compiler
bulwahn [Mon, 22 Mar 2010 08:30:13 +0100] rev 35880
a new simpler random compilation for the predicate compiler
2010-03-22 reviving the classical depth-limited computation in the predicate compiler
bulwahn [Mon, 22 Mar 2010 08:30:13 +0100] rev 35879
reviving the classical depth-limited computation in the predicate compiler
2010-03-22 cleaning the function flattening
bulwahn [Mon, 22 Mar 2010 08:30:13 +0100] rev 35878
cleaning the function flattening
2010-03-22 generalized split transformation in the function flattening
bulwahn [Mon, 22 Mar 2010 08:30:13 +0100] rev 35877
generalized split transformation in the function flattening
2010-03-22 only adding lifted arguments to item net in the function flattening; correcting indentation; removing dead code
bulwahn [Mon, 22 Mar 2010 08:30:12 +0100] rev 35876
only adding lifted arguments to item net in the function flattening; correcting indentation; removing dead code
2010-03-22 restructuring function flattening
bulwahn [Mon, 22 Mar 2010 08:30:12 +0100] rev 35875
restructuring function flattening
2010-03-22 renaming mk_prems to flatten in the function flattening
bulwahn [Mon, 22 Mar 2010 08:30:12 +0100] rev 35874
renaming mk_prems to flatten in the function flattening
2010-03-22 simplifying function flattening
bulwahn [Mon, 22 Mar 2010 08:30:12 +0100] rev 35873
simplifying function flattening
2010-03-22 removed warning_count (known causes for warnings have been resolved)
boehmes [Mon, 22 Mar 2010 11:45:09 +0100] rev 35872
removed warning_count (known causes for warnings have been resolved)
2010-03-22 remove the iteration counter from Sledgehammer's minimizer
blanchet [Mon, 22 Mar 2010 10:38:28 +0100] rev 35871
remove the iteration counter from Sledgehammer's minimizer
2010-03-22 merged
blanchet [Mon, 22 Mar 2010 10:25:44 +0100] rev 35870
merged
2010-03-22 start work on direct proof reconstruction for Sledgehammer
blanchet [Mon, 22 Mar 2010 10:25:07 +0100] rev 35869
start work on direct proof reconstruction for Sledgehammer
2010-03-19 renamed "e_full" and "vampire_full" to "e_isar" and "vampire_isar";
blanchet [Fri, 19 Mar 2010 16:04:15 +0100] rev 35868
renamed "e_full" and "vampire_full" to "e_isar" and "vampire_isar"; "full" sounds like "full types" or something, not like a structured Isar proof -- at some point I hope to make this an option that's orthogonal to the prover
2010-03-19 move all ATP setup code into ATP_Wrapper
blanchet [Fri, 19 Mar 2010 15:33:18 +0100] rev 35867
move all ATP setup code into ATP_Wrapper
2010-03-19 move the Sledgehammer Isar commands together into one file;
blanchet [Fri, 19 Mar 2010 15:07:44 +0100] rev 35866
move the Sledgehammer Isar commands together into one file; this will make easier to add options and reorganize them later
2010-03-19 more Sledgehammer refactoring
blanchet [Fri, 19 Mar 2010 13:02:18 +0100] rev 35865
more Sledgehammer refactoring
2010-03-22 use a proof context instead of a local theory
boehmes [Mon, 22 Mar 2010 09:54:22 +0100] rev 35864
use a proof context instead of a local theory
2010-03-22 provide a hook to safely manipulate verification conditions
boehmes [Mon, 22 Mar 2010 09:46:04 +0100] rev 35863
provide a hook to safely manipulate verification conditions
2010-03-22 replaced old-style Drule.add_axiom by Specification.axiomatization
boehmes [Mon, 22 Mar 2010 09:40:11 +0100] rev 35862
replaced old-style Drule.add_axiom by Specification.axiomatization
2010-03-22 removed e-mail address from error message
boehmes [Mon, 22 Mar 2010 09:39:10 +0100] rev 35861
removed e-mail address from error message
2010-03-22 merged
haftmann [Mon, 22 Mar 2010 09:32:28 +0100] rev 35860
merged
2010-03-21 tuned whitespace
haftmann [Sun, 21 Mar 2010 08:46:50 +0100] rev 35859
tuned whitespace
2010-03-21 handle hidden polymorphism in class target (without class target syntax, though)
haftmann [Sun, 21 Mar 2010 08:46:49 +0100] rev 35858
handle hidden polymorphism in class target (without class target syntax, though)
2010-03-21 replaced Theory.add_axioms(_i) by more primitive Theory.add_axiom;
wenzelm [Mon, 22 Mar 2010 00:51:18 +0100] rev 35857
replaced Theory.add_axioms(_i) by more primitive Theory.add_axiom;
2010-03-21 replaced PureThy.add_axioms by more basic Drule.add_axiom, which is old-style nonetheless;
wenzelm [Mon, 22 Mar 2010 00:48:56 +0100] rev 35856
replaced PureThy.add_axioms by more basic Drule.add_axiom, which is old-style nonetheless;
2010-03-21 add_axiom: axiomatize "unconstrained" version, with explicit of_class premises;
wenzelm [Sun, 21 Mar 2010 22:24:04 +0100] rev 35855
add_axiom: axiomatize "unconstrained" version, with explicit of_class premises; more uniform add_axiom/add_def;
2010-03-21 Logic.mk_of_sort convenience;
wenzelm [Sun, 21 Mar 2010 22:13:31 +0100] rev 35854
Logic.mk_of_sort convenience;
2010-03-21 more explicit invented name;
wenzelm [Sun, 21 Mar 2010 19:30:19 +0100] rev 35853
more explicit invented name;
2010-03-21 minor renovation of old-style 'axioms' -- make it an alias of iterated 'axiomatization';
wenzelm [Sun, 21 Mar 2010 19:28:25 +0100] rev 35852
minor renovation of old-style 'axioms' -- make it an alias of iterated 'axiomatization';
2010-03-21 do not open ML structures;
wenzelm [Sun, 21 Mar 2010 19:04:46 +0100] rev 35851
do not open ML structures;
2010-03-21 modernized overloaded definitions;
wenzelm [Sun, 21 Mar 2010 17:28:35 +0100] rev 35850
modernized overloaded definitions;
2010-03-21 standard headers;
wenzelm [Sun, 21 Mar 2010 17:12:31 +0100] rev 35849
standard headers;
2010-03-21 slightly more uniform definitions -- eliminated old-style meta-equality;
wenzelm [Sun, 21 Mar 2010 16:51:37 +0100] rev 35848
slightly more uniform definitions -- eliminated old-style meta-equality;
2010-03-21 eliminated old constdefs;
wenzelm [Sun, 21 Mar 2010 15:57:40 +0100] rev 35847
eliminated old constdefs;
2010-03-21 corrected setup for of_list
haftmann [Sun, 21 Mar 2010 06:59:23 +0100] rev 35846
corrected setup for of_list
2010-03-20 renamed varify/unvarify operations to varify_global/unvarify_global to emphasize that these only work in a global situation;
wenzelm [Sat, 20 Mar 2010 17:33:11 +0100] rev 35845
renamed varify/unvarify operations to varify_global/unvarify_global to emphasize that these only work in a global situation;
2010-03-20 added lemma infinite_Un
Christian Urban <urbanc@in.tum.de> [Sat, 20 Mar 2010 02:23:41 +0100] rev 35844
added lemma infinite_Un
2010-03-19 Check that argument is not a 'Bound' before calling fastype_of.
Cezary Kaliszyk <kaliszyk@in.tum.de> [Fri, 19 Mar 2010 06:14:37 +0100] rev 35843
Check that argument is not a 'Bound' before calling fastype_of.
2010-03-18 typedef etc.: no constraints;
wenzelm [Fri, 19 Mar 2010 00:47:23 +0100] rev 35842
typedef etc.: no constraints;
2010-03-18 allow sort constraints in HOL/typedef;
wenzelm [Fri, 19 Mar 2010 00:46:08 +0100] rev 35841
allow sort constraints in HOL/typedef;
2010-03-18 allow sort constraints in HOL/typedef and related HOLCF variants;
wenzelm [Fri, 19 Mar 2010 00:43:49 +0100] rev 35840
allow sort constraints in HOL/typedef and related HOLCF variants;
2010-03-18 OuterParse.type_args_constrained;
wenzelm [Fri, 19 Mar 2010 00:42:17 +0100] rev 35839
OuterParse.type_args_constrained;
2010-03-18 support type arguments with sort constraints;
wenzelm [Fri, 19 Mar 2010 00:41:34 +0100] rev 35838
support type arguments with sort constraints;
2010-03-18 typedecl: no sort constraints;
wenzelm [Thu, 18 Mar 2010 23:08:52 +0100] rev 35837
typedecl: no sort constraints; prefer Name.invents over old-style Name.variant_list;
2010-03-18 eliminated slightly odd typedecl_wrt in favour of explicit predeclare_constraints;
wenzelm [Thu, 18 Mar 2010 23:00:18 +0100] rev 35836
eliminated slightly odd typedecl_wrt in favour of explicit predeclare_constraints;
2010-03-18 typedecl: no sort constraints;
wenzelm [Thu, 18 Mar 2010 22:59:44 +0100] rev 35835
typedecl: no sort constraints;
2010-03-18 eliminated slightly odd typedecl_wrt in favour of explicit predeclare_constraints (which also works for recursive types);
wenzelm [Thu, 18 Mar 2010 22:56:32 +0100] rev 35834
eliminated slightly odd typedecl_wrt in favour of explicit predeclare_constraints (which also works for recursive types); allow sort constraints; misc tuning and clarification;
2010-03-16 Added product measure space
hoelzl [Tue, 16 Mar 2010 16:27:28 +0100] rev 35833
Added product measure space
2010-03-18 added type constraints to make SML/NJ happy
blanchet [Thu, 18 Mar 2010 14:52:11 +0100] rev 35832
added type constraints to make SML/NJ happy
2010-03-18 merged
blanchet [Thu, 18 Mar 2010 13:59:20 +0100] rev 35831
merged
2010-03-18 fix Mirabelle after renaming Sledgehammer structures
blanchet [Thu, 18 Mar 2010 13:43:50 +0100] rev 35830
fix Mirabelle after renaming Sledgehammer structures
2010-03-18 merged
blanchet [Thu, 18 Mar 2010 13:14:54 +0100] rev 35829
merged
2010-03-18 now use "Named_Thms" for "noatp", and renamed "noatp" to "no_atp"
blanchet [Thu, 18 Mar 2010 12:58:52 +0100] rev 35828
now use "Named_Thms" for "noatp", and renamed "noatp" to "no_atp"
2010-03-17 renamed "ATP_Linkup" theory to "Sledgehammer"
blanchet [Wed, 17 Mar 2010 19:37:44 +0100] rev 35827
renamed "ATP_Linkup" theory to "Sledgehammer"
2010-03-17 renamed Sledgehammer structures
blanchet [Wed, 17 Mar 2010 19:26:05 +0100] rev 35826
renamed Sledgehammer structures
2010-03-17 move Sledgehammer files in a directory of their own
blanchet [Wed, 17 Mar 2010 18:16:31 +0100] rev 35825
move Sledgehammer files in a directory of their own
2010-03-18 merged
haftmann [Thu, 18 Mar 2010 13:57:00 +0100] rev 35824
merged
2010-03-18 dropped odd interpretation of comm_monoid_mult into comm_monoid_add
haftmann [Thu, 18 Mar 2010 13:56:34 +0100] rev 35823
dropped odd interpretation of comm_monoid_mult into comm_monoid_add
2010-03-18 lemma swap_inj_on, swap_product
haftmann [Thu, 18 Mar 2010 13:56:34 +0100] rev 35822
lemma swap_inj_on, swap_product
2010-03-18 meaningful transfer certificate
haftmann [Thu, 18 Mar 2010 13:56:33 +0100] rev 35821
meaningful transfer certificate
2010-03-18 dropped odd interpretation of comm_monoid_mult into comm_monoid_add; consider Min.insert_idem as default simp rule
haftmann [Thu, 18 Mar 2010 13:56:33 +0100] rev 35820
dropped odd interpretation of comm_monoid_mult into comm_monoid_add; consider Min.insert_idem as default simp rule
2010-03-18 updated certificate
haftmann [Thu, 18 Mar 2010 13:56:32 +0100] rev 35819
updated certificate
2010-03-18 dropped odd interpretation of comm_monoid_mult into comm_monoid_add
haftmann [Thu, 18 Mar 2010 13:56:32 +0100] rev 35818
dropped odd interpretation of comm_monoid_mult into comm_monoid_add
2010-03-18 added locales folding_one_(idem); various streamlining and tuning
haftmann [Thu, 18 Mar 2010 13:56:32 +0100] rev 35817
added locales folding_one_(idem); various streamlining and tuning
2010-03-18 generic locale for big operators in monoids; dropped odd interpretation of comm_monoid_mult into comm_monoid_add
haftmann [Thu, 18 Mar 2010 13:56:31 +0100] rev 35816
generic locale for big operators in monoids; dropped odd interpretation of comm_monoid_mult into comm_monoid_add
2010-03-17 tuned proofs (to avoid linarith error message caused by bootstrapping of HOL)
boehmes [Wed, 17 Mar 2010 19:55:07 +0100] rev 35815
tuned proofs (to avoid linarith error message caused by bootstrapping of HOL)
2010-03-17 added one-entry cache around Kodkod invocation
blanchet [Wed, 17 Mar 2010 17:23:45 +0100] rev 35814
added one-entry cache around Kodkod invocation
2010-03-17 merged
blanchet [Wed, 17 Mar 2010 16:27:11 +0100] rev 35813
merged
2010-03-17 solve error in "Nitpick_Mono" + short path when no finite functions are inferred
blanchet [Wed, 17 Mar 2010 16:26:08 +0100] rev 35812
solve error in "Nitpick_Mono" + short path when no finite functions are inferred
2010-03-17 minor additions to Nitpick docs
blanchet [Wed, 17 Mar 2010 16:11:48 +0100] rev 35811
minor additions to Nitpick docs
2010-03-17 NEWS: Nat_Bijection library
huffman [Wed, 17 Mar 2010 08:11:24 -0700] rev 35810
NEWS: Nat_Bijection library
2010-03-17 document "nitpick_choice_spec" attribute
blanchet [Wed, 17 Mar 2010 12:21:54 +0100] rev 35809
document "nitpick_choice_spec" attribute
2010-03-17 fix typo in "nitpick_choice_spec" attribute name (singular, not plural)
blanchet [Wed, 17 Mar 2010 12:01:01 +0100] rev 35808
fix typo in "nitpick_choice_spec" attribute name (singular, not plural)
2010-03-17 added support for "specification" and "ax_specification" constructs to Nitpick
blanchet [Wed, 17 Mar 2010 09:14:43 +0100] rev 35807
added support for "specification" and "ax_specification" constructs to Nitpick
2010-03-16 rollback of local typedef until problem with type-variables can be sorted out; fixed header
Christian Urban <urbanc@in.tum.de> [Tue, 16 Mar 2010 08:45:08 +0100] rev 35806
rollback of local typedef until problem with type-variables can be sorted out; fixed header
2010-03-16 adjusted to changes in Finite_Set
haftmann [Tue, 16 Mar 2010 06:55:01 +0100] rev 35805
adjusted to changes in Finite_Set
2010-03-15 merged
wenzelm [Mon, 15 Mar 2010 22:22:28 +0100] rev 35804
merged
2010-03-15 merged
nipkow [Mon, 15 Mar 2010 17:34:03 +0100] rev 35803
merged
2010-03-15 tuned inductions
nipkow [Mon, 15 Mar 2010 17:33:41 +0100] rev 35802
tuned inductions
2010-03-15 tuned;
wenzelm [Mon, 15 Mar 2010 21:59:28 +0100] rev 35801
tuned;
2010-03-15 moved old Sign.intern_term to the place where it is still used;
wenzelm [Mon, 15 Mar 2010 21:57:35 +0100] rev 35800
moved old Sign.intern_term to the place where it is still used;
2010-03-15 preserve full const name more carefully, and avoid slightly odd Sign.intern_term;
wenzelm [Mon, 15 Mar 2010 20:27:23 +0100] rev 35799
preserve full const name more carefully, and avoid slightly odd Sign.intern_term;
2010-03-15 replaced type_syntax/term_syntax by uniform syntax_declaration;
wenzelm [Mon, 15 Mar 2010 18:59:16 +0100] rev 35798
replaced type_syntax/term_syntax by uniform syntax_declaration;
2010-03-15 merged
haftmann [Mon, 15 Mar 2010 15:13:22 +0100] rev 35797
merged
2010-03-15 corrected disastrous syntax declarations
haftmann [Mon, 15 Mar 2010 15:13:07 +0100] rev 35796
corrected disastrous syntax declarations
2010-03-15 added stmaryrd for isasymSqinter
haftmann [Mon, 15 Mar 2010 13:59:34 +0100] rev 35795
added stmaryrd for isasymSqinter
2010-03-15 use headers consistently
huffman [Sun, 14 Mar 2010 19:48:33 -0700] rev 35794
use headers consistently
2010-03-15 no_document for theory Countable
huffman [Sun, 14 Mar 2010 19:47:13 -0700] rev 35793
no_document for theory Countable
2010-03-14 old domain package also defines map functions
huffman [Sun, 14 Mar 2010 14:10:36 -0700] rev 35792
old domain package also defines map functions
2010-03-14 separate map-related code into new function define_map_functions
huffman [Sun, 14 Mar 2010 14:10:05 -0700] rev 35791
separate map-related code into new function define_map_functions
2010-03-14 removed Local_Theory.theory_result by using local Typedef.add_typedef
Christian Urban <urbanc@in.tum.de> [Sun, 14 Mar 2010 15:50:17 +0100] rev 35790
removed Local_Theory.theory_result by using local Typedef.add_typedef
2010-03-14 tuned comment;
wenzelm [Sun, 14 Mar 2010 14:36:56 +0100] rev 35789
tuned comment;
(0) -30000 -10000 -3000 -1000 -240 +240 +1000 +3000 +10000 +30000 tip