Mercurial
Mercurial
>
repos
>
isabelle
/ graph
summary
|
shortlog
|
changelog
| graph |
tags
|
bookmarks
|
branches
|
files
|
gz
|
help
less
more
|
(0)
-30000
-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.
merged
2009-06-02, by wenzelm
use algebra_simps instead of ring_simps
2009-06-02, by hoelzl
merged, resolving conflict in src/Pure/Isar/attrib.ML;
2009-06-02, by wenzelm
Generalized Integral_add
2009-06-02, by hoelzl
Added theorems about distinct & concat, map & replicate and concat & replicate
2009-06-02, by hoelzl
merged
2009-06-02, by berghofe
Fixed broken code dealing with alternative names.
2009-06-02, by berghofe
Enclosed parts of subsection in @{text ...} to make LaTeX happy.
2009-06-02, by berghofe
Added Convex_Euclidean_Space.thy again.
2009-06-02, by berghofe
made SML/NJ happy
2009-06-02, by haftmann
declare Bfun_def [code del]
2009-06-01, by huffman
simp del -> code del
2009-06-01, by huffman
limits of inverse using filters
2009-06-01, by huffman
merged
2009-06-01, by huffman
add [code del] declarations
2009-06-01, by huffman
add dependency on Limits.thy
2009-06-01, by huffman
new lemma
2009-06-01, by nipkow
merged
2009-05-31, by huffman
new theory of filters and limits; prove LIMSEQ and LIM lemmas using filters
2009-05-31, by huffman
more abstract properties of eventually
2009-05-31, by huffman
new lemmas about eventually; rewrite Lim proofs to use more abstract properties of eventually
2009-05-31, by huffman
generalize at function to class perfect_space
2009-05-29, by huffman
generalize topological notions to class metric_space; add class perfect_space
2009-05-29, by huffman
instance ^ :: (metric_space, finite) metric_space
2009-05-29, by huffman
generalize tendsto and related constants to class metric_space
2009-05-29, by huffman
add lemmas Lim_at_iff_LIM, Lim_sequentially_iff_LIMSEQ
2009-05-29, by huffman
remove duplicate cauchy constant
2009-05-29, by huffman
fix reference to LIM_def
2009-05-29, by huffman
instance * :: (metric_space, metric_space) metric_space; generalize lemmas to class metric_space
2009-05-29, by huffman
generalize constants from Lim.thy to class metric_space
2009-05-29, by huffman
LIMSEQ_def -> LIMSEQ_iff
2009-05-28, by huffman
generalize constants in SEQ.thy to class metric_space
2009-05-28, by huffman
early setup of secure operations (again, cf. deddd77112b7) -- NB: fix_ints is required for bootstrap;
2009-06-02, by wenzelm
structure ML_Compiler;
2009-06-01, by wenzelm
added structure ML_Compiler: runtime compilation, with advanced version for Poly/ML 5.3 (formerly ML_Test);
2009-06-01, by wenzelm
added flatten;
2009-06-01, by wenzelm
tuned signature;
2009-06-01, by wenzelm
export secure_mltext;
2009-06-01, by wenzelm
tuned comments;
2009-06-01, by wenzelm
maintain tokens within common ML environment;
2009-06-01, by wenzelm
ML_Env;
2009-06-01, by wenzelm
slightly later setup of ML and secure operations;
2009-06-01, by wenzelm
moved local ML environment to separate module ML_Env;
2009-06-01, by wenzelm
removed print function from global ML name space, to reduce risk of surprises;
2009-06-01, by wenzelm
made SML/NJ happy;
2009-06-01, by wenzelm
attempt to eliminate adhoc makestring at runtime (which is not well-defined);
2009-05-31, by wenzelm
eliminated misleading dummy versions of print/makestring, cf. 6974449ddea9;
2009-05-31, by wenzelm
provide local dummy version of makestring -- NB: makestring is fragile and not portable, it should not occur in repository sources;
2009-05-31, by wenzelm
no longer open PolyML -- to avoid surprises within the global name space;
2009-05-31, by wenzelm
explicit PolyML qualification;
2009-05-31, by wenzelm
removed "compress" option from isabelle-process and isabelle usedir -- this is always enabled;
2009-05-31, by wenzelm
test experimental Poly/ML 5.3;
2009-05-31, by wenzelm
removed obsolete COPYDB flag;
2009-05-31, by wenzelm
explicit PolyML.install_pp;
2009-05-31, by wenzelm
renamed polyml_pp.ML to pp_polyml.ML;
2009-05-31, by wenzelm
more modular setup of runtime compilation;
2009-05-31, by wenzelm
more precise version information;
2009-05-31, by wenzelm
uniform treatment of shellscript mode;
2009-05-31, by wenzelm
updated example settings;
2009-05-31, by wenzelm
discontinued support for Poly/ML 4.x versions;
2009-05-31, by wenzelm
ISABELLE_USEDIR_OPTIONS: proper word splitting of quoted options (via array variable and special expansion, cf. "$@");
2009-05-30, by wenzelm
eliminated old Attrib.add_attributes (and Attrib.syntax);
2009-05-30, by wenzelm
modernized attribute setup;
2009-05-30, by wenzelm
eliminated old Method.add_method(s);
2009-05-30, by wenzelm
removed obsolete combinators for method args;
2009-05-30, by wenzelm
proper signature constraint;
2009-05-30, by wenzelm
minimal signature cleanup;
2009-05-30, by wenzelm
modernized method setup;
2009-05-30, by wenzelm
modernized method setup;
2009-05-30, by wenzelm
tuned;
2009-05-30, by wenzelm
tuned;
2009-05-30, by wenzelm
simps with mandatory name prefix
2009-05-30, by haftmann
corrected bound/unbounded flag for nat numerals
2009-05-30, by haftmann
removed dead theory Relation_Power
2009-05-29, by haftmann
fix reference to dist_def
2009-05-28, by huffman
definition of dist for complex
2009-05-28, by huffman
fix references to dist_def
2009-05-28, by huffman
define dist for products
2009-05-28, by huffman
move dist operation to new metric_space class
2009-05-28, by huffman
remove hard tabs, fix indentation
2009-05-28, by huffman
use class field_char_0
2009-05-28, by huffman
merged
2009-05-28, by huffman
generalize dist function to class real_normed_vector
2009-05-28, by huffman
added remark to code
2009-05-28, by bulwahn
Removed Convex_Euclidean_Space.thy from Library.
2009-05-28, by himmelma
Moved some lemmas about intervals to Topology
2009-05-28, by himmelma
Corrected definition of is_interval
2009-05-28, by himmelma
corrected problem in Determinants
2009-05-28, by himmelma
Corrected error in Convex_Euclidean_Space
2009-05-28, by himmelma
Added Convex_Euclidean_Space to Library.thy and Library/IsaMakefile
2009-05-28, by himmelma
merged
2009-05-28, by himmelma
Added Convex_Euclidean_Space.thy
2009-05-28, by himmelma
Changed prioriy of vector_scalar_mult
2009-05-28, by himmelma
addition formulas for fps_sin, fps_cos
2009-05-28, by huffman
use class field_char_0 for fps definitions
2009-05-28, by huffman
merged
2009-05-27, by huffman
add constants sin_coeff, cos_coeff
2009-05-27, by huffman
merged
2009-05-27, by wenzelm
tuned signature of add_primrec_simple
2009-05-27, by haftmann
added lemma select_weight_cons_zero
2009-05-27, by haftmann
added lemma beyond_zero; hide constants
2009-05-27, by haftmann
added lemma about 0 - 1
2009-05-27, by haftmann
merged
2009-05-27, by wenzelm
more lemmas
2009-05-27, by nipkow
merged
2009-05-27, by haftmann
add_primrec_simple
2009-05-26, by haftmann
dropped superfluos prefixes
2009-05-26, by haftmann
separate module for quickcheck generators
2009-05-26, by haftmann
encode gauge-fine partitions with lists instead of functions; remove lots of unnecessary lemmas
2009-05-26, by huffman
listsum lemmas
2009-05-26, by huffman
clean up some rsum proofs
2009-05-26, by huffman
weakend references to old axclass
2009-05-26, by haftmann
clarified benefit of interpretation
2009-05-26, by haftmann
documented print_codeproc command
2009-05-26, by haftmann
use interval sets with gauge predicate
2009-05-25, by huffman
clean up some proofs
2009-05-25, by huffman
tuned whitespace
2009-05-24, by haftmann
funpow_yield; tuned
2009-05-24, by haftmann
tuned class user space type system code
2009-05-24, by haftmann
dropped Id
2009-05-24, by haftmann
less
more
|
(0)
-30000
-10000
-3000
-1000
-120
+120
+1000
+3000
+10000
+30000
tip