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