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.
remove unnecessary finiteness assumptions from lemmas about setsum
2014-03-18, by huffman
adapt to Isabelle/c726ecfb22b6
2014-03-18, by huffman
fix HOL-NSA; move lemmas
2014-03-18, by hoelzl
cleanup Series: sorted according to typeclass hierarchy, use {..<_} instead of {0..<_}
2014-03-18, by hoelzl
changed policy when to define constants
2014-03-18, by traytel
tuned proofs; removed duplicated facts
2014-03-18, by traytel
additional lemmas
2014-03-18, by immler
removed dependencies on theory Ordered_Euclidean_Space
2014-03-18, by immler
use cbox to relax class constraints
2014-03-18, by immler
merged
2014-03-17, by wenzelm
tuned;
2014-03-17, by wenzelm
more antiquotations;
2014-03-17, by wenzelm
more robust machine-generated ML sources: constructors for typ and term sometimes occur elsewhere;
2014-03-17, by wenzelm
remove sums_seq, it is not used
2014-03-17, by hoelzl
update syntax of has_*derivative to infix 50; fixed proofs
2014-03-17, by hoelzl
unify syntax for has_derivative and differentiable
2014-03-17, by hoelzl
tuned proofs
2014-03-17, by haftmann
tuned internal construction
2014-03-17, by traytel
a few new theorems
2014-03-17, by paulson
proper flags for main action (amending 638b29331549);
2014-03-17, by wenzelm
tuned rendering -- avoid flashing background of aux. files that are disconnected from the document model;
2014-03-17, by wenzelm
merge semantic and syntax completion;
2014-03-17, by wenzelm
tuned;
2014-03-17, by wenzelm
tuned signature;
2014-03-17, by wenzelm
tuned signature;
2014-03-17, by wenzelm
clarified key event propagation, in accordance to outer_key_listener;
2014-03-17, by wenzelm
allow implicit semantic completion, notably after delay that exceeds usual round-trip time;
2014-03-17, by wenzelm
reject internal names, notably from Term.free_dummy_patterns;
2014-03-17, by wenzelm
more uniform alias vs. hide: proper check, allow to hide global names as well;
2014-03-17, by wenzelm
tuned proofs
2014-03-16, by huffman
normalising simp rules for compound operators
2014-03-16, by haftmann
tuned markup;
2014-03-15, by wenzelm
minor tuning;
2014-03-15, by wenzelm
more markup;
2014-03-15, by wenzelm
clarified completion ordering: prefer local names;
2014-03-15, by wenzelm
tuned signature;
2014-03-15, by wenzelm
tuned -- avoid vacuous reports;
2014-03-15, by wenzelm
clarified local facts;
2014-03-15, by wenzelm
more explicit treatment of verbose mode, which includes concealed entries;
2014-03-15, by wenzelm
removed dead code;
2014-03-15, by wenzelm
clarified retrieve_generic: local error takes precedence, which is relevant for completion;
2014-03-15, by wenzelm
clarified print_local_facts;
2014-03-15, by wenzelm
more complete set of lemmas wrt. image and composition
2014-03-15, by haftmann
merge
2014-03-15, by panny
add error messages for invalid inputs
2014-03-15, by panny
add lemmas about nhds filter; tuned proof
2014-03-14, by huffman
remove unused lemma which was a direct consequence of tendsto_intros
2014-03-14, by huffman
merged
2014-03-14, by wenzelm
merged
2014-03-14, by wenzelm
prefer more robust Synchronized.var;
2014-03-14, by wenzelm
discontinued somewhat pointless "thy_script" keyword kind;
2014-03-14, by wenzelm
conceal improper cases, e.g. relevant for completion (and potentially for markup);
2014-03-14, by wenzelm
conceal somewhat obscure internal facts, e.g. relevant for 'print_theorems', 'find_theorems';
2014-03-14, by wenzelm
more accurate resolution of hybrid facts, which actually changes the sort order of results;
2014-03-14, by wenzelm
tuned -- command 'text' was localized some years ago;
2014-03-14, by wenzelm
back to a form of hybrid facts, to reduce performance impact of ed92ce2ac88e;
2014-03-14, by wenzelm
just one cumulative Proof_Context.facts, with uniform retrieval (including PIDE markup, completion etc.);
2014-03-14, by wenzelm
more frugal recording of changes: join merely requires information from one side;
2014-03-13, by wenzelm
do not test details of error messages;
2014-03-13, by wenzelm
minor tuning -- NB: props are usually empty for global facts;
2014-03-13, by wenzelm
even smarter Path.smart_implode;
2014-03-13, by wenzelm
added ML antiquotation @{path};
2014-03-13, by wenzelm
clarified Path.smart_implode;
2014-03-13, by wenzelm
generalization of differential_zero_maxmin to class real_normed_vector
2014-03-14, by huffman
delayed construction of command (and of noncommercial check) + tuning
2014-03-14, by blanchet
tuning
2014-03-14, by blanchet
consolidate consecutive steps that prove the same formula
2014-03-14, by blanchet
remove '__' skolem suffixes before showing terms to users
2014-03-14, by blanchet
undo rewrite rules (e.g. for 'fun_app') in Isar
2014-03-14, by blanchet
debugging stuff
2014-03-14, by blanchet
more simplification of trivial steps
2014-03-14, by blanchet
tuning
2014-03-14, by blanchet
tuned wording (pun)
2014-03-14, by blanchet
document the new 'nonexhaustive' option (cf. 52e8f110fec3)
2014-03-14, by blanchet
made SML/NJ happier
2014-03-14, by blanchet
print warning if some constructors are missing;
2014-03-14, by panny
updated Sledgehammer docs w.r.t. 'smt2' and 'z3_new'
2014-03-14, by blanchet
updated documentation w.r.t. 'z3_non_commercial' option in Isabelle/jEdit
2014-03-14, by blanchet
updated NEWS and CONTRIBUTORS (BNF, SMT2, Sledgehammer)
2014-03-14, by blanchet
remove ordered_euclidean_space constraint from brouwer/derivative lemmas;
2014-03-13, by huffman
typos
2014-03-13, by nipkow
merged
2014-03-13, by traytel
tuned tactics
2014-03-13, by traytel
simplified internal codatatype construction
2014-03-13, by traytel
updated SMT2 examples and certificates
2014-03-13, by blanchet
updated SMT2 certificates
2014-03-13, by blanchet
added Z3 4.3.0 as component (for use with 'smt2' method)
2014-03-13, by blanchet
updated SMT example certificates
2014-03-13, by blanchet
added 'smt2_status' to keywords
2014-03-13, by blanchet
avoid name clash
2014-03-13, by blanchet
simplify index handling
2014-03-13, by blanchet
more robust indices
2014-03-13, by blanchet
correctly reconstruct helper facts (e.g. 'nat_int') in Isar proofs
2014-03-13, by blanchet
move lemmas to theory file, towards textual proof reconstruction
2014-03-13, by blanchet
simpler translation of 'div' and 'mod' for Z3
2014-03-13, by blanchet
tuning
2014-03-13, by blanchet
tuning
2014-03-13, by blanchet
thread through step IDs from Z3 to Sledgehammer
2014-03-13, by blanchet
adapted to ML structure renaming
2014-03-13, by blanchet
tuning
2014-03-13, by blanchet
avoid names that may clash with Z3's output (e.g. '')
2014-03-13, by blanchet
do less work in 'filter' mode
2014-03-13, by blanchet
let exception pass through in debug mode
2014-03-13, by blanchet
simplified preplaying information
2014-03-13, by blanchet
renamed (hardly used) 'prod_pred' and 'option_pred' to 'pred_prod' and 'pred_option'
2014-03-13, by blanchet
simplified solution parsing
2014-03-13, by blanchet
adapted to renamed ML files
2014-03-13, by blanchet
renamed ML files
2014-03-13, by blanchet
reintroduced old model reconstruction code -- still needs to be ported
2014-03-13, by blanchet
slacker error code policy for Z3
2014-03-13, by blanchet
repaired 'if' logic
2014-03-13, by blanchet
killed a few 'metis' calls
2014-03-13, by blanchet
honor the fact that the new Z3 can generate Isar proofs
2014-03-13, by blanchet
have Sledgehammer generate Isar proofs from Z3 proofs
2014-03-13, by blanchet
tuned ML interface
2014-03-13, by blanchet
integrate SMT2 with Sledgehammer
2014-03-13, by blanchet
removed tracing output
2014-03-13, by blanchet
use 'smt2' in SMT examples as much as currently possible
2014-03-13, by blanchet
moved 'SMT2' (SMT-LIB-2-based SMT module) into Isabelle
2014-03-13, by blanchet
tuned proofs
2014-03-13, by haftmann
less
more
|
(0)
-30000
-10000
-3000
-1000
-120
+120
+1000
+3000
+10000
tip