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.
formalisation of my PhD (the result was correct, but the proof needed several corrections)
2007-05-24, by urbanc
add an option in fresh_fun_simp to prevent rewriting in assumptions
2007-05-24, by narboux
fixes tvar issue in type inference
2007-05-24, by haftmann
tuned
2007-05-24, by haftmann
tuned warning
2007-05-24, by haftmann
rudimentary class target implementation
2007-05-24, by haftmann
tuned Pure/General/name_space.ML
2007-05-24, by haftmann
Introduced new classes monoid_add and group_add
2007-05-24, by nipkow
add lemma complete_algebra_summable_geometric
2007-05-23, by huffman
formatting
2007-05-23, by paulson
generalize powerseries and termdiffs lemmas using axclasses
2007-05-23, by huffman
remove unused simproc definition
2007-05-23, by huffman
remove redundant simproc; remove legacy ML bindings
2007-05-23, by huffman
remove redundant simproc
2007-05-23, by huffman
new simp rule Infinitesimal_of_hypreal_iff
2007-05-22, by huffman
removed redundant lemmas
2007-05-22, by huffman
generalize uniqueness of limits to class real_normed_algebra_1
2007-05-22, by huffman
Some hacks for SPASS format
2007-05-22, by paulson
some optimizations, cleanup
2007-05-22, by krauss
add missing instance declarations
2007-05-22, by huffman
adjusted to change in Provers/Arith/combine_numerals.ML
2007-05-22, by haftmann
adjusted to change in Provers/Arith/combine_numerals.ML
2007-05-22, by haftmann
regression tests: send failure reports to krauss@in.tum.de, too
2007-05-22, by krauss
rename lemmas LIM_ident, isCont_ident, DERIV_ident
2007-05-22, by huffman
remove obsolete CSeries.thy
2007-05-22, by huffman
generalized ring_eq_cancel simprocs to class idom; removed redundant field_eq_cancel simprocs
2007-05-22, by huffman
new field_combine_numerals simproc, which uses fractions as coefficients
2007-05-21, by huffman
search bottom up to get the inner fresh fun
2007-05-21, by narboux
add a bottom up search function
2007-05-21, by narboux
tuned
2007-05-21, by haftmann
evaluation for integers
2007-05-21, by haftmann
added lemma divAlg_div_mof
2007-05-21, by haftmann
improved code for rev
2007-05-21, by haftmann
min/max
2007-05-21, by haftmann
generalize CombineNumerals functor to allow coefficients with types other than IntInf.int
2007-05-21, by huffman
add lemmas divide_numeral_1 and inverse_numeral_1
2007-05-21, by huffman
fixed signature
2007-05-21, by krauss
Method "lexicographic_order" now takes the same arguments as "auto"
2007-05-21, by krauss
change fresh_fun_simp to treat occurences in assumptions and try to solve the generated subgoals
2007-05-21, by narboux
define pi with THE instead of SOME; cleaned up
2007-05-20, by huffman
add lemmas for sin,cos,tan of 30,45,60 degrees; cleaned up
2007-05-20, by huffman
add lemma power2_eq_imp_eq
2007-05-20, by huffman
added lemma for permutations on strings
2007-05-20, by urbanc
moved sqrt lemmas from Transcendental.thy to NthRoot.thy
2007-05-20, by huffman
remove obsolete DERIV_ln lemmas
2007-05-20, by huffman
add realpow_pos_nth2 back in
2007-05-20, by huffman
add odd_real_root lemmas
2007-05-20, by huffman
add lemmas about inverse functions; cleaned up proof of polar_ex
2007-05-20, by huffman
change premises of DERIV_inverse_function lemma
2007-05-20, by huffman
rearranged sections
2007-05-20, by huffman
add lemmas about continuity and derivatives of roots
2007-05-20, by huffman
add lemma DERIV_inverse_function
2007-05-20, by huffman
add lemmas LIM_compose2, isCont_LIM_compose2
2007-05-20, by huffman
improved aliassing
2007-05-19, by haftmann
more robust thm handling
2007-05-19, by haftmann
added a set of NNF normalization lemmas and nnf_conv
2007-05-19, by chaieb
added lt and some other infix operation analogous to Ocaml's num library
2007-05-19, by chaieb
added a generic conversion for quantifier elimination and a special useful instance
2007-05-19, by chaieb
added binop_conv, aconvc
2007-05-19, by chaieb
added cpat antiquotation for reading certified patterns
2007-05-19, by chaieb
unfold min/max in Stefans code generator
2007-05-19, by nipkow
added code generation based on Isabelle's rat type.
2007-05-19, by nipkow
Disabled Stefancs code generator - already enabled in RealDef.
2007-05-19, by nipkow
constant op @ now named append
2007-05-19, by haftmann
fixed comment
2007-05-19, by haftmann
dropped legacy
2007-05-19, by haftmann
improved eta expansion
2007-05-19, by haftmann
dropped nonsense comment
2007-05-19, by haftmann
fixed text
2007-05-19, by haftmann
eliminated name clash with List.append
2007-05-19, by haftmann
added qualification for ambiguous definition names
2007-05-19, by haftmann
tuned
2007-05-19, by haftmann
typ_of instance for int
2007-05-19, by haftmann
hide locale predicate "field" from HOL library
2007-05-19, by haftmann
no special treatment in naming of locale predicates stemming form classes
2007-05-19, by haftmann
uniform module names for code generation
2007-05-19, by haftmann
added Executable_Real
2007-05-19, by haftmann
updated
2007-05-19, by haftmann
Had to replace "case 1/2" by "case base/step". No idea why.
2007-05-19, by nipkow
*** empty log message ***
2007-05-19, by nipkow
remove dependence on Hilbert_Choice.thy
2007-05-19, by huffman
use THE instead of SOME
2007-05-19, by huffman
minimize imports
2007-05-18, by huffman
Prove existence of nth roots using Intermediate Value Theorem
2007-05-18, by huffman
avoid using real_mult_inverse_left; cleaned up
2007-05-18, by huffman
use mult_strict_mono instead of real_mult_less_mono
2007-05-18, by huffman
Fixed bug in subst causing primrec functions returning functions
2007-05-18, by berghofe
dropped word_setup.ML
2007-05-18, by haftmann
added files
2007-05-17, by krauss
updated
2007-05-17, by krauss
moved lemmas to Nat.thy
2007-05-17, by krauss
added induction principles for induction "backwards": P (Suc n) ==> P n
2007-05-17, by krauss
added pointer to new Unification theory
2007-05-17, by krauss
Added unification case study (using new function package)
2007-05-17, by krauss
avoid using redundant lemmas from RealDef.thy
2007-05-17, by huffman
canonical prefixing of class constants
2007-05-17, by haftmann
dropped beta/eta normalization of defining equations
2007-05-17, by haftmann
refined pow function
2007-05-17, by haftmann
abstract size function in hologic.ML
2007-05-17, by haftmann
tuned
2007-05-17, by haftmann
add classes ring_no_zero_divisors and dom
2007-05-17, by huffman
generalize class restrictions on some lemmas
2007-05-17, by huffman
added classes ring_no_zero_divisors and dom (non-commutative version of idom);
2007-05-17, by huffman
Added three items to the signature
2007-05-17, by paulson
generalize some lemmas from field to division_ring
2007-05-17, by huffman
instance division_ring < no_zero_divisors; clean up field instance proofs
2007-05-17, by huffman
remove redundant instance declaration
2007-05-17, by huffman
cleaned up proof of Maclaurin_sin_bound
2007-05-17, by huffman
section labels
2007-05-16, by huffman
minimize imports
2007-05-16, by huffman
dropped |R
2007-05-16, by chaieb
A verified theory for rational numbers representation and simple calculations;
2007-05-15, by chaieb
Fixed bug that caused proof of induction theorem to fail if
2007-05-15, by berghofe
minimize imports
2007-05-15, by huffman
clean up polar_Ex proofs; remove unnecessary lemmas
2007-05-15, by huffman
remove simp attribute from various polar_Ex lemmas
2007-05-15, by huffman
tuned proofs
2007-05-14, by huffman
spelling: rename arcos -> arccos
2007-05-14, by huffman
tuned proofs
2007-05-14, by huffman
add lemma sgn_mult; declare real_scaleR_def and scaleR_eq_0_iff as simp rules
2007-05-14, by huffman
less
more
|
(0)
-10000
-3000
-1000
-120
+120
+1000
+3000
+10000
+30000
tip