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.
more robust Par_Exn.make, especially relevant for SML/NJ trying to use Par_Exn.release_all;
2013-03-14, by wenzelm
proper use of "member", without embarking on delicate questions about SML equality types;
2013-03-14, by wenzelm
made SML/NJ happy;
2013-03-14, by wenzelm
tuned
2013-03-14, by nipkow
merged
2013-03-13, by wenzelm
clarified parallel_subproofs_saturation (blind guess) vs. parallel_subproofs_threshold (precient timing estimate);
2013-03-13, by wenzelm
proper formatting, to facilitate line-based diff;
2013-03-13, by wenzelm
more uniform session descriptions, which show up in chapter index;
2013-03-13, by wenzelm
proper index for HOL-Proofs, which is also in chapter "HOL";
2013-03-13, by wenzelm
include only README.html, not historic README, which tends towards surprises like src/HOL/SPARK/Examples/README;
2013-03-13, by wenzelm
more accurate handling of global browser info at the very end (without races), subject to no_build and info.browser_info;
2013-03-13, by wenzelm
sessions may be organized via 'chapter' in ROOT;
2013-03-13, by wenzelm
do not absorb I/O errors;
2013-03-13, by wenzelm
show expanded path, to avoid odd /foo/bar/$ISABELLE_BROWSER_INFO/baz;
2013-03-13, by wenzelm
new lemma subset_decode_imp_le
2013-03-13, by paulson
merged
2013-03-13, by kleing
more IMP snippets
2013-03-13, by kleing
rename fset_member to fmember and prove parametricity
2013-03-13, by kuncar
BNF uses fset defined via Lifting/Transfer rather than Quotient
2013-03-13, by traytel
nitpick setup and code generation for streams
2013-03-13, by traytel
merged
2013-03-13, by nipkow
tuned
2013-03-13, by nipkow
proper path -- I/O was hidden due to permissiveness;
2013-03-12, by wenzelm
merged
2013-03-12, by wenzelm
removed odd cvs artifacts;
2013-03-12, by wenzelm
refurbished some old README.html files as session descriptions, which show up in chapter index;
2013-03-12, by wenzelm
include session description in chapter index;
2013-03-12, by wenzelm
tuned;
2013-03-12, by wenzelm
more accurate theory links;
2013-03-12, by wenzelm
discontinued "isabelle usedir" option -r (reset session path);
2013-03-12, by wenzelm
discontinued "isabelle usedir" option -P (remote path);
2013-03-11, by wenzelm
support for 'chapter' specifications within session ROOT;
2013-03-11, by wenzelm
added latex markup
2013-03-12, by nipkow
merged
2013-03-12, by kleing
more snippets
2013-03-12, by kleing
added pairs
2013-03-12, by nipkow
extended set comprehension notation with {pttrn : A . P}
2013-03-12, by nipkow
tuned
2013-03-11, by nipkow
more factorisation of Step & Co
2013-03-11, by nipkow
factored out Step
2013-03-10, by nipkow
merged
2013-03-10, by nipkow
stepwise instantiation is more modular
2013-03-10, by nipkow
generalized subclass relation;
2013-03-10, by haftmann
termination proof for narrowing: fewer assumptions
2013-03-10, by nipkow
accomodate encrypted file-system on linux;
2013-03-09, by wenzelm
tuned;
2013-03-09, by wenzelm
discontinued theory src/HOL/Library/Eval_Witness -- assumptions do not longer hold in presence of abstract types
2013-03-09, by haftmann
updated keywords (cf. 84d01fd733cf);
2013-03-08, by wenzelm
proper type inference for default values
2013-03-08, by blanchet
convert mappings to parametric lifting
2013-03-08, by kuncar
setup_lifting doesn't support a type variable as a raw type
2013-03-08, by kuncar
add [relator_mono] and [relator_distr] rules
2013-03-08, by kuncar
simplify Lift_FSet because we have parametricity in Lifting now
2013-03-08, by kuncar
patch Isabelle ditribution to conform to changes regarding the parametricity
2013-03-08, by kuncar
lift_definition and setup_lifting generate parametric transfer rules if parametricity theorems are provided
2013-03-08, by kuncar
merged
2013-03-08, by nipkow
simplified basic termination proof
2013-03-08, by nipkow
some simp rules for fset
2013-03-08, by traytel
avoid -Infinity which confuses JFreeChart histogram;
2013-03-07, by wenzelm
tuned proofs -- more structure, less warnings;
2013-03-07, by wenzelm
tuned signature -- prefer terminology of Scala and Axiom;
2013-03-07, by wenzelm
better message (type-unsoundnesses are becoming rare, usually the issue is elsewhere, e.g. in the TSTP proof parser)
2013-03-07, by blanchet
avoid using Arith_Data.dest_sum in extended-nat simprocs (it treats 'x - y' as 'x + - y', which is not valid for enat)
2013-03-06, by huffman
netlimit is abbreviation for Lim
2013-03-06, by hoelzl
tuned proofs
2013-03-06, by hoelzl
changed has_derivative_intros into a named theorems collection
2013-03-06, by hoelzl
changed continuous_on_intros into a named theorems collection
2013-03-06, by hoelzl
changed continuous_intros into a named theorems collection
2013-03-06, by hoelzl
add tendsto_eq_intros: they add an additional rewriting step at the rhs of --->
2013-03-06, by hoelzl
major redesign: order instead of preorder, new definition of intervals as quotients
2013-03-06, by nipkow
added lemma
2013-03-06, by nipkow
extended numerals
2013-03-06, by nipkow
merged
2013-03-05, by wenzelm
merged
2013-03-05, by wenzelm
removed unused Future.flat, while leaving its influence of Future.map (see bcd6b1aa4db5);
2013-03-05, by wenzelm
extended stream library a little more
2013-03-05, by traytel
extended stream library
2013-03-05, by traytel
generalized lemmas in Extended_Real_Limits
2013-03-05, by hoelzl
eventually nhds represented using sequentially
2013-03-05, by hoelzl
generalized compact_Times to topological_space
2013-03-05, by hoelzl
move lemma Inf to usage point
2013-03-05, by hoelzl
tuned proof of Edelstein fixed point theorem (use continuity of dist and attains_sup)
2013-03-05, by hoelzl
tuned proofs (used continuity of infdist, dist and continuous_attains_sup)
2013-03-05, by hoelzl
generalized continuous/compact_attains_inf/sup from real to linorder_topology
2013-03-05, by hoelzl
continuity of pair operations
2013-03-05, by hoelzl
use generate_topology for second countable topologies, does not require intersection stable basis
2013-03-05, by hoelzl
generalized isGlb_unique
2013-03-05, by hoelzl
complete_linorder is also a complete_distrib_lattice
2013-03-05, by hoelzl
move Liminf / Limsup lemmas on complete_lattices to its own file
2013-03-05, by hoelzl
merged
2013-03-05, by nipkow
New theory of infinity-extended types; should replace Extended_xyz eventually
2013-03-05, by nipkow
Avoid ML warning about unreferenced identifier.
2013-03-05, by webertj
polymorphic SPASS is also SPASS
2013-03-05, by blanchet
allow more general coercion maps; tuned;
2013-03-05, by traytel
more lemmas about intervals
2013-03-05, by nipkow
merged
2013-03-04, by wenzelm
refined parallel_proofs = 2: fork whole Isar sub-proofs, not just terminal ones;
2013-03-04, by wenzelm
join all proofs before scheduling present phase (ordered according to weight);
2013-03-04, by wenzelm
more explicit datatype result;
2013-03-04, by wenzelm
split dense into inner_dense_order and no_top/no_bot
2013-02-20, by hoelzl
move auxiliary lemmas from Library/Extended_Reals to HOL image
2013-02-20, by hoelzl
tuned (extend datatype to inline option)
2013-03-04, by traytel
prefer more systematic Future.flat;
2013-03-03, by wenzelm
more uniform Future.map: always internalize failure;
2013-03-03, by wenzelm
uniform treatment of global/local proofs;
2013-03-03, by wenzelm
tuned;
2013-03-03, by wenzelm
clarified Toplevel.element_result wrt. Toplevel.is_ignored;
2013-03-03, by wenzelm
more Thy_Syntax.element operations;
2013-03-03, by wenzelm
coercion-invariant arguments at work
2013-03-01, by traytel
constants with coercion-invariant arguments (possibility to disable/reenable
2013-03-01, by traytel
simplified Proof.future_proof;
2013-02-28, by wenzelm
provide explicit dummy names (cf. dfe469293eb4);
2013-02-28, by wenzelm
discontinued empty name bindings in 'axiomatization';
2013-02-28, by wenzelm
provide common HOLogic.conj_conv and HOLogic.eq_conv;
2013-02-28, by wenzelm
just one HOLogic.Trueprop_conv, with regular exception CTERM;
2013-02-28, by wenzelm
discontinued obsolete 'axioms' command;
2013-02-28, by wenzelm
more robust build error handling, e.g. missing outer syntax commands;
2013-02-28, by wenzelm
eliminated legacy 'axioms';
2013-02-28, by wenzelm
eliminated legacy 'axioms';
2013-02-28, by wenzelm
eliminated legacy 'axioms';
2013-02-28, by wenzelm
less
more
|
(0)
-30000
-10000
-3000
-1000
-120
+120
+1000
+3000
+10000
+30000
tip