Mercurial
Mercurial
>
repos
>
isabelle
/ graph
summary
|
shortlog
|
changelog
| graph |
tags
|
bookmarks
|
branches
|
files
|
gz
|
help
less
more
|
(0)
-30000
-10000
-3000
-1000
-240
+240
+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.
Better approximation of cos around pi.
2009-06-08, by hoelzl
merged
2009-06-08, by huffman
merged
2009-06-07, by huffman
new lemma
2009-06-08, by nipkow
merged
2009-06-08, by haftmann
merged
2009-06-08, by haftmann
proper deresolving of class relations and class parameters in SML
2009-06-08, by haftmann
New lemma
2009-06-08, by nipkow
eliminated hardwired Cygwin setup;
2009-06-08, by wenzelm
Accessing the Cygwin installation.
2009-06-08, by wenzelm
static IsabelleSystem.charset;
2009-06-07, by wenzelm
isabelle getenv: option -d;
2009-06-07, by wenzelm
no parallel make jobs on macbroy23, which is the machine where SML/XL is tested -- attempt to consume less resources;
2009-06-06, by wenzelm
updated version;
2009-06-06, by wenzelm
fix type of open
2009-06-07, by huffman
new setL2 lemmas; instance ^ :: (topological_space, finite) topological_space
2009-06-07, by huffman
replace 'topo' with 'open'; add extra type constraint for 'open'
2009-06-07, by huffman
generalize tendsto lemmas for products
2009-06-07, by huffman
move definitions of open, closed to RealVector.thy
2009-06-07, by huffman
lemmas islimptI, islimptE; generalize open_inter_closure_subset
2009-06-06, by huffman
generalize tendsto to class topological_space
2009-06-06, by huffman
put syntax for tendsto in Limits.thy; rename variables
2009-06-05, by huffman
constant "chars" of all characters
2009-06-08, by haftmann
added infrastructure for definitorial construction of generators for datatypes
2009-06-08, by haftmann
constant "chars" of all characters
2009-06-08, by haftmann
added generator for char and trivial generator for String.literal
2009-06-08, by haftmann
using constant "chars"
2009-06-08, by haftmann
method linarith
2009-06-08, by haftmann
reraise exceptions to preserve position information;
2009-06-06, by wenzelm
ML_Compiler.exn_message;
2009-06-06, by wenzelm
ML_Compiler.exn_message;
2009-06-06, by wenzelm
added exn_message (formerly in toplevel.ML);
2009-06-06, by wenzelm
moved Isar toplevel runtime support to runtime.ML, which is loaded early (before ml_compiler.ML);
2009-06-06, by wenzelm
report_parse_tree: ML_open, ML_struct;
2009-06-06, by wenzelm
export end_pos_of;
2009-06-06, by wenzelm
use: tuned error;
2009-06-06, by wenzelm
added markup ML_open, ML_struct;
2009-06-06, by wenzelm
use_text: pass file name to compiler, tuned;
2009-06-06, by wenzelm
tuned comments;
2009-06-06, by wenzelm
removed obsolete YXML/XML.detect;
2009-06-05, by wenzelm
Approximation: Corrected precision of ln on all real values
2009-06-05, by hoelzl
Approximation: Implemented argument reduction for cosine. Sinus is now implemented in terms of cosine. Sqrt computes on the entire real numbers
2009-06-04, by hoelzl
CONTRIBUTORS
2009-06-05, by haftmann
merged
2009-06-05, by haftmann
tuned proofs
2009-06-05, by haftmann
added mk_valtermify_app and mk_random
2009-06-05, by haftmann
Set.insert with authentic syntax
2009-06-05, by haftmann
merged
2009-06-05, by haftmann
Set.insert with authentic syntax
2009-06-05, by haftmann
added trees implementing mappings
2009-06-04, by haftmann
avoid Library.foldl_map
2009-06-04, by haftmann
class replaces axclass
2009-06-04, by haftmann
insert now qualified and with authentic syntax
2009-06-04, by haftmann
lemma about List.foldl and Finite_Set.fold
2009-06-04, by haftmann
dropped legacy ML bindings; tuned
2009-06-04, by haftmann
lemmas about basic set operations and Finite_Set.fold
2009-06-04, by haftmann
merged
2009-06-05, by nipkow
new lemma
2009-06-05, by nipkow
merged
2009-06-05, by huffman
fix type of hnorm
2009-06-05, by huffman
define netlimit in terms of eventually
2009-06-04, by huffman
generalize type of 'at' to topological_space; generalize some lemmas
2009-06-04, by huffman
add extra type constraints for dist, norm
2009-06-04, by huffman
generalize norm method to work over class real_normed_vector
2009-06-04, by huffman
example settings for Poly/ML 5.3 (experimental);
2009-06-04, by wenzelm
uniform (short) ids on both sides;
2009-06-04, by wenzelm
merged
2009-06-04, by wenzelm
finite lemmas
2009-06-04, by nipkow
made SML/NJ happy
2009-06-04, by haftmann
merged
2009-06-04, by nipkow
A few finite lemmas
2009-06-04, by nipkow
removed unused location_of;
2009-06-04, by wenzelm
retrieve ML source files;
2009-06-04, by wenzelm
export file_name;
2009-06-04, by wenzelm
more robust treatment of bootstrap source positions;
2009-06-04, by wenzelm
less experimental polyml-5.3;
2009-06-04, by wenzelm
just one ROOT.ML without any cd or ".." -- simplifies ML environment references to bootstrap sources;
2009-06-04, by wenzelm
exn_message/raised: ML_Compiler.exception_position;
2009-06-04, by wenzelm
eliminated costly registration of tokens;
2009-06-04, by wenzelm
convert explicitly between Position.T/PolyML.location, without costly registration of tokens;
2009-06-04, by wenzelm
added exception_position (dummy);
2009-06-04, by wenzelm
reraise exceptions to preserve original position (ML system specific);
2009-06-04, by wenzelm
tuned signature;
2009-06-04, by wenzelm
export esc;
2009-06-04, by wenzelm
export value;
2009-06-04, by wenzelm
uniform default settings for E, Vampire, SPASS;
2009-06-04, by wenzelm
merged
2009-06-03, by huffman
add classes for t0, t1, and t2 spaces
2009-06-03, by huffman
generalize type of islimpt
2009-06-03, by huffman
more [code del] declarations
2009-06-03, by huffman
generalize some constants and lemmas to class topological_space
2009-06-03, by huffman
replace class open with class topo
2009-06-03, by huffman
open_dist instance for vectors
2009-06-03, by huffman
instance * :: topological_space
2009-06-03, by huffman
class real_inner derives from open_dist
2009-06-03, by huffman
introduce class topological_space as a superclass of metric_space
2009-06-03, by huffman
Converted reification to use fold_map instead of Library.foldl_map. Use antiquotations.
2009-06-03, by hoelzl
additional debugging
2009-06-03, by immler
include chain-ths in every prover-call
2009-06-03, by immler
split preparing clauses and writing problemfile;
2009-06-03, by immler
merged
2009-06-03, by huffman
merged
2009-06-02, by huffman
instance ^ :: complete_space
2009-06-02, by huffman
instance * :: complete_space; generalize continuity lemmas for fst, snd, Pair
2009-06-02, by huffman
generalize type of constant lim
2009-06-02, by huffman
class complete_space
2009-06-02, by huffman
generalize constant uniformly_continuous_on
2009-06-02, by huffman
generalize more constants
2009-06-02, by huffman
generalize type of bounded
2009-06-02, by huffman
generalize lemma norm_pastecart
2009-06-02, by huffman
generalize lemma norm_triangle_sub
2009-06-02, by huffman
generalize lemma Lim_unique
2009-06-02, by huffman
generalize lemma closed_cball
2009-06-02, by huffman
generalize Lim_transform lemmas
2009-06-02, by huffman
generalize lemma interior_closed_Un_empty_interior
2009-06-02, by huffman
reuse definition of nets from Limits.thy
2009-06-02, by huffman
replace filters with filter bases
2009-06-02, by huffman
generalize type of 'at' to metric_space
2009-06-02, by huffman
redefine nets as filter bases
2009-06-02, by huffman
new lemmas
2009-06-02, by huffman
limits of Pair using filters
2009-06-01, by huffman
Removed usage of reference in reification
2009-06-03, by hoelzl
corrected spacing in reflection
2009-06-02, by hoelzl
switch at-sml-dev-e back to full test on macbroy23
2009-06-03, by kleing
IsabelleProcess: emit status "ready" after initialization and reports;
2009-06-02, by wenzelm
moved restrict_map_insert to theory Map
2009-06-02, by haftmann
merged
2009-06-02, by haftmann
added Landau theory
2009-06-02, by haftmann
added/moved lemmas by Andreas Lochbihler
2009-06-02, by haftmann
added Fin_Fun theory
2009-06-02, by haftmann
tuned code generator test theories
2009-06-02, by haftmann
OCaml builtin intergers are elusive; avoid
2009-06-02, by haftmann
more aggresive bracketing of let expressions
2009-06-02, by haftmann
tuned whitespace
2009-06-02, by haftmann
merged
2009-06-02, by wenzelm
merged
2009-06-02, by wenzelm
merged
2009-06-02, by chaieb
merged
2009-06-02, by chaieb
merged
2009-06-02, by chaieb
Reverses idempotent; radical of E; generalized logarithm;
2009-06-01, by chaieb
made SML/NJ happy;
2009-06-02, by wenzelm
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
less
more
|
(0)
-30000
-10000
-3000
-1000
-240
+240
+1000
+3000
+10000
+30000
tip