2013-03-26 |
hoelzl |
Series.thy is based on Limits.thy and not Deriv.thy
|
changeset |
files
|
2013-03-26 |
hoelzl |
move Ln.thy and Log.thy to Transcendental.thy
|
changeset |
files
|
2013-03-26 |
hoelzl |
move SEQ.thy and Lim.thy to Limits.thy
|
changeset |
files
|
2013-03-26 |
hoelzl |
HOL-NSA should only import Complex_Main
|
changeset |
files
|
2013-03-26 |
hoelzl |
rename RealVector.thy to Real_Vector_Spaces.thy
|
changeset |
files
|
2013-03-26 |
hoelzl |
rename RealDef to Real
|
changeset |
files
|
2013-03-26 |
hoelzl |
remove Real.thy
|
changeset |
files
|
2013-03-26 |
hoelzl |
merge RComplete into RealDef
|
changeset |
files
|
2013-03-26 |
hoelzl |
move real_isLub_unique to isLub_unique in Lubs; real_sum_of_halves to RealDef; abs_diff_less_iff to Rings
|
changeset |
files
|
2013-03-26 |
hoelzl |
remove posreal_complete
|
changeset |
files
|
2013-03-26 |
hoelzl |
separate SupInf into Conditional_Complete_Lattice, move instantiation of real to RealDef
|
changeset |
files
|
2013-03-25 |
ballarin |
Discontinued theories src/HOL/Algebra/abstract and .../poly.
|
changeset |
files
|
2013-03-25 |
ballarin |
Remove obsolete URLs in documentation of HOL-Algebra.
|
changeset |
files
|
2013-03-25 |
ballarin |
Fix issue related to mixins in roundup.
|
changeset |
files
|
2013-03-25 |
kleing |
simp_const -> afold; bfold -> fold'; bsimp_const -> bfold
|
changeset |
files
|
2013-03-25 |
nipkow |
added lemmas
|
changeset |
files
|
2013-03-25 |
wenzelm |
merged
|
changeset |
files
|
2013-03-25 |
wenzelm |
clarified text_fold vs. fbrk;
|
changeset |
files
|
2013-03-25 |
wenzelm |
tuned print_classes: more standard order, markup, formatting;
|
changeset |
files
|
2013-03-25 |
wenzelm |
tuned message;
|
changeset |
files
|
2013-03-25 |
wenzelm |
actually exit on scalac failure;
|
changeset |
files
|
2013-03-25 |
wenzelm |
tuned signature;
|
changeset |
files
|
2013-03-25 |
kleing |
removed obsolete uses of ext
|
changeset |
files
|
2013-03-24 |
wenzelm |
prefer preset = 3 -- much faster and less memory requirement;
|
changeset |
files
|
2013-03-24 |
wenzelm |
basic support for xz files;
|
changeset |
files
|
2013-03-24 |
wenzelm |
added component xz-java-1.2;
|
changeset |
files
|
2013-03-24 |
wenzelm |
more "quick start" hints;
|
changeset |
files
|
2013-03-24 |
traytel |
simple case syntax for stream (stolen from AFP/Coinductive)
|
changeset |
files
|
2013-03-23 |
wenzelm |
prefer plain \<^sub> for better rendering (both in Isabelle/jEdit and LaTeX);
|
changeset |
files
|
2013-03-23 |
wenzelm |
merged
|
changeset |
files
|
2013-03-23 |
wenzelm |
reverted most of 5944b20c41bf -- tends to cause race condition of synchronous vs. asynchronous version;
|
changeset |
files
|
2013-03-23 |
wenzelm |
no censorship of "view.fracFontMetrics", although it often degrades rendering quality;
|
changeset |
files
|
2013-03-23 |
wenzelm |
retain original tooltip range, to avoid repeated window popup when the mouse is moved over the same content;
|
changeset |
files
|
2013-03-23 |
wenzelm |
apply small result immediately, to avoid visible delay of text update after window move;
|
changeset |
files
|
2013-03-23 |
wenzelm |
structural equality for Command.Results;
|
changeset |
files
|
2013-03-23 |
wenzelm |
allow fractional pretty margin -- avoid premature rounding;
|
changeset |
files
|
2013-03-23 |
wenzelm |
more explicit Pretty.Metric, with clear distinction of unit (space width) vs. average char width (for visual adjustments) -- NB: Pretty formatting works via full space characters (despite a981a5c8a505 and 70f7483df9cb);
|
changeset |
files
|
2013-03-23 |
wenzelm |
tuned;
|
changeset |
files
|
2013-03-23 |
haftmann |
spelling
|
changeset |
files
|
2013-03-23 |
haftmann |
fundamental revision of big operators on sets
|
changeset |
files
|
2013-03-23 |
haftmann |
tuned proof
|
changeset |
files
|
2013-03-23 |
haftmann |
locales for abstract orders
|
changeset |
files
|
2013-03-23 |
krauss |
merged
|
changeset |
files
|
2013-03-21 |
krauss |
added rudimentary induction rule for partial_function (heap)
|
changeset |
files
|
2013-03-21 |
krauss |
allow induction predicates with arbitrary arity (not just binary)
|
changeset |
files
|
2013-03-22 |
hoelzl |
modernized definition of root: use the_inv, handle positive and negative case uniformly, and 0-th root is constant 0
|
changeset |
files
|
2013-03-22 |
hoelzl |
arcsin and arccos are continuous on {0 .. 1} (including the endpoints)
|
changeset |
files
|
2013-03-22 |
hoelzl |
move continuous_on_inv to HOL image (simplifies isCont_inverse_function)
|
changeset |
files
|
2013-03-22 |
hoelzl |
move connected to HOL image; used to show intermediate value theorem
|
changeset |
files
|
2013-03-22 |
hoelzl |
move compact to the HOL image; prove compactness of real closed intervals; show that continuous functions attain supremum and infimum on compact sets
|
changeset |
files
|
2013-03-22 |
hoelzl |
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
|
changeset |
files
|
2013-03-22 |
hoelzl |
clean up lemma_nest_unique and renamed to nested_sequence_unique
|
changeset |
files
|
2013-03-22 |
hoelzl |
simplify proof of the Bolzano bisection lemma; use more meta-logic to state it; renamed lemma_Bolzano to Bolzano
|
changeset |
files
|
2013-03-22 |
hoelzl |
introduct the conditional_complete_lattice type class; generalize theorems about real Sup and Inf to it
|
changeset |
files
|
2013-03-22 |
hoelzl |
generalize Bfun and Bseq to metric spaces; Bseq is an abbreviation for Bfun
|
changeset |
files
|
2013-03-22 |
hoelzl |
move first_countable_topology to the HOL image
|
changeset |
files
|
2013-03-22 |
hoelzl |
move metric_space to its own theory
|
changeset |
files
|
2013-03-22 |
hoelzl |
move topological_space to its own theory
|
changeset |
files
|
2013-03-21 |
wenzelm |
proper metric for blanks -- NB: 70f7483df9cb discontinues coincidence of char_width with space width;
|
changeset |
files
|
2013-03-21 |
wenzelm |
eliminated char_width_int to avoid unclear rounding;
|
changeset |
files
|