Mercurial
Mercurial
>
repos
>
isabelle
/ graph
summary
|
shortlog
|
changelog
| graph |
tags
|
bookmarks
|
branches
|
files
|
gz
|
help
less
more
|
(0)
-30000
-10000
-3000
-1000
-112
+112
+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.
bypass slow check for inlined files, where it is not really required;
2012-09-03, by wenzelm
more direct access to all-important chunks for text painting;
2012-09-03, by wenzelm
merged
2012-09-03, by nipkow
added annotations after condition in if and while
2012-09-03, by nipkow
merge, resolving trivial conflict;
2012-09-03, by wenzelm
forgot to add lemmas
2012-08-30, by Christian Sternagel
hide newly introduced constant Sublist.sub to allow for name sub in TreeFsetI
2012-08-30, by Christian Sternagel
reverted (accidentally commited) changes from changeset fd4aef9bc7a9
2012-08-30, by Christian Sternagel
reverted (accidentally commited) changes from changeset fd4aef9bc7a9
2012-08-30, by Christian Sternagel
added theory instantiating type class order for list prefixes
2012-08-30, by Christian Sternagel
Main is implicitly imported via Sublist
2012-08-30, by Christian Sternagel
added author
2012-08-30, by Christian Sternagel
List is implicitly imported by Main
2012-08-30, by Christian Sternagel
introduced "sub" as abbreviation for "emb (op =)";
2012-08-29, by Christian Sternagel
base Sublist_Order on Sublist (using a simplified form of embedding as sublist relation)
2012-08-29, by Christian Sternagel
dropped ord and bot instance for list prefixes (use locale interpretation instead, which allows users to decide what order to use on lists)
2012-08-29, by Christian Sternagel
more lemmas on suffixes and embedding
2012-08-29, by Christian Sternagel
changed arguement order of suffixeq (to facilitate reading "suffixeq xs ys" as "xs is a (possibly empty) suffix of ys)
2012-08-29, by Christian Sternagel
added embedding for lists (constant emb)
2012-08-29, by Christian Sternagel
renamed (in Sublist): postfix ~> suffixeq, and dropped infix syntax >>=
2012-08-29, by Christian Sternagel
renamed (in Sublist): prefix ~> prefixeq, strict_prefix ~> prefix
2012-08-29, by Christian Sternagel
renamed theory List_Prefix into Sublist (since it is not only about prefixes)
2012-08-29, by Christian Sternagel
compile
2012-09-03, by blanchet
rearrange dependencies
2012-09-03, by blanchet
renamed three BNF/(co)datatype-related commands
2012-09-03, by blanchet
tuned boundary cases of command-line;
2012-09-03, by wenzelm
"isabelle logo" produces EPS and PDF format simultaneously;
2012-09-03, by wenzelm
actually reset output when there is no valid command span here (especially relevant at very end of jEdit buffer, which lacks the terminating newline);
2012-09-03, by wenzelm
tuned proofs;
2012-09-03, by wenzelm
some parallel ML;
2012-09-03, by wenzelm
proper classpath on windows;
2012-09-02, by wenzelm
proper classpath for Java FX;
2012-09-02, by wenzelm
basic setup for HTML5 panel;
2012-09-02, by wenzelm
basic support for Java FX;
2012-09-02, by wenzelm
maintain stable state of node entries from last round -- bypass slightly different Thm.join_theory_proofs;
2012-09-02, by wenzelm
removed unused material;
2012-09-01, by wenzelm
discontinued complicated/unreliable notion of recent proofs within context;
2012-09-01, by wenzelm
central management of forked goals wrt. transaction id;
2012-09-01, by wenzelm
merged
2012-08-31, by wenzelm
always register proofs, even for empty binding;
2012-08-31, by wenzelm
tuned signature;
2012-08-31, by wenzelm
made parser a bit more flexible
2012-08-31, by blanchet
tuning
2012-08-31, by blanchet
pad the selectors' list with default names
2012-08-31, by blanchet
generate default names for selectors
2012-08-31, by blanchet
renamed "disc_disjoint" property "disj_exclus"
2012-08-31, by blanchet
optimized "mk_split_tac" + use "notes"
2012-08-31, by blanchet
optimized "mk_case_disc_tac" further
2012-08-31, by blanchet
optimized "mk_case_disc_tac"
2012-08-31, by blanchet
tuning
2012-08-31, by blanchet
rationalized data structure for distinctness theorems
2012-08-31, by blanchet
optimized "case_cong" proof
2012-08-31, by blanchet
allow default names for selectors via wildcard (_) + fix wrong index (k)
2012-08-31, by blanchet
minor fixes (for compatibility with existing datatype package)
2012-08-31, by blanchet
generate "split_asm" property
2012-08-31, by blanchet
generate "split" property
2012-08-31, by blanchet
more precise register_proofs for local goals;
2012-08-31, by wenzelm
more informative error message from failed goal forks (violating old-style TTY protocol!);
2012-08-31, by wenzelm
avoid empty tooltips;
2012-08-31, by wenzelm
clarified command status (again);
2012-08-31, by wenzelm
recovered ScrollPane from d899be1cfe6d;
2012-08-31, by wenzelm
more markup for failed goal forks, reusing "bad";
2012-08-31, by wenzelm
further refinement of command status, to accomodate forked proofs;
2012-08-31, by wenzelm
merged;
2012-08-30, by wenzelm
make parallel list indexing possible for inject theorems
2012-08-30, by blanchet
generate "weak_case_cong" property
2012-08-30, by blanchet
generate "case_cong" property
2012-08-30, by blanchet
generate "case_disc" property
2012-08-30, by blanchet
generate "ctr_sels" theorems
2012-08-30, by blanchet
generate "disc_exhaust" property
2012-08-30, by blanchet
generate "disc_distinct" theorems
2012-08-30, by blanchet
added discriminator theorems
2012-08-30, by blanchet
adjust example
2012-08-30, by blanchet
more work on sugar
2012-08-30, by blanchet
updated Java-related error message
2012-08-30, by blanchet
changed order of arguments to "bnf_sugar"
2012-08-30, by blanchet
define selectors and discriminators
2012-08-30, by blanchet
tuning
2012-08-30, by blanchet
more work on BNF sugar -- up to derivation of nchotomy
2012-08-30, by blanchet
more work on BNF sugar
2012-08-30, by blanchet
renamed ML function for consistency
2012-08-30, by blanchet
started work on datatype sugar
2012-08-30, by blanchet
killed obsolete "bnf_of_typ" command
2012-08-30, by blanchet
removed dead code
2012-08-30, by blanchet
have "bnf_of_typ" command seal the BNF
2012-08-30, by blanchet
register proofs of Isar goals, to enable recovery from unstable command states after interactive cancellation;
2012-08-30, by wenzelm
refined treatment of forked proofs at transaction boundaries, including proof commands (see also 7ee000ce5390);
2012-08-30, by wenzelm
some support for registering forked proofs within Proof.state, using its bottom context;
2012-08-30, by wenzelm
tuned signature;
2012-08-30, by wenzelm
refined status of forked goals;
2012-08-30, by wenzelm
proper merge of promises to avoid exponential blow-up in pathologic situations (e.g. lack of PThm wrapping);
2012-08-30, by wenzelm
tuned message;
2012-08-29, by wenzelm
discontinued old init_components script, superseded by init_components shell function as explained in README_REPOSITORY;
2012-08-29, by wenzelm
approximative build of pdf documents in 1 pass instead of 3;
2012-08-29, by wenzelm
more formal isabelle makedist from repository;
2012-08-29, by wenzelm
removed remains of generated material, which tends to rot;
2012-08-29, by wenzelm
one more round to ensure that base images are already there, without producing document output themselves;
2012-08-29, by wenzelm
more robust document setup;
2012-08-29, by wenzelm
provide polyml-5.4.1 as regular component;
2012-08-29, by wenzelm
clarified handling of raw output messages;
2012-08-29, by wenzelm
no attempt to build documentation for now -- requires ML_HOME etc. which is not present here;
2012-08-29, by wenzelm
command 'use' is legacy;
2012-08-29, by wenzelm
clarified separated_chunks vs. space_explode;
2012-08-29, by wenzelm
more precise indentation;
2012-08-29, by wenzelm
modernized specifications;
2012-08-29, by wenzelm
tuned signature;
2012-08-29, by wenzelm
renamed Position.str_of to Position.here;
2012-08-29, by wenzelm
init components from local clone that is used to produce the test distribition, which itself lacks Admin;
2012-08-29, by wenzelm
discontinued centralistic changelog;
2012-08-28, by wenzelm
discontinued odd copy of eps logos (cf. 8fc3828fdc8a);
2012-08-28, by wenzelm
prefer cp over mv, to reduce assumptions about file-system boundaries and GNU vs. non-GNU tools;
2012-08-28, by wenzelm
removed odd left-over file;
2012-08-28, by wenzelm
less
more
|
(0)
-30000
-10000
-3000
-1000
-112
+112
+1000
+3000
+10000
+30000
tip