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.
remove outdated comment
2011-11-23, by huffman
NEWS;
2011-11-21, by wenzelm
simplified read_instantiate -- no longer need to assign values, since rule attributes are now static;
2011-11-21, by wenzelm
drop vacuous decls;
2011-11-21, by wenzelm
tuned;
2011-11-21, by wenzelm
tuned header;
2011-11-21, by wenzelm
misspelled name
2011-11-21, by kuncar
eliminated obsolete "standard";
2011-11-20, by wenzelm
eliminated obsolete "standard";
2011-11-20, by wenzelm
eliminated obsolete "standard";
2011-11-20, by wenzelm
eliminated obsolete "standard";
2011-11-20, by wenzelm
eliminated obsolete "standard";
2011-11-20, by wenzelm
explicit is better than implicit;
2011-11-20, by wenzelm
eliminated obsolete "standard";
2011-11-20, by wenzelm
tuned signature;
2011-11-20, by wenzelm
'lemmas' / 'theorems' commands allow 'for' fixes and standardize the result before storing;
2011-11-20, by wenzelm
updated comment;
2011-11-20, by wenzelm
more uniform signature;
2011-11-20, by wenzelm
uniform cert_vars/read_vars;
2011-11-20, by wenzelm
eliminated dead code;
2011-11-20, by wenzelm
clarified certify vs. sharing;
2011-11-20, by wenzelm
tuned;
2011-11-20, by wenzelm
NEWS;
2011-11-19, by wenzelm
added ML antiquotation @{attributes};
2011-11-19, by wenzelm
merged
2011-11-19, by wenzelm
made SML/NJ happy
2011-11-19, by blanchet
simplified Locale.add_thmss, after partial evaluation of attributes;
2011-11-19, by wenzelm
misc tuning;
2011-11-19, by wenzelm
tuned;
2011-11-19, by wenzelm
refined partial evaluation of attributes: avoid duplication of facts for plain declarations;
2011-11-19, by wenzelm
discontinued slightly odd write_prv, which would still write .prv files the first time, and deprive add-on tools from date stamp change (cf. 157e74588c49);
2011-11-19, by wenzelm
do not store vacuous theorem specifications -- relevant for frugal local theory content;
2011-11-19, by wenzelm
put structural attributes of 'obtains' in outer declarations, to make it actually work in local theory;
2011-11-19, by wenzelm
sequential lemmas to accomodate static rule attributes;
2011-11-18, by wenzelm
partial evaluation of locale facts leads to static scoping of rule attributes;
2011-11-18, by wenzelm
tuned message;
2011-11-18, by wenzelm
gave SML/NJ a chance
2011-11-18, by blanchet
more robust options
2011-11-18, by blanchet
adding another example for lifting definitions
2011-11-18, by bulwahn
improving header
2011-11-18, by bulwahn
more "metis" calls in example
2011-11-18, by blanchet
be more silent when auto minimizing
2011-11-18, by blanchet
less offensive terminology
2011-11-18, by blanchet
more "metis" calls in example
2011-11-18, by blanchet
minor textual improvement
2011-11-18, by blanchet
pull variables (Var) out of lambdas, so that the Isabelle theorems closely mirror the Metis lambda-lifted ones
2011-11-18, by blanchet
wrap lambdas earlier, to get more control over beta/eta
2011-11-18, by blanchet
move eta-contraction to before translation to Metis, to ensure everything stays in sync
2011-11-18, by blanchet
avoid that var names get changed by resolution in Metis lambda-lifting
2011-11-18, by blanchet
better threading of type encodings between Sledgehammer and "metis"
2011-11-18, by blanchet
fixed bugs in lambda-lifting code -- ensure distinct names for variables
2011-11-18, by blanchet
protect prefix against variant mutations
2011-11-18, by blanchet
example cleanup
2011-11-18, by blanchet
example cleanup
2011-11-18, by blanchet
don't propagate user-set "type_enc" or "lam_trans" to Metis calls
2011-11-18, by blanchet
don't needlessly pass "lam_lifted" option to "metis" call for SMT proof
2011-11-18, by blanchet
avoid spurious messages in "lam_lifting" mode
2011-11-18, by blanchet
eta-contract to avoid needless "lambda" wrappers
2011-11-18, by blanchet
quiet down SMT
2011-11-18, by blanchet
more aggressive lambda hiding (if we anyway need to pass an option to Metis)
2011-11-18, by blanchet
updated Sledgehammer docs
2011-11-18, by blanchet
don't pass "lam_lifted" option to "metis" unless there's a good reason
2011-11-18, by blanchet
no needless reconstructors
2011-11-18, by blanchet
removed more clutter
2011-11-18, by blanchet
removed needless baggage
2011-11-18, by blanchet
Word.thy: reduce usage of numeral-representation-dependent thms like number_of_is_id in proofs
2011-11-18, by huffman
merged
2011-11-18, by huffman
Groups.thy: generalize several lemmas from class ab_group_add to class group_add
2011-11-17, by huffman
HOL-Word: removed more duplicate theorems
2011-11-17, by huffman
HOL-Word: removed many duplicate theorems (see NEWS)
2011-11-17, by huffman
Word.thy: rearrange to instantiate arithmetic classes together with arithmetic operations
2011-11-17, by huffman
move definitions of bitwise operators into appropriate document section
2011-11-17, by huffman
HOL-Word: add simp rules for bin_rest, bin_last; shorten several proofs
2011-11-17, by huffman
HOL-NSA: add number_semiring instance, reformulate several lemmas using '2' instead of '1+1'
2011-11-17, by huffman
simplify implementation of approx_reorient_simproc
2011-11-17, by huffman
name simp theorems st_0 and st_1
2011-11-17, by huffman
remove redundant simp rules plus_enat_0
2011-11-17, by huffman
eliminated slightly odd Rep' with dynamically-scoped [simplified];
2011-11-17, by wenzelm
partial evaluation in invisible context;
2011-11-17, by wenzelm
adding a preliminary example to show how the quotient_definition package can be generalized
2011-11-17, by bulwahn
tuned header
2011-11-17, by bulwahn
adding database of abs and rep terms to the quotient package; registering abs and rep terms in quotient_type and using them in quotient_definition
2011-11-17, by bulwahn
simplify some proofs
2011-11-17, by huffman
Int.thy: remove duplicate lemmas double_less_0_iff and odd_less_0, use {even,odd}_less_0_iff instead
2011-11-17, by huffman
merged
2011-11-17, by huffman
rewrite integer numeral div/mod simprocs to not return conditional rewrites; add regression tests
2011-11-16, by huffman
remove redundant lemmas bin_last_mod and bin_rest_div, use bin_last_def and bin_rest_def instead
2011-11-16, by huffman
simplify proof of word_of_int; remove several now-unused lemmas about Rep_Integ
2011-11-16, by huffman
retain mixed attributes as dynamic theorem expression, but disallow subsequent static rules;
2011-11-16, by wenzelm
clarified Attrib.partial_evaluation;
2011-11-16, by wenzelm
tagging is not stable under morphisms and need to be replayed dynamically (mixed_attribute);
2011-11-16, by wenzelm
compile
2011-11-16, by blanchet
compile
2011-11-16, by blanchet
compile
2011-11-16, by blanchet
give each time slice its own lambda translation
2011-11-16, by blanchet
thread in additional options to minimizer
2011-11-16, by blanchet
make metis reconstruction handling more flexible
2011-11-16, by blanchet
document metis options better
2011-11-16, by blanchet
fixed typo
2011-11-16, by blanchet
document "lam_trans" option
2011-11-16, by blanchet
nicer bullets
2011-11-16, by blanchet
parse lambda translation option in Metis
2011-11-16, by blanchet
rename the lambda translation schemes, so that they are understandable out of context
2011-11-15, by blanchet
rename configuration option to more reasonable length
2011-11-15, by blanchet
continued implementation of lambda-lifting in Metis
2011-11-15, by blanchet
disable debugging output
2011-11-15, by blanchet
use consts, not frees, for lambda-lifting
2011-11-15, by blanchet
started implementing lambda-lifting in Metis
2011-11-15, by blanchet
improved generators for rational numbers to generate negative numbers;
2011-11-15, by bulwahn
tuned
2011-11-15, by bulwahn
remove one more old-style semicolon
2011-11-15, by huffman
Metis_Examples/Big_O.thy: add number_ring class constraints, adapt proofs to use cancellation simprocs
2011-11-15, by huffman
less
more
|
(0)
-30000
-10000
-3000
-1000
-112
+112
+1000
+3000
+10000
+30000
tip