Wed, 18 Mar 2009 11:57:28 +0100 tuned interpunctation
haftmann [Wed, 18 Mar 2009 11:57:28 +0100] rev 30569
tuned interpunctation
Tue, 17 Mar 2009 19:53:57 +0100 strip_abss: always strip abstractions as far as possible, without keeping alternatives (which appear to be redundant anyway, but cause significant slowdown since discrimination nets collapse abstractions);
wenzelm [Tue, 17 Mar 2009 19:53:57 +0100] rev 30568
strip_abss: always strip abstractions as far as possible, without keeping alternatives (which appear to be redundant anyway, but cause significant slowdown since discrimination nets collapse abstractions);
Tue, 17 Mar 2009 19:06:04 +0100 close/all_assm_tac: finish all subgoals from left to right (cf. Proof.goal_tac a28d83e903ce) -- NB: ALLGOALS/THEN_ALL_NEW operate from right to left;
wenzelm [Tue, 17 Mar 2009 19:06:04 +0100] rev 30567
close/all_assm_tac: finish all subgoals from left to right (cf. Proof.goal_tac a28d83e903ce) -- NB: ALLGOALS/THEN_ALL_NEW operate from right to left;
Tue, 17 Mar 2009 16:55:21 +0100 reverted abbreviations: improved performance via Item_Net.T;
wenzelm [Tue, 17 Mar 2009 16:55:21 +0100] rev 30566
reverted abbreviations: improved performance via Item_Net.T;
Tue, 17 Mar 2009 15:35:27 +0100 export match_rew -- useful for implementing "procs" for rewrite_term;
wenzelm [Tue, 17 Mar 2009 15:35:27 +0100] rev 30565
export match_rew -- useful for implementing "procs" for rewrite_term;
Tue, 17 Mar 2009 15:34:42 +0100 tuned comment;
wenzelm [Tue, 17 Mar 2009 15:34:42 +0100] rev 30564
tuned comment;
Tue, 17 Mar 2009 14:14:25 +0100 merged
wenzelm [Tue, 17 Mar 2009 14:14:25 +0100] rev 30563
merged
Mon, 16 Mar 2009 15:58:41 -0700 document new additions to HOL/Library
huffman [Mon, 16 Mar 2009 15:58:41 -0700] rev 30562
document new additions to HOL/Library
Mon, 16 Mar 2009 15:10:59 -0700 clean up proofs
huffman [Mon, 16 Mar 2009 15:10:59 -0700] rev 30561
clean up proofs
Tue, 17 Mar 2009 14:12:43 +0100 adapted to general Item_Net;
wenzelm [Tue, 17 Mar 2009 14:12:43 +0100] rev 30560
adapted to general Item_Net;
Tue, 17 Mar 2009 14:12:06 +0100 turned structure NetRules into general Item_Net, which is loaded earlier;
wenzelm [Tue, 17 Mar 2009 14:12:06 +0100] rev 30559
turned structure NetRules into general Item_Net, which is loaded earlier;
Tue, 17 Mar 2009 14:09:20 +0100 renamed Tactic.taglist/untaglist/orderlist to tag_list/untag_list/order_list (in library.ML);
wenzelm [Tue, 17 Mar 2009 14:09:20 +0100] rev 30558
renamed Tactic.taglist/untaglist/orderlist to tag_list/untag_list/order_list (in library.ML);
Tue, 17 Mar 2009 13:33:21 +0100 goal_tac: finish marked assumptions from left to right -- corresponds better with the strategy of etac, with significant performance gains in some situations;
wenzelm [Tue, 17 Mar 2009 13:33:21 +0100] rev 30557
goal_tac: finish marked assumptions from left to right -- corresponds better with the strategy of etac, with significant performance gains in some situations;
Tue, 17 Mar 2009 12:10:42 +0100 eq_assumption: slightly more efficient by checking (open) result of Logic.assum_problems directly;
wenzelm [Tue, 17 Mar 2009 12:10:42 +0100] rev 30556
eq_assumption: slightly more efficient by checking (open) result of Logic.assum_problems directly; tuned;
Tue, 17 Mar 2009 12:09:43 +0100 tuned aeconv: test plain aconv before expensive eta_contract;
wenzelm [Tue, 17 Mar 2009 12:09:43 +0100] rev 30555
tuned aeconv: test plain aconv before expensive eta_contract;
Mon, 16 Mar 2009 23:52:30 +0100 substantial speedup of assumption and elim-resolution: Logic.assum_problems refrains from eager application of parameters, discriminate via Term.could_unify before invoking full unification (assumes terms in beta-normal form, as do higher term net operations anyway);
wenzelm [Mon, 16 Mar 2009 23:52:30 +0100] rev 30554
substantial speedup of assumption and elim-resolution: Logic.assum_problems refrains from eager application of parameters, discriminate via Term.could_unify before invoking full unification (assumes terms in beta-normal form, as do higher term net operations anyway);
Mon, 16 Mar 2009 23:39:44 +0100 refined is_norm_hhf: reject beta-redexes (rules based on term nets or could_unify assume normal form), also potentially faster by avoiding expensive Envir.beta_eta_contract;
wenzelm [Mon, 16 Mar 2009 23:39:44 +0100] rev 30553
refined is_norm_hhf: reject beta-redexes (rules based on term nets or could_unify assume normal form), also potentially faster by avoiding expensive Envir.beta_eta_contract;
Mon, 16 Mar 2009 23:36:55 +0100 provide Simplifier.norm_hhf(_protect) as regular simplifier operation;
wenzelm [Mon, 16 Mar 2009 23:36:55 +0100] rev 30552
provide Simplifier.norm_hhf(_protect) as regular simplifier operation;
Mon, 16 Mar 2009 19:40:03 +0100 method parser: pass proper context;
wenzelm [Mon, 16 Mar 2009 19:40:03 +0100] rev 30551
method parser: pass proper context;
Mon, 16 Mar 2009 18:24:39 +0100 merged
wenzelm [Mon, 16 Mar 2009 18:24:39 +0100] rev 30550
merged
Mon, 16 Mar 2009 18:24:30 +0100 simplified method setup;
wenzelm [Mon, 16 Mar 2009 18:24:30 +0100] rev 30549
simplified method setup;
Mon, 16 Mar 2009 17:51:24 +0100 updated generated file;
wenzelm [Mon, 16 Mar 2009 17:51:24 +0100] rev 30548
updated generated file;
Mon, 16 Mar 2009 17:51:07 +0100 simplifief 'method_setup' command;
wenzelm [Mon, 16 Mar 2009 17:51:07 +0100] rev 30547
simplifief 'method_setup' command;
Mon, 16 Mar 2009 17:48:02 +0100 spelling;
wenzelm [Mon, 16 Mar 2009 17:48:02 +0100] rev 30546
spelling;
Mon, 16 Mar 2009 17:47:26 +0100 export method parser;
wenzelm [Mon, 16 Mar 2009 17:47:26 +0100] rev 30545
export method parser;
Mon, 16 Mar 2009 17:46:49 +0100 adapted 'method_setup' command to Method.setup;
wenzelm [Mon, 16 Mar 2009 17:46:49 +0100] rev 30544
adapted 'method_setup' command to Method.setup;
Mon, 16 Mar 2009 17:46:11 +0100 tuned signature;
wenzelm [Mon, 16 Mar 2009 17:46:11 +0100] rev 30543
tuned signature;
Mon, 16 Mar 2009 14:26:30 +0100 have remote script interrupted like the other provers
immler@in.tum.de [Mon, 16 Mar 2009 14:26:30 +0100] rev 30542
have remote script interrupted like the other provers
Sun, 15 Mar 2009 20:25:58 +0100 simplified method setup;
wenzelm [Sun, 15 Mar 2009 20:25:58 +0100] rev 30541
simplified method setup;
Sun, 15 Mar 2009 20:19:14 +0100 export section, sections;
wenzelm [Sun, 15 Mar 2009 20:19:14 +0100] rev 30540
export section, sections; tuned signature;
Sun, 15 Mar 2009 16:59:17 +0100 merged
wenzelm [Sun, 15 Mar 2009 16:59:17 +0100] rev 30539
merged
Sat, 14 Mar 2009 17:52:53 +0100 updated NEWS
immler@in.tum.de [Sat, 14 Mar 2009 17:52:53 +0100] rev 30538
updated NEWS
Sat, 14 Mar 2009 16:50:25 +0100 use goal instead of Proof State
immler@in.tum.de [Sat, 14 Mar 2009 16:50:25 +0100] rev 30537
use goal instead of Proof State
Sat, 14 Mar 2009 16:46:23 +0100 split relevance-filter and writing of problem-files;
immler@in.tum.de [Sat, 14 Mar 2009 16:46:23 +0100] rev 30536
split relevance-filter and writing of problem-files; perform relevance-filtering for only one subgoal; added additional explicit timeout to provers
Sat, 14 Mar 2009 15:45:45 +0100 show certain errors to the user
immler@in.tum.de [Sat, 14 Mar 2009 15:45:45 +0100] rev 30535
show certain errors to the user
Sat, 14 Mar 2009 15:15:44 +0100 removed connection check;
immler@in.tum.de [Sat, 14 Mar 2009 15:15:44 +0100] rev 30534
removed connection check; adapted times
Sun, 15 Mar 2009 16:02:22 +0100 merged
wenzelm [Sun, 15 Mar 2009 16:02:22 +0100] rev 30533
merged
Sat, 14 Mar 2009 12:51:13 +0100 merged
haftmann [Sat, 14 Mar 2009 12:51:13 +0100] rev 30532
merged
Sat, 14 Mar 2009 12:50:29 +0100 reverted to old version of Set.thy -- strange effects have to be traced first
haftmann [Sat, 14 Mar 2009 12:50:29 +0100] rev 30531
reverted to old version of Set.thy -- strange effects have to be traced first
Sun, 15 Mar 2009 15:59:45 +0100 simplified attribute and method setup;
wenzelm [Sun, 15 Mar 2009 15:59:45 +0100] rev 30530
simplified attribute and method setup;
Sun, 15 Mar 2009 15:59:44 +0100 simplified attribute setup;
wenzelm [Sun, 15 Mar 2009 15:59:44 +0100] rev 30529
simplified attribute setup; replaced add_args by add parser;
Sun, 15 Mar 2009 15:59:44 +0100 simplified attribute setup;
wenzelm [Sun, 15 Mar 2009 15:59:44 +0100] rev 30528
simplified attribute setup;
Sun, 15 Mar 2009 15:59:44 +0100 updated generated files;
wenzelm [Sun, 15 Mar 2009 15:59:44 +0100] rev 30527
updated generated files;
Sun, 15 Mar 2009 15:59:43 +0100 added 'attribute_setup' command;
wenzelm [Sun, 15 Mar 2009 15:59:43 +0100] rev 30526
added 'attribute_setup' command;
Sun, 15 Mar 2009 15:59:43 +0100 added setup and attribute_setup -- expect plain parser instead of syntax function;
wenzelm [Sun, 15 Mar 2009 15:59:43 +0100] rev 30525
added setup and attribute_setup -- expect plain parser instead of syntax function; aded add_del parser;
Sun, 15 Mar 2009 15:59:43 +0100 ML_Syntax.make_binding;
wenzelm [Sun, 15 Mar 2009 15:59:43 +0100] rev 30524
ML_Syntax.make_binding;
Sun, 15 Mar 2009 15:59:42 +0100 added make_binding;
wenzelm [Sun, 15 Mar 2009 15:59:42 +0100] rev 30523
added make_binding;
Sat, 14 Mar 2009 00:13:50 +0100 removed obsolete no_base_names naming policy;
wenzelm [Sat, 14 Mar 2009 00:13:50 +0100] rev 30522
removed obsolete no_base_names naming policy;
Fri, 13 Mar 2009 23:56:07 +0100 merged
wenzelm [Fri, 13 Mar 2009 23:56:07 +0100] rev 30521
merged
Fri, 13 Mar 2009 19:18:07 +0100 merged
haftmann [Fri, 13 Mar 2009 19:18:07 +0100] rev 30520
merged
Fri, 13 Mar 2009 19:17:58 +0100 coherent binding policy with primitive target operations
haftmann [Fri, 13 Mar 2009 19:17:58 +0100] rev 30519
coherent binding policy with primitive target operations
Fri, 13 Mar 2009 19:17:57 +0100 moved some generic nonsense to arith_data.ML
haftmann [Fri, 13 Mar 2009 19:17:57 +0100] rev 30518
moved some generic nonsense to arith_data.ML
Fri, 13 Mar 2009 19:17:57 +0100 tuned ML code
haftmann [Fri, 13 Mar 2009 19:17:57 +0100] rev 30517
tuned ML code
Fri, 13 Mar 2009 10:14:47 -0700 remove legacy ML bindings
huffman [Fri, 13 Mar 2009 10:14:47 -0700] rev 30516
remove legacy ML bindings
Fri, 13 Mar 2009 23:50:05 +0100 simplified method setup;
wenzelm [Fri, 13 Mar 2009 23:50:05 +0100] rev 30515
simplified method setup;
Fri, 13 Mar 2009 23:32:40 +0100 simplified goal_spec: default to first goal;
wenzelm [Fri, 13 Mar 2009 23:32:40 +0100] rev 30514
simplified goal_spec: default to first goal;
Fri, 13 Mar 2009 21:25:15 +0100 eliminated type Args.T;
wenzelm [Fri, 13 Mar 2009 21:25:15 +0100] rev 30513
eliminated type Args.T; pervasive types 'a parser and 'a context_parser;
Fri, 13 Mar 2009 21:24:21 +0100 added simplified setup;
wenzelm [Fri, 13 Mar 2009 21:24:21 +0100] rev 30512
added simplified setup; eliminated type Args.T; pervasive types 'a parser and 'a context_parser;
Fri, 13 Mar 2009 21:22:45 +0100 pervasive types 'a parser and 'a context_parser;
wenzelm [Fri, 13 Mar 2009 21:22:45 +0100] rev 30511
pervasive types 'a parser and 'a context_parser;
Fri, 13 Mar 2009 19:58:26 +0100 unified type Proof.method and pervasive METHOD combinators;
wenzelm [Fri, 13 Mar 2009 19:58:26 +0100] rev 30510
unified type Proof.method and pervasive METHOD combinators;
(0) -30000 -10000 -3000 -1000 -300 -100 -60 +60 +100 +300 +1000 +3000 +10000 +30000 tip