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
Wed, 24 Mar 2010 17:40:44 +0100 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
Wed, 24 Mar 2010 17:40:44 +0100 adopting examples to Library move
bulwahn [Wed, 24 Mar 2010 17:40:44 +0100] rev 35954
adopting examples to Library move
Wed, 24 Mar 2010 17:40:43 +0100 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
Wed, 24 Mar 2010 17:40:43 +0100 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
Wed, 24 Mar 2010 17:40:43 +0100 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
Wed, 24 Mar 2010 17:40:43 +0100 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
Wed, 24 Mar 2010 21:55:30 +0100 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;
Wed, 24 Mar 2010 07:50:21 -0700 remove ancient continuity tactic
huffman [Wed, 24 Mar 2010 07:50:21 -0700] rev 35948
remove ancient continuity tactic
Wed, 24 Mar 2010 15:21:42 +0100 removed Cache_IO component
boehmes [Wed, 24 Mar 2010 15:21:42 +0100] rev 35947
removed Cache_IO component
Wed, 24 Mar 2010 14:08:07 +0100 updated SMT certificates
boehmes [Wed, 24 Mar 2010 14:08:07 +0100] rev 35946
updated SMT certificates
Wed, 24 Mar 2010 14:03:52 +0100 inhibit invokation of external SMT solver
boehmes [Wed, 24 Mar 2010 14:03:52 +0100] rev 35945
inhibit invokation of external SMT solver
Wed, 24 Mar 2010 12:30:21 +0100 more precise dependencies
boehmes [Wed, 24 Mar 2010 12:30:21 +0100] rev 35944
more precise dependencies
Wed, 24 Mar 2010 09:44:47 +0100 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
Wed, 24 Mar 2010 09:43:34 +0100 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
Wed, 24 Mar 2010 08:22:43 +0100 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)
Tue, 23 Mar 2010 19:03:05 -0700 merged
huffman [Tue, 23 Mar 2010 19:03:05 -0700] rev 35940
merged
Tue, 23 Mar 2010 13:42:12 -0700 minimize dependencies
huffman [Tue, 23 Mar 2010 13:42:12 -0700] rev 35939
minimize dependencies
Tue, 23 Mar 2010 12:20:27 -0700 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
Tue, 23 Mar 2010 22:43:53 +0100 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
Tue, 23 Mar 2010 20:46:47 +0100 merged
boehmes [Tue, 23 Mar 2010 20:46:47 +0100] rev 35936
merged
Tue, 23 Mar 2010 20:46:08 +0100 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
Tue, 23 Mar 2010 19:35:33 +0100 merged
wenzelm [Tue, 23 Mar 2010 19:35:33 +0100] rev 35934
merged
Tue, 23 Mar 2010 10:07:39 -0700 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
Tue, 23 Mar 2010 09:39:21 -0700 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
Tue, 23 Mar 2010 19:35:03 +0100 more accurate dependencies;
wenzelm [Tue, 23 Mar 2010 19:35:03 +0100] rev 35931
more accurate dependencies;
Tue, 23 Mar 2010 17:26:41 +0100 even less ambitious isatest for smlnj;
wenzelm [Tue, 23 Mar 2010 17:26:41 +0100] rev 35930
even less ambitious isatest for smlnj;
Tue, 23 Mar 2010 16:18:44 +0100 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.
Tue, 23 Mar 2010 16:17:41 +0100 Generate image for HOL-Probability
hoelzl [Tue, 23 Mar 2010 16:17:41 +0100] rev 35928
Generate image for HOL-Probability
Tue, 23 Mar 2010 12:29:41 +0100 updated Thm.add_axiom/add_def;
wenzelm [Tue, 23 Mar 2010 12:29:41 +0100] rev 35927
updated Thm.add_axiom/add_def;
Mon, 22 Mar 2010 23:34:23 -0700 completely remove constants cpair, cfst, csnd
huffman [Mon, 22 Mar 2010 23:34:23 -0700] rev 35926
completely remove constants cpair, cfst, csnd
Mon, 22 Mar 2010 23:33:23 -0700 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
Mon, 22 Mar 2010 23:33:02 -0700 use Pair instead of cpair
huffman [Mon, 22 Mar 2010 23:33:02 -0700] rev 35924
use Pair instead of cpair
Mon, 22 Mar 2010 23:02:43 -0700 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
Mon, 22 Mar 2010 22:55:26 -0700 define csplit using fst, snd
huffman [Mon, 22 Mar 2010 22:55:26 -0700] rev 35922
define csplit using fst, snd
Mon, 22 Mar 2010 22:43:21 -0700 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
Mon, 22 Mar 2010 22:42:34 -0700 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
Mon, 22 Mar 2010 22:41:41 -0700 add lemmas fst_monofun, snd_monofun
huffman [Mon, 22 Mar 2010 22:41:41 -0700] rev 35919
add lemmas fst_monofun, snd_monofun
Mon, 22 Mar 2010 21:37:48 -0700 use Pair instead of cpair
huffman [Mon, 22 Mar 2010 21:37:48 -0700] rev 35918
use Pair instead of cpair
Mon, 22 Mar 2010 21:33:31 -0700 use fixrec_simp instead of fixpat
huffman [Mon, 22 Mar 2010 21:33:31 -0700] rev 35917
use fixrec_simp instead of fixpat
Mon, 22 Mar 2010 21:31:32 -0700 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
Mon, 22 Mar 2010 21:11:54 -0700 remove admw predicate
huffman [Mon, 22 Mar 2010 21:11:54 -0700] rev 35915
remove admw predicate
Mon, 22 Mar 2010 20:54:52 -0700 remove contlub predicate
huffman [Mon, 22 Mar 2010 20:54:52 -0700] rev 35914
remove contlub predicate
Mon, 22 Mar 2010 16:02:51 -0700 merged
huffman [Mon, 22 Mar 2010 16:02:51 -0700] rev 35913
merged
Mon, 22 Mar 2010 15:53:25 -0700 error -> raise Fail
huffman [Mon, 22 Mar 2010 15:53:25 -0700] rev 35912
error -> raise Fail
Mon, 22 Mar 2010 23:48:27 +0100 merged
wenzelm [Mon, 22 Mar 2010 23:48:27 +0100] rev 35911
merged
Mon, 22 Mar 2010 23:20:55 +0100 merged
wenzelm [Mon, 22 Mar 2010 23:20:55 +0100] rev 35910
merged
Mon, 22 Mar 2010 22:56:46 +0100 merged
wenzelm [Mon, 22 Mar 2010 22:56:46 +0100] rev 35909
merged
Mon, 22 Mar 2010 15:45:54 -0700 remove unused adm_tac.ML
huffman [Mon, 22 Mar 2010 15:45:54 -0700] rev 35908
remove unused adm_tac.ML
Mon, 22 Mar 2010 15:42:07 -0700 avoid dependence on adm_tac solver
huffman [Mon, 22 Mar 2010 15:42:07 -0700] rev 35907
avoid dependence on adm_tac solver
Mon, 22 Mar 2010 15:23:16 -0700 remove obsolete holcf_logic.ML
huffman [Mon, 22 Mar 2010 15:23:16 -0700] rev 35906
remove obsolete holcf_logic.ML
Mon, 22 Mar 2010 15:05:20 -0700 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
Mon, 22 Mar 2010 14:58:21 -0700 fix ML warnings in repdef.ML
huffman [Mon, 22 Mar 2010 14:58:21 -0700] rev 35904
fix ML warnings in repdef.ML
Mon, 22 Mar 2010 14:44:37 -0700 fix ML warnings in fixrec.ML
huffman [Mon, 22 Mar 2010 14:44:37 -0700] rev 35903
fix ML warnings in fixrec.ML
Mon, 22 Mar 2010 14:11:13 -0700 fix ML warnings in pcpodef.ML
huffman [Mon, 22 Mar 2010 14:11:13 -0700] rev 35902
fix ML warnings in pcpodef.ML
Mon, 22 Mar 2010 13:27:35 -0700 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
Mon, 22 Mar 2010 12:52:51 -0700 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
Mon, 22 Mar 2010 20:59:22 +0100 explicit Simplifier.global_context;
wenzelm [Mon, 22 Mar 2010 20:59:22 +0100] rev 35899
explicit Simplifier.global_context;
Mon, 22 Mar 2010 20:58:52 +0100 recovered header;
wenzelm [Mon, 22 Mar 2010 20:58:52 +0100] rev 35898
recovered header;
Mon, 22 Mar 2010 19:29:11 +0100 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;
Mon, 22 Mar 2010 19:26:12 +0100 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;
Mon, 22 Mar 2010 19:25:14 +0100 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);
Mon, 22 Mar 2010 19:23:03 +0100 added Specification.axiom convenience;
wenzelm [Mon, 22 Mar 2010 19:23:03 +0100] rev 35894
added Specification.axiom convenience;
Mon, 22 Mar 2010 15:07:07 +0100 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)
Mon, 22 Mar 2010 13:48:15 +0100 merged
bulwahn [Mon, 22 Mar 2010 13:48:15 +0100] rev 35892
merged
Mon, 22 Mar 2010 08:30:13 +0100 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
Mon, 22 Mar 2010 08:30:13 +0100 removed unused Predicate_Compile_Set
bulwahn [Mon, 22 Mar 2010 08:30:13 +0100] rev 35890
removed unused Predicate_Compile_Set
Mon, 22 Mar 2010 08:30:13 +0100 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
Mon, 22 Mar 2010 08:30:13 +0100 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
Mon, 22 Mar 2010 08:30:13 +0100 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
Mon, 22 Mar 2010 08:30:13 +0100 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
Mon, 22 Mar 2010 08:30:13 +0100 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
Mon, 22 Mar 2010 08:30:13 +0100 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
Mon, 22 Mar 2010 08:30:13 +0100 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
Mon, 22 Mar 2010 08:30:13 +0100 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
Mon, 22 Mar 2010 08:30:13 +0100 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
Mon, 22 Mar 2010 08:30:13 +0100 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
Mon, 22 Mar 2010 08:30:13 +0100 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
Mon, 22 Mar 2010 08:30:13 +0100 cleaning the function flattening
bulwahn [Mon, 22 Mar 2010 08:30:13 +0100] rev 35878
cleaning the function flattening
Mon, 22 Mar 2010 08:30:13 +0100 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
Mon, 22 Mar 2010 08:30:12 +0100 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
Mon, 22 Mar 2010 08:30:12 +0100 restructuring function flattening
bulwahn [Mon, 22 Mar 2010 08:30:12 +0100] rev 35875
restructuring function flattening
Mon, 22 Mar 2010 08:30:12 +0100 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
Mon, 22 Mar 2010 08:30:12 +0100 simplifying function flattening
bulwahn [Mon, 22 Mar 2010 08:30:12 +0100] rev 35873
simplifying function flattening
Mon, 22 Mar 2010 11:45:09 +0100 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)
Mon, 22 Mar 2010 10:38:28 +0100 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
Mon, 22 Mar 2010 10:25:44 +0100 merged
blanchet [Mon, 22 Mar 2010 10:25:44 +0100] rev 35870
merged
Mon, 22 Mar 2010 10:25:07 +0100 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
Fri, 19 Mar 2010 16:04:15 +0100 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
Fri, 19 Mar 2010 15:33:18 +0100 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
Fri, 19 Mar 2010 15:07:44 +0100 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
Fri, 19 Mar 2010 13:02:18 +0100 more Sledgehammer refactoring
blanchet [Fri, 19 Mar 2010 13:02:18 +0100] rev 35865
more Sledgehammer refactoring
Mon, 22 Mar 2010 09:54:22 +0100 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
Mon, 22 Mar 2010 09:46:04 +0100 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
Mon, 22 Mar 2010 09:40:11 +0100 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
Mon, 22 Mar 2010 09:39:10 +0100 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
Mon, 22 Mar 2010 09:32:28 +0100 merged
haftmann [Mon, 22 Mar 2010 09:32:28 +0100] rev 35860
merged
Sun, 21 Mar 2010 08:46:50 +0100 tuned whitespace
haftmann [Sun, 21 Mar 2010 08:46:50 +0100] rev 35859
tuned whitespace
Sun, 21 Mar 2010 08:46:49 +0100 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)
Mon, 22 Mar 2010 00:51:18 +0100 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;
Mon, 22 Mar 2010 00:48:56 +0100 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;
Sun, 21 Mar 2010 22:24:04 +0100 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;
Sun, 21 Mar 2010 22:13:31 +0100 Logic.mk_of_sort convenience;
wenzelm [Sun, 21 Mar 2010 22:13:31 +0100] rev 35854
Logic.mk_of_sort convenience;
Sun, 21 Mar 2010 19:30:19 +0100 more explicit invented name;
wenzelm [Sun, 21 Mar 2010 19:30:19 +0100] rev 35853
more explicit invented name;
Sun, 21 Mar 2010 19:28:25 +0100 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';
Sun, 21 Mar 2010 19:04:46 +0100 do not open ML structures;
wenzelm [Sun, 21 Mar 2010 19:04:46 +0100] rev 35851
do not open ML structures;
Sun, 21 Mar 2010 17:28:35 +0100 modernized overloaded definitions;
wenzelm [Sun, 21 Mar 2010 17:28:35 +0100] rev 35850
modernized overloaded definitions;
Sun, 21 Mar 2010 17:12:31 +0100 standard headers;
wenzelm [Sun, 21 Mar 2010 17:12:31 +0100] rev 35849
standard headers;
Sun, 21 Mar 2010 16:51:37 +0100 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;
Sun, 21 Mar 2010 15:57:40 +0100 eliminated old constdefs;
wenzelm [Sun, 21 Mar 2010 15:57:40 +0100] rev 35847
eliminated old constdefs;
Sun, 21 Mar 2010 06:59:23 +0100 corrected setup for of_list
haftmann [Sun, 21 Mar 2010 06:59:23 +0100] rev 35846
corrected setup for of_list
Sat, 20 Mar 2010 17:33:11 +0100 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;
Sat, 20 Mar 2010 02:23:41 +0100 added lemma infinite_Un
Christian Urban <urbanc@in.tum.de> [Sat, 20 Mar 2010 02:23:41 +0100] rev 35844
added lemma infinite_Un
Fri, 19 Mar 2010 06:14:37 +0100 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.
Fri, 19 Mar 2010 00:47:23 +0100 typedef etc.: no constraints;
wenzelm [Fri, 19 Mar 2010 00:47:23 +0100] rev 35842
typedef etc.: no constraints;
Fri, 19 Mar 2010 00:46:08 +0100 allow sort constraints in HOL/typedef;
wenzelm [Fri, 19 Mar 2010 00:46:08 +0100] rev 35841
allow sort constraints in HOL/typedef;
Fri, 19 Mar 2010 00:43:49 +0100 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;
Fri, 19 Mar 2010 00:42:17 +0100 OuterParse.type_args_constrained;
wenzelm [Fri, 19 Mar 2010 00:42:17 +0100] rev 35839
OuterParse.type_args_constrained;
Fri, 19 Mar 2010 00:41:34 +0100 support type arguments with sort constraints;
wenzelm [Fri, 19 Mar 2010 00:41:34 +0100] rev 35838
support type arguments with sort constraints;
Thu, 18 Mar 2010 23:08:52 +0100 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;
Thu, 18 Mar 2010 23:00:18 +0100 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;
Thu, 18 Mar 2010 22:59:44 +0100 typedecl: no sort constraints;
wenzelm [Thu, 18 Mar 2010 22:59:44 +0100] rev 35835
typedecl: no sort constraints;
Thu, 18 Mar 2010 22:56:32 +0100 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;
Tue, 16 Mar 2010 16:27:28 +0100 Added product measure space
hoelzl [Tue, 16 Mar 2010 16:27:28 +0100] rev 35833
Added product measure space
Thu, 18 Mar 2010 14:52:11 +0100 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
Thu, 18 Mar 2010 13:59:20 +0100 merged
blanchet [Thu, 18 Mar 2010 13:59:20 +0100] rev 35831
merged
Thu, 18 Mar 2010 13:43:50 +0100 fix Mirabelle after renaming Sledgehammer structures
blanchet [Thu, 18 Mar 2010 13:43:50 +0100] rev 35830
fix Mirabelle after renaming Sledgehammer structures
Thu, 18 Mar 2010 13:14:54 +0100 merged
blanchet [Thu, 18 Mar 2010 13:14:54 +0100] rev 35829
merged
Thu, 18 Mar 2010 12:58:52 +0100 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"
Wed, 17 Mar 2010 19:37:44 +0100 renamed "ATP_Linkup" theory to "Sledgehammer"
blanchet [Wed, 17 Mar 2010 19:37:44 +0100] rev 35827
renamed "ATP_Linkup" theory to "Sledgehammer"
Wed, 17 Mar 2010 19:26:05 +0100 renamed Sledgehammer structures
blanchet [Wed, 17 Mar 2010 19:26:05 +0100] rev 35826
renamed Sledgehammer structures
Wed, 17 Mar 2010 18:16:31 +0100 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
Thu, 18 Mar 2010 13:57:00 +0100 merged
haftmann [Thu, 18 Mar 2010 13:57:00 +0100] rev 35824
merged
Thu, 18 Mar 2010 13:56:34 +0100 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
Thu, 18 Mar 2010 13:56:34 +0100 lemma swap_inj_on, swap_product
haftmann [Thu, 18 Mar 2010 13:56:34 +0100] rev 35822
lemma swap_inj_on, swap_product
Thu, 18 Mar 2010 13:56:33 +0100 meaningful transfer certificate
haftmann [Thu, 18 Mar 2010 13:56:33 +0100] rev 35821
meaningful transfer certificate
Thu, 18 Mar 2010 13:56:33 +0100 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
Thu, 18 Mar 2010 13:56:32 +0100 updated certificate
haftmann [Thu, 18 Mar 2010 13:56:32 +0100] rev 35819
updated certificate
Thu, 18 Mar 2010 13:56:32 +0100 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
Thu, 18 Mar 2010 13:56:32 +0100 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
Thu, 18 Mar 2010 13:56:31 +0100 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
Wed, 17 Mar 2010 19:55:07 +0100 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)
Wed, 17 Mar 2010 17:23:45 +0100 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
Wed, 17 Mar 2010 16:27:11 +0100 merged
blanchet [Wed, 17 Mar 2010 16:27:11 +0100] rev 35813
merged
Wed, 17 Mar 2010 16:26:08 +0100 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
Wed, 17 Mar 2010 16:11:48 +0100 minor additions to Nitpick docs
blanchet [Wed, 17 Mar 2010 16:11:48 +0100] rev 35811
minor additions to Nitpick docs
Wed, 17 Mar 2010 08:11:24 -0700 NEWS: Nat_Bijection library
huffman [Wed, 17 Mar 2010 08:11:24 -0700] rev 35810
NEWS: Nat_Bijection library
Wed, 17 Mar 2010 12:21:54 +0100 document "nitpick_choice_spec" attribute
blanchet [Wed, 17 Mar 2010 12:21:54 +0100] rev 35809
document "nitpick_choice_spec" attribute
Wed, 17 Mar 2010 12:01:01 +0100 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)
Wed, 17 Mar 2010 09:14:43 +0100 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
Tue, 16 Mar 2010 08:45:08 +0100 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
Tue, 16 Mar 2010 06:55:01 +0100 adjusted to changes in Finite_Set
haftmann [Tue, 16 Mar 2010 06:55:01 +0100] rev 35805
adjusted to changes in Finite_Set
Mon, 15 Mar 2010 22:22:28 +0100 merged
wenzelm [Mon, 15 Mar 2010 22:22:28 +0100] rev 35804
merged
Mon, 15 Mar 2010 17:34:03 +0100 merged
nipkow [Mon, 15 Mar 2010 17:34:03 +0100] rev 35803
merged
Mon, 15 Mar 2010 17:33:41 +0100 tuned inductions
nipkow [Mon, 15 Mar 2010 17:33:41 +0100] rev 35802
tuned inductions
Mon, 15 Mar 2010 21:59:28 +0100 tuned;
wenzelm [Mon, 15 Mar 2010 21:59:28 +0100] rev 35801
tuned;
Mon, 15 Mar 2010 21:57:35 +0100 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;
Mon, 15 Mar 2010 20:27:23 +0100 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;
Mon, 15 Mar 2010 18:59:16 +0100 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;
Mon, 15 Mar 2010 15:13:22 +0100 merged
haftmann [Mon, 15 Mar 2010 15:13:22 +0100] rev 35797
merged
Mon, 15 Mar 2010 15:13:07 +0100 corrected disastrous syntax declarations
haftmann [Mon, 15 Mar 2010 15:13:07 +0100] rev 35796
corrected disastrous syntax declarations
Mon, 15 Mar 2010 13:59:34 +0100 added stmaryrd for isasymSqinter
haftmann [Mon, 15 Mar 2010 13:59:34 +0100] rev 35795
added stmaryrd for isasymSqinter
Sun, 14 Mar 2010 19:48:33 -0700 use headers consistently
huffman [Sun, 14 Mar 2010 19:48:33 -0700] rev 35794
use headers consistently
Sun, 14 Mar 2010 19:47:13 -0700 no_document for theory Countable
huffman [Sun, 14 Mar 2010 19:47:13 -0700] rev 35793
no_document for theory Countable
Sun, 14 Mar 2010 14:10:36 -0700 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
Sun, 14 Mar 2010 14:10:05 -0700 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
Sun, 14 Mar 2010 15:50:17 +0100 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
Sun, 14 Mar 2010 14:36:56 +0100 tuned comment;
wenzelm [Sun, 14 Mar 2010 14:36:56 +0100] rev 35789
tuned comment;
Sun, 14 Mar 2010 14:31:24 +0100 observe standard header format;
wenzelm [Sun, 14 Mar 2010 14:31:24 +0100] rev 35788
observe standard header format;
Sun, 14 Mar 2010 14:29:30 +0100 expose formal text;
wenzelm [Sun, 14 Mar 2010 14:29:30 +0100] rev 35787
expose formal text;
Sun, 14 Mar 2010 14:10:21 +0100 localized @{class} and @{type};
wenzelm [Sun, 14 Mar 2010 14:10:21 +0100] rev 35786
localized @{class} and @{type};
Sun, 14 Mar 2010 00:51:58 -0800 move functions into holcf_library.ML
huffman [Sun, 14 Mar 2010 00:51:58 -0800] rev 35785
move functions into holcf_library.ML
Sun, 14 Mar 2010 00:40:04 -0800 simplify definition of when combinators
huffman [Sun, 14 Mar 2010 00:40:04 -0800] rev 35784
simplify definition of when combinators
Sat, 13 Mar 2010 22:00:34 -0800 declare case_names for various induction rules
huffman [Sat, 13 Mar 2010 22:00:34 -0800] rev 35783
declare case_names for various induction rules
Sat, 13 Mar 2010 21:07:20 -0800 add case name 'adm' for infinite induction rules
huffman [Sat, 13 Mar 2010 21:07:20 -0800] rev 35782
add case name 'adm' for infinite induction rules
Sat, 13 Mar 2010 20:15:25 -0800 renamed some lemmas generated by the domain package
huffman [Sat, 13 Mar 2010 20:15:25 -0800] rev 35781
renamed some lemmas generated by the domain package
Sat, 13 Mar 2010 19:06:18 -0800 use Simplifier.context to avoid 'no proof context in simpset' errors from fixrec_simp after theory merge
huffman [Sat, 13 Mar 2010 19:06:18 -0800] rev 35780
use Simplifier.context to avoid 'no proof context in simpset' errors from fixrec_simp after theory merge
Sat, 13 Mar 2010 18:16:48 -0800 fixpat command prints legacy_feature warning
huffman [Sat, 13 Mar 2010 18:16:48 -0800] rev 35779
fixpat command prints legacy_feature warning
Sat, 13 Mar 2010 17:36:53 -0800 merged
huffman [Sat, 13 Mar 2010 17:36:53 -0800] rev 35778
merged
Sat, 13 Mar 2010 17:05:34 -0800 pass binding as argument to add_domain_constructors; proper binding for case combinator
huffman [Sat, 13 Mar 2010 17:05:34 -0800] rev 35777
pass binding as argument to add_domain_constructors; proper binding for case combinator
Sat, 13 Mar 2010 16:48:57 -0800 pass domain binding as argument to Domain_Theorems.theorems; proper qualified bindings for theorem names
huffman [Sat, 13 Mar 2010 16:48:57 -0800] rev 35776
pass domain binding as argument to Domain_Theorems.theorems; proper qualified bindings for theorem names
Sat, 13 Mar 2010 15:51:12 -0800 pass take_info as argument to Domain_Theorems.theorems
huffman [Sat, 13 Mar 2010 15:51:12 -0800] rev 35775
pass take_info as argument to Domain_Theorems.theorems
Sat, 13 Mar 2010 15:18:25 -0800 replace some string arguments with bindings
huffman [Sat, 13 Mar 2010 15:18:25 -0800] rev 35774
replace some string arguments with bindings
Sat, 13 Mar 2010 14:30:38 -0800 more consistent use of qualified bindings
huffman [Sat, 13 Mar 2010 14:30:38 -0800] rev 35773
more consistent use of qualified bindings
Sat, 13 Mar 2010 14:26:26 -0800 avoid unnecessary primed variable names
huffman [Sat, 13 Mar 2010 14:26:26 -0800] rev 35772
avoid unnecessary primed variable names
Sat, 13 Mar 2010 12:24:50 -0800 remove redundant lemmas
huffman [Sat, 13 Mar 2010 12:24:50 -0800] rev 35771
remove redundant lemmas
Sat, 13 Mar 2010 10:38:38 -0800 fixes to allow using fixrec_simp inside a locale, with test in ex/Fixrec_ex.thy
huffman [Sat, 13 Mar 2010 10:38:38 -0800] rev 35770
fixes to allow using fixrec_simp inside a locale, with test in ex/Fixrec_ex.thy
Sat, 13 Mar 2010 10:00:45 -0800 fixrec now generates qualified theorem names
huffman [Sat, 13 Mar 2010 10:00:45 -0800] rev 35769
fixrec now generates qualified theorem names
Sat, 13 Mar 2010 09:32:19 -0800 no_document for Infinite_Set in HOLCF
huffman [Sat, 13 Mar 2010 09:32:19 -0800] rev 35768
no_document for Infinite_Set in HOLCF
Sat, 13 Mar 2010 20:44:12 +0100 removed unused Args.maxidx_values and Element.generalize_facts;
wenzelm [Sat, 13 Mar 2010 20:44:12 +0100] rev 35767
removed unused Args.maxidx_values and Element.generalize_facts;
(0) -30000 -10000 -3000 -1000 -240 +240 +1000 +3000 +10000 +30000 tip