wenzelm [Thu, 05 Jul 2007 20:01:26 +0200] rev 23590
renamed ObjectLogic.atomize_tac to ObjectLogic.atomize_prems_tac;
aspinall [Thu, 05 Jul 2007 19:59:01 +0200] rev 23589
Revert body of pgml to match schema for now [change bad for Broker]
aspinall [Thu, 05 Jul 2007 19:57:19 +0200] rev 23588
Classify -- comments as ordinary comments (no undo)
wenzelm [Thu, 05 Jul 2007 00:15:44 +0200] rev 23587
tuned;
wenzelm [Thu, 05 Jul 2007 00:06:25 +0200] rev 23586
avoid polymorphic equality;
added dest_judgment;
wenzelm [Thu, 05 Jul 2007 00:06:24 +0200] rev 23585
sort_le: tuned eq case;
wenzelm [Thu, 05 Jul 2007 00:06:23 +0200] rev 23584
tuned goal conversion interfaces;
wenzelm [Thu, 05 Jul 2007 00:06:22 +0200] rev 23583
else_conv: only handle THM | CTERM | TERM | TYPE;
prems_conv: no index;
renamed goal_conv_rule to gconv_rule;
wenzelm [Thu, 05 Jul 2007 00:06:20 +0200] rev 23582
avoid polymorphic equality;
Numeral.mk_cnumber;
wenzelm [Thu, 05 Jul 2007 00:06:19 +0200] rev 23581
tuned;
wenzelm [Thu, 05 Jul 2007 00:06:18 +0200] rev 23580
moved mk_cnumeral/mk_cnumber to Tools/numeral.ML;
tuned;
wenzelm [Thu, 05 Jul 2007 00:06:17 +0200] rev 23579
avoid polymorphic equality;
do not export ring_conv (which is not a conversion anyway);
renamed algebra_tac to ring_tac;
ring_tac: simplified tactic wrapper, no longer handles ERROR;
wenzelm [Thu, 05 Jul 2007 00:06:16 +0200] rev 23578
avoid polymorphic equality;
removed dead code;
wenzelm [Thu, 05 Jul 2007 00:06:14 +0200] rev 23577
avoid polymorphic equality;
wenzelm [Thu, 05 Jul 2007 00:06:13 +0200] rev 23576
removed dest_cTrueprop (cf. ObjectLogic.dest_judgment);
wenzelm [Thu, 05 Jul 2007 00:06:12 +0200] rev 23575
Logical operations on numerals (see also HOL/hologic.ML).
wenzelm [Thu, 05 Jul 2007 00:06:11 +0200] rev 23574
added Tools/numeral.ML;
wenzelm [Thu, 05 Jul 2007 00:06:10 +0200] rev 23573
common normalizer_funs, avoid cterm_of;
wenzelm [Thu, 05 Jul 2007 00:06:09 +0200] rev 23572
Numeral.mk_cnumber;
aspinall [Wed, 04 Jul 2007 21:20:23 +0200] rev 23571
PGML abstraction, draft version
aspinall [Wed, 04 Jul 2007 21:19:34 +0200] rev 23570
Use pgml
obua [Wed, 04 Jul 2007 17:21:02 +0200] rev 23569
fixed argument order in calls to Integer.pow
wenzelm [Wed, 04 Jul 2007 16:49:36 +0200] rev 23568
added binop_cong_rule;
wenzelm [Wed, 04 Jul 2007 16:49:35 +0200] rev 23567
export dlo_conv;
removed redundant auxiliary operations;
tuned exceptions -- avoid error here;
simplified tactic wrapper (CSUBGOAL, CONVERSION);
merge_ss: recover simpset context;
tuned;
wenzelm [Wed, 04 Jul 2007 16:49:34 +0200] rev 23566
replaced HOLogic.Trueprop_conv by ObjectLogic.judgment_conv;
nipkow [Wed, 04 Jul 2007 14:21:00 +0200] rev 23565
*** empty log message ***
nipkow [Wed, 04 Jul 2007 14:10:01 +0200] rev 23564
*** empty log message ***
paulson [Wed, 04 Jul 2007 13:56:26 +0200] rev 23563
simplified a proof
wenzelm [Tue, 03 Jul 2007 23:00:42 +0200] rev 23562
tuned;
wenzelm [Tue, 03 Jul 2007 22:27:30 +0200] rev 23561
CONVERSION: handle TYPE | TERM | CTERM | THM;
wenzelm [Tue, 03 Jul 2007 22:27:27 +0200] rev 23560
proper use of ioa_package.ML;
wenzelm [Tue, 03 Jul 2007 22:27:25 +0200] rev 23559
tuned;
wenzelm [Tue, 03 Jul 2007 22:27:19 +0200] rev 23558
tuned is_comb/is_binop -- avoid construction of cterms;
removed conjunction rules (cf. HOLogic.conj_XXX);
wenzelm [Tue, 03 Jul 2007 22:27:16 +0200] rev 23557
HOLogic.conj_intr/elims;
removed obsolete assocd/assoc;
removed dead string_of_pol;
tuned;
wenzelm [Tue, 03 Jul 2007 22:27:13 +0200] rev 23556
use mucke_oracle.ML only once;
wenzelm [Tue, 03 Jul 2007 22:27:11 +0200] rev 23555
assume basic HOL context for compilation (antiquotations);
added dest_cTrueprop;
tuned Trueprop_conv;
added low-level conj_intr/elim/elis (dire need for @{rule} antiquotation!);
wenzelm [Tue, 03 Jul 2007 22:27:08 +0200] rev 23554
proper use of function_package ML files;
wenzelm [Tue, 03 Jul 2007 22:27:05 +0200] rev 23553
use hologic.ML in basic HOL context;
tuned proofs;
paulson [Tue, 03 Jul 2007 21:56:25 +0200] rev 23552
to handle non-atomic assumptions
wenzelm [Tue, 03 Jul 2007 20:26:08 +0200] rev 23551
rename class dom to ring_1_no_zero_divisors (cf. HOL/Ring_and_Field.thy 1.84 by huffman);
huffman [Tue, 03 Jul 2007 18:42:09 +0200] rev 23550
convert instance proofs to Isar style
chaieb [Tue, 03 Jul 2007 18:00:57 +0200] rev 23549
Dependency on reflection_data.ML to build HOL-ex
chaieb [Tue, 03 Jul 2007 17:50:00 +0200] rev 23548
Generalized case for atoms. Selection of environment lists is allowed more than once.
chaieb [Tue, 03 Jul 2007 17:49:58 +0200] rev 23547
More examples
chaieb [Tue, 03 Jul 2007 17:49:55 +0200] rev 23546
reflection and reification methods now manage Context data
chaieb [Tue, 03 Jul 2007 17:49:53 +0200] rev 23545
Context Data for the reflection and reification methods
huffman [Tue, 03 Jul 2007 17:28:36 +0200] rev 23544
rename class dom to ring_1_no_zero_divisors
wenzelm [Tue, 03 Jul 2007 17:17:17 +0200] rev 23543
rewrite_goal_tac;
wenzelm [Tue, 03 Jul 2007 17:17:16 +0200] rev 23542
replaced Conv.goals_conv by Conv.prems_conv;
wenzelm [Tue, 03 Jul 2007 17:17:15 +0200] rev 23541
exported meta_rewrite_conv;
CONVERSION tactical;
wenzelm [Tue, 03 Jul 2007 17:17:15 +0200] rev 23540
CONVERSION tactical;
MetaSimplifier.rewrite_goal_tac;
wenzelm [Tue, 03 Jul 2007 17:17:13 +0200] rev 23539
removed obsolete eta_long_tac;
wenzelm [Tue, 03 Jul 2007 17:17:13 +0200] rev 23538
added CONVERSION tactical;
tuned signature;
wenzelm [Tue, 03 Jul 2007 17:17:11 +0200] rev 23537
tuned rotate_prems;
tuned comments;
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);
wenzelm [Tue, 03 Jul 2007 17:17:09 +0200] rev 23535
removed obsolete mk_conjunction_list, intr/elim_list;
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;
wenzelm [Tue, 03 Jul 2007 17:17:07 +0200] rev 23533
Conjunction.intr/elim_balanced;
CONVERSION tactical;
tuned;
wenzelm [Tue, 03 Jul 2007 17:17:07 +0200] rev 23532
CONVERSION tactical;
Simplifier.rewrite_goal_tac;
wenzelm [Tue, 03 Jul 2007 17:17:06 +0200] rev 23531
Conjunction.mk_conjunction_balanced;
wenzelm [Tue, 03 Jul 2007 17:17:04 +0200] rev 23530
CONVERSION tactical;
nipkow [Tue, 03 Jul 2007 15:23:11 +0200] rev 23529
Fixed problem with patterns in lambdas
krauss [Tue, 03 Jul 2007 14:48:27 +0200] rev 23528
fixed an issue with mutual recursion
huffman [Tue, 03 Jul 2007 01:26:06 +0200] rev 23527
instance pordered_comm_ring < pordered_ring
nipkow [Mon, 02 Jul 2007 23:14:06 +0200] rev 23526
Added pattern maatching for lambda abstraction
paulson [Mon, 02 Jul 2007 16:42:37 +0200] rev 23525
revised the discussion of type classes
chaieb [Mon, 02 Jul 2007 10:43:20 +0200] rev 23524
Generic QE need no Context anymore
chaieb [Mon, 02 Jul 2007 10:43:19 +0200] rev 23523
Handle exception TYPE
chaieb [Mon, 02 Jul 2007 10:43:17 +0200] rev 23522
Tuned proofs
obua [Sat, 30 Jun 2007 17:30:10 +0200] rev 23521
added ordered_ring and ordered_semiring
haftmann [Fri, 29 Jun 2007 21:23:05 +0200] rev 23520
tuned arithmetic modules
paulson [Fri, 29 Jun 2007 18:21:25 +0200] rev 23519
bug fixes to proof reconstruction
haftmann [Fri, 29 Jun 2007 16:05:00 +0200] rev 23518
dropped local cg cmd
haftmann [Thu, 28 Jun 2007 19:09:43 +0200] rev 23517
dropped toplevel lcm, gcd
haftmann [Thu, 28 Jun 2007 19:09:41 +0200] rev 23516
proper collapse_let
haftmann [Thu, 28 Jun 2007 19:09:38 +0200] rev 23515
new code generator framework
haftmann [Thu, 28 Jun 2007 19:09:36 +0200] rev 23514
dropped Library.lcm
haftmann [Thu, 28 Jun 2007 19:09:35 +0200] rev 23513
tuned
haftmann [Thu, 28 Jun 2007 19:09:34 +0200] rev 23512
code generation for dvd
haftmann [Thu, 28 Jun 2007 19:09:32 +0200] rev 23511
simplified keyword setup
paulson [Wed, 27 Jun 2007 12:41:36 +0200] rev 23510
GPL -> BSD
nipkow [Wed, 27 Jun 2007 11:06:43 +0200] rev 23509
*** empty log message ***
paulson [Tue, 26 Jun 2007 18:32:53 +0200] rev 23508
updated for metis method
paulson [Tue, 26 Jun 2007 18:32:24 +0200] rev 23507
recoded
paulson [Tue, 26 Jun 2007 18:28:40 +0200] rev 23506
simplified
paulson [Tue, 26 Jun 2007 15:48:24 +0200] rev 23505
completed some references
paulson [Tue, 26 Jun 2007 15:48:09 +0200] rev 23504
changes for type class ring_no_zero_divisors
nipkow [Tue, 26 Jun 2007 13:02:28 +0200] rev 23503
*** empty log message ***
nipkow [Tue, 26 Jun 2007 13:01:48 +0200] rev 23502
added NBE
nipkow [Tue, 26 Jun 2007 08:42:04 +0200] rev 23501
removed removed lemmas
wenzelm [Tue, 26 Jun 2007 00:35:14 +0200] rev 23500
fixed undo: try undos_proof first!
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;
nipkow [Mon, 25 Jun 2007 16:56:41 +0200] rev 23498
removed theorem
nipkow [Mon, 25 Jun 2007 15:19:34 +0200] rev 23497
removed redundant lemma
nipkow [Mon, 25 Jun 2007 15:19:18 +0200] rev 23496
removed redundant lemmas
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
krauss [Mon, 25 Jun 2007 12:16:27 +0200] rev 23494
removed "sum_tools.ML" in favour of BalancedTree
wenzelm [Mon, 25 Jun 2007 00:36:42 +0200] rev 23493
added eta_long_conversion;
wenzelm [Mon, 25 Jun 2007 00:36:41 +0200] rev 23492
added eta_long_tac;
wenzelm [Mon, 25 Jun 2007 00:36:40 +0200] rev 23491
added reasonably efficient add_cterm_frees;
wenzelm [Mon, 25 Jun 2007 00:36:39 +0200] rev 23490
made type conv pervasive;
removed obsolete eta_conv (cf. Thm.eta_long_conv);
wenzelm [Mon, 25 Jun 2007 00:36:38 +0200] rev 23489
made type conv pervasive;
Thm.eta_long_conversion;
Thm.add_cterm_frees;
tuned;
wenzelm [Mon, 25 Jun 2007 00:36:37 +0200] rev 23488
Thm.eta_long_conversion;
wenzelm [Mon, 25 Jun 2007 00:36:36 +0200] rev 23487
made type conv pervasive;
Thm.add_cterm_frees;
wenzelm [Mon, 25 Jun 2007 00:36:35 +0200] rev 23486
Thm.add_cterm_frees;
wenzelm [Mon, 25 Jun 2007 00:36:34 +0200] rev 23485
made type conv pervasive;
wenzelm [Mon, 25 Jun 2007 00:36:33 +0200] rev 23484
made type conv pervasive;
tuned;
nipkow [Sun, 24 Jun 2007 21:15:55 +0200] rev 23483
tex problem fixed
nipkow [Sun, 24 Jun 2007 20:55:41 +0200] rev 23482
tuned and used field_simps
nipkow [Sun, 24 Jun 2007 20:47:05 +0200] rev 23481
*** empty log message ***
nipkow [Sun, 24 Jun 2007 20:18:20 +0200] rev 23480
*** empty log message ***
nipkow [Sun, 24 Jun 2007 15:17:54 +0200] rev 23479
new lemmas
nipkow [Sun, 24 Jun 2007 10:33:49 +0200] rev 23478
*** empty log message ***
nipkow [Sat, 23 Jun 2007 19:33:22 +0200] rev 23477
tuned and renamed group_eq_simps and ring_eq_simps
huffman [Fri, 22 Jun 2007 22:41:17 +0200] rev 23476
fix looping simp rule
huffman [Fri, 22 Jun 2007 20:19:39 +0200] rev 23475
reinstate real_root_less_iff [simp]
chaieb [Fri, 22 Jun 2007 16:16:23 +0200] rev 23474
merge is now identity
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.
huffman [Thu, 21 Jun 2007 23:49:26 +0200] rev 23472
section headings
huffman [Thu, 21 Jun 2007 23:33:10 +0200] rev 23471
add thm antiquotations