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
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.
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
less
more
|
(0)
-30000
-10000
-3000
-1000
-120
+120
+1000
+3000
+10000
tip