Tue, 13 Jan 2009 08:58:56 -0800 define polynomial multiplication using poly_rec
huffman [Tue, 13 Jan 2009 08:58:56 -0800] rev 29474
define polynomial multiplication using poly_rec
Tue, 13 Jan 2009 08:20:12 -0800 merged.
huffman [Tue, 13 Jan 2009 08:20:12 -0800] rev 29473
merged.
Tue, 13 Jan 2009 08:19:14 -0800 declare smult rules [simp]
huffman [Tue, 13 Jan 2009 08:19:14 -0800] rev 29472
declare smult rules [simp]
Tue, 13 Jan 2009 07:40:05 -0800 simplify proof of coeff_mult_degree_sum
huffman [Tue, 13 Jan 2009 07:40:05 -0800] rev 29471
simplify proof of coeff_mult_degree_sum
Tue, 13 Jan 2009 06:57:08 -0800 convert Deriv.thy to use new Polynomial library (incomplete)
huffman [Tue, 13 Jan 2009 06:57:08 -0800] rev 29470
convert Deriv.thy to use new Polynomial library (incomplete)
Tue, 13 Jan 2009 06:55:13 -0800 Integration imports ATP_Linkup (for metis)
huffman [Tue, 13 Jan 2009 06:55:13 -0800] rev 29469
Integration imports ATP_Linkup (for metis)
Tue, 13 Jan 2009 22:20:49 +0100 misc internal rearrangements;
wenzelm [Tue, 13 Jan 2009 22:20:49 +0100] rev 29468
misc internal rearrangements; fold_entries: really start from start, or optional position; added find_first_entries, find_first_entries; insert_entry: always invalidate next state; added refresh_states (partial version);
Tue, 13 Jan 2009 17:34:12 +0100 replaced sys_error by plain error;
wenzelm [Tue, 13 Jan 2009 17:34:12 +0100] rev 29467
replaced sys_error by plain error; some basic operations on command entries within a document;
Tue, 13 Jan 2009 14:31:02 +0100 merged
wenzelm [Tue, 13 Jan 2009 14:31:02 +0100] rev 29466
merged
Mon, 12 Jan 2009 23:36:30 -0800 change dvd_minus_iff, minus_dvd_iff from [iff] to [simp] (due to problems with Library/Primes.thy)
huffman [Mon, 12 Jan 2009 23:36:30 -0800] rev 29465
change dvd_minus_iff, minus_dvd_iff from [iff] to [simp] (due to problems with Library/Primes.thy)
Mon, 12 Jan 2009 22:41:08 -0800 convert Fundamental_Theorem_Algebra.thy to use new Polynomial library
huffman [Mon, 12 Jan 2009 22:41:08 -0800] rev 29464
convert Fundamental_Theorem_Algebra.thy to use new Polynomial library
Mon, 12 Jan 2009 22:18:51 -0800 add Polynomial.thy to makefile
huffman [Mon, 12 Jan 2009 22:18:51 -0800] rev 29463
add Polynomial.thy to makefile
Mon, 12 Jan 2009 22:16:35 -0800 add lemmas poly_power, poly_roots_finite
huffman [Mon, 12 Jan 2009 22:16:35 -0800] rev 29462
add lemmas poly_power, poly_roots_finite
Mon, 12 Jan 2009 12:10:41 -0800 declare dvd_minus_iff and minus_dvd_iff [iff]
huffman [Mon, 12 Jan 2009 12:10:41 -0800] rev 29461
declare dvd_minus_iff and minus_dvd_iff [iff]
Mon, 12 Jan 2009 12:09:54 -0800 new lemmas about synthetic_div; declare degree_pCons_eq_if [simp]
huffman [Mon, 12 Jan 2009 12:09:54 -0800] rev 29460
new lemmas about synthetic_div; declare degree_pCons_eq_if [simp]
Tue, 13 Jan 2009 13:47:35 +0100 added Isar/isar_document.ML: Interactive Isar documents.
wenzelm [Tue, 13 Jan 2009 13:47:35 +0100] rev 29459
added Isar/isar_document.ML: Interactive Isar documents.
Tue, 13 Jan 2009 13:46:30 +0100 export list;
wenzelm [Tue, 13 Jan 2009 13:46:30 +0100] rev 29458
export list;
Mon, 12 Jan 2009 10:09:23 -0800 correctness and uniqueness of synthetic division
huffman [Mon, 12 Jan 2009 10:09:23 -0800] rev 29457
correctness and uniqueness of synthetic division
Mon, 12 Jan 2009 09:35:15 -0800 add synthetic division algorithm for polynomials
huffman [Mon, 12 Jan 2009 09:35:15 -0800] rev 29456
add synthetic division algorithm for polynomials
Mon, 12 Jan 2009 09:04:25 -0800 add list-style syntax for pCons
huffman [Mon, 12 Jan 2009 09:04:25 -0800] rev 29455
add list-style syntax for pCons
Mon, 12 Jan 2009 08:46:07 -0800 add recursion combinator poly_rec; define poly function using poly_rec
huffman [Mon, 12 Jan 2009 08:46:07 -0800] rev 29454
add recursion combinator poly_rec; define poly function using poly_rec
Mon, 12 Jan 2009 08:15:07 -0800 add lemmas degree_{add,diff}_less
huffman [Mon, 12 Jan 2009 08:15:07 -0800] rev 29453
add lemmas degree_{add,diff}_less
Sun, 11 Jan 2009 21:50:05 +0100 merged
wenzelm [Sun, 11 Jan 2009 21:50:05 +0100] rev 29452
merged
Sun, 11 Jan 2009 12:05:50 -0800 new theory of polynomials
huffman [Sun, 11 Jan 2009 12:05:50 -0800] rev 29451
new theory of polynomials
Sun, 11 Jan 2009 21:49:59 +0100 tuned categories;
wenzelm [Sun, 11 Jan 2009 21:49:59 +0100] rev 29450
tuned categories;
Sun, 11 Jan 2009 20:40:09 +0100 added outer_keyword.scala: Isar command keyword classification;
wenzelm [Sun, 11 Jan 2009 20:40:09 +0100] rev 29449
added outer_keyword.scala: Isar command keyword classification;
Sun, 11 Jan 2009 18:18:35 +0100 added Goal.future_enabled abstraction -- now also checks that this is already
wenzelm [Sun, 11 Jan 2009 18:18:35 +0100] rev 29448
added Goal.future_enabled abstraction -- now also checks that this is already a future task, which excludes interactive commands of the old toplevel;
Sun, 11 Jan 2009 17:34:02 +0100 load main entry points sequentially, for reduced memory demands;
wenzelm [Sun, 11 Jan 2009 17:34:02 +0100] rev 29447
load main entry points sequentially, for reduced memory demands;
Sun, 11 Jan 2009 16:56:59 +0100 merged
wenzelm [Sun, 11 Jan 2009 16:56:59 +0100] rev 29446
merged
Sun, 11 Jan 2009 14:23:54 +0100 merged
wenzelm [Sun, 11 Jan 2009 14:23:54 +0100] rev 29445
merged
Sun, 11 Jan 2009 16:41:48 +0100 less ambitious ML_OPTIONS;
wenzelm [Sun, 11 Jan 2009 16:41:48 +0100] rev 29444
less ambitious ML_OPTIONS;
Sun, 11 Jan 2009 14:22:34 +0100 merged
wenzelm [Sun, 11 Jan 2009 14:22:34 +0100] rev 29443
merged
Sun, 11 Jan 2009 14:18:32 +0100 merged
haftmann [Sun, 11 Jan 2009 14:18:32 +0100] rev 29442
merged
Sun, 11 Jan 2009 14:18:17 +0100 explicit bookkeeping of intro rules and axiom
haftmann [Sun, 11 Jan 2009 14:18:17 +0100] rev 29441
explicit bookkeeping of intro rules and axiom
Sun, 11 Jan 2009 14:18:16 +0100 stripped Id
haftmann [Sun, 11 Jan 2009 14:18:16 +0100] rev 29440
stripped Id
Sun, 11 Jan 2009 14:18:16 +0100 construct explicit class morphism
haftmann [Sun, 11 Jan 2009 14:18:16 +0100] rev 29439
construct explicit class morphism
Sun, 11 Jan 2009 13:48:11 +0100 less ambitious ML_OPTIONS;
wenzelm [Sun, 11 Jan 2009 13:48:11 +0100] rev 29438
less ambitious ML_OPTIONS;
Sat, 10 Jan 2009 23:56:11 +0100 schedule_futures: save memory for non-parallel proofs, by applying after_load as soon as possible here;
wenzelm [Sat, 10 Jan 2009 23:56:11 +0100] rev 29437
schedule_futures: save memory for non-parallel proofs, by applying after_load as soon as possible here;
Sat, 10 Jan 2009 21:47:02 +0100 future_result: avoid expensive norm_proof (consider usedir option -Q false in low-memory situations);
wenzelm [Sat, 10 Jan 2009 21:47:02 +0100] rev 29436
future_result: avoid expensive norm_proof (consider usedir option -Q false in low-memory situations);
Sat, 10 Jan 2009 21:32:30 +0100 added parallel_proofs flag (default true, cf. usedir option -Q), which can be disabled in low-memory situations;
wenzelm [Sat, 10 Jan 2009 21:32:30 +0100] rev 29435
added parallel_proofs flag (default true, cf. usedir option -Q), which can be disabled in low-memory situations;
Sat, 10 Jan 2009 16:58:56 +0100 remove_thy: perform PureThy.cancel_proofs;
wenzelm [Sat, 10 Jan 2009 16:58:56 +0100] rev 29434
remove_thy: perform PureThy.cancel_proofs; schedule_futures: PureThy.join_proofs before after_load -- achieves parallel error messages;
Sat, 10 Jan 2009 16:55:46 +0100 added cancel_proofs, based on task groups of "entered" proofs;
wenzelm [Sat, 10 Jan 2009 16:55:46 +0100] rev 29433
added cancel_proofs, based on task groups of "entered" proofs;
Sat, 10 Jan 2009 16:54:55 +0100 added pending_groups -- accumulates task groups of local derivations only;
wenzelm [Sat, 10 Jan 2009 16:54:55 +0100] rev 29432
added pending_groups -- accumulates task groups of local derivations only;
Sat, 10 Jan 2009 16:53:12 +0100 added cancel_group;
wenzelm [Sat, 10 Jan 2009 16:53:12 +0100] rev 29431
added cancel_group;
Sat, 10 Jan 2009 16:00:34 +0100 merged
wenzelm [Sat, 10 Jan 2009 16:00:34 +0100] rev 29430
merged
Sat, 10 Jan 2009 13:11:56 +0100 schedule_futures: tuned final consolidation, explicit after_load phase;
wenzelm [Sat, 10 Jan 2009 13:11:56 +0100] rev 29429
schedule_futures: tuned final consolidation, explicit after_load phase;
Sat, 10 Jan 2009 13:10:38 +0100 load_thy: explicit after_load phase for presentation;
wenzelm [Sat, 10 Jan 2009 13:10:38 +0100] rev 29428
load_thy: explicit after_load phase for presentation;
Sat, 10 Jan 2009 13:10:07 +0100 excursion: commit_exit internally -- checkpoints are fully persistent now;
wenzelm [Sat, 10 Jan 2009 13:10:07 +0100] rev 29427
excursion: commit_exit internally -- checkpoints are fully persistent now; excursion: do not force intermediate result states yet -- great performance improvement;
Sat, 10 Jan 2009 15:55:19 +0100 slightly more robust matching of session name;
wenzelm [Sat, 10 Jan 2009 15:55:19 +0100] rev 29426
slightly more robust matching of session name;
Sat, 10 Jan 2009 01:28:31 +0100 merged
wenzelm [Sat, 10 Jan 2009 01:28:31 +0100] rev 29425
merged
Sat, 10 Jan 2009 01:06:32 +0100 fixed proof involving dvd;
wenzelm [Sat, 10 Jan 2009 01:06:32 +0100] rev 29424
fixed proof involving dvd;
Sat, 10 Jan 2009 01:28:18 +0100 tuned;
wenzelm [Sat, 10 Jan 2009 01:28:18 +0100] rev 29423
tuned;
Sat, 10 Jan 2009 01:28:03 +0100 added force_result;
wenzelm [Sat, 10 Jan 2009 01:28:03 +0100] rev 29422
added force_result;
Sat, 10 Jan 2009 00:25:31 +0100 use_thys: perform consolidate_thy on loaded theories, which removes failed nodes in post-hoc fashion;
wenzelm [Sat, 10 Jan 2009 00:25:31 +0100] rev 29421
use_thys: perform consolidate_thy on loaded theories, which removes failed nodes in post-hoc fashion;
Sat, 10 Jan 2009 00:24:07 +0100 simplified join_proofs;
wenzelm [Sat, 10 Jan 2009 00:24:07 +0100] rev 29420
simplified join_proofs;
Fri, 09 Jan 2009 23:39:53 +0100 merged
wenzelm [Fri, 09 Jan 2009 23:39:53 +0100] rev 29419
merged
Fri, 09 Jan 2009 23:34:36 +0100 added split_thy_path;
wenzelm [Fri, 09 Jan 2009 23:34:36 +0100] rev 29418
added split_thy_path;
Fri, 09 Jan 2009 23:33:59 +0100 added running task markup;
wenzelm [Fri, 09 Jan 2009 23:33:59 +0100] rev 29417
added running task markup;
Thu, 08 Jan 2009 13:18:34 +0100 tuned;
wenzelm [Thu, 08 Jan 2009 13:18:34 +0100] rev 29416
tuned;
Thu, 08 Jan 2009 12:15:23 +0100 merged
wenzelm [Thu, 08 Jan 2009 12:15:23 +0100] rev 29415
merged
Fri, 09 Jan 2009 19:41:33 +0100 merged
wenzelm [Fri, 09 Jan 2009 19:41:33 +0100] rev 29414
merged
Fri, 09 Jan 2009 09:49:01 -0800 merged.
huffman [Fri, 09 Jan 2009 09:49:01 -0800] rev 29413
merged.
Fri, 09 Jan 2009 09:34:49 -0800 fix proof broken by changes in dvd theory
huffman [Fri, 09 Jan 2009 09:34:49 -0800] rev 29412
fix proof broken by changes in dvd theory
Thu, 08 Jan 2009 21:13:40 -0800 merged.
huffman [Thu, 08 Jan 2009 21:13:40 -0800] rev 29411
merged.
Thu, 08 Jan 2009 12:25:22 -0800 remove type-specific proofs
huffman [Thu, 08 Jan 2009 12:25:22 -0800] rev 29410
remove type-specific proofs
Thu, 08 Jan 2009 10:43:09 -0800 add lemma dvd_diff to class comm_ring_1
huffman [Thu, 08 Jan 2009 10:43:09 -0800] rev 29409
add lemma dvd_diff to class comm_ring_1
Thu, 08 Jan 2009 10:26:50 -0800 add lemmas dvd_minus_iff and minus_dvd_iff in class comm_ring_1
huffman [Thu, 08 Jan 2009 10:26:50 -0800] rev 29408
add lemmas dvd_minus_iff and minus_dvd_iff in class comm_ring_1
Thu, 08 Jan 2009 10:07:39 -0800 move lemmas mult_minus{left,right} inside class ring
huffman [Thu, 08 Jan 2009 10:07:39 -0800] rev 29407
move lemmas mult_minus{left,right} inside class ring
Thu, 08 Jan 2009 09:58:36 -0800 clean up division_ring proofs
huffman [Thu, 08 Jan 2009 09:58:36 -0800] rev 29406
clean up division_ring proofs
Thu, 08 Jan 2009 09:12:29 -0800 add class ring_div; generalize mod/diff/minus proofs for class ring_div
huffman [Thu, 08 Jan 2009 09:12:29 -0800] rev 29405
add class ring_div; generalize mod/diff/minus proofs for class ring_div
Thu, 08 Jan 2009 08:36:16 -0800 generalize zmod_zmod_cancel -> mod_mod_cancel
huffman [Thu, 08 Jan 2009 08:36:16 -0800] rev 29404
generalize zmod_zmod_cancel -> mod_mod_cancel
Thu, 08 Jan 2009 08:24:08 -0800 generalize some div/mod lemmas; remove type-specific proofs
huffman [Thu, 08 Jan 2009 08:24:08 -0800] rev 29403
generalize some div/mod lemmas; remove type-specific proofs
Wed, 07 Jan 2009 08:13:56 -0800 add tracing for domain package proofs
huffman [Wed, 07 Jan 2009 08:13:56 -0800] rev 29402
add tracing for domain package proofs
Tue, 06 Jan 2009 11:49:23 -0800 rename abbreviation square -> power2, to match theorem names
huffman [Tue, 06 Jan 2009 11:49:23 -0800] rev 29401
rename abbreviation square -> power2, to match theorem names
Fri, 09 Jan 2009 08:22:44 +0100 merged
haftmann [Fri, 09 Jan 2009 08:22:44 +0100] rev 29400
merged
Thu, 08 Jan 2009 17:10:41 +0100 split of Imperative_HOL theories from HOL-Library
haftmann [Thu, 08 Jan 2009 17:10:41 +0100] rev 29399
split of Imperative_HOL theories from HOL-Library
Thu, 08 Jan 2009 17:25:06 +0100 NEWS and CONTRIBUTORS
haftmann [Thu, 08 Jan 2009 17:25:06 +0100] rev 29398
NEWS and CONTRIBUTORS
Thu, 08 Jan 2009 10:53:48 +0100 dded code_thm antiquotation
haftmann [Thu, 08 Jan 2009 10:53:48 +0100] rev 29397
dded code_thm antiquotation
Thu, 08 Jan 2009 08:06:11 +0100 made SML/NJ happy
haftmann [Thu, 08 Jan 2009 08:06:11 +0100] rev 29396
made SML/NJ happy
Wed, 07 Jan 2009 23:56:56 +0100 merged
wenzelm [Wed, 07 Jan 2009 23:56:56 +0100] rev 29395
merged
Wed, 07 Jan 2009 22:33:04 +0100 merged
haftmann [Wed, 07 Jan 2009 22:33:04 +0100] rev 29394
merged
Wed, 07 Jan 2009 22:31:37 +0100 tuned siganture of locale.ML
haftmann [Wed, 07 Jan 2009 22:31:37 +0100] rev 29393
tuned siganture of locale.ML
Wed, 07 Jan 2009 22:31:36 +0100 tuned signature; internal code reorganisation
haftmann [Wed, 07 Jan 2009 22:31:36 +0100] rev 29392
tuned signature; internal code reorganisation
Wed, 07 Jan 2009 22:31:36 +0100 tuned signature; changed locale predicate name convention
haftmann [Wed, 07 Jan 2009 22:31:36 +0100] rev 29391
tuned signature; changed locale predicate name convention
Wed, 07 Jan 2009 22:31:34 +0100 changed locale predicate name convention
haftmann [Wed, 07 Jan 2009 22:31:34 +0100] rev 29390
changed locale predicate name convention
Wed, 07 Jan 2009 23:53:08 +0100 inductive: added fork_mono flag;
wenzelm [Wed, 07 Jan 2009 23:53:08 +0100] rev 29389
inductive: added fork_mono flag;
Wed, 07 Jan 2009 23:52:18 +0100 added fork_mono flag, which is usually enabled in batch-mode only;
wenzelm [Wed, 07 Jan 2009 23:52:18 +0100] rev 29388
added fork_mono flag, which is usually enabled in batch-mode only; mono rule: unnamed LocalTheory.node ensures proper joining of pending proofs;
Wed, 07 Jan 2009 20:27:55 +0100 Proof.global_future_terminal_proof;
wenzelm [Wed, 07 Jan 2009 20:27:55 +0100] rev 29387
Proof.global_future_terminal_proof;
Wed, 07 Jan 2009 20:27:23 +0100 Proof.global_future_proof;
wenzelm [Wed, 07 Jan 2009 20:27:23 +0100] rev 29386
Proof.global_future_proof;
Wed, 07 Jan 2009 20:27:05 +0100 future_proof: refined version covers local_future_proof and global_future_proof;
wenzelm [Wed, 07 Jan 2009 20:27:05 +0100] rev 29385
future_proof: refined version covers local_future_proof and global_future_proof; future_proof: refrain from full Variable.auto_fixes -- not all contexts in the stack are in body mode; refined is_relevant: mode check; added local/global_future_terminal_proof;
Wed, 07 Jan 2009 17:26:03 +0100 more robust propagation of errors through bulk jobs;
wenzelm [Wed, 07 Jan 2009 17:26:03 +0100] rev 29384
more robust propagation of errors through bulk jobs;
Wed, 07 Jan 2009 16:22:10 +0100 qed/after_qed: singleton result;
wenzelm [Wed, 07 Jan 2009 16:22:10 +0100] rev 29383
qed/after_qed: singleton result;
Wed, 07 Jan 2009 12:10:22 +0100 Proof.future_terminal_proof: no fork for interactive mode -- proofs need to be checked immediately here;
wenzelm [Wed, 07 Jan 2009 12:10:22 +0100] rev 29382
Proof.future_terminal_proof: no fork for interactive mode -- proofs need to be checked immediately here;
Wed, 07 Jan 2009 12:09:39 +0100 future_terminal_proof: no fork for interactive mode, assert_backward;
wenzelm [Wed, 07 Jan 2009 12:09:39 +0100] rev 29381
future_terminal_proof: no fork for interactive mode, assert_backward;
Wed, 07 Jan 2009 12:08:22 +0100 added local_theory';
wenzelm [Wed, 07 Jan 2009 12:08:22 +0100] rev 29380
added local_theory';
Wed, 07 Jan 2009 08:04:12 +0100 merged
haftmann [Wed, 07 Jan 2009 08:04:12 +0100] rev 29379
merged
Wed, 07 Jan 2009 08:03:25 +0100 proper local_theory after Class.class
haftmann [Wed, 07 Jan 2009 08:03:25 +0100] rev 29378
proper local_theory after Class.class
Tue, 06 Jan 2009 22:08:42 +0100 more parallel loading;
wenzelm [Tue, 06 Jan 2009 22:08:42 +0100] rev 29377
more parallel loading;
Tue, 06 Jan 2009 21:55:51 +0100 more parallel loading;
wenzelm [Tue, 06 Jan 2009 21:55:51 +0100] rev 29376
more parallel loading;
Tue, 06 Jan 2009 21:17:43 +0100 merged
wenzelm [Tue, 06 Jan 2009 21:17:43 +0100] rev 29375
merged
Tue, 06 Jan 2009 09:18:02 -0800 merged.
huffman [Tue, 06 Jan 2009 09:18:02 -0800] rev 29374
merged.
Tue, 06 Jan 2009 09:03:37 -0800 make cont_proc handle eta-contracted terms
huffman [Tue, 06 Jan 2009 09:03:37 -0800] rev 29373
make cont_proc handle eta-contracted terms
Tue, 06 Jan 2009 09:02:18 -0800 implement is_closed_term using Term.loose_bvar
huffman [Tue, 06 Jan 2009 09:02:18 -0800] rev 29372
implement is_closed_term using Term.loose_bvar
Mon, 05 Jan 2009 15:26:57 -0800 use Thm.close_derivation instead of standard
huffman [Mon, 05 Jan 2009 15:26:57 -0800] rev 29371
use Thm.close_derivation instead of standard
Tue, 06 Jan 2009 21:17:37 +0100 tuned;
wenzelm [Tue, 06 Jan 2009 21:17:37 +0100] rev 29370
tuned;
Tue, 06 Jan 2009 14:45:45 +0100 merged
wenzelm [Tue, 06 Jan 2009 14:45:45 +0100] rev 29369
merged
Tue, 06 Jan 2009 14:43:35 +0100 renamed structure ParList to Par_List;
wenzelm [Tue, 06 Jan 2009 14:43:35 +0100] rev 29368
renamed structure ParList to Par_List;
Tue, 06 Jan 2009 14:33:49 +0100 parallelized merge_data;
wenzelm [Tue, 06 Jan 2009 14:33:49 +0100] rev 29367
parallelized merge_data;
Tue, 06 Jan 2009 13:46:48 +0100 tuned map: reduced overhead due to bulk jobs;
wenzelm [Tue, 06 Jan 2009 13:46:48 +0100] rev 29366
tuned map: reduced overhead due to bulk jobs; tuned join_results: reduced overhead for finished futures; tuned;
Tue, 06 Jan 2009 13:43:17 +0100 added is_valid;
wenzelm [Tue, 06 Jan 2009 13:43:17 +0100] rev 29365
added is_valid; added extend: support bulk jobs; tuned;
Tue, 06 Jan 2009 13:36:42 +0100 future_terminal_proof: check Future.enabled;
wenzelm [Tue, 06 Jan 2009 13:36:42 +0100] rev 29364
future_terminal_proof: check Future.enabled;
Tue, 06 Jan 2009 08:50:12 +0100 merged
haftmann [Tue, 06 Jan 2009 08:50:12 +0100] rev 29363
merged
Tue, 06 Jan 2009 08:50:02 +0100 locale -> old_locale, new_locale -> locale
haftmann [Tue, 06 Jan 2009 08:50:02 +0100] rev 29362
locale -> old_locale, new_locale -> locale
Mon, 05 Jan 2009 15:55:51 +0100 locale -> old_locale, new_locale -> locale
haftmann [Mon, 05 Jan 2009 15:55:51 +0100] rev 29361
locale -> old_locale, new_locale -> locale
Mon, 05 Jan 2009 15:55:04 +0100 locale -> old_locale, new_locale -> locale
haftmann [Mon, 05 Jan 2009 15:55:04 +0100] rev 29360
locale -> old_locale, new_locale -> locale
Mon, 05 Jan 2009 15:37:49 +0100 removed locale adaption layer
haftmann [Mon, 05 Jan 2009 15:37:49 +0100] rev 29359
removed locale adaption layer
Mon, 05 Jan 2009 15:36:24 +0100 rearranged target theories
haftmann [Mon, 05 Jan 2009 15:36:24 +0100] rev 29358
rearranged target theories
Mon, 05 Jan 2009 15:35:42 +0100 removed locale adaption layer
haftmann [Mon, 05 Jan 2009 15:35:42 +0100] rev 29357
removed locale adaption layer
Mon, 05 Jan 2009 19:37:15 +0100 merged
wenzelm [Mon, 05 Jan 2009 19:37:15 +0100] rev 29356
merged
Mon, 05 Jan 2009 18:13:26 +0100 misc tuning and modernization;
wenzelm [Mon, 05 Jan 2009 18:13:26 +0100] rev 29355
misc tuning and modernization;
(0) -10000 -3000 -1000 -120 +120 +1000 +3000 +10000 +30000 tip