Tue, 03 Jul 2007 17:17:17 +0200 rewrite_goal_tac;
wenzelm [Tue, 03 Jul 2007 17:17:17 +0200] rev 23543
rewrite_goal_tac;
Tue, 03 Jul 2007 17:17:16 +0200 replaced Conv.goals_conv by Conv.prems_conv;
wenzelm [Tue, 03 Jul 2007 17:17:16 +0200] rev 23542
replaced Conv.goals_conv by Conv.prems_conv;
Tue, 03 Jul 2007 17:17:15 +0200 exported meta_rewrite_conv;
wenzelm [Tue, 03 Jul 2007 17:17:15 +0200] rev 23541
exported meta_rewrite_conv; CONVERSION tactical;
Tue, 03 Jul 2007 17:17:15 +0200 CONVERSION tactical;
wenzelm [Tue, 03 Jul 2007 17:17:15 +0200] rev 23540
CONVERSION tactical; MetaSimplifier.rewrite_goal_tac;
Tue, 03 Jul 2007 17:17:13 +0200 removed obsolete eta_long_tac;
wenzelm [Tue, 03 Jul 2007 17:17:13 +0200] rev 23539
removed obsolete eta_long_tac;
Tue, 03 Jul 2007 17:17:13 +0200 added CONVERSION tactical;
wenzelm [Tue, 03 Jul 2007 17:17:13 +0200] rev 23538
added CONVERSION tactical; tuned signature;
Tue, 03 Jul 2007 17:17:11 +0200 tuned rotate_prems;
wenzelm [Tue, 03 Jul 2007 17:17:11 +0200] rev 23537
tuned rotate_prems; tuned comments;
Tue, 03 Jul 2007 17:17:11 +0200 moved (asm_)rewrite_goal_tac from goal.ML to meta_simplifier.ML (no longer depends on SELECT_GOAL);
wenzelm [Tue, 03 Jul 2007 17:17:11 +0200] rev 23536
moved (asm_)rewrite_goal_tac from goal.ML to meta_simplifier.ML (no longer depends on SELECT_GOAL);
Tue, 03 Jul 2007 17:17:09 +0200 removed obsolete mk_conjunction_list, intr/elim_list;
wenzelm [Tue, 03 Jul 2007 17:17:09 +0200] rev 23535
removed obsolete mk_conjunction_list, intr/elim_list;
Tue, 03 Jul 2007 17:17:09 +0200 removed obsolete goals_conv (cf. prems_conv);
wenzelm [Tue, 03 Jul 2007 17:17:09 +0200] rev 23534
removed obsolete goals_conv (cf. prems_conv); added efficient goal_conv_rule; tuned comments;
Tue, 03 Jul 2007 17:17:07 +0200 Conjunction.intr/elim_balanced;
wenzelm [Tue, 03 Jul 2007 17:17:07 +0200] rev 23533
Conjunction.intr/elim_balanced; CONVERSION tactical; tuned;
Tue, 03 Jul 2007 17:17:07 +0200 CONVERSION tactical;
wenzelm [Tue, 03 Jul 2007 17:17:07 +0200] rev 23532
CONVERSION tactical; Simplifier.rewrite_goal_tac;
Tue, 03 Jul 2007 17:17:06 +0200 Conjunction.mk_conjunction_balanced;
wenzelm [Tue, 03 Jul 2007 17:17:06 +0200] rev 23531
Conjunction.mk_conjunction_balanced;
Tue, 03 Jul 2007 17:17:04 +0200 CONVERSION tactical;
wenzelm [Tue, 03 Jul 2007 17:17:04 +0200] rev 23530
CONVERSION tactical;
Tue, 03 Jul 2007 15:23:11 +0200 Fixed problem with patterns in lambdas
nipkow [Tue, 03 Jul 2007 15:23:11 +0200] rev 23529
Fixed problem with patterns in lambdas
Tue, 03 Jul 2007 14:48:27 +0200 fixed an issue with mutual recursion
krauss [Tue, 03 Jul 2007 14:48:27 +0200] rev 23528
fixed an issue with mutual recursion
Tue, 03 Jul 2007 01:26:06 +0200 instance pordered_comm_ring < pordered_ring
huffman [Tue, 03 Jul 2007 01:26:06 +0200] rev 23527
instance pordered_comm_ring < pordered_ring
Mon, 02 Jul 2007 23:14:06 +0200 Added pattern maatching for lambda abstraction
nipkow [Mon, 02 Jul 2007 23:14:06 +0200] rev 23526
Added pattern maatching for lambda abstraction
Mon, 02 Jul 2007 16:42:37 +0200 revised the discussion of type classes
paulson [Mon, 02 Jul 2007 16:42:37 +0200] rev 23525
revised the discussion of type classes
Mon, 02 Jul 2007 10:43:20 +0200 Generic QE need no Context anymore
chaieb [Mon, 02 Jul 2007 10:43:20 +0200] rev 23524
Generic QE need no Context anymore
Mon, 02 Jul 2007 10:43:19 +0200 Handle exception TYPE
chaieb [Mon, 02 Jul 2007 10:43:19 +0200] rev 23523
Handle exception TYPE
Mon, 02 Jul 2007 10:43:17 +0200 Tuned proofs
chaieb [Mon, 02 Jul 2007 10:43:17 +0200] rev 23522
Tuned proofs
Sat, 30 Jun 2007 17:30:10 +0200 added ordered_ring and ordered_semiring
obua [Sat, 30 Jun 2007 17:30:10 +0200] rev 23521
added ordered_ring and ordered_semiring
Fri, 29 Jun 2007 21:23:05 +0200 tuned arithmetic modules
haftmann [Fri, 29 Jun 2007 21:23:05 +0200] rev 23520
tuned arithmetic modules
Fri, 29 Jun 2007 18:21:25 +0200 bug fixes to proof reconstruction
paulson [Fri, 29 Jun 2007 18:21:25 +0200] rev 23519
bug fixes to proof reconstruction
Fri, 29 Jun 2007 16:05:00 +0200 dropped local cg cmd
haftmann [Fri, 29 Jun 2007 16:05:00 +0200] rev 23518
dropped local cg cmd
Thu, 28 Jun 2007 19:09:43 +0200 dropped toplevel lcm, gcd
haftmann [Thu, 28 Jun 2007 19:09:43 +0200] rev 23517
dropped toplevel lcm, gcd
Thu, 28 Jun 2007 19:09:41 +0200 proper collapse_let
haftmann [Thu, 28 Jun 2007 19:09:41 +0200] rev 23516
proper collapse_let
Thu, 28 Jun 2007 19:09:38 +0200 new code generator framework
haftmann [Thu, 28 Jun 2007 19:09:38 +0200] rev 23515
new code generator framework
Thu, 28 Jun 2007 19:09:36 +0200 dropped Library.lcm
haftmann [Thu, 28 Jun 2007 19:09:36 +0200] rev 23514
dropped Library.lcm
Thu, 28 Jun 2007 19:09:35 +0200 tuned
haftmann [Thu, 28 Jun 2007 19:09:35 +0200] rev 23513
tuned
Thu, 28 Jun 2007 19:09:34 +0200 code generation for dvd
haftmann [Thu, 28 Jun 2007 19:09:34 +0200] rev 23512
code generation for dvd
Thu, 28 Jun 2007 19:09:32 +0200 simplified keyword setup
haftmann [Thu, 28 Jun 2007 19:09:32 +0200] rev 23511
simplified keyword setup
Wed, 27 Jun 2007 12:41:36 +0200 GPL -> BSD
paulson [Wed, 27 Jun 2007 12:41:36 +0200] rev 23510
GPL -> BSD
Wed, 27 Jun 2007 11:06:43 +0200 *** empty log message ***
nipkow [Wed, 27 Jun 2007 11:06:43 +0200] rev 23509
*** empty log message ***
Tue, 26 Jun 2007 18:32:53 +0200 updated for metis method
paulson [Tue, 26 Jun 2007 18:32:53 +0200] rev 23508
updated for metis method
Tue, 26 Jun 2007 18:32:24 +0200 recoded
paulson [Tue, 26 Jun 2007 18:32:24 +0200] rev 23507
recoded
Tue, 26 Jun 2007 18:28:40 +0200 simplified
paulson [Tue, 26 Jun 2007 18:28:40 +0200] rev 23506
simplified
Tue, 26 Jun 2007 15:48:24 +0200 completed some references
paulson [Tue, 26 Jun 2007 15:48:24 +0200] rev 23505
completed some references
Tue, 26 Jun 2007 15:48:09 +0200 changes for type class ring_no_zero_divisors
paulson [Tue, 26 Jun 2007 15:48:09 +0200] rev 23504
changes for type class ring_no_zero_divisors
Tue, 26 Jun 2007 13:02:28 +0200 *** empty log message ***
nipkow [Tue, 26 Jun 2007 13:02:28 +0200] rev 23503
*** empty log message ***
Tue, 26 Jun 2007 13:01:48 +0200 added NBE
nipkow [Tue, 26 Jun 2007 13:01:48 +0200] rev 23502
added NBE
Tue, 26 Jun 2007 08:42:04 +0200 removed removed lemmas
nipkow [Tue, 26 Jun 2007 08:42:04 +0200] rev 23501
removed removed lemmas
Tue, 26 Jun 2007 00:35:14 +0200 fixed undo: try undos_proof first!
wenzelm [Tue, 26 Jun 2007 00:35:14 +0200] rev 23500
fixed undo: try undos_proof first!
Mon, 25 Jun 2007 22:46:55 +0200 tactics: more robust addressing of subgoal using (C)SUBGOAL/THEN_ALL_NEW;
wenzelm [Mon, 25 Jun 2007 22:46:55 +0200] rev 23499
tactics: more robust addressing of subgoal using (C)SUBGOAL/THEN_ALL_NEW; eta_long_tac; tuned;
Mon, 25 Jun 2007 16:56:41 +0200 removed theorem
nipkow [Mon, 25 Jun 2007 16:56:41 +0200] rev 23498
removed theorem
Mon, 25 Jun 2007 15:19:34 +0200 removed redundant lemma
nipkow [Mon, 25 Jun 2007 15:19:34 +0200] rev 23497
removed redundant lemma
Mon, 25 Jun 2007 15:19:18 +0200 removed redundant lemmas
nipkow [Mon, 25 Jun 2007 15:19:18 +0200] rev 23496
removed redundant lemmas
Mon, 25 Jun 2007 14:49:32 +0200 commented changes in HOL/Ring_and_Field.thy, and in HOL/Real/RealPow.thy
obua [Mon, 25 Jun 2007 14:49:32 +0200] rev 23495
commented changes in HOL/Ring_and_Field.thy, and in HOL/Real/RealPow.thy
Mon, 25 Jun 2007 12:16:27 +0200 removed "sum_tools.ML" in favour of BalancedTree
krauss [Mon, 25 Jun 2007 12:16:27 +0200] rev 23494
removed "sum_tools.ML" in favour of BalancedTree
Mon, 25 Jun 2007 00:36:42 +0200 added eta_long_conversion;
wenzelm [Mon, 25 Jun 2007 00:36:42 +0200] rev 23493
added eta_long_conversion;
Mon, 25 Jun 2007 00:36:41 +0200 added eta_long_tac;
wenzelm [Mon, 25 Jun 2007 00:36:41 +0200] rev 23492
added eta_long_tac;
Mon, 25 Jun 2007 00:36:40 +0200 added reasonably efficient add_cterm_frees;
wenzelm [Mon, 25 Jun 2007 00:36:40 +0200] rev 23491
added reasonably efficient add_cterm_frees;
Mon, 25 Jun 2007 00:36:39 +0200 made type conv pervasive;
wenzelm [Mon, 25 Jun 2007 00:36:39 +0200] rev 23490
made type conv pervasive; removed obsolete eta_conv (cf. Thm.eta_long_conv);
Mon, 25 Jun 2007 00:36:38 +0200 made type conv pervasive;
wenzelm [Mon, 25 Jun 2007 00:36:38 +0200] rev 23489
made type conv pervasive; Thm.eta_long_conversion; Thm.add_cterm_frees; tuned;
Mon, 25 Jun 2007 00:36:37 +0200 Thm.eta_long_conversion;
wenzelm [Mon, 25 Jun 2007 00:36:37 +0200] rev 23488
Thm.eta_long_conversion;
Mon, 25 Jun 2007 00:36:36 +0200 made type conv pervasive;
wenzelm [Mon, 25 Jun 2007 00:36:36 +0200] rev 23487
made type conv pervasive; Thm.add_cterm_frees;
Mon, 25 Jun 2007 00:36:35 +0200 Thm.add_cterm_frees;
wenzelm [Mon, 25 Jun 2007 00:36:35 +0200] rev 23486
Thm.add_cterm_frees;
Mon, 25 Jun 2007 00:36:34 +0200 made type conv pervasive;
wenzelm [Mon, 25 Jun 2007 00:36:34 +0200] rev 23485
made type conv pervasive;
Mon, 25 Jun 2007 00:36:33 +0200 made type conv pervasive;
wenzelm [Mon, 25 Jun 2007 00:36:33 +0200] rev 23484
made type conv pervasive; tuned;
Sun, 24 Jun 2007 21:15:55 +0200 tex problem fixed
nipkow [Sun, 24 Jun 2007 21:15:55 +0200] rev 23483
tex problem fixed
Sun, 24 Jun 2007 20:55:41 +0200 tuned and used field_simps
nipkow [Sun, 24 Jun 2007 20:55:41 +0200] rev 23482
tuned and used field_simps
Sun, 24 Jun 2007 20:47:05 +0200 *** empty log message ***
nipkow [Sun, 24 Jun 2007 20:47:05 +0200] rev 23481
*** empty log message ***
Sun, 24 Jun 2007 20:18:20 +0200 *** empty log message ***
nipkow [Sun, 24 Jun 2007 20:18:20 +0200] rev 23480
*** empty log message ***
Sun, 24 Jun 2007 15:17:54 +0200 new lemmas
nipkow [Sun, 24 Jun 2007 15:17:54 +0200] rev 23479
new lemmas
Sun, 24 Jun 2007 10:33:49 +0200 *** empty log message ***
nipkow [Sun, 24 Jun 2007 10:33:49 +0200] rev 23478
*** empty log message ***
Sat, 23 Jun 2007 19:33:22 +0200 tuned and renamed group_eq_simps and ring_eq_simps
nipkow [Sat, 23 Jun 2007 19:33:22 +0200] rev 23477
tuned and renamed group_eq_simps and ring_eq_simps
Fri, 22 Jun 2007 22:41:17 +0200 fix looping simp rule
huffman [Fri, 22 Jun 2007 22:41:17 +0200] rev 23476
fix looping simp rule
Fri, 22 Jun 2007 20:19:39 +0200 reinstate real_root_less_iff [simp]
huffman [Fri, 22 Jun 2007 20:19:39 +0200] rev 23475
reinstate real_root_less_iff [simp]
Fri, 22 Jun 2007 16:16:23 +0200 merge is now identity
chaieb [Fri, 22 Jun 2007 16:16:23 +0200] rev 23474
merge is now identity
Fri, 22 Jun 2007 10:23:37 +0200 new method "elim_to_cases" provides ad-hoc conversion of obtain-style
krauss [Fri, 22 Jun 2007 10:23:37 +0200] rev 23473
new method "elim_to_cases" provides ad-hoc conversion of obtain-style elimination goals to a disjunction of existentials.
Thu, 21 Jun 2007 23:49:26 +0200 section headings
huffman [Thu, 21 Jun 2007 23:49:26 +0200] rev 23472
section headings
Thu, 21 Jun 2007 23:33:10 +0200 add thm antiquotations
huffman [Thu, 21 Jun 2007 23:33:10 +0200] rev 23471
add thm antiquotations
Thu, 21 Jun 2007 23:28:44 +0200 spelling
huffman [Thu, 21 Jun 2007 23:28:44 +0200] rev 23470
spelling
Thu, 21 Jun 2007 22:52:22 +0200 add thm antiquotations
huffman [Thu, 21 Jun 2007 22:52:22 +0200] rev 23469
add thm antiquotations
Thu, 21 Jun 2007 22:30:58 +0200 changed simp rules for of_nat
huffman [Thu, 21 Jun 2007 22:30:58 +0200] rev 23468
changed simp rules for of_nat
Thu, 21 Jun 2007 22:10:16 +0200 tuned proofs -- avoid implicit prems;
wenzelm [Thu, 21 Jun 2007 22:10:16 +0200] rev 23467
tuned proofs -- avoid implicit prems;
Thu, 21 Jun 2007 20:48:48 +0200 moved quantifier elimination tools to Tools/Qelim/;
wenzelm [Thu, 21 Jun 2007 20:48:48 +0200] rev 23466
moved quantifier elimination tools to Tools/Qelim/;
Thu, 21 Jun 2007 20:48:47 +0200 moved Presburger setup back to Presburger.thy;
wenzelm [Thu, 21 Jun 2007 20:48:47 +0200] rev 23465
moved Presburger setup back to Presburger.thy;
Thu, 21 Jun 2007 20:07:26 +0200 tuned proofs -- avoid implicit prems;
wenzelm [Thu, 21 Jun 2007 20:07:26 +0200] rev 23464
tuned proofs -- avoid implicit prems;
Thu, 21 Jun 2007 17:28:53 +0200 tuned proofs -- avoid implicit prems;
wenzelm [Thu, 21 Jun 2007 17:28:53 +0200] rev 23463
tuned proofs -- avoid implicit prems;
Thu, 21 Jun 2007 17:28:50 +0200 renamed NatSimprocs.thy to Arith_Tools.thy;
wenzelm [Thu, 21 Jun 2007 17:28:50 +0200] rev 23462
renamed NatSimprocs.thy to Arith_Tools.thy; incorporated HOL/Presburger.thy into NatSimprocs.thy;
Thu, 21 Jun 2007 15:42:15 +0200 tuned;
wenzelm [Thu, 21 Jun 2007 15:42:15 +0200] rev 23461
tuned;
Thu, 21 Jun 2007 15:42:14 +0200 adapted tool setup;
wenzelm [Thu, 21 Jun 2007 15:42:14 +0200] rev 23460
adapted tool setup;
Thu, 21 Jun 2007 15:42:13 +0200 added Ferrante-Rackoff setup;
wenzelm [Thu, 21 Jun 2007 15:42:13 +0200] rev 23459
added Ferrante-Rackoff setup;
Thu, 21 Jun 2007 15:42:12 +0200 tuned comments;
wenzelm [Thu, 21 Jun 2007 15:42:12 +0200] rev 23458
tuned comments;
Thu, 21 Jun 2007 15:42:11 +0200 moved HOL/Tools/Presburger/qelim.ML to HOL/Tools/qelim.ML;
wenzelm [Thu, 21 Jun 2007 15:42:11 +0200] rev 23457
moved HOL/Tools/Presburger/qelim.ML to HOL/Tools/qelim.ML;
Thu, 21 Jun 2007 15:42:10 +0200 Ferrante-Rackoff quantifier elimination.
wenzelm [Thu, 21 Jun 2007 15:42:10 +0200] rev 23456
Ferrante-Rackoff quantifier elimination.
Thu, 21 Jun 2007 15:42:09 +0200 Context data for Ferrante-Rackoff quantifier elimination.
wenzelm [Thu, 21 Jun 2007 15:42:09 +0200] rev 23455
Context data for Ferrante-Rackoff quantifier elimination.
Thu, 21 Jun 2007 15:42:07 +0200 replaced Real/Ferrante-Rackoff tool by generic version in Main HOL;
wenzelm [Thu, 21 Jun 2007 15:42:07 +0200] rev 23454
replaced Real/Ferrante-Rackoff tool by generic version in Main HOL;
Thu, 21 Jun 2007 15:42:06 +0200 Dense linear order witout endpoints
wenzelm [Thu, 21 Jun 2007 15:42:06 +0200] rev 23453
Dense linear order witout endpoints and a quantifier elimination procedure in Ferrante and Rackoff style.
Thu, 21 Jun 2007 13:53:53 +0200 renamed metis-env.ML to metis_env.ML;
wenzelm [Thu, 21 Jun 2007 13:53:53 +0200] rev 23452
renamed metis-env.ML to metis_env.ML;
Thu, 21 Jun 2007 13:53:23 +0200 added Id;
wenzelm [Thu, 21 Jun 2007 13:53:23 +0200] rev 23451
added Id;
Thu, 21 Jun 2007 13:49:27 +0200 fine tune automatic generation of inversion lemmas
narboux [Thu, 21 Jun 2007 13:49:27 +0200] rev 23450
fine tune automatic generation of inversion lemmas
Thu, 21 Jun 2007 13:23:33 +0200 integration of Metis prover
paulson [Thu, 21 Jun 2007 13:23:33 +0200] rev 23449
integration of Metis prover
Thu, 21 Jun 2007 12:01:27 +0200 renamed metis-env to metis-env.ML;
wenzelm [Thu, 21 Jun 2007 12:01:27 +0200] rev 23448
renamed metis-env to metis-env.ML;
Wed, 20 Jun 2007 23:19:18 +0200 tuned comments;
wenzelm [Wed, 20 Jun 2007 23:19:18 +0200] rev 23447
tuned comments;
Wed, 20 Jun 2007 23:19:17 +0200 obsolete (cf. ATP_Linkup.thy);
wenzelm [Wed, 20 Jun 2007 23:19:17 +0200] rev 23446
obsolete (cf. ATP_Linkup.thy);
Wed, 20 Jun 2007 23:19:17 +0200 added Tools/metis_tools.ML;
wenzelm [Wed, 20 Jun 2007 23:19:17 +0200] rev 23445
added Tools/metis_tools.ML;
Wed, 20 Jun 2007 23:19:16 +0200 added Metis setup (from Metis.thy);
wenzelm [Wed, 20 Jun 2007 23:19:16 +0200] rev 23444
added Metis setup (from Metis.thy);
Wed, 20 Jun 2007 23:15:25 +0200 added HOL-Nominal-Examples;
wenzelm [Wed, 20 Jun 2007 23:15:25 +0200] rev 23443
added HOL-Nominal-Examples;
Wed, 20 Jun 2007 22:07:52 +0200 The Metis prover (slightly modified version from Larry);
wenzelm [Wed, 20 Jun 2007 22:07:52 +0200] rev 23442
The Metis prover (slightly modified version from Larry);
Wed, 20 Jun 2007 19:49:14 +0200 avoid using implicit prems in assumption
huffman [Wed, 20 Jun 2007 19:49:14 +0200] rev 23441
avoid using implicit prems in assumption
Wed, 20 Jun 2007 17:34:44 +0200 Added flexflex_first_order and tidied first_order_resolution
paulson [Wed, 20 Jun 2007 17:34:44 +0200] rev 23440
Added flexflex_first_order and tidied first_order_resolution
Wed, 20 Jun 2007 17:32:53 +0200 A more robust flexflex_unique
paulson [Wed, 20 Jun 2007 17:32:53 +0200] rev 23439
A more robust flexflex_unique
Wed, 20 Jun 2007 17:28:55 +0200 remove simp attribute from of_nat_diff, for backward compatibility with zdiff_int
huffman [Wed, 20 Jun 2007 17:28:55 +0200] rev 23438
remove simp attribute from of_nat_diff, for backward compatibility with zdiff_int
Wed, 20 Jun 2007 17:02:57 +0200 tuned error msg
krauss [Wed, 20 Jun 2007 17:02:57 +0200] rev 23437
tuned error msg
Wed, 20 Jun 2007 15:10:34 +0200 Remove dedicated flag setting elements in favour of setproverflag.
aspinall [Wed, 20 Jun 2007 15:10:34 +0200] rev 23436
Remove dedicated flag setting elements in favour of setproverflag.
Wed, 20 Jun 2007 15:10:02 +0200 Remove dedicated flag setting elements in favour of setproverflag. Restore displayconfig response in askpgip.
aspinall [Wed, 20 Jun 2007 15:10:02 +0200] rev 23435
Remove dedicated flag setting elements in favour of setproverflag. Restore displayconfig response in askpgip.
Wed, 20 Jun 2007 15:07:42 +0200 Synchronize schema with current version
aspinall [Wed, 20 Jun 2007 15:07:42 +0200] rev 23434
Synchronize schema with current version
Wed, 20 Jun 2007 14:38:24 +0200 added lemmas
nipkow [Wed, 20 Jun 2007 14:38:24 +0200] rev 23433
added lemmas
Wed, 20 Jun 2007 08:09:56 +0200 added meta_impE
nipkow [Wed, 20 Jun 2007 08:09:56 +0200] rev 23432
added meta_impE
(0) -10000 -3000 -1000 -112 +112 +1000 +3000 +10000 +30000 tip