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, reverting workarounds on both sides;
2009-06-11, by wenzelm
theory Predicate_Compile_ex: enable quick_and_dirty for now, to make it work with internal cheat_tac invocations;
2009-06-11, by wenzelm
added sporadic (Local)Theory.checkpoint, to enable parallel proof checking;
2009-06-11, by wenzelm
merged
2009-06-11, by wenzelm
merged
2009-06-10, by wenzelm
making isatest happy; but misunderstanding remains
2009-06-11, by bulwahn
code_pred command now also requires proofs for dependent predicates; changed handling of parameters in introrules of executable function
2009-06-10, by bulwahn
tuned; corrected exception handling
2009-06-10, by bulwahn
tuned;
2009-06-10, by wenzelm
discontinued escaped symbols;
2009-06-10, by wenzelm
eliminated escaped symbols;
2009-06-10, by wenzelm
discontinued escaped symbols such as \\<forall> -- only one backslash should be used;
2009-06-10, by wenzelm
updated generated files;
2009-06-10, by wenzelm
allow Isabelle symbols within low-level ML source;
2009-06-10, by wenzelm
reraise exceptions to preserve position information;
2009-06-10, by wenzelm
simplified Graph.extend;
2009-06-10, by wenzelm
removed unused make;
2009-06-10, by wenzelm
merged
2009-06-09, by wenzelm
merged
2009-06-09, by huffman
instance heine_borel < complete_space; generalize many lemmas to class heine_borel
2009-06-09, by huffman
new class heine_borel for lemma bounded_closed_imp_compact; instances for real, ^
2009-06-09, by huffman
generalize compact/closure lemmas
2009-06-08, by huffman
add lemma complete_imp_closed
2009-06-08, by huffman
generalize constant 'bounded' to class metric_space
2009-06-08, by huffman
generalize lemmas compact_imp_bounded, compact_imp_closed
2009-06-08, by huffman
generalize more lemmas
2009-06-08, by huffman
generalize constant 'indirection'
2009-06-08, by huffman
lemmas about linear, bilinear
2009-06-08, by huffman
generalize constant 'complete'
2009-06-08, by huffman
generalize lemmas eventually_within_interior, lim_within_interior
2009-06-08, by huffman
generalize more lemmas
2009-06-08, by huffman
generalize some lemmas
2009-06-08, by huffman
avoiding duplicate definitions of executable functions
2009-06-09, by bulwahn
tuned;
2009-06-09, by wenzelm
more native Scala style;
2009-06-09, by wenzelm
tuned;
2009-06-09, by wenzelm
simplified IsabelleSystem.platform_path for cygwin;
2009-06-09, by wenzelm
merged
2009-06-09, by wenzelm
removed duplicate lemmas
2009-06-09, by himmelma
removed general graph functions in the predicate compiler
2009-06-09, by bulwahn
added graph builders
2009-06-09, by bulwahn
removed debug messages
2009-06-09, by bulwahn
refactoring the predicate compiler
2009-06-09, by bulwahn
merged
2009-06-09, by chaieb
Tuned sos tactic to reject non SOS goals
2009-06-09, by chaieb
tuned
2009-06-09, by boehmes
fast_lin_arith uses proper multiplication instead of unfolding to additions
2009-06-08, by boehmes
more lemmas
2009-06-08, by nipkow
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
less
more
|
(0)
-30000
-10000
-3000
-1000
-120
+120
+1000
+3000
+10000
+30000
tip