Thu, 18 Aug 2011 13:55:26 +0200 observe distinction between sets and predicates more properly
haftmann [Thu, 18 Aug 2011 13:55:26 +0200] rev 44278
observe distinction between sets and predicates more properly
Thu, 18 Aug 2011 13:25:17 +0200 moved fundamental lemma fun_eq_iff to theory HOL; tuned whitespace
haftmann [Thu, 18 Aug 2011 13:25:17 +0200] rev 44277
moved fundamental lemma fun_eq_iff to theory HOL; tuned whitespace
Thu, 18 Aug 2011 13:10:24 +0200 avoid case-sensitive name for example theory
haftmann [Thu, 18 Aug 2011 13:10:24 +0200] rev 44276
avoid case-sensitive name for example theory
Thu, 18 Aug 2011 17:42:35 +0200 merged
nipkow [Thu, 18 Aug 2011 17:42:35 +0200] rev 44275
merged
Thu, 18 Aug 2011 17:42:18 +0200 case_names NEWS
nipkow [Thu, 18 Aug 2011 17:42:18 +0200] rev 44274
case_names NEWS
Thu, 18 Aug 2011 17:00:15 +0200 adding documentation about simps equation in the inductive package
bulwahn [Thu, 18 Aug 2011 17:00:15 +0200] rev 44273
adding documentation about simps equation in the inductive package
Thu, 18 Aug 2011 12:06:17 +0200 activating narrowing-based quickcheck by default
bulwahn [Thu, 18 Aug 2011 12:06:17 +0200] rev 44272
activating narrowing-based quickcheck by default
Thu, 18 Aug 2011 18:07:40 +0200 more precise treatment of exception nesting and serial numbers;
wenzelm [Thu, 18 Aug 2011 18:07:40 +0200] rev 44271
more precise treatment of exception nesting and serial numbers;
Thu, 18 Aug 2011 17:53:32 +0200 more careful treatment of exception serial numbers, with propagation to message channel;
wenzelm [Thu, 18 Aug 2011 17:53:32 +0200] rev 44270
more careful treatment of exception serial numbers, with propagation to message channel;
Thu, 18 Aug 2011 17:30:47 +0200 updated sequential version (cf. b94951f06e48);
wenzelm [Thu, 18 Aug 2011 17:30:47 +0200] rev 44269
updated sequential version (cf. b94951f06e48);
Thu, 18 Aug 2011 16:07:58 +0200 tuned comments;
wenzelm [Thu, 18 Aug 2011 16:07:58 +0200] rev 44268
tuned comments;
Thu, 18 Aug 2011 15:51:34 +0200 tuned document;
wenzelm [Thu, 18 Aug 2011 15:51:34 +0200] rev 44267
tuned document; tuned proofs;
Thu, 18 Aug 2011 15:39:00 +0200 clarified Par_Exn.release_first: prefer plain exn, before falling back on full pack of parallel exceptions;
wenzelm [Thu, 18 Aug 2011 15:39:00 +0200] rev 44266
clarified Par_Exn.release_first: prefer plain exn, before falling back on full pack of parallel exceptions;
Thu, 18 Aug 2011 15:37:01 +0200 export Par_List.managed_results, to enable specific treatment of results apart from default Par_Exn.release_first;
wenzelm [Thu, 18 Aug 2011 15:37:01 +0200] rev 44265
export Par_List.managed_results, to enable specific treatment of results apart from default Par_Exn.release_first;
Thu, 18 Aug 2011 15:15:43 +0200 tune Par_Exn.make: balance merge;
wenzelm [Thu, 18 Aug 2011 15:15:43 +0200] rev 44264
tune Par_Exn.make: balance merge; clarified Par_Exn.dest: later exceptions first;
Thu, 18 Aug 2011 16:52:19 +0900 Quotient_Examples/DList: explicit proof of remdups_eq_member_eq needed for explicit set type.
Cezary Kaliszyk <kaliszyk@in.tum.de> [Thu, 18 Aug 2011 16:52:19 +0900] rev 44263
Quotient_Examples/DList: explicit proof of remdups_eq_member_eq needed for explicit set type.
Wed, 17 Aug 2011 15:12:34 -0700 merged
huffman [Wed, 17 Aug 2011 15:12:34 -0700] rev 44262
merged
Wed, 17 Aug 2011 15:03:30 -0700 HOL-IMP: respect set/pred distinction
huffman [Wed, 17 Aug 2011 15:03:30 -0700] rev 44261
HOL-IMP: respect set/pred distinction
Wed, 17 Aug 2011 15:02:17 -0700 Determinants.thy: avoid using mem_def/Collect_def
huffman [Wed, 17 Aug 2011 15:02:17 -0700] rev 44260
Determinants.thy: avoid using mem_def/Collect_def
Wed, 17 Aug 2011 14:42:59 -0700 Wfrec.thy: respect set/pred distinction
huffman [Wed, 17 Aug 2011 14:42:59 -0700] rev 44259
Wfrec.thy: respect set/pred distinction
Thu, 18 Aug 2011 00:02:44 +0200 follow updates of Isabelle/Pure;
wenzelm [Thu, 18 Aug 2011 00:02:44 +0200] rev 44258
follow updates of Isabelle/Pure;
Wed, 17 Aug 2011 23:41:47 +0200 merged
wenzelm [Wed, 17 Aug 2011 23:41:47 +0200] rev 44257
merged
Wed, 17 Aug 2011 14:32:48 -0700 IsaMakefile: target HOLCF-Library now compiles HOL/HOLCF/Library instead of HOL/Library
huffman [Wed, 17 Aug 2011 14:32:48 -0700] rev 44256
IsaMakefile: target HOLCF-Library now compiles HOL/HOLCF/Library instead of HOL/Library
Wed, 17 Aug 2011 13:10:49 -0700 merged
huffman [Wed, 17 Aug 2011 13:10:49 -0700] rev 44255
merged
Wed, 17 Aug 2011 13:10:11 -0700 Lim.thy: generalize and simplify proofs of LIM/LIMSEQ theorems
huffman [Wed, 17 Aug 2011 13:10:11 -0700] rev 44254
Lim.thy: generalize and simplify proofs of LIM/LIMSEQ theorems
Wed, 17 Aug 2011 11:39:09 -0700 add lemma tendsto_compose_eventually; use it to shorten some proofs
huffman [Wed, 17 Aug 2011 11:39:09 -0700] rev 44253
add lemma tendsto_compose_eventually; use it to shorten some proofs
Wed, 17 Aug 2011 11:07:32 -0700 Topology_Euclidean_Space.thy: simplify some proofs
huffman [Wed, 17 Aug 2011 11:07:32 -0700] rev 44252
Topology_Euclidean_Space.thy: simplify some proofs
Wed, 17 Aug 2011 11:06:39 -0700 add lemma metric_tendsto_imp_tendsto
huffman [Wed, 17 Aug 2011 11:06:39 -0700] rev 44251
add lemma metric_tendsto_imp_tendsto
Wed, 17 Aug 2011 09:59:10 -0700 simplify proofs of lemmas open_interval, closed_interval
huffman [Wed, 17 Aug 2011 09:59:10 -0700] rev 44250
simplify proofs of lemmas open_interval, closed_interval
Wed, 17 Aug 2011 23:37:23 +0200 identify parallel exceptions where they emerge first -- to achieve unique results within evaluation graph;
wenzelm [Wed, 17 Aug 2011 23:37:23 +0200] rev 44249
identify parallel exceptions where they emerge first -- to achieve unique results within evaluation graph;
Wed, 17 Aug 2011 22:25:00 +0200 clarified Par_Exn.release_first: traverse topmost list structure only, not arbitrary depths of nested Par_Exn;
wenzelm [Wed, 17 Aug 2011 22:25:00 +0200] rev 44248
clarified Par_Exn.release_first: traverse topmost list structure only, not arbitrary depths of nested Par_Exn;
Wed, 17 Aug 2011 22:14:22 +0200 more systematic handling of parallel exceptions;
wenzelm [Wed, 17 Aug 2011 22:14:22 +0200] rev 44247
more systematic handling of parallel exceptions; distinguish exception concatanation EXCEPTIONS from parallel Par_Exn;
Wed, 17 Aug 2011 20:08:36 +0200 tuned signature;
wenzelm [Wed, 17 Aug 2011 20:08:36 +0200] rev 44246
tuned signature;
Wed, 17 Aug 2011 18:52:21 +0200 merged
haftmann [Wed, 17 Aug 2011 18:52:21 +0200] rev 44245
merged
Wed, 17 Aug 2011 18:51:27 +0200 merged
haftmann [Wed, 17 Aug 2011 18:51:27 +0200] rev 44244
merged
Wed, 17 Aug 2011 07:13:13 +0200 merged
haftmann [Wed, 17 Aug 2011 07:13:13 +0200] rev 44243
merged
Tue, 16 Aug 2011 19:47:50 +0200 avoid Collect_def in proof
haftmann [Tue, 16 Aug 2011 19:47:50 +0200] rev 44242
avoid Collect_def in proof
Wed, 17 Aug 2011 18:05:31 +0200 modernized signature of Term.absfree/absdummy;
wenzelm [Wed, 17 Aug 2011 18:05:31 +0200] rev 44241
modernized signature of Term.absfree/absdummy; eliminated obsolete Term.list_abs_free;
Wed, 17 Aug 2011 16:46:58 +0200 improved default context for ML toplevel pretty-printing;
wenzelm [Wed, 17 Aug 2011 16:46:58 +0200] rev 44240
improved default context for ML toplevel pretty-printing;
Wed, 17 Aug 2011 16:30:38 +0200 less verbosity for 'function' and 'fun': observe "int" flag more carefully (cf. a32ca9165928);
wenzelm [Wed, 17 Aug 2011 16:30:38 +0200] rev 44239
less verbosity for 'function' and 'fun': observe "int" flag more carefully (cf. a32ca9165928);
Wed, 17 Aug 2011 16:01:27 +0200 some convenience actions/shortcuts for control symbols;
wenzelm [Wed, 17 Aug 2011 16:01:27 +0200] rev 44238
some convenience actions/shortcuts for control symbols;
Wed, 17 Aug 2011 15:14:48 +0200 export Function_Fun.fun_config for user convenience;
wenzelm [Wed, 17 Aug 2011 15:14:48 +0200] rev 44237
export Function_Fun.fun_config for user convenience;
Wed, 17 Aug 2011 13:14:20 +0200 moved theory Nested_Environment to HOL-Unix (a bit too specific for HOL-Library);
wenzelm [Wed, 17 Aug 2011 13:14:20 +0200] rev 44236
moved theory Nested_Environment to HOL-Unix (a bit too specific for HOL-Library);
Wed, 17 Aug 2011 10:03:58 +0200 distinguish THF syntax with and without choice (Satallax vs. LEO-II)
blanchet [Wed, 17 Aug 2011 10:03:58 +0200] rev 44235
distinguish THF syntax with and without choice (Satallax vs. LEO-II)
Tue, 16 Aug 2011 15:02:20 -0700 merged
huffman [Tue, 16 Aug 2011 15:02:20 -0700] rev 44234
merged
Tue, 16 Aug 2011 09:31:23 -0700 add simp rules for isCont
huffman [Tue, 16 Aug 2011 09:31:23 -0700] rev 44233
add simp rules for isCont
Tue, 16 Aug 2011 23:39:58 +0200 updated keywords -- old codegen is no longer in Pure;
wenzelm [Tue, 16 Aug 2011 23:39:58 +0200] rev 44232
updated keywords -- old codegen is no longer in Pure;
Tue, 16 Aug 2011 23:39:30 +0200 include HOL-Library keywords for the sake of recdef;
wenzelm [Tue, 16 Aug 2011 23:39:30 +0200] rev 44231
include HOL-Library keywords for the sake of recdef;
Tue, 16 Aug 2011 23:25:02 +0200 merged
wenzelm [Tue, 16 Aug 2011 23:25:02 +0200] rev 44230
merged
Tue, 16 Aug 2011 13:07:52 -0700 Multivariate_Analysis includes Determinants.thy, but doesn't import it by default
huffman [Tue, 16 Aug 2011 13:07:52 -0700] rev 44229
Multivariate_Analysis includes Determinants.thy, but doesn't import it by default
Tue, 16 Aug 2011 07:56:17 -0700 get Multivariate_Analysis/Determinants.thy compiled and working again
huffman [Tue, 16 Aug 2011 07:56:17 -0700] rev 44228
get Multivariate_Analysis/Determinants.thy compiled and working again
Tue, 16 Aug 2011 07:06:54 -0700 get Library/Permutations.thy compiled and working again
huffman [Tue, 16 Aug 2011 07:06:54 -0700] rev 44227
get Library/Permutations.thy compiled and working again
Tue, 16 Aug 2011 23:17:26 +0200 workaround for Cygwin, to make it work in the important special case without extra files;
wenzelm [Tue, 16 Aug 2011 23:17:26 +0200] rev 44226
workaround for Cygwin, to make it work in the important special case without extra files;
Tue, 16 Aug 2011 22:48:31 +0200 more robust Thy_Header.base_name, with minimal assumptions about path syntax;
wenzelm [Tue, 16 Aug 2011 22:48:31 +0200] rev 44225
more robust Thy_Header.base_name, with minimal assumptions about path syntax; Isabelle.buffer_path: keep platform syntax;
Tue, 16 Aug 2011 21:54:06 +0200 tuned message;
wenzelm [Tue, 16 Aug 2011 21:54:06 +0200] rev 44224
tuned message;
Tue, 16 Aug 2011 21:50:53 +0200 more robust treatment of node dependencies in incremental edits;
wenzelm [Tue, 16 Aug 2011 21:50:53 +0200] rev 44223
more robust treatment of node dependencies in incremental edits;
Tue, 16 Aug 2011 21:13:52 +0200 use full .thy file name as node name, which makes MiscUtilities.resolveSymlinks/File.getCanonicalPath more predictable;
wenzelm [Tue, 16 Aug 2011 21:13:52 +0200] rev 44222
use full .thy file name as node name, which makes MiscUtilities.resolveSymlinks/File.getCanonicalPath more predictable; more robust treatment of node dependencies; misc tuning;
Tue, 16 Aug 2011 12:06:49 +0200 omit MiscUtilities.resolveSymlinks for now -- odd effects on case-insensible file-system;
wenzelm [Tue, 16 Aug 2011 12:06:49 +0200] rev 44221
omit MiscUtilities.resolveSymlinks for now -- odd effects on case-insensible file-system;
Mon, 15 Aug 2011 19:42:52 -0700 merged
huffman [Mon, 15 Aug 2011 19:42:52 -0700] rev 44220
merged
Mon, 15 Aug 2011 18:35:36 -0700 generalize lemmas open_Collect_less, closed_Collect_le, closed_Collect_eq to class topological_space
huffman [Mon, 15 Aug 2011 18:35:36 -0700] rev 44219
generalize lemmas open_Collect_less, closed_Collect_le, closed_Collect_eq to class topological_space
Mon, 15 Aug 2011 16:48:05 -0700 add lemma tendsto_compose
huffman [Mon, 15 Aug 2011 16:48:05 -0700] rev 44218
add lemma tendsto_compose
Mon, 15 Aug 2011 16:18:13 -0700 remove extraneous subsection heading
huffman [Mon, 15 Aug 2011 16:18:13 -0700] rev 44217
remove extraneous subsection heading
Mon, 15 Aug 2011 15:11:55 -0700 generalized lemma closed_Collect_eq
huffman [Mon, 15 Aug 2011 15:11:55 -0700] rev 44216
generalized lemma closed_Collect_eq
Mon, 15 Aug 2011 14:50:24 -0700 remove duplicate lemma disjoint_iff
huffman [Mon, 15 Aug 2011 14:50:24 -0700] rev 44215
remove duplicate lemma disjoint_iff
Mon, 15 Aug 2011 14:29:17 -0700 Library/Product_Vector.thy: class instances for t0_space, t1_space, and t2_space
huffman [Mon, 15 Aug 2011 14:29:17 -0700] rev 44214
Library/Product_Vector.thy: class instances for t0_space, t1_space, and t2_space
Mon, 15 Aug 2011 14:09:39 -0700 add lemmas open_Collect_less, closed_Collect_le, closed_Collect_eq;
huffman [Mon, 15 Aug 2011 14:09:39 -0700] rev 44213
add lemmas open_Collect_less, closed_Collect_le, closed_Collect_eq; simplify and generalize some proofs;
Mon, 15 Aug 2011 12:18:34 -0700 generalize lemma continuous_uniform_limit to class metric_space
huffman [Mon, 15 Aug 2011 12:18:34 -0700] rev 44212
generalize lemma continuous_uniform_limit to class metric_space
Mon, 15 Aug 2011 12:13:46 -0700 remove duplicate lemmas eventually_conjI, eventually_and, eventually_false
huffman [Mon, 15 Aug 2011 12:13:46 -0700] rev 44211
remove duplicate lemmas eventually_conjI, eventually_and, eventually_false
Mon, 15 Aug 2011 10:49:48 -0700 Topology_Euclidean_Space.thy: organize section headings
huffman [Mon, 15 Aug 2011 10:49:48 -0700] rev 44210
Topology_Euclidean_Space.thy: organize section headings
Mon, 15 Aug 2011 09:08:17 -0700 simplify some proofs
huffman [Mon, 15 Aug 2011 09:08:17 -0700] rev 44209
simplify some proofs
Sun, 14 Aug 2011 13:04:57 -0700 generalize lemma convergent_subseq_convergent
huffman [Sun, 14 Aug 2011 13:04:57 -0700] rev 44208
generalize lemma convergent_subseq_convergent
Sun, 14 Aug 2011 11:44:12 -0700 locale-ize some definitions, so perfect_space and heine_borel can inherit from the proper superclasses
huffman [Sun, 14 Aug 2011 11:44:12 -0700] rev 44207
locale-ize some definitions, so perfect_space and heine_borel can inherit from the proper superclasses
Sun, 14 Aug 2011 10:47:47 -0700 locale-ize some constant definitions, so complete_space can inherit from metric_space
huffman [Sun, 14 Aug 2011 10:47:47 -0700] rev 44206
locale-ize some constant definitions, so complete_space can inherit from metric_space
Sun, 14 Aug 2011 10:25:43 -0700 generalize constant 'lim' and limit uniqueness theorems to class t2_space
huffman [Sun, 14 Aug 2011 10:25:43 -0700] rev 44205
generalize constant 'lim' and limit uniqueness theorems to class t2_space
Tue, 16 Aug 2011 07:17:15 +0900 Quotient Package: make quotient_type work with separate set type
Cezary Kaliszyk <kaliszyk@in.tum.de> [Tue, 16 Aug 2011 07:17:15 +0900] rev 44204
Quotient Package: make quotient_type work with separate set type
Mon, 15 Aug 2011 22:31:17 +0200 updated README;
wenzelm [Mon, 15 Aug 2011 22:31:17 +0200] rev 44203
updated README;
Mon, 15 Aug 2011 21:54:32 +0200 touch descendants of edited nodes;
wenzelm [Mon, 15 Aug 2011 21:54:32 +0200] rev 44202
touch descendants of edited nodes; more precise handling of Graph exceptions;
Mon, 15 Aug 2011 21:05:30 +0200 parellel scheduling of node edits and execution;
wenzelm [Mon, 15 Aug 2011 21:05:30 +0200] rev 44201
parellel scheduling of node edits and execution;
Mon, 15 Aug 2011 20:38:16 +0200 tuned error message;
wenzelm [Mon, 15 Aug 2011 20:38:16 +0200] rev 44200
tuned error message;
Mon, 15 Aug 2011 20:19:41 +0200 retrieve imports from document state, with fall-back on theory loader for preloaded theories;
wenzelm [Mon, 15 Aug 2011 20:19:41 +0200] rev 44199
retrieve imports from document state, with fall-back on theory loader for preloaded theories; misc tuning;
Mon, 15 Aug 2011 19:27:55 +0200 explicit check of finished evaluation;
wenzelm [Mon, 15 Aug 2011 19:27:55 +0200] rev 44198
explicit check of finished evaluation;
Mon, 15 Aug 2011 16:38:42 +0200 refined Document.edit: less stateful update via Graph.schedule;
wenzelm [Mon, 15 Aug 2011 16:38:42 +0200] rev 44197
refined Document.edit: less stateful update via Graph.schedule; clarified node result -- more direct get_theory; clarified Document.joint_commands;
Mon, 15 Aug 2011 14:54:36 +0200 simplified exec: eliminated unused status flag;
wenzelm [Mon, 15 Aug 2011 14:54:36 +0200] rev 44196
simplified exec: eliminated unused status flag;
Sun, 14 Aug 2011 08:45:38 -0700 consistently use variable name 'F' for filters
huffman [Sun, 14 Aug 2011 08:45:38 -0700] rev 44195
consistently use variable name 'F' for filters
Sun, 14 Aug 2011 07:54:24 -0700 generalize lemmas about LIM and LIMSEQ to tendsto
huffman [Sun, 14 Aug 2011 07:54:24 -0700] rev 44194
generalize lemmas about LIM and LIMSEQ to tendsto
Sat, 13 Aug 2011 18:10:14 -0700 HOL-Nominal-Examples: respect distinction between sets and functions
huffman [Sat, 13 Aug 2011 18:10:14 -0700] rev 44193
HOL-Nominal-Examples: respect distinction between sets and functions
Sat, 13 Aug 2011 22:04:07 +0200 less verbosity in batch mode -- spam reduction and notable performance improvement;
wenzelm [Sat, 13 Aug 2011 22:04:07 +0200] rev 44192
less verbosity in batch mode -- spam reduction and notable performance improvement; clarified Proof_Display.print_consts;
Sat, 13 Aug 2011 21:28:01 +0200 merged
wenzelm [Sat, 13 Aug 2011 21:28:01 +0200] rev 44191
merged
Sat, 13 Aug 2011 07:56:55 -0700 HOL-Hahn_Banach: use Set_Algebras library
huffman [Sat, 13 Aug 2011 07:56:55 -0700] rev 44190
HOL-Hahn_Banach: use Set_Algebras library
Sat, 13 Aug 2011 07:39:35 -0700 ex/Quickcheck_Examples.thy: respect distinction between sets and functions
huffman [Sat, 13 Aug 2011 07:39:35 -0700] rev 44189
ex/Quickcheck_Examples.thy: respect distinction between sets and functions
Sat, 13 Aug 2011 21:06:01 +0200 clarified Toplevel.end_theory;
wenzelm [Sat, 13 Aug 2011 21:06:01 +0200] rev 44188
clarified Toplevel.end_theory;
Sat, 13 Aug 2011 20:49:41 +0200 simplified Toplevel.init_theory: discontinued special name argument;
wenzelm [Sat, 13 Aug 2011 20:49:41 +0200] rev 44187
simplified Toplevel.init_theory: discontinued special name argument;
Sat, 13 Aug 2011 20:41:29 +0200 simplified Toplevel.init_theory: discontinued special master argument;
wenzelm [Sat, 13 Aug 2011 20:41:29 +0200] rev 44186
simplified Toplevel.init_theory: discontinued special master argument;
Sat, 13 Aug 2011 20:20:36 +0200 provide node header via Scala layer;
wenzelm [Sat, 13 Aug 2011 20:20:36 +0200] rev 44185
provide node header via Scala layer; clarified node edit Clear: retain header information; run_command: node info via document model, error handling within transaction; node names without ".thy" suffix, to coincide with traditional theory loader treatment;
Sat, 13 Aug 2011 16:07:26 +0200 reduced verbosity;
wenzelm [Sat, 13 Aug 2011 16:07:26 +0200] rev 44184
reduced verbosity;
Sat, 13 Aug 2011 16:04:28 +0200 tuned signature;
wenzelm [Sat, 13 Aug 2011 16:04:28 +0200] rev 44183
tuned signature;
Sat, 13 Aug 2011 15:59:26 +0200 clarified node header -- exclude master_dir;
wenzelm [Sat, 13 Aug 2011 15:59:26 +0200] rev 44182
clarified node header -- exclude master_dir;
Sat, 13 Aug 2011 13:48:26 +0200 tuned;
wenzelm [Sat, 13 Aug 2011 13:48:26 +0200] rev 44181
tuned;
Sat, 13 Aug 2011 13:42:35 +0200 maintain node header;
wenzelm [Sat, 13 Aug 2011 13:42:35 +0200] rev 44180
maintain node header; misc tuning and clarification;
Sat, 13 Aug 2011 12:23:51 +0200 removed unused lemma; removed old-style ;
kleing [Sat, 13 Aug 2011 12:23:51 +0200] rev 44179
removed unused lemma; removed old-style ;
Sat, 13 Aug 2011 12:05:52 +0200 point isatest-statistics to the right afp log files
kleing [Sat, 13 Aug 2011 12:05:52 +0200] rev 44178
point isatest-statistics to the right afp log files
Sat, 13 Aug 2011 11:57:13 +0200 IMP/Util distinguishes between sets and functions again; imported only where used.
kleing [Sat, 13 Aug 2011 11:57:13 +0200] rev 44177
IMP/Util distinguishes between sets and functions again; imported only where used.
Fri, 12 Aug 2011 20:55:22 -0700 remove redundant lemma setsum_norm in favor of norm_setsum;
huffman [Fri, 12 Aug 2011 20:55:22 -0700] rev 44176
remove redundant lemma setsum_norm in favor of norm_setsum; remove finiteness assumption from setsum_norm_le;
Fri, 12 Aug 2011 16:47:53 -0700 merged
huffman [Fri, 12 Aug 2011 16:47:53 -0700] rev 44175
merged
Fri, 12 Aug 2011 14:45:50 -0700 make more HOL theories work with separate set type
huffman [Fri, 12 Aug 2011 14:45:50 -0700] rev 44174
make more HOL theories work with separate set type
Sat, 13 Aug 2011 00:34:54 +0200 immediate fork of initial workers -- avoid 5 ticks (250ms) for adaptive scheme (a07558eb5029);
wenzelm [Sat, 13 Aug 2011 00:34:54 +0200] rev 44173
immediate fork of initial workers -- avoid 5 ticks (250ms) for adaptive scheme (a07558eb5029); more careful treatment of last_round on startup/shutdown;
Fri, 12 Aug 2011 23:29:28 +0200 merged
wenzelm [Fri, 12 Aug 2011 23:29:28 +0200] rev 44172
merged
Fri, 12 Aug 2011 09:17:30 -0700 merged
huffman [Fri, 12 Aug 2011 09:17:30 -0700] rev 44171
merged
Fri, 12 Aug 2011 09:17:24 -0700 make Multivariate_Analysis work with separate set type
huffman [Fri, 12 Aug 2011 09:17:24 -0700] rev 44170
make Multivariate_Analysis work with separate set type
Fri, 12 Aug 2011 07:18:28 -0700 make HOLCF work with separate set type
huffman [Fri, 12 Aug 2011 07:18:28 -0700] rev 44169
make HOLCF work with separate set type
Fri, 12 Aug 2011 07:13:12 -0700 merged
huffman [Fri, 12 Aug 2011 07:13:12 -0700] rev 44168
merged
Thu, 11 Aug 2011 14:24:05 -0700 avoid duplicate rule warnings
huffman [Thu, 11 Aug 2011 14:24:05 -0700] rev 44167
avoid duplicate rule warnings
Thu, 11 Aug 2011 13:05:56 -0700 modify euclidean_space class to include basis set
huffman [Thu, 11 Aug 2011 13:05:56 -0700] rev 44166
modify euclidean_space class to include basis set
Thu, 11 Aug 2011 09:11:15 -0700 remove lemma stupid_ext
huffman [Thu, 11 Aug 2011 09:11:15 -0700] rev 44165
remove lemma stupid_ext
Fri, 12 Aug 2011 17:01:30 +0200 documented extended version of case_names attribute
nipkow [Fri, 12 Aug 2011 17:01:30 +0200] rev 44164
documented extended version of case_names attribute
Fri, 12 Aug 2011 22:10:49 +0200 normalized theory dependencies wrt. file_store;
wenzelm [Fri, 12 Aug 2011 22:10:49 +0200] rev 44163
normalized theory dependencies wrt. file_store;
Fri, 12 Aug 2011 20:32:25 +0200 general Graph.schedule;
wenzelm [Fri, 12 Aug 2011 20:32:25 +0200] rev 44162
general Graph.schedule;
Fri, 12 Aug 2011 15:30:12 +0200 allow "$" within basic path elements (NB: initial "$" refers to path variable);
wenzelm [Fri, 12 Aug 2011 15:30:12 +0200] rev 44161
allow "$" within basic path elements (NB: initial "$" refers to path variable);
Fri, 12 Aug 2011 15:28:30 +0200 clarified document model header: master_dir (native wrt. editor, potentially URL) and node_name (full canonical path);
wenzelm [Fri, 12 Aug 2011 15:28:30 +0200] rev 44160
clarified document model header: master_dir (native wrt. editor, potentially URL) and node_name (full canonical path);
Fri, 12 Aug 2011 12:03:17 +0200 simplified class Thy_Header;
wenzelm [Fri, 12 Aug 2011 12:03:17 +0200] rev 44159
simplified class Thy_Header;
(0) -30000 -10000 -3000 -1000 -120 +120 +1000 +3000 +10000 +30000 tip