Mercurial
Mercurial
>
repos
>
isabelle
/ graph
summary
|
shortlog
|
changelog
| graph |
tags
|
bookmarks
|
branches
|
files
|
gz
|
help
less
more
|
(0)
-30000
-10000
-3000
-1000
-480
+480
+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.
generate "id" rather than (%v. v)
2012-09-11, by blanchet
correctly generate sel_coiter and sel_corec theorems
2012-09-11, by blanchet
generate "sel_coiters" and friends
2012-09-10, by blanchet
sanity check
2012-09-10, by blanchet
implemented and use "mk_sum_casesN_balanced"
2012-09-10, by blanchet
fixed general case of "mk_sumEN_balanced"
2012-09-10, by blanchet
debug
2012-09-10, by blanchet
fixed base case of "mk_sumEN_balanced"
2012-09-10, by blanchet
prevent inconsistent selector types
2012-09-10, by blanchet
minor optimization
2012-09-10, by blanchet
allow same selector name for several constructors
2012-09-10, by blanchet
removed done TODO
2012-09-10, by blanchet
avoid type inference + tuning
2012-09-10, by blanchet
use balanced sums for constructors (to gracefully handle 100 constructors or more)
2012-09-10, by blanchet
busted -- let's use more neutral names
2012-09-10, by blanchet
replacing own dummy value by Haskell's Prelude.undefined
2012-09-10, by bulwahn
prefer global default font over IsabelleText of jEdit TextArea;
2012-09-11, by wenzelm
uniform operation on initial delay;
2012-09-11, by wenzelm
option jedit_load_delay;
2012-09-10, by wenzelm
dynamic evaluation of time (e.g. via options);
2012-09-10, by wenzelm
proper multi-line tooltip;
2012-09-10, by wenzelm
more detailed option tooltip;
2012-09-10, by wenzelm
more systematic JEdit_Options.make_component;
2012-09-10, by wenzelm
manage Isabelle/jEdit options as Isabelle/Scala options (with persistent preferences);
2012-09-10, by wenzelm
formal markup for @{file} (for hyperlinks etc.) -- interpret path wrt. master directory as usual;
2012-09-10, by wenzelm
more explicit indication of legacy features;
2012-09-10, by wenzelm
more explicit indication of legacy features;
2012-09-10, by wenzelm
simplify "Process" example even further
2012-09-10, by traytel
stabilized generation of parameterized theorem
2012-09-10, by traytel
added snippets
2012-09-10, by nipkow
simplify "Process" example further
2012-09-09, by blanchet
simplify "Process" example
2012-09-09, by blanchet
full name of a type as key in bnf table
2012-09-09, by traytel
fixed bug with one-value codatatype "codata 'a dead_foo = A"
2012-09-09, by blanchet
tuning
2012-09-09, by blanchet
fixed and reenabled "corecs" theorems
2012-09-09, by blanchet
fixed and enabled generation of "coiters" theorems, including the recursive case
2012-09-09, by blanchet
generate "fld_unf_corecs" as well
2012-09-09, by blanchet
reactivated generation of "coiters" theorems
2012-09-09, by blanchet
use map_id, not map_id', to allow better composition
2012-09-09, by blanchet
open typedefs everywhere in the package
2012-09-09, by traytel
open typedef for datatypes
2012-09-09, by traytel
fixed and enabled iterator/recursor theorems
2012-09-08, by blanchet
renamed for consistency
2012-09-08, by blanchet
oops
2012-09-08, by blanchet
tuning
2012-09-08, by blanchet
for compatiblity with old datatype package: not only "recs" with "s", but also "iters" and their "fld_"/"unf_" variants
2012-09-08, by blanchet
fixed bug with one-value types with phantom type arguments
2012-09-08, by blanchet
imported patch debugging
2012-09-08, by blanchet
repaired "nofail4" example
2012-09-08, by blanchet
renamed xxxBNF to pre_xxx
2012-09-08, by blanchet
fixed handling of map of "fun"
2012-09-08, by blanchet
comment out code that's not ready
2012-09-08, by blanchet
tuning
2012-09-08, by blanchet
construct the right iterator theorem in the recursive case
2012-09-08, by blanchet
some work on coiter tactic
2012-09-08, by blanchet
more sugar on codatatypes
2012-09-08, by blanchet
define corecursors
2012-09-08, by blanchet
define coiterators
2012-09-08, by blanchet
TODO
2012-09-08, by blanchet
tuning
2012-09-08, by blanchet
completed iter/rec proofs
2012-09-08, by blanchet
TODOs
2012-09-08, by blanchet
implemented "mk_iter_or_rec_tac"
2012-09-08, by blanchet
generate iter/rec goals
2012-09-08, by blanchet
repaired constant types
2012-09-08, by blanchet
some work towards iterator and recursor properties
2012-09-08, by blanchet
tuning
2012-09-08, by blanchet
correctly curry recursor arguments
2012-09-08, by blanchet
added high-level recursor, not yet curried
2012-09-08, by blanchet
merged
2012-09-07, by wenzelm
tuned proofs;
2012-09-07, by wenzelm
postpone update of text overview panel after incoming session edits, to improve reactivity of editing massive theories like src/HOL/Multivariate_Analysis;
2012-09-07, by wenzelm
more explicit Delay operations;
2012-09-07, by wenzelm
tuned proofs;
2012-09-07, by wenzelm
clearer names for functions in Quickcheck's narrowing engine
2012-09-07, by bulwahn
merged
2012-09-07, by nipkow
tuned latex
2012-09-07, by nipkow
lattice instances for option type
2012-09-07, by haftmann
combinator Option.these
2012-09-07, by haftmann
adjusted examples
2012-09-07, by nipkow
countable_datatype method: pre-instantiate induction rule to avoid failure with e.g. datatype a = A "b list" and b = B "a"
2012-09-06, by huffman
handle type constructors not known to be a BNF using the DEADID BNF
2012-09-06, by traytel
respect order of/additional type variables supplied by the user in fixed point constructions;
2012-09-06, by traytel
gracefully handle shadowing case (fourth step of sugar localization)
2012-09-06, by blanchet
careful about constructor types w.r.t. fake context (third step of localization)
2012-09-06, by blanchet
read the real types off the constant types, rather than using the fake parser types (second step of sugar localization)
2012-09-06, by blanchet
tuning
2012-09-06, by blanchet
use "add_type" rather than "add_types_global"
2012-09-06, by blanchet
don't throw away the context when hacking the theory (first step to localize the sugar code)
2012-09-06, by blanchet
tuning
2012-09-06, by blanchet
introduced and used "mk_Freesss", and simplified "mk_Freess(')"
2012-09-06, by blanchet
construct high-level iterator RHS
2012-09-06, by blanchet
option for discarding build results, enabled in particular for Isabelle_makeall
2012-09-06, by krauss
by default, only generate one discriminator for a two-value datatype
2012-09-05, by blanchet
eliminated potentially confusing terminology of Scala "layer";
2012-09-05, by wenzelm
merged
2012-09-05, by wenzelm
tuned proofs;
2012-09-05, by wenzelm
discontinued obsolete fork_mono to loosen some brakes -- NB: TTY interaction has Goal.future_proofs disabled due to missing Future.worker_task;
2012-09-05, by wenzelm
honor mixfix specifications
2012-09-05, by blanchet
code indentation
2012-09-05, by blanchet
print timing information
2012-09-05, by blanchet
adapted example
2012-09-05, by blanchet
check type variables on rhs
2012-09-05, by blanchet
proper subsexp projection of Isabelle_Markup.Path, in correspondence to 5d0cd770828e;
2012-09-05, by wenzelm
added tooltip to reveal jEdit platform file name;
2012-09-05, by wenzelm
commented out slow examples again
2012-09-05, by blanchet
fixed (n + 1)st bug in "mk_exhaust_tac" -- arose with uncurried constructors
2012-09-05, by blanchet
fixed "mk_exhaust_tac" for the nth time
2012-09-05, by blanchet
updated README
2012-09-05, by blanchet
ported "Misc_Codata" to new syntax
2012-09-05, by blanchet
ported "Misc_Data" to new syntax
2012-09-05, by blanchet
error message only in case of an error
2012-09-05, by traytel
do not trivialize important internal theorem in quick_and_dirty mode
2012-09-05, by traytel
merged
2012-09-05, by wenzelm
made "mk_case_eq_tac" work in the case where the first constructor is an "alternate" constructor (in which case its discriminator paradoxically starts with a negation)
2012-09-05, by blanchet
tuning (systematic 1-based indices)
2012-09-05, by blanchet
reindented code
2012-09-05, by blanchet
added TODO
2012-09-05, by blanchet
tell "select_prem_tac" not to thin any further premisses -- the "rotate_tac" otherwise confuses it
2012-09-05, by blanchet
fixed "mk_alternate_disc_def_tac" in the case where the constructors are swapped compared with the common Nil/Cons case
2012-09-05, by blanchet
don't get confused by extraneous premisses
2012-09-05, by blanchet
added a check
2012-09-05, by blanchet
NEWS; CONTRIBUTORS
2012-09-04, by Christian Sternagel
misc tuning;
2012-09-05, by wenzelm
no need to wait 3h on macbroy30 (unlike former macbroy6, cf. 6e5b994070c1);
2012-09-05, by wenzelm
more conservative rechecking of processed constraints in subtyping constraint simplification
2012-09-05, by traytel
added comment for Dmitriy
2012-09-05, by blanchet
fixed bug in type instantiation of case theorem
2012-09-05, by blanchet
use empty binding rather than "*" for default
2012-09-05, by blanchet
tuned
2012-09-05, by nipkow
fixed bugs in one-constructor case
2012-09-05, by blanchet
smoothly handle one-constructor types
2012-09-04, by blanchet
fixed some type issues in sugar "exhaust_tac"
2012-09-04, by blanchet
optionally provide extra dead variables to the FP constructions
2012-09-04, by blanchet
merged
2012-09-04, by wenzelm
added robustness
2012-09-04, by blanchet
added build option -R;
2012-09-04, by wenzelm
implemented "mk_case_tac" -- and got rid of "cheat_tac"
2012-09-04, by blanchet
define "case" constant
2012-09-04, by blanchet
renamed low-level (co)iterators and (co)recursors with "fld_"/"unf_" prefix
2012-09-04, by blanchet
implemented "mk_half_distinct_tac"
2012-09-04, by blanchet
implemented "mk_inject_tac"
2012-09-04, by blanchet
implemented "mk_exhaust_tac"
2012-09-04, by blanchet
more work on FP sugar
2012-09-04, by blanchet
more work on sugar + simplify Trueprop + eq idiom everywhere
2012-09-04, by blanchet
renamed "disc_exclus" theorem to "disc_exclude"
2012-09-04, by blanchet
more work on FP sugar
2012-09-04, by blanchet
smarter "*" syntax -- fallback on "_" if "*" is impossible
2012-09-04, by blanchet
more work on FP sugar
2012-09-04, by blanchet
renamed theorem
2012-09-04, by blanchet
tuned TODO comment
2012-09-04, by blanchet
allow pseudo-definition of is_Cons in terms of is_Nil (and similarly for other two-constructor datatypes)
2012-09-04, by blanchet
removed oddities
2012-09-04, by blanchet
allow "*" to indicate no discriminator
2012-09-04, by blanchet
tuned TODOs
2012-09-04, by blanchet
started work on sugared "(co)data" commands
2012-09-04, by blanchet
export "wrap" function
2012-09-04, by blanchet
eliminated obsolete "parallel_proofs = 0" restriction (cf. 0e5b859e1c91)
2012-09-04, by traytel
no more aliases for Local_Theory.note; use Thm.close_derivation in internal theorems;
2012-09-04, by traytel
enable parallel terminal proofs in interaction;
2012-09-04, by wenzelm
misc tuning;
2012-09-03, by wenzelm
merged
2012-09-03, by wenzelm
killed internal output
2012-09-03, by traytel
generate coinductive witnesses for codatatypes
2012-09-03, by traytel
generalized signature
2012-09-03, by traytel
added examples for testing of coinductive witnesses
2012-09-03, by traytel
continue with more robust dummy session after failed startup;
2012-09-03, by wenzelm
prefer old startup dialog scheme (cf. 514bb82514df);
2012-09-03, by wenzelm
more permissive handling of plugin startup failure;
2012-09-03, by wenzelm
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
update on "isabelle build" and "isabelle build_doc";
2012-08-28, by wenzelm
renamed doc-src to src/Doc;
2012-08-28, by wenzelm
do not hardwire document output options -- to be provided by the user;
2012-08-28, by wenzelm
more permanent update of keywords (cf. 3517d6f50b12);
2012-08-28, by wenzelm
merged
2012-08-28, by wenzelm
updated keywords
2012-08-28, by blanchet
fixed import paths in examples
2012-08-28, by blanchet
fixed import paths
2012-08-28, by blanchet
tuning
2012-08-28, by blanchet
updated NEWS and CONTRIBUTORS
2012-08-28, by blanchet
documentation cleanup
2012-08-28, by blanchet
added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
2012-08-28, by blanchet
Typo fixed.
2012-08-28, by webertj
updated .hgignore to reflect to (almost) clean result of build_doc;
2012-08-28, by wenzelm
more formal build_doc tool (Admin only);
2012-08-28, by wenzelm
prepare document more uniformly;
2012-08-28, by wenzelm
prefer \input which actually checks file existence;
2012-08-28, by wenzelm
tuned;
2012-08-28, by wenzelm
prefer (old) isa-index as provided here, to get exactly the same index layout as in Isabelle2012;
2012-08-28, by wenzelm
removed old stuff;
2012-08-28, by wenzelm
more standard document preparation within session context: avoid clashes with generated .tex files, even on case-insensible file-system;
2012-08-28, by wenzelm
removed old stuff;
2012-08-28, by wenzelm
removed historic manual;
2012-08-28, by wenzelm
more standard document preparation within session context;
2012-08-28, by wenzelm
more standard document preparation within session context;
2012-08-28, by wenzelm
updated IsarRef/document/style.sty;
2012-08-28, by wenzelm
missing file;
2012-08-28, by wenzelm
removed junk;
2012-08-28, by wenzelm
more standard document preparation within session context;
2012-08-28, by wenzelm
removed outdated IsarRef/Thy/HOLCF_Specific.thy -- make IsarRef depend on HOL only;
2012-08-28, by wenzelm
prefer doc-src/pdfsetup.sty;
2012-08-28, by wenzelm
more official way to set margin;
2012-08-27, by wenzelm
avoid clash with generated Adaptation.tex on case-insensible file-systems;
2012-08-27, by wenzelm
missing file;
2012-08-27, by wenzelm
deactivate updated doc-src sessions, to make Admin/build doc and makedist work for now;
2012-08-27, by wenzelm
more standard document preparation within session context;
2012-08-27, by wenzelm
more standard document preparation within session context;
2012-08-27, by wenzelm
more standard document preparation within session context;
2012-08-27, by wenzelm
more standard document preparation within session context;
2012-08-27, by wenzelm
more standard document preparation within session context;
2012-08-27, by wenzelm
more standard document preparation within session context;
2012-08-27, by wenzelm
more standard document preparation within session context;
2012-08-27, by wenzelm
more standard document preparation within session context;
2012-08-27, by wenzelm
more standard document preparation within session context;
2012-08-27, by wenzelm
more standard document preparation within session context;
2012-08-27, by wenzelm
more standard document preparation within session context;
2012-08-27, by wenzelm
more portable perl invocation;
2012-08-27, by wenzelm
more standard document preparation within session context;
2012-08-27, by wenzelm
more standard document preparation within session context;
2012-08-27, by wenzelm
more standard document preparation within session context;
2012-08-27, by wenzelm
clarified "isabelle logo";
2012-08-27, by wenzelm
clarified document directories: browser_info as backdrop vs. optional output directory in the foreground;
2012-08-27, by wenzelm
less ambitious test -- terminate more quickly;
2012-08-27, by wenzelm
tuned;
2012-08-27, by wenzelm
actual use of (sos remote_csdp) via ISABELLE_FULL_TEST;
2012-08-19, by wenzelm
test with many add-ons;
2012-08-27, by wenzelm
updated Theory.begin_theory;
2012-08-26, by wenzelm
entity markup for theory Pure, to enable hyperlinks etc.;
2012-08-26, by wenzelm
more accurate defining position of theory;
2012-08-26, by wenzelm
theory def/ref position reports, which enable hyperlinks etc.;
2012-08-26, by wenzelm
fixed theory dependency
2012-08-26, by nipkow
more convenient switching of buffers;
2012-08-24, by wenzelm
report source path and let front-end resolve implicit master location (e.g. URL);
2012-08-24, by wenzelm
prefer jEdit file name representation (potentially via VFS);
2012-08-24, by wenzelm
more precise counting of line/column;
2012-08-24, by wenzelm
support for direct hyperlinks, without the Hyperlinks plugin;
2012-08-24, by wenzelm
tuned signature;
2012-08-24, by wenzelm
some markup for inlined files;
2012-08-24, by wenzelm
check side-comments of command spans (normally filtered out in Outer_Syntax.toplevel_source);
2012-08-24, by wenzelm
updated READMEs -- most Mac OS X problems are gone thanks to jdk-7u6;
2012-08-24, by wenzelm
clarified syntax boundary cases and errors;
2012-08-24, by wenzelm
simplified JVM startup, based on stronger assumptions about the Java version provided as Isabelle component;
2012-08-23, by wenzelm
eliminated obsolete byte_reader -- theory headers + body files are parsed in full;
2012-08-23, by wenzelm
more direct File.read_bytes -- avoid cumulative copying of StringBuilder;
2012-08-23, by wenzelm
improved errors of parser combinators;
2012-08-23, by wenzelm
tuned messages: end-of-input rarely means physical end-of-file from the past;
2012-08-23, by wenzelm
merged
2012-08-23, by wenzelm
remove Hoare dependency from Fold.thy
2012-08-23, by Gerwin Klein
added specific 'spark_open_vcg' and 'spark_open_siv' with formal management of corresponding source files;
2012-08-23, by wenzelm
turned 'boogie_open' into thy_load command, without any declarations of 'uses';
2012-08-23, by wenzelm
tuned signature;
2012-08-23, by wenzelm
clarified type Token.file;
2012-08-23, by wenzelm
expand all files uniformly;
2012-08-23, by wenzelm
added build option -l (list files);
2012-08-23, by wenzelm
prefer classic take_prefix/take_suffix over chop_while (cf. 0659e84bdc5f);
2012-08-23, by wenzelm
more basic file dependencies -- no load command here;
2012-08-23, by wenzelm
tuned signature (again, cf. ff9cd47be39b);
2012-08-23, by wenzelm
updated Thy_Load.check_thy;
2012-08-23, by wenzelm
simplified Thy_Load.check_thy (again) -- no need to pass keywords nor find files in body text;
2012-08-23, by wenzelm
tuned signature;
2012-08-23, by wenzelm
simplified Thy_Load.provide: do not store full path;
2012-08-23, by wenzelm
prefer ML_file over old uses;
2012-08-22, by wenzelm
merged
2012-08-22, by wenzelm
abstracted lemmas
2012-08-21, by nipkow
prefer ML_file over old uses;
2012-08-22, by wenzelm
prefer ML_file over old uses;
2012-08-22, by wenzelm
'ML_file' evaluates ML text from a file directly within the theory, without predeclaration via 'uses';
2012-08-22, by wenzelm
add keywords of this node as well (e.g. relevant for Pure.thy);
2012-08-22, by wenzelm
tuned;
2012-08-22, by wenzelm
tuned message -- dynamic loading happens routinely, e.g. in TTY/PG interaction;
2012-08-22, by wenzelm
discontinued separate list of required files -- maintain only provided files as they occur at runtime;
2012-08-22, by wenzelm
find files via load commands within theory text;
2012-08-22, by wenzelm
clarified global get_recent_syntax: session always has its base_syntax, but it might be absent itself;
2012-08-22, by wenzelm
pass syntax through check_thy;
2012-08-22, by wenzelm
use Thy_Header.read on explicit text only -- potentially via File.read, not Scan.byte_reader;
2012-08-22, by wenzelm
clarified Parse.path vs. Parse.explode -- prefer errors in proper transaction context;
2012-08-22, by wenzelm
tuned;
2012-08-22, by wenzelm
clarified bootstrapping of Pure;
2012-08-22, by wenzelm
tuned errors;
2012-08-22, by wenzelm
prefer File.full_path in accordance to check_file;
2012-08-21, by wenzelm
more standard Thy_Load.check_thy for Pure.thy, relying on its header;
2012-08-21, by wenzelm
updated Thy_Load.check_thy;
2012-08-21, by wenzelm
refined Thy_Load.check_thy: find more uses in body text, based on keywords;
2012-08-21, by wenzelm
more direct cumulation of (sparse) keywords;
2012-08-21, by wenzelm
some support for thy_load_commands;
2012-08-21, by wenzelm
tuned signature;
2012-08-21, by wenzelm
clarified initialization of Thy_Load, Thy_Info, Session;
2012-08-21, by wenzelm
tuned;
2012-08-21, by wenzelm
more robust cleaning of "% tag" and "-- cmt";
2012-08-20, by wenzelm
some support for inlining file content into outer syntax token language;
2012-08-20, by wenzelm
tuned comment;
2012-08-20, by wenzelm
tuned;
2012-08-20, by wenzelm
added keyword kind "thy_load" (with optional list of file extensions);
2012-08-20, by wenzelm
updated generated files;
2012-08-20, by wenzelm
more strict syntax, according to manual;
2012-08-20, by wenzelm
abstracted lemma
2012-08-20, by nipkow
retain unknown options within preferences;
2012-08-19, by wenzelm
more comprehensible platform family name;
2012-08-19, by wenzelm
tuned message;
2012-08-19, by wenzelm
fewer components, more roots;
2012-08-19, by wenzelm
actually remove makeall (cf. 292b97e17fb7);
2012-08-19, by wenzelm
tuned;
2012-08-17, by wenzelm
Backed out changeset ec82c33c75f8;
2012-08-17, by wenzelm
Typo fixed.
2012-08-17, by webertj
merged
2012-08-17, by wenzelm
merged
2012-08-17, by nipkow
fixed lemmas
2012-08-17, by nipkow
abstracted lemmas
2012-08-16, by nipkow
updated to new init_components, hoping that mira can digest that;
2012-08-17, by wenzelm
some explanations on component categories;
2012-08-17, by wenzelm
specific cygwin components;
2012-08-17, by wenzelm
obsolete;
2012-08-17, by wenzelm
some explanations on isabelle components;
2012-08-17, by wenzelm
some grouping of components;
2012-08-17, by wenzelm
renamed components to components_old, to make room for some directory of the same name;
2012-08-17, by wenzelm
minor robustification;
2012-08-17, by wenzelm
added "isabelle components" tool;
2012-08-17, by wenzelm
tuned;
2012-08-17, by wenzelm
direct support for component forests via init_components;
2012-08-17, by wenzelm
allow to provide external ISABELLE_IDENTIFIER for repository clone -- potentially relevant for isatest and mira;
2012-08-17, by wenzelm
tuned;
2012-08-17, by wenzelm
tuned;
2012-08-17, by wenzelm
updated component repository;
2012-08-17, by wenzelm
updates on 32 bit vs. 64 bit platforms;
2012-08-17, by wenzelm
updated to jedit_build-20120813, pointing to another contrib directory as a change;
2012-08-17, by wenzelm
merged
2012-08-16, by wenzelm
tuned proofs;
2012-08-16, by wenzelm
look in current directory first before looking up includes in the TPTP directory, as required by Geoff
2012-08-16, by blanchet
prefer eta-expanded code equations for fold, to accomodate tail recursion optimisation in Scala
2012-08-16, by haftmann
more robust multi-platform support;
2012-08-16, by wenzelm
updated to jdk-7u6 and jedit_build-20120813 -- NB: plain Isabelle/Scala still happens to work with jdk-6;
2012-08-16, by wenzelm
support for jdk-7u6 component;
2012-08-16, by wenzelm
Clarification: free variables allowed in interpreted locale instances.
2012-08-15, by ballarin
merged
2012-08-15, by nipkow
fixed proof
2012-08-15, by nipkow
abstracted lemmas
2012-08-15, by nipkow
Backed out changeset 6cf7a9d8bbaf
2012-08-15, by nipkow
abstracted lemmas
2012-08-15, by nipkow
merged
2012-08-15, by webertj
Turned into Admin tool download_components.
2012-08-15, by webertj
tuned;
2012-08-15, by wenzelm
tuned;
2012-08-15, by wenzelm
some updates of "Presenting theories", using mkroot/build instead of former mkdir/make/usedir (which are still present in "Misc");
2012-08-15, by wenzelm
tuned;
2012-08-15, by wenzelm
fixed handling of "int" in the wake of its port to the quotient package
2012-08-15, by blanchet
removed dead code
2012-08-15, by blanchet
merged
2012-08-15, by webertj
Added various options, notably -c to download components listed in Admin/components. Also, curl instead of wget.
2012-08-15, by webertj
ignore some administrative files on newer Mercurial versions as well;
2012-08-14, by wenzelm
some support for persistent user preferences;
2012-08-14, by wenzelm
merged
2012-08-14, by wenzelm
explicit document_output directory, without implicit purge of default in ISABELLE_BROWSER_INFO;
2012-08-14, by wenzelm
more direct interpretation of document_variants for build (unchanged for usedir);
2012-08-14, by wenzelm
tone down "z3_tptp", now that Z3 (starting with 4.1) no longer supports TPTP TFF0
2012-08-14, by blanchet
fixed then-else confusion
2012-08-14, by blanchet
tweak Vampire setup in the light of new evaluation
2012-08-14, by blanchet
improved set of reconstructor methods
2012-08-14, by blanchet
warn users about unused "using" facts
2012-08-14, by blanchet
be less aggressive at kicking out chained facts
2012-08-14, by blanchet
recognize bus errors as crash
2012-08-14, by blanchet
consider removing chained facts last, so that they're more likely to be kept
2012-08-14, by blanchet
clarified format of etc/options: only declarations, not re-definitions;
2012-08-14, by wenzelm
check_errors for cumulative session content;
2012-08-14, by wenzelm
even more defensive path expansion (see also 8d381fdef898);
2012-08-14, by wenzelm
support for 'typ' with explicit sort constraint;
2012-08-14, by wenzelm
added jedit option -d;
2012-08-14, by wenzelm
always retain doc-src (as regular component);
2012-08-14, by wenzelm
merged
2012-08-13, by wenzelm
less
more
|
(0)
-30000
-10000
-3000
-1000
-480
+480
+1000
+3000
+10000
+30000
tip