Mon, 29 Mar 2010 17:30:36 +0200 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
Mon, 29 Mar 2010 17:30:36 +0200 added new compilation to predicate_compiler
bulwahn [Mon, 29 Mar 2010 17:30:36 +0200] rev 36018
added new compilation to predicate_compiler
Mon, 29 Mar 2010 17:30:34 +0200 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
Tue, 30 Mar 2010 00:47:52 +0200 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;
Tue, 30 Mar 2010 00:13:27 +0200 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;
Tue, 30 Mar 2010 00:12:42 +0200 auto update by Netbeans 6.8;
wenzelm [Tue, 30 Mar 2010 00:12:42 +0200] rev 36014
auto update by Netbeans 6.8;
Tue, 30 Mar 2010 00:11:41 +0200 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;
Mon, 29 Mar 2010 22:55:57 +0200 replaced some deprecated methods;
wenzelm [Mon, 29 Mar 2010 22:55:57 +0200] rev 36012
replaced some deprecated methods;
Mon, 29 Mar 2010 22:43:56 +0200 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;
Mon, 29 Mar 2010 01:07:01 -0700 merged
huffman [Mon, 29 Mar 2010 01:07:01 -0700] rev 36010
merged
Sun, 28 Mar 2010 12:50:38 -0700 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
Sun, 28 Mar 2010 12:49:14 -0700 add/change some lemmas about lattices
huffman [Sun, 28 Mar 2010 12:49:14 -0700] rev 36008
add/change some lemmas about lattices
Sun, 28 Mar 2010 10:34:02 -0700 cleaned up some proofs
huffman [Sun, 28 Mar 2010 10:34:02 -0700] rev 36007
cleaned up some proofs
Mon, 29 Mar 2010 09:06:34 +0200 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
Sun, 28 Mar 2010 19:34:08 +0200 merged
wenzelm [Sun, 28 Mar 2010 19:34:08 +0200] rev 36005
merged
Sun, 28 Mar 2010 19:20:52 +0200 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;
Sun, 28 Mar 2010 18:39:27 +0200 make SML/NJ happy
blanchet [Sun, 28 Mar 2010 18:39:27 +0200] rev 36003
make SML/NJ happy
Sun, 28 Mar 2010 17:43:09 +0200 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;
Sun, 28 Mar 2010 16:59:06 +0200 static defaults for configuration options;
wenzelm [Sun, 28 Mar 2010 16:59:06 +0200] rev 36001
static defaults for configuration options;
Sun, 28 Mar 2010 16:13:29 +0200 configuration options admit dynamic default values;
wenzelm [Sun, 28 Mar 2010 16:13:29 +0200] rev 36000
configuration options admit dynamic default values;
Sun, 28 Mar 2010 16:29:51 +0200 tuned;
wenzelm [Sun, 28 Mar 2010 16:29:51 +0200] rev 35999
tuned;
Sun, 28 Mar 2010 15:38:07 +0200 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;
Sun, 28 Mar 2010 15:13:19 +0200 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;
Sat, 27 Mar 2010 21:46:10 +0100 merged
wenzelm [Sat, 27 Mar 2010 21:46:10 +0100] rev 35996
merged
Sat, 27 Mar 2010 21:34:28 +0100 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)
Sat, 27 Mar 2010 21:38:38 +0100 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;
Sat, 27 Mar 2010 18:43:11 +0100 merged
nipkow [Sat, 27 Mar 2010 18:43:11 +0100] rev 35993
merged
Sat, 27 Mar 2010 18:42:27 +0100 added reference to Trace Simp Depth.
nipkow [Sat, 27 Mar 2010 18:42:27 +0100] rev 35992
added reference to Trace Simp Depth.
Sat, 27 Mar 2010 18:12:02 +0100 merged
wenzelm [Sat, 27 Mar 2010 18:12:02 +0100] rev 35991
merged
Sat, 27 Mar 2010 14:48:46 +0100 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
Sat, 27 Mar 2010 18:07:21 +0100 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;
Sat, 27 Mar 2010 17:36:32 +0100 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;
Sat, 27 Mar 2010 16:01:45 +0100 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;
Sat, 27 Mar 2010 15:47:57 +0100 added Term.fold_atyps_sorts convenience;
wenzelm [Sat, 27 Mar 2010 15:47:57 +0100] rev 35986
added Term.fold_atyps_sorts convenience;
Sat, 27 Mar 2010 15:20:31 +0100 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;
Sat, 27 Mar 2010 14:10:37 +0100 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;
Sat, 27 Mar 2010 02:10:00 +0100 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)
Sat, 27 Mar 2010 00:08:39 +0100 merged
boehmes [Sat, 27 Mar 2010 00:08:39 +0100] rev 35982
merged
Fri, 26 Mar 2010 23:58:27 +0100 updated SMT certificates
boehmes [Fri, 26 Mar 2010 23:58:27 +0100] rev 35981
updated SMT certificates
Fri, 26 Mar 2010 23:57:35 +0100 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)
Fri, 26 Mar 2010 23:46:22 +0100 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
Fri, 26 Mar 2010 20:30:03 +0100 merged
wenzelm [Fri, 26 Mar 2010 20:30:03 +0100] rev 35978
merged
Fri, 26 Mar 2010 18:03:01 +0100 Added finite measure space.
hoelzl [Fri, 26 Mar 2010 18:03:01 +0100] rev 35977
Added finite measure space.
Fri, 26 Mar 2010 20:30:05 +0100 tuned white space;
wenzelm [Fri, 26 Mar 2010 20:30:05 +0100] rev 35976
tuned white space;
Fri, 26 Mar 2010 20:28:15 +0100 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;
Fri, 26 Mar 2010 17:59:11 +0100 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);
Thu, 25 Mar 2010 23:18:42 +0100 merged
wenzelm [Thu, 25 Mar 2010 23:18:42 +0100] rev 35973
merged
Thu, 25 Mar 2010 17:56:31 +0100 merged
blanchet [Thu, 25 Mar 2010 17:56:31 +0100] rev 35972
merged
Thu, 25 Mar 2010 17:55:55 +0100 make Mirabelle happy again
blanchet [Thu, 25 Mar 2010 17:55:55 +0100] rev 35971
make Mirabelle happy again
Wed, 24 Mar 2010 14:51:36 +0100 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
Wed, 24 Mar 2010 14:49:32 +0100 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
Wed, 24 Mar 2010 14:43:35 +0100 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
Wed, 24 Mar 2010 12:31:37 +0100 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
Wed, 24 Mar 2010 12:30:33 +0100 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
Tue, 23 Mar 2010 14:43:22 +0100 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".
Tue, 23 Mar 2010 11:40:46 +0100 leverage code now in Sledgehammer
blanchet [Tue, 23 Mar 2010 11:40:46 +0100] rev 35964
leverage code now in Sledgehammer
Tue, 23 Mar 2010 11:39:21 +0100 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
Mon, 22 Mar 2010 15:23:18 +0100 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
Thu, 25 Mar 2010 21:27:04 +0100 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;
Thu, 25 Mar 2010 21:14:15 +0100 removed unused AxClass.of_sort derivation;
wenzelm [Thu, 25 Mar 2010 21:14:15 +0100] rev 35960
removed unused AxClass.of_sort derivation;
Wed, 24 Mar 2010 22:30:33 +0100 more precise dependencies;
wenzelm [Wed, 24 Mar 2010 22:30:33 +0100] rev 35959
more precise dependencies;
Wed, 24 Mar 2010 22:08:03 +0100 merged
wenzelm [Wed, 24 Mar 2010 22:08:03 +0100] rev 35958
merged
Wed, 24 Mar 2010 17:41:25 +0100 merged
bulwahn [Wed, 24 Mar 2010 17:41:25 +0100] rev 35957
merged
Wed, 24 Mar 2010 17:40:44 +0100 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
(0) -30000 -10000 -3000 -1000 -300 -100 -64 +64 +100 +300 +1000 +3000 +10000 +30000 tip