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
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.
Added tag Isabelle2013-2-RC3 for changeset aeb21314d078
2013-12-01, by wenzelm
prefer transparent application icon (like Mac OS X);
2013-12-01, by wenzelm
specific application name for official bundle (as for Mac OS X);
2013-12-01, by wenzelm
prefer isabelle application icon;
2013-12-01, by wenzelm
more isabelle logos (from isabelle.ico);
2013-12-01, by wenzelm
prefer 32x32 icon like jedit (image from isabelle.ico);
2013-11-30, by wenzelm
updated isabelle.ico for the record (see also 84177f8372f9);
2013-11-30, by wenzelm
updated icon of Isabelle.exe, using http://convertico.org/image_to_icon_converter on lib/logo/isabelle.gif (approx. 256x256 pixels according to Windows 7 format);
2013-11-30, by wenzelm
further encouragement to read jEdit documentation;
2013-11-30, by wenzelm
clarified view.title;
2013-11-30, by wenzelm
NEWS;
2013-11-30, by wenzelm
non-focusable button, to avoid second interpretation of SPACE in C+e SPACE (isabelle.set-node-required);
2013-11-30, by wenzelm
more thorough read_pid with extra delay, to give external process a chance to write pid file before attempting to terminate it -- especially relevant for PIDE document processing, where interrupts can happen in the range of milliseconds;
2013-11-30, by wenzelm
Added tag Isabelle2013-2-RC2 for changeset 99b9249b3e05
2013-11-28, by wenzelm
more official task context via Task_Queue.enroll, which is required to participate in group cancellation (e.g. to terminate command exec);
2013-11-28, by wenzelm
NEWS;
2013-11-25, by wenzelm
more defensive order of Markup.failed vs. Markup.finished -- more informative status in Isabelle/Scala, although it is not rendered in Isabelle/jEdit;
2013-11-25, by wenzelm
more robust status reports: avoid loosing information about physical events (see also 28d207ba9340, 2bc5924b117f, 9edfd36a0355) -- NB: TTY and Proof General ignore Output.status and Output.report;
2013-11-25, by wenzelm
more robust and portable invocation of kill as bash builtin, instead of external executable -- NB: /bin/kill on Mac OS X Mountain Lion chokes on Linux workaround from 3610ae73cfdb;
2013-11-25, by wenzelm
Added tag Isabelle2013-2-RC1 for changeset 57aefb80b639
2013-11-24, by wenzelm
more on GTK;
2013-11-23, by wenzelm
reintroduced e2d08b9c9047, lost in 54e290da6da8 + e13b0c88c798 (clone of f6ffe53387ef);
2013-11-22, by wenzelm
NEWS;
2013-11-21, by wenzelm
back to Status.FINISHED and immediate remove_overlay (reverting 6e69f9ca8f1c), which is important to avoid restart of print function after edits + re-assignment of located command;
2013-11-21, by wenzelm
updated to Isabelle2013-2;
2013-11-20, by wenzelm
compile on Windows (clone of d04576557400);
2013-11-20, by wenzelm
register actual group of nested worker context -- relevant for insulated cancellation of exec_ids (see also 78693e46a237, e0169f13bd37);
2013-11-20, by wenzelm
updated mirror script for Cambridge
2013-12-05, by paulson
proper code generation for discriminators/selectors
2013-12-05, by blanchet
reverted 141cb34744de and e78e7df36690 -- better provide nicer "eta-expanded" definitions for discriminators and selectors, since users might want to unfold them
2013-12-05, by blanchet
experiment
2013-12-05, by blanchet
make sure acyclicity axiom gets generated in the case where the problem involves mutually recursive datatypes
2013-12-05, by blanchet
news
2013-12-05, by Andreas Lochbihler
restrict admissibility to non-empty chains to allow more syntax-directed proof rules
2013-12-05, by Andreas Lochbihler
merge
2013-12-03, by panny
generate "code" theorems for incomplete definitions
2013-12-02, by panny
updated keywords
2013-12-02, by blanchet
added 'no_code' option
2013-12-02, by blanchet
killed obsolete artifact
2013-12-02, by blanchet
revert making 'map_cong' a 'cong' -- it breaks too many proofs in the AFP
2013-12-02, by blanchet
avoid user-level 'Specification.definition' for low-level definitions
2013-12-02, by blanchet
repaired inconsistency introduced in transiting to 'Local_Theory.define'
2013-12-02, by blanchet
docs for forgotten BNF theorems
2013-12-02, by blanchet
tuning
2013-12-02, by blanchet
added 'cong' attribute to 'map_cong'
2013-12-02, by blanchet
avoid user-level 'Specification.definition' for internal constructions (to avoid e.g. automatic code generation behavior)
2013-12-02, by blanchet
don't try to register code equations in a locale with assumptions
2013-12-02, by blanchet
minor doc update
2013-12-02, by blanchet
generalized datatype code generation code so that it works with old-style and new-style (co)datatypes (as long as they are not local)
2013-12-02, by blanchet
simpler code
2013-12-02, by blanchet
more work towards "exhaustive"
2013-12-01, by panny
Backed out changeset: a8ad7f6dd217---bypassing Main breaks theories that use \<inf> or \<sup>
2013-11-29, by traytel
set_comprehension_pointfree simproc causes to many surprises if enabled by default
2013-11-29, by traytel
tuned
2013-11-28, by nipkow
updated docs
2013-11-28, by blanchet
added Riss3g
2013-11-28, by blanchet
reduce dependency (toward move to 'HOL')
2013-11-28, by blanchet
cleaned up indirect dependency
2013-11-28, by blanchet
tuned
2013-11-28, by nipkow
prefer sort-stripping const_typ over Sign.the_const_type whenever appropriate
2013-11-28, by haftmann
prefer name-normalizing devarify over unvarifyT whenever appropriate
2013-11-28, by haftmann
some documentation
2013-11-27, by traytel
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
2013-11-27, by traytel
remove junk
2013-11-27, by Andreas Lochbihler
revert 4af7c82463d3 and document type class problem in Haskell
2013-11-27, by Andreas Lochbihler
merged
2013-11-27, by Andreas Lochbihler
no ord instance for String.literal in Haskell when list is also ordered lexicographically
2013-11-20, by Andreas Lochbihler
implement comparisons on String.literal by target-language comparisons
2013-11-20, by Andreas Lochbihler
instantiate linorder for String.literal by lexicographic order
2013-11-20, by Andreas Lochbihler
setup lifting/transfer for String.literal
2013-11-20, by Andreas Lochbihler
add predicate version of lexicographic order on lists
2013-11-20, by Andreas Lochbihler
merge
2013-11-26, by panny
prevent exception when equations for a function are missing;
2013-11-25, by panny
Add Zorn to HOL-Library
2013-11-26, by hoelzl
made SML/NJ happier
2013-11-26, by traytel
NEWS
2013-11-26, by traytel
even more precise NEWS
2013-11-25, by haftmann
mreged
2013-11-25, by paulson
Small simplifications to proofs
2013-11-25, by paulson
possibility to fold coercion inference error messages; tuned;
2013-11-25, by traytel
tweaks to the documentation
2013-11-25, by paulson
MaSH files should be ignored
2013-11-25, by paulson
eliminated dependence of Cardinals_FP on Set_Intervals, more precise imports
2013-11-25, by traytel
adapt to 9733ab5c1df6
2013-11-25, by traytel
drop theorem duplicates
2013-11-25, by traytel
eliminated dependence of BNF on Infinite_Set by moving 3 theorems from the latter to Main
2013-11-25, by traytel
typos
2013-11-25, by nipkow
tidied more proofs
2013-11-25, by paulson
cleaned up more messy proofs
2013-11-24, by paulson
merged
2013-11-24, by paulson
cleaned up some messy proofs
2013-11-24, by paulson
tuned
2013-11-24, by nipkow
replaced bad example
2013-11-24, by nipkow
polished some ancient proofs
2013-11-24, by paulson
merged
2013-11-23, by paulson
Simplified, tidied and generalised proofs esp of Binomial Theorem.
2013-11-23, by paulson
more uniform / rigid checking of Goal.prove_common vs. Proof.conclude_goal -- NB: Goal.prove_common cannot check hyps right now, e.g. due to undeclared Simplifier prems;
2013-11-23, by wenzelm
more accurate goal context;
2013-11-23, by wenzelm
tuned;
2013-11-23, by wenzelm
more accurate goal context;
2013-11-23, by wenzelm
more official option;
2013-11-23, by wenzelm
clarified node edits sent to prover -- Clear/Blob only required for text edits within editor;
2013-11-22, by wenzelm
exclude gzipped files from document model, to avoid confusion about actual file name and content;
2013-11-22, by wenzelm
more .hgignore;
2013-11-22, by wenzelm
tuned messages;
2013-11-22, by wenzelm
more total master_directory -- NB: this is used outside command transactions (see also 92961f196d9e);
2013-11-22, by wenzelm
correctly account for dead variables when naming set functions
2013-11-22, by blanchet
compile
2013-11-21, by blanchet
rationalize imports
2013-11-21, by blanchet
eliminated Sledgehammer's dependency on old-style datatypes
2013-11-21, by blanchet
moved meson up the dependency chain
2013-11-21, by blanchet
moving 'Order_Relation' to 'HOL' (since it's a BNF dependency)
2013-11-21, by blanchet
fixed apparent copy-paste bug
2013-11-21, by blanchet
merged
2013-11-21, by wenzelm
actually expose errors of cumulative theory dependencies;
2013-11-21, by wenzelm
proper concatenation of messages;
2013-11-21, by wenzelm
renamed TFF0/THF0 to three-letter acronyms, in keeping with new TPTP policy
2013-11-21, by blanchet
fixed spying so that the envirnoment variables are queried at run-time not at build-time
2013-11-21, by blanchet
effectively reverted d25fc4c0ff62, to avoid quasi-cyclic dependencies with HOL-Cardinals and minimize BNF dependencies
2013-11-20, by blanchet
killed more needless thms
2013-11-20, by blanchet
killed needless thm
2013-11-20, by blanchet
mention docs
2013-11-20, by blanchet
took out warning (BNF is still under development, but it is finished enough)
2013-11-20, by blanchet
moved 'coinduction' proof method to 'HOL'
2013-11-20, by blanchet
move registration of countable set type as BNF to its own theory file (+ renamed theory)
2013-11-20, by blanchet
factor 'List_Prefix' out of 'Sublist' and move to 'Main' (needed for codatatypes)
2013-11-20, by blanchet
fixed LaTeX missing }
2013-11-20, by blanchet
compile
2013-11-20, by blanchet
support Negated_Conjecture as a TPTP role as well (e.g. for SMT proofs)
2013-11-20, by blanchet
tuning
2013-11-20, by blanchet
NEWS;
2013-11-20, by wenzelm
merged
2013-11-20, by wenzelm
restrict node_required status and Theories panel to actual theories;
2013-11-20, by wenzelm
ranges of thy_load commands count as visible within perspective;
2013-11-20, by wenzelm
tuned;
2013-11-20, by wenzelm
refer to thy_load command of auxiliary file;
2013-11-20, by wenzelm
proper static resolution of files via Thy_Load.load_thy, instead of TTY fall-back;
2013-11-20, by wenzelm
load files that are not provided by PIDE blobs;
2013-11-20, by wenzelm
tuned;
2013-11-20, by wenzelm
more explicit indication of missing files;
2013-11-19, by wenzelm
more uniform handling of inlined files;
2013-11-19, by wenzelm
tuned signature;
2013-11-19, by wenzelm
clarified Document.Blobs environment vs. actual edits of auxiliary files;
2013-11-19, by wenzelm
release file errors at runtime: Command.eval instead of Command.read;
2013-11-19, by wenzelm
maintain blobs within document state: digest + text in ML, digest-only in Scala;
2013-11-19, by wenzelm
always reparse nodes with thy_load commands, to update inlined files;
2013-11-19, by wenzelm
proper Thy_Load.append of auxiliary file names;
2013-11-19, by wenzelm
proper theory name vs. node name;
2013-11-19, by wenzelm
clarified boundary cases of Document.Node.Name;
2013-11-19, by wenzelm
clarified Thy_Load.node_name;
2013-11-18, by wenzelm
inline blobs into command, via SHA1 digest;
2013-11-18, by wenzelm
persistent value;
2013-11-18, by wenzelm
caching of blob;
2013-11-18, by wenzelm
tuned;
2013-11-18, by wenzelm
maintain document model for all files, with document view for theory only, and special blob for non-theory files;
2013-11-18, by wenzelm
tuned
2013-11-20, by nipkow
whitespace tuning
2013-11-19, by blanchet
tuning
2013-11-19, by blanchet
more refactoring to accommodate SMT proofs
2013-11-19, by blanchet
tuning
2013-11-19, by blanchet
tuning
2013-11-19, by blanchet
more correct NEWS
2013-11-19, by haftmann
simplified old code
2013-11-19, by blanchet
refactoring
2013-11-19, by blanchet
refactoring
2013-11-19, by blanchet
merged
2013-11-19, by hoelzl
BNF/Examples/Stream: rename same to sconst; define same, fromN in terms of siterate
2013-11-18, by hoelzl
add lemmas Suc_funpow and id_funpow to simpset; add lemma map_add_upt
2013-11-18, by hoelzl
refactored
2013-11-19, by blanchet
updated docs
2013-11-19, by blanchet
use type suffixes instead of prefixes for 'case', '(un)fold', '(co)rec'
2013-11-19, by blanchet
prefix internal names as well
2013-11-19, by blanchet
case_if -> case_eq_if + docs
2013-11-19, by blanchet
use suffix '_list' etc. instead of prefix 'list_' for constants not present in the old package
2013-11-19, by blanchet
eliminiated neg_numeral in favour of - (numeral _)
2013-11-19, by haftmann
more tuning for speed
2013-11-19, by blanchet
tuning
2013-11-19, by blanchet
tuned proofs
2013-11-19, by blanchet
killed more needless theorems
2013-11-19, by blanchet
killed unused lemmas
2013-11-19, by blanchet
optimized more bad apples
2013-11-19, by blanchet
optimized 'bad apple' method calls
2013-11-19, by blanchet
compile
2013-11-18, by blanchet
no need for 3-way split with GFP for a handful of theorems
2013-11-18, by blanchet
moved more theorems out of LFP
2013-11-18, by blanchet
moved theorems out of LFP
2013-11-18, by blanchet
moved theorems out of LFP
2013-11-18, by blanchet
moved theorems out of LFP
2013-11-18, by blanchet
moved theorems out of LFP
2013-11-18, by blanchet
split 'Cardinal_Arithmetic' 3-way
2013-11-18, by blanchet
started three-way split of 'HOL-Cardinals'
2013-11-18, by blanchet
send output of "tptp_translate" to standard output, to simplify Geoff Sutcliffe's life
2013-11-18, by blanchet
merged
2013-11-18, by traytel
show all involved subtyping constraints that cause coercion inference to fail
2013-11-18, by traytel
additional lemmas in BNF/Examples/Stream
2013-11-18, by hoelzl
reintroduced e2d08b9c9047, lost in 54e290da6da8 + e13b0c88c798
2013-11-18, by traytel
comments by Sean Seefried
2013-11-18, by nipkow
more robust example;
2013-11-17, by wenzelm
tuned proofs;
2013-11-17, by wenzelm
tuned;
2013-11-17, by wenzelm
tuned proofs;
2013-11-17, by wenzelm
explicit indication of thy_load commands;
2013-11-17, by wenzelm
centralized management of pending buffer edits;
2013-11-17, by wenzelm
merged
2013-11-17, by nipkow
added functions all and exists to IArray
2013-11-16, by nipkow
prefer explicit "document" flag -- eliminated stateful Present.no_document;
2013-11-16, by wenzelm
simplified HTML linefeed (again, see 041dc6d8d344);
2013-11-16, by wenzelm
simplified HTML theory presentation;
2013-11-16, by wenzelm
removed remains of HTML presentation of auxiliary files -- inactive since Isabelle2013;
2013-11-16, by wenzelm
tuned;
2013-11-16, by wenzelm
merged
2013-11-16, by wenzelm
tuned proofs;
2013-11-16, by wenzelm
tuned signature;
2013-11-16, by wenzelm
tuned signature -- clarified Proof General legacy;
2013-11-16, by wenzelm
toplevel function "use" refers to raw ML bootstrap environment;
2013-11-16, by wenzelm
obsolete;
2013-11-16, by wenzelm
proper thy_load command 'boogie_file' -- avoid direct access to file-system;
2013-11-16, by wenzelm
tuned signature;
2013-11-16, by wenzelm
updated example;
2013-11-16, by wenzelm
prefer UTF8.decode_permissive;
2013-11-16, by wenzelm
more distinctive Isabelle_Process.Output vs. Isabelle_Process.Protocol_Output;
2013-11-16, by wenzelm
more specific Protocol_Output: empty message.body, main content via bytes/text;
2013-11-15, by wenzelm
tuned imports;
2013-11-14, by wenzelm
tuned signature;
2013-11-14, by wenzelm
immutable byte vectors versus UTF8 strings;
2013-11-14, by wenzelm
dropped duplicate of of_bool
2013-11-15, by haftmann
proper code equations for Gcd and Lcm on nat and int
2013-11-15, by haftmann
tuned
2013-11-16, by nipkow
fixed type variable confusion in 'datatype_new_compat'
2013-11-14, by blanchet
implemented 'tptp_translate'
2013-11-14, by blanchet
reintroduced (unimplemented) 'tptp_translate' tool
2013-11-14, by blanchet
have MaSh support nameless facts (i.e. proofs) and use that support
2013-11-14, by blanchet
made SML/NJ happy
2013-11-14, by blanchet
renamed thm
2013-11-14, by blanchet
explicit inclusion of data refinement theory into HOL-Library session
2013-11-14, by haftmann
tuned to improve automation (for REPEAT)
2013-11-14, by nipkow
separated comparision on bit operations into separate theory
2013-11-13, by haftmann
prohibit locally fixed type variables in bnf definitions
2013-11-13, by traytel
tuned
2013-11-13, by traytel
standard relator for list bnf
2013-11-13, by traytel
less
more
|
(0)
-30000
-10000
-3000
-1000
-240
+240
+1000
+3000
+10000
tip