Tue, 12 Jun 2007 23:14:29 +0200 huffman add lemma inj_of_nat
Tue, 12 Jun 2007 21:59:40 +0200 huffman thm antiquotations
Tue, 12 Jun 2007 20:49:56 +0200 chaieb Unfortunately needed patch due to incompatibility with SML -- oo is infix and hence can not appear on the left handside of patterns
Tue, 12 Jun 2007 20:49:50 +0200 chaieb changed int stuff into integer for SMLNJ compatibility
Tue, 12 Jun 2007 17:20:30 +0200 huffman more of_rat lemmas
Tue, 12 Jun 2007 17:04:26 +0200 huffman add function of_rat and related lemmas
Tue, 12 Jun 2007 12:00:03 +0200 chaieb turned curry (op opr) into curry op opr --- because of smlnj
Tue, 12 Jun 2007 11:01:16 +0200 wenzelm De-overloaded operations for int and real.
Tue, 12 Jun 2007 11:00:18 +0200 wenzelm SML basis with type int representing proper integers, not machine words.
Tue, 12 Jun 2007 10:40:44 +0200 chaieb Tuned proofs : now use 'algebra ad: ...'
Tue, 12 Jun 2007 10:15:58 +0200 chaieb cooper_tac takes now two lists of theorems to be added/deleted from the simpset dor pre-simplification
Tue, 12 Jun 2007 10:15:52 +0200 chaieb changed val restriction to local due to smlnj
Tue, 12 Jun 2007 10:15:48 +0200 chaieb 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;
Tue, 12 Jun 2007 10:15:45 +0200 chaieb Added algebra_tac; tuned;
Tue, 12 Jun 2007 10:15:40 +0200 chaieb Method now takes theorems to be added or deleted from a simpset for simplificatio before the core method starts
Tue, 12 Jun 2007 10:15:32 +0200 chaieb 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
Mon, 11 Jun 2007 18:34:12 +0200 nipkow nex example
Mon, 11 Jun 2007 18:28:16 +0200 chaieb Conversion for computation on constants now depends on the context
Mon, 11 Jun 2007 18:28:15 +0200 chaieb tuned setup for the fields instantiation for Groebner Bases;
Mon, 11 Jun 2007 18:26:44 +0200 chaieb Added dependency on file Groebner_Basis.thy
Mon, 11 Jun 2007 16:23:17 +0200 chaieb Added instantiation of algebra method to fields
Mon, 11 Jun 2007 16:21:03 +0200 nipkow hid constant "dom"
Mon, 11 Jun 2007 11:10:04 +0200 chaieb Removed from CVS, since obselete in the new Presburger Method;
Mon, 11 Jun 2007 11:07:18 +0200 chaieb Generated reflected QE procedure for Presburger Arithmetic-- Cooper's Algorithm -- see HOL/ex/Reflected_Presburger.thy
Mon, 11 Jun 2007 11:06:23 +0200 chaieb Added more examples
Mon, 11 Jun 2007 11:06:21 +0200 chaieb Now only contains generic conversion for quantifier elimination in HOL
Mon, 11 Jun 2007 11:06:19 +0200 chaieb A new tactic for Presburger;
Mon, 11 Jun 2007 11:06:18 +0200 chaieb tuned
Mon, 11 Jun 2007 11:06:17 +0200 chaieb Temporarily added theorems for QE that were in old Presburger.thy ; This will diseappear with the new Ferrante and Rackoff shortly;
Mon, 11 Jun 2007 11:06:15 +0200 chaieb tuned tactic
Mon, 11 Jun 2007 11:06:13 +0200 chaieb Temporarily use int instead of IntInf.int but Code generator should map HOL's int to ML's IntInf.int --- To be fixed
Mon, 11 Jun 2007 11:06:11 +0200 chaieb tuned Proof and Document
Mon, 11 Jun 2007 11:06:04 +0200 chaieb tuned Proof
Mon, 11 Jun 2007 11:06:00 +0200 chaieb A new and cleaned up Theory for QE. for Presburger arithmetic
Mon, 11 Jun 2007 11:05:59 +0200 chaieb Added new files for Presburger (cooper_data.ML, cooper.ML) and deleted old unused ones cooper_dec, cooper_proof, reflected_cooper etc..
Mon, 11 Jun 2007 11:05:57 +0200 chaieb explicitely depends on file groebner.ML
Mon, 11 Jun 2007 11:05:56 +0200 chaieb Context Data for the new presburger Method
Mon, 11 Jun 2007 11:05:54 +0200 chaieb A new simpler and cleaner implementation of proof Synthesis for Presburger Arithmetic --- Cooper's Algorithm
Mon, 11 Jun 2007 07:10:06 +0200 huffman remove references to constant int::nat=>int
Mon, 11 Jun 2007 06:14:32 +0200 huffman simplify int proofs
Mon, 11 Jun 2007 05:20:05 +0200 huffman modify proofs to avoid referring to int::nat=>int
Mon, 11 Jun 2007 02:25:55 +0200 huffman add int_of_nat versions of lemmas about int::nat=>int
Mon, 11 Jun 2007 02:24:39 +0200 huffman add lemma of_nat_power
Mon, 11 Jun 2007 01:22:29 +0200 huffman add int_of_nat versions of lemmas about int::nat=>int
Mon, 11 Jun 2007 00:53:18 +0200 huffman add abbreviation int_of_nat for of_nat::nat=>int;
Sun, 10 Jun 2007 23:48:27 +0200 wenzelm disabled theory "Reflected_Presburger" for smlnj (temporarily);
Sun, 10 Jun 2007 21:06:59 +0200 wenzelm disabled theories MIR and ReflectedFerrack for smlnj (temporarily);
Sun, 10 Jun 2007 10:23:42 +0200 nipkow *** empty log message ***
Sat, 09 Jun 2007 02:38:51 +0200 huffman remove dependencies of proofs on constant int::nat=>int, preparing to remove it
Sat, 09 Jun 2007 00:28:47 +0200 wenzelm eqtype int -- explicitly encourage overloaded equality;
Sat, 09 Jun 2007 00:28:46 +0200 wenzelm simplified type integer;
Fri, 08 Jun 2007 18:13:58 +0200 berghofe Adapted Proofterm.bicompose_proof to Larry's changes in
Fri, 08 Jun 2007 18:09:37 +0200 chaieb Method "algebra" solves polynomial equations over (semi)rings
Fri, 08 Jun 2007 03:24:27 +0200 huffman generalize zpower_number_of_{even,odd} lemmas
Thu, 07 Jun 2007 17:21:43 +0200 obua deleted comments
Thu, 07 Jun 2007 14:26:05 +0200 obua deleted legacy lemmas
Thu, 07 Jun 2007 11:25:27 +0200 nipkow somebody elses problem fixed
Thu, 07 Jun 2007 11:25:05 +0200 nipkow filter syntax change
Thu, 07 Jun 2007 04:33:15 +0200 huffman remove redundant lemmas
Thu, 07 Jun 2007 03:45:56 +0200 huffman remove references to preal-specific theorems
Thu, 07 Jun 2007 03:11:31 +0200 huffman define (1::preal); clean up instance declarations
Thu, 07 Jun 2007 02:34:37 +0200 huffman tuned
Thu, 07 Jun 2007 01:44:35 +0200 huffman instance preal :: ordered_cancel_ab_semigroup_add
Wed, 06 Jun 2007 23:06:29 +0200 huffman use new-style class for sq_ord; rename op << to sq_le
Wed, 06 Jun 2007 21:24:35 +0200 urbanc take out Class.thy again, because it does not yet compile cleanly
Wed, 06 Jun 2007 20:49:04 +0200 huffman add axclass semiring_char_0 for types where of_nat is injective
Wed, 06 Jun 2007 19:12:59 +0200 nipkow changed filter syntax from : to <-
Wed, 06 Jun 2007 19:12:40 +0200 nipkow hide filter
Wed, 06 Jun 2007 19:12:07 +0200 nipkow tuned list comprehension, changed filter syntax from : to <-
Wed, 06 Jun 2007 18:32:05 +0200 huffman clean up proofs of exp_zero, sin_zero, cos_zero
Wed, 06 Jun 2007 17:01:33 +0200 huffman generalize class constraints on some lemmas
Wed, 06 Jun 2007 17:00:09 +0200 huffman generalize of_nat and related constants to class semiring_1
Wed, 06 Jun 2007 16:42:39 +0200 huffman declare complex_diff as simp rule
Wed, 06 Jun 2007 16:12:08 +0200 chaieb New Reflected Presburger added to HOL/ex
Tue, 05 Jun 2007 22:47:49 +0200 wenzelm Groebner Basis Examples.
Tue, 05 Jun 2007 22:46:59 +0200 wenzelm print_antiquotations: sort_strings;
Tue, 05 Jun 2007 22:46:58 +0200 wenzelm tuned document;
Tue, 05 Jun 2007 22:46:57 +0200 wenzelm tuned source deps;
Tue, 05 Jun 2007 22:46:56 +0200 wenzelm simplified/renamed add_numerals;
Tue, 05 Jun 2007 22:46:55 +0200 wenzelm renamed ex/Eval_Examples.thy;
Tue, 05 Jun 2007 22:46:55 +0200 wenzelm added ex/Groebner_Examples.thy;
Tue, 05 Jun 2007 22:46:53 +0200 wenzelm tuned document;
Tue, 05 Jun 2007 20:46:25 +0200 chaieb Added two examples in Complex/ex :Reflected QE for linear real arith and QE for mixed integer real linear arithmetic
Tue, 05 Jun 2007 20:44:12 +0200 chaieb Added twe Examples for Quantifier elimination ofer linear real arithmetic and over the mixed theory of linear real artihmetic with integers
Tue, 05 Jun 2007 19:23:09 +0200 haftmann tuned boostrap
Tue, 05 Jun 2007 19:22:01 +0200 haftmann eliminated Code_Generator.thy
Tue, 05 Jun 2007 19:19:30 +0200 haftmann tuned integers
Tue, 05 Jun 2007 18:36:10 +0200 wenzelm tuned;
Tue, 05 Jun 2007 18:36:09 +0200 wenzelm fixed type int vs. integer;
Tue, 05 Jun 2007 18:36:07 +0200 wenzelm renamed locale ring/semiring to gb_ring/gb_semiring to avoid clash with Ring_and_Field versions;
Tue, 05 Jun 2007 17:16:41 +0200 huffman add new lemmas
Tue, 05 Jun 2007 16:32:16 +0200 chaieb Polynomials now only depend on Deriv; Definition of degree changed
Tue, 05 Jun 2007 16:31:10 +0200 chaieb lemma lemma_DERIV_subst moved to Deriv.thy
Tue, 05 Jun 2007 16:26:07 +0200 wenzelm tuned proofs;
Tue, 05 Jun 2007 16:26:06 +0200 wenzelm tuned comments;
Tue, 05 Jun 2007 16:26:04 +0200 wenzelm Semiring normalization and Groebner Bases.
Tue, 05 Jun 2007 15:17:02 +0200 haftmann moved generic algebra modules
Tue, 05 Jun 2007 15:16:11 +0200 haftmann updated documentation
Tue, 05 Jun 2007 15:16:10 +0200 haftmann fixed broken execption handling
Tue, 05 Jun 2007 15:16:09 +0200 haftmann simplified notion of "operational classes"
Tue, 05 Jun 2007 15:16:08 +0200 haftmann merged Code_Generator.thy into HOL.thy
Tue, 05 Jun 2007 12:12:25 +0200 chaieb added a function partition and a few lemmas
Tue, 05 Jun 2007 11:00:04 +0200 chaieb added a few theorems about foldl and set
Tue, 05 Jun 2007 10:42:31 +0200 chaieb added lcm, ilcm (lcm for integers) and some lemmas about them;
Tue, 05 Jun 2007 09:56:19 +0200 urbanc included Class.thy in the compiling process for Nominal/Examples
Tue, 05 Jun 2007 07:58:50 +0200 huffman remove simp attribute from lemma_STAR theorems
Tue, 05 Jun 2007 00:54:03 +0200 huffman add lemma exp_of_real
Mon, 04 Jun 2007 22:27:18 +0200 nipkow tuned list comprehension
Mon, 04 Jun 2007 21:04:20 +0200 wenzelm tuned;
Mon, 04 Jun 2007 21:04:19 +0200 wenzelm added is_atomic;
Mon, 04 Jun 2007 21:04:19 +0200 wenzelm added assume_rule_tac;
Mon, 04 Jun 2007 15:43:32 +0200 haftmann reverted appnd to append
Mon, 04 Jun 2007 15:43:31 +0200 haftmann authentic syntax for List.append
Mon, 04 Jun 2007 15:43:30 +0200 haftmann tuned comments
Mon, 04 Jun 2007 13:22:22 +0200 urbanc added a few comments to the proofs
Mon, 04 Jun 2007 11:39:19 +0200 chaieb removed fixmes
Mon, 04 Jun 2007 11:38:34 +0200 chaieb opaque-constraint removed
Mon, 04 Jun 2007 09:57:02 +0200 chaieb tuned;
Sun, 03 Jun 2007 23:16:57 +0200 wenzelm monomorphic equality: let ML work out the details;
Sun, 03 Jun 2007 23:16:56 +0200 wenzelm added gen_merge_lists/merge_lists/merge_alists (legacy operations from library.ML);
(0) -10000 -3000 -1000 -120 +120 +1000 +3000 +10000 +30000 tip