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
huffman [Thu, 21 Jun 2007 23:28:44 +0200] rev 23470
spelling
huffman [Thu, 21 Jun 2007 22:52:22 +0200] rev 23469
add thm antiquotations
huffman [Thu, 21 Jun 2007 22:30:58 +0200] rev 23468
changed simp rules for of_nat
wenzelm [Thu, 21 Jun 2007 22:10:16 +0200] rev 23467
tuned proofs -- avoid implicit prems;
wenzelm [Thu, 21 Jun 2007 20:48:48 +0200] rev 23466
moved quantifier elimination tools to Tools/Qelim/;
wenzelm [Thu, 21 Jun 2007 20:48:47 +0200] rev 23465
moved Presburger setup back to Presburger.thy;
wenzelm [Thu, 21 Jun 2007 20:07:26 +0200] rev 23464
tuned proofs -- avoid implicit prems;
wenzelm [Thu, 21 Jun 2007 17:28:53 +0200] rev 23463
tuned proofs -- avoid implicit prems;
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;
wenzelm [Thu, 21 Jun 2007 15:42:15 +0200] rev 23461
tuned;
wenzelm [Thu, 21 Jun 2007 15:42:14 +0200] rev 23460
adapted tool setup;
wenzelm [Thu, 21 Jun 2007 15:42:13 +0200] rev 23459
added Ferrante-Rackoff setup;
wenzelm [Thu, 21 Jun 2007 15:42:12 +0200] rev 23458
tuned comments;
wenzelm [Thu, 21 Jun 2007 15:42:11 +0200] rev 23457
moved HOL/Tools/Presburger/qelim.ML to HOL/Tools/qelim.ML;
wenzelm [Thu, 21 Jun 2007 15:42:10 +0200] rev 23456
Ferrante-Rackoff quantifier elimination.
wenzelm [Thu, 21 Jun 2007 15:42:09 +0200] rev 23455
Context data for Ferrante-Rackoff quantifier elimination.
wenzelm [Thu, 21 Jun 2007 15:42:07 +0200] rev 23454
replaced Real/Ferrante-Rackoff tool by generic version in Main HOL;
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.
wenzelm [Thu, 21 Jun 2007 13:53:53 +0200] rev 23452
renamed metis-env.ML to metis_env.ML;
wenzelm [Thu, 21 Jun 2007 13:53:23 +0200] rev 23451
added Id;
narboux [Thu, 21 Jun 2007 13:49:27 +0200] rev 23450
fine tune automatic generation of inversion lemmas
paulson [Thu, 21 Jun 2007 13:23:33 +0200] rev 23449
integration of Metis prover
wenzelm [Thu, 21 Jun 2007 12:01:27 +0200] rev 23448
renamed metis-env to metis-env.ML;
wenzelm [Wed, 20 Jun 2007 23:19:18 +0200] rev 23447
tuned comments;
wenzelm [Wed, 20 Jun 2007 23:19:17 +0200] rev 23446
obsolete (cf. ATP_Linkup.thy);
wenzelm [Wed, 20 Jun 2007 23:19:17 +0200] rev 23445
added Tools/metis_tools.ML;
wenzelm [Wed, 20 Jun 2007 23:19:16 +0200] rev 23444
added Metis setup (from Metis.thy);
wenzelm [Wed, 20 Jun 2007 23:15:25 +0200] rev 23443
added HOL-Nominal-Examples;
wenzelm [Wed, 20 Jun 2007 22:07:52 +0200] rev 23442
The Metis prover (slightly modified version from Larry);
huffman [Wed, 20 Jun 2007 19:49:14 +0200] rev 23441
avoid using implicit prems in assumption
paulson [Wed, 20 Jun 2007 17:34:44 +0200] rev 23440
Added flexflex_first_order and tidied first_order_resolution
paulson [Wed, 20 Jun 2007 17:32:53 +0200] rev 23439
A more robust flexflex_unique
huffman [Wed, 20 Jun 2007 17:28:55 +0200] rev 23438
remove simp attribute from of_nat_diff, for backward compatibility with zdiff_int
krauss [Wed, 20 Jun 2007 17:02:57 +0200] rev 23437
tuned error msg
aspinall [Wed, 20 Jun 2007 15:10:34 +0200] rev 23436
Remove dedicated flag setting elements in favour of setproverflag.
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.
aspinall [Wed, 20 Jun 2007 15:07:42 +0200] rev 23434
Synchronize schema with current version
nipkow [Wed, 20 Jun 2007 14:38:24 +0200] rev 23433
added lemmas
nipkow [Wed, 20 Jun 2007 08:09:56 +0200] rev 23432
added meta_impE
huffman [Wed, 20 Jun 2007 05:18:39 +0200] rev 23431
change simp rules for of_nat to work like int did previously (reorient of_nat_Suc, remove of_nat_mult [simp]); preserve original variable names in legacy int theorems
huffman [Wed, 20 Jun 2007 05:06:56 +0200] rev 23430
section headings
huffman [Wed, 20 Jun 2007 05:06:16 +0200] rev 23429
simplify some proofs
wenzelm [Tue, 19 Jun 2007 23:21:39 +0200] rev 23428
oops -- fixed profiling;
wenzelm [Tue, 19 Jun 2007 23:16:14 +0200] rev 23427
Balanced binary trees (material from library.ML);
wenzelm [Tue, 19 Jun 2007 23:15:59 +0200] rev 23426
profiling: observe no_timing;
wenzelm [Tue, 19 Jun 2007 23:15:57 +0200] rev 23425
added raw_tactic;
wenzelm [Tue, 19 Jun 2007 23:15:54 +0200] rev 23424
moved balanced tree operations to General/balanced_tree.ML;
wenzelm [Tue, 19 Jun 2007 23:15:51 +0200] rev 23423
added with_subgoal;
wenzelm [Tue, 19 Jun 2007 23:15:49 +0200] rev 23422
balanced conjunctions;
tuned interfaces;
tuned;
wenzelm [Tue, 19 Jun 2007 23:15:47 +0200] rev 23421
balanced conjunctions;
added split_defined (from conjunction.ML);
wenzelm [Tue, 19 Jun 2007 23:15:43 +0200] rev 23420
added General/balanced_tree.ML;
wenzelm [Tue, 19 Jun 2007 23:15:38 +0200] rev 23419
BalancedTree;
wenzelm [Tue, 19 Jun 2007 23:15:27 +0200] rev 23418
balanced conjunctions;
wenzelm [Tue, 19 Jun 2007 23:15:23 +0200] rev 23417
tuned;
krauss [Tue, 19 Jun 2007 18:00:49 +0200] rev 23416
generalized proofs so that call graphs can have any node type.
wenzelm [Tue, 19 Jun 2007 00:02:16 +0200] rev 23415
macbroy5: trying -j 2;
wenzelm [Mon, 18 Jun 2007 23:30:46 +0200] rev 23414
tuned conjunction tactics: slightly smaller proof terms;
nipkow [Sun, 17 Jun 2007 18:47:03 +0200] rev 23413
tuned laws for cancellation in divisions for fields.
chaieb [Sun, 17 Jun 2007 13:39:50 +0200] rev 23412
moved nonzero_mult_divide_cancel_right to Ring_and_Field as nonzero_mult_divide_cancel_right'; tuned proofs
chaieb [Sun, 17 Jun 2007 13:39:48 +0200] rev 23411
Added eta_conv and eta-expansion conversion: waiting for it to be in thm.ML; exported is_refl
chaieb [Sun, 17 Jun 2007 13:39:45 +0200] rev 23410
gen_qelim_conv now reduces the universal quatifier to the existential one; Now also deals with Ex f for eta-contracted f;
chaieb [Sun, 17 Jun 2007 13:39:39 +0200] rev 23409
thin_prems_tac first max-scopes universal quantifiers; eta_conv moved to Pure/conv.ML
chaieb [Sun, 17 Jun 2007 13:39:34 +0200] rev 23408
Tuned error messages; tuned;
chaieb [Sun, 17 Jun 2007 13:39:32 +0200] rev 23407
normalizer conversions depend on the proof context; added functions for conversion and wrapper that sill depend on the variable ordering (_ord)
chaieb [Sun, 17 Jun 2007 13:39:29 +0200] rev 23406
added theorems nonzero_mult_divide_cancel_right' nonzero_mult_divide_cancel_left' ordered_field_no_lb ordered_field_no_ub
chaieb [Sun, 17 Jun 2007 13:39:27 +0200] rev 23405
moved lemma all_not_ex to HOL.thy ; tuned proofs
chaieb [Sun, 17 Jun 2007 13:39:25 +0200] rev 23404
Tuned instantiation of Groebner bases to fields
chaieb [Sun, 17 Jun 2007 13:39:22 +0200] rev 23403
added Theorem all_not_ex
nipkow [Sun, 17 Jun 2007 08:56:13 +0200] rev 23402
renamed vars in zle_trans for compatibility
nipkow [Sat, 16 Jun 2007 16:27:35 +0200] rev 23401
tuned
nipkow [Sat, 16 Jun 2007 15:01:54 +0200] rev 23400
The simprocs "divide_cancel_factor" and "ring_eq_cancel_factor" no
longer need class numeral_ring. This made a number of special
simp-thms redundant.
berghofe [Fri, 15 Jun 2007 19:19:23 +0200] rev 23399
Locally added definition of "int :: nat => int" again to make
code generation work.
nipkow [Fri, 15 Jun 2007 15:10:32 +0200] rev 23398
made divide_self a simp rule
nipkow [Fri, 15 Jun 2007 09:10:06 +0200] rev 23397
Removed thunk from Fun
nipkow [Fri, 15 Jun 2007 09:09:06 +0200] rev 23396
Church numerals added
wenzelm [Thu, 14 Jun 2007 23:04:40 +0200] rev 23395
method assumption: uniform treatment of prems as legacy feature;
wenzelm [Thu, 14 Jun 2007 23:04:39 +0200] rev 23394
tuned proofs;
wenzelm [Thu, 14 Jun 2007 23:04:36 +0200] rev 23393
tuned proofs: avoid implicit prems;
chaieb [Thu, 14 Jun 2007 22:59:42 +0200] rev 23392
fixed term_constants (impact on is_relevant); terms in generalize_tac are sorted before we abstract over them (to *try* to avoid the case when a term to be abstracted over already occurs in an other)
chaieb [Thu, 14 Jun 2007 22:59:40 +0200] rev 23391
no computation rules in the pre-simplifiaction set
chaieb [Thu, 14 Jun 2007 22:59:39 +0200] rev 23390
Added some lemmas to default presburger simpset; tuned proofs
wenzelm [Thu, 14 Jun 2007 18:33:31 +0200] rev 23389
tuned proofs: avoid implicit prems;
wenzelm [Thu, 14 Jun 2007 18:33:29 +0200] rev 23388
tuned proofs: avoid implicit prems;
tuned partition proofs;
paulson [Thu, 14 Jun 2007 13:19:50 +0200] rev 23387
Now ResHolClause also does first-order problems!
paulson [Thu, 14 Jun 2007 13:18:59 +0200] rev 23386
Now also handles FO problems
paulson [Thu, 14 Jun 2007 13:18:24 +0200] rev 23385
Deleted unused code
paulson [Thu, 14 Jun 2007 13:16:44 +0200] rev 23384
tidied
wenzelm [Thu, 14 Jun 2007 10:38:48 +0200] rev 23383
tuned proofs: avoid implicit prems;
kleing [Thu, 14 Jun 2007 09:54:14 +0200] rev 23382
clarified who we consider to be a contributor
chaieb [Thu, 14 Jun 2007 09:37:38 +0200] rev 23381
Fixed Problem with ML-bindings for thm names;
nipkow [Thu, 14 Jun 2007 07:27:55 +0200] rev 23380
fixed filter syntax
wenzelm [Thu, 14 Jun 2007 00:48:42 +0200] rev 23379
updated 'find_theorems' -- moved ProofGeneral specifics to ProofGeneral/CHANGES;
wenzelm [Thu, 14 Jun 2007 00:22:45 +0200] rev 23378
tuned proofs: avoid implicit prems;
huffman [Wed, 13 Jun 2007 19:14:51 +0200] rev 23377
int abbreviates of_nat
wenzelm [Wed, 13 Jun 2007 18:30:17 +0200] rev 23376
tuned proofs: avoid implicit prems;
tuned;
wenzelm [Wed, 13 Jun 2007 18:30:16 +0200] rev 23375
tuned proofs: avoid implicit prems;
major cleanup of proofs/document;
wenzelm [Wed, 13 Jun 2007 18:30:15 +0200] rev 23374
tuned comments;
wenzelm [Wed, 13 Jun 2007 18:30:11 +0200] rev 23373
tuned proofs: avoid implicit prems;
huffman [Wed, 13 Jun 2007 16:43:02 +0200] rev 23372
clean up instance proofs; reorganize section headings
wenzelm [Wed, 13 Jun 2007 14:21:54 +0200] rev 23371
reactivated theory Class;
urbanc [Wed, 13 Jun 2007 12:22:02 +0200] rev 23370
added the Q_Unit rule (was missing) and adjusted the proof accordingly
wenzelm [Wed, 13 Jun 2007 11:54:03 +0200] rev 23369
* Isar: method "assumption" (implicit closing of subproofs) takes non-atomic goal assumptions into account;
* Isar: implicit use of prems from the Isar proof context is considered a legacy feature;
narboux [Wed, 13 Jun 2007 11:16:24 +0200] rev 23368
generate_fresh works even if there is no free variable in the goal
wenzelm [Wed, 13 Jun 2007 10:44:35 +0200] rev 23367
tuned;
wenzelm [Wed, 13 Jun 2007 10:43:38 +0200] rev 23366
tuned proofs: avoid implicit prems;
huffman [Wed, 13 Jun 2007 03:31:11 +0200] rev 23365
removed constant int :: nat => int;
int is now an abbreviation for of_nat :: nat => int
huffman [Wed, 13 Jun 2007 03:28:21 +0200] rev 23364
thm antiquotations
wenzelm [Wed, 13 Jun 2007 00:02:06 +0200] rev 23363
transaction: context_position (non-destructive only);
wenzelm [Wed, 13 Jun 2007 00:02:05 +0200] rev 23362
added map_current;
simplified internal type proof;
wenzelm [Wed, 13 Jun 2007 00:02:04 +0200] rev 23361
tuned msg;
wenzelm [Wed, 13 Jun 2007 00:02:03 +0200] rev 23360
apply_method/end_proof: pass position;
Method.Basic: include position;
wenzelm [Wed, 13 Jun 2007 00:02:02 +0200] rev 23359
renamed map to map_current;
wenzelm [Wed, 13 Jun 2007 00:02:01 +0200] rev 23358
tuned;
wenzelm [Wed, 13 Jun 2007 00:02:00 +0200] rev 23357
removed unused is_atomic;
wenzelm [Wed, 13 Jun 2007 00:01:59 +0200] rev 23356
renamed prove_raw to prove_internal;
tuned;
wenzelm [Wed, 13 Jun 2007 00:01:58 +0200] rev 23355
merge/merge_refs: plain error instead of exception TERM;
wenzelm [Wed, 13 Jun 2007 00:01:57 +0200] rev 23354
Context positions.
wenzelm [Wed, 13 Jun 2007 00:01:56 +0200] rev 23353
added context_position.ML;
wenzelm [Wed, 13 Jun 2007 00:01:54 +0200] rev 23352
renamed Goal.prove_raw to Goal.prove_internal;
wenzelm [Wed, 13 Jun 2007 00:01:51 +0200] rev 23351
Method.Basic: include position;
wenzelm [Wed, 13 Jun 2007 00:01:41 +0200] rev 23350
tuned proofs: avoid implicit prems;
wenzelm [Wed, 13 Jun 2007 00:01:38 +0200] rev 23349
Basic text: include position;
assumption/close: refer to non-atomic assumptions as well, implicit use of prems now considered legacy feature;
huffman [Tue, 12 Jun 2007 23:39:02 +0200] rev 23348
thm antiquotations
huffman [Tue, 12 Jun 2007 23:14:29 +0200] rev 23347
add lemma inj_of_nat
huffman [Tue, 12 Jun 2007 21:59:40 +0200] rev 23346
thm antiquotations
chaieb [Tue, 12 Jun 2007 20:49:56 +0200] rev 23345
Unfortunately needed patch due to incompatibility with SML -- oo is infix and hence can not appear on the left handside of patterns
chaieb [Tue, 12 Jun 2007 20:49:50 +0200] rev 23344
changed int stuff into integer for SMLNJ compatibility
huffman [Tue, 12 Jun 2007 17:20:30 +0200] rev 23343
more of_rat lemmas
huffman [Tue, 12 Jun 2007 17:04:26 +0200] rev 23342
add function of_rat and related lemmas
chaieb [Tue, 12 Jun 2007 12:00:03 +0200] rev 23341
turned curry (op opr) into curry op opr --- because of smlnj
wenzelm [Tue, 12 Jun 2007 11:01:16 +0200] rev 23340
De-overloaded operations for int and real.
wenzelm [Tue, 12 Jun 2007 11:00:18 +0200] rev 23339
SML basis with type int representing proper integers, not machine words.
chaieb [Tue, 12 Jun 2007 10:40:44 +0200] rev 23338
Tuned proofs : now use 'algebra ad: ...'
chaieb [Tue, 12 Jun 2007 10:15:58 +0200] rev 23337
cooper_tac takes now two lists of theorems to be added/deleted from the simpset dor pre-simplification
chaieb [Tue, 12 Jun 2007 10:15:52 +0200] rev 23336
changed val restriction to local due to smlnj
chaieb [Tue, 12 Jun 2007 10:15:48 +0200] rev 23335
Changed normalizer Data to contain a simpset besides the list of instances; Before the method starts, it simplifies with this simpset; Added attribute 'algebra' to add and delete theorems from the simpset above;
chaieb [Tue, 12 Jun 2007 10:15:45 +0200] rev 23334
Added algebra_tac; tuned;
chaieb [Tue, 12 Jun 2007 10:15:40 +0200] rev 23333
Method now takes theorems to be added or deleted from a simpset for simplificatio before the core method starts
chaieb [Tue, 12 Jun 2007 10:15:32 +0200] rev 23332
algebra_tac moved to file Tools/Groebner_Basis/groebner.ML; Method now takes theorems to be added or deleted from a simpset for simplificatio *before* the core method starts
nipkow [Mon, 11 Jun 2007 18:34:12 +0200] rev 23331
nex example
chaieb [Mon, 11 Jun 2007 18:28:16 +0200] rev 23330
Conversion for computation on constants now depends on the context
chaieb [Mon, 11 Jun 2007 18:28:15 +0200] rev 23329
tuned setup for the fields instantiation for Groebner Bases;
chaieb [Mon, 11 Jun 2007 18:26:44 +0200] rev 23328
Added dependency on file Groebner_Basis.thy
chaieb [Mon, 11 Jun 2007 16:23:17 +0200] rev 23327
Added instantiation of algebra method to fields
nipkow [Mon, 11 Jun 2007 16:21:03 +0200] rev 23326
hid constant "dom"
chaieb [Mon, 11 Jun 2007 11:10:04 +0200] rev 23325
Removed from CVS, since obselete in the new Presburger Method;
chaieb [Mon, 11 Jun 2007 11:07:18 +0200] rev 23324
Generated reflected QE procedure for Presburger Arithmetic-- Cooper's Algorithm -- see HOL/ex/Reflected_Presburger.thy