Mercurial
Mercurial
>
repos
>
isabelle
/ graph
summary
|
shortlog
|
changelog
| graph |
tags
|
bookmarks
|
branches
|
files
|
gz
|
help
less
more
|
(0)
-30000
-10000
-3000
-1000
-224
+224
+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
remove old-style semicolons
2011-11-15, by huffman
avoid theorem references like 'semiring_norm(111)'
2011-11-15, by huffman
merged
2011-11-15, by huffman
merged
2011-11-14, by huffman
Parametric_Ferrante_Rackoff.thy: restrict to class number_ring, replace '1+1' with '2' everywhere
2011-11-14, by huffman
avoid numeral-representation-specific rules in metis proof
2011-11-14, by huffman
merged
2011-11-14, by wenzelm
remove sorry, otherwise it breaks the testboard
2011-11-14, by hoelzl
cleaned up float theories; removed duplicate definitions and theorems
2011-11-14, by hoelzl
enforce quick_and_dirty in Code_Real_Approx_By_Float
2011-11-14, by hoelzl
some support for partial evaluation of attributed facts;
2011-11-14, by wenzelm
tuned;
2011-11-14, by wenzelm
eliminated dead code;
2011-11-14, by wenzelm
inner syntax positions for string literals;
2011-11-14, by wenzelm
less confusion subexpression markup;
2011-11-14, by wenzelm
pass positions for named targets, for formal links in the document model;
2011-11-14, by wenzelm
simplified Runtime.exn_messages: always print detailed version of low-level exeptions, which should not occur in regular user errors anyway;
2011-11-14, by wenzelm
more detailed exception_trace: in Poly/ML 5.4.x intermediate handlers reset the trace (cf. Poly/ML SVN 1110);
2011-11-14, by wenzelm
merged
2011-11-14, by bulwahn
setting up exhaustive generators which are used for the smart generators
2011-11-14, by bulwahn
add Code_Real_Approx_By_Float
2011-11-14, by hoelzl
merged
2011-11-14, by huffman
remove lemma float_remove_real_numeral, which duplicated Float.float_number_of
2011-11-13, by huffman
remove unnecessary number-representation-specific rules from metis calls;
2011-11-13, by huffman
avoid confusing selector output
2011-11-13, by blanchet
remove unsound line in Nitpick's "rat" setup
2011-11-13, by blanchet
tuned proofs;
2011-11-12, by wenzelm
merged
2011-11-12, by wenzelm
removed some old-style semicolons
2011-11-12, by huffman
index markup elements for more efficient cumulate/select operations;
2011-11-12, by wenzelm
tuned;
2011-11-12, by wenzelm
tuned markup -- prefer user-perspective;
2011-11-12, by wenzelm
tuned specifications and proofs;
2011-11-12, by wenzelm
more precise type;
2011-11-12, by wenzelm
refined Markup_Tree implementation: stacked markup within each entry;
2011-11-12, by wenzelm
tuned signature;
2011-11-12, by wenzelm
tuned signature;
2011-11-12, by wenzelm
merged
2011-11-11, by wenzelm
merged
2011-11-11, by huffman
abel_cancel.ML: avoid canceling zeros, which would cause the simproc to return a trivial rewrite;
2011-11-11, by huffman
use simproc_setup for the remaining nat_numeral simprocs
2011-11-11, by huffman
use simproc_setup for more nat_numeral simprocs; add simproc tests
2011-11-11, by huffman
using more conventional names for monad plus operations
2011-11-11, by bulwahn
more tooltip content;
2011-11-11, by wenzelm
added markup_cumulate operator;
2011-11-11, by wenzelm
depth-first proof forking for improved locality (wrt. cancellation and overall memory usage);
2011-11-11, by wenzelm
tuned;
2011-11-11, by wenzelm
more abstract Markup_Tree;
2011-11-11, by wenzelm
prefer statically typed Text.Markup;
2011-11-11, by wenzelm
discontinued entity text color, notably historic red for classes;
2011-11-11, by wenzelm
more scalable Proof_Context.prepare_sorts;
2011-11-11, by wenzelm
increasing values_timeout to avoid failures of isatest with HOL-IMP
2011-11-11, by bulwahn
renaming example invocations: tester predicate_compile is renamed to smart_exhaustive
2011-11-11, by bulwahn
adding CPS compilation to predicate compiler;
2011-11-11, by bulwahn
adding option allow_function_inversion to quickcheck options
2011-11-11, by bulwahn
more efficient prepare_sorts -- bypass encoded positions;
2011-11-10, by wenzelm
suppress irrelevant positions;
2011-11-10, by wenzelm
more generous margin;
2011-11-10, by wenzelm
pass term positions into check phase, where resulting types are reported accordingly, and eventually shown as tooltips;
2011-11-10, by wenzelm
tuned signature;
2011-11-10, by wenzelm
discontinued unused Thm.compress (again);
2011-11-10, by wenzelm
renewed prolog-quickcheck
2011-11-10, by bulwahn
adding some test cases for preprocessing and narrowing
2011-11-10, by bulwahn
adding a minimalistic preprocessing rewriting common boolean operators; tuned
2011-11-10, by bulwahn
merged
2011-11-10, by huffman
merged
2011-11-09, by huffman
tune post-processing of simproc-generated rules so they won't produce Numeral0 or Numeral1
2011-11-09, by huffman
use simproc_setup for some nat_numeral simprocs; add simproc tests
2011-11-09, by huffman
add ring_char_0 class constraints to several simprocs (internal proofs of #n ~= 0 fail for type
2011-11-09, by huffman
simultaneous check;
2011-11-10, by wenzelm
avoid separate typ_check phases, integrate into main term_check 0 instead (cf. its Syntax.check_typs in Type_Infer_Context.prepare);
2011-11-09, by wenzelm
clarified singleton_fixate: intersection with supersort is identity, only replace actual type inference parameters;
2011-11-09, by wenzelm
misc tuning and simplification;
2011-11-09, by wenzelm
misc tuning;
2011-11-09, by wenzelm
tuned signature;
2011-11-09, by wenzelm
quickcheck invocations in mutabelle must not catch codegenerator errors internally
2011-11-09, by bulwahn
sort assignment before simultaneous term_check, not isolated parse_term;
2011-11-09, by wenzelm
tuned;
2011-11-09, by wenzelm
avoid inconsistent sort constraints;
2011-11-09, by wenzelm
localized Record.decode_type: use standard Proof_Context.get_sort;
2011-11-09, by wenzelm
tuned signature -- emphasize internal role of these operations;
2011-11-09, by wenzelm
proper configuration option;
2011-11-09, by wenzelm
tuned layout;
2011-11-09, by wenzelm
more precise messages with the tester's name in quickcheck; tuned
2011-11-09, by bulwahn
quickcheck fails with code generator errors only if one tester is invoked
2011-11-09, by bulwahn
removing extra arguments
2011-11-09, by bulwahn
removing deactivated timeout handling; catching compilation errors and only outputing an urgent message to enable parallel sucessful quickcheck compilations and runs to present their result
2011-11-09, by bulwahn
tuned
2011-11-09, by bulwahn
more fragments to export, removed the one from Com
2011-11-09, by kleing
updated functor Named_Thms;
2011-11-08, by wenzelm
disabled Thm.compress (again) -- costs for building tables tend to be higher than potential benefit;
2011-11-08, by wenzelm
entity markup for bound variables;
2011-11-08, by wenzelm
merged
2011-11-08, by wenzelm
made SML/NJ happy
2011-11-08, by boehmes
adding some documentation about the values command to the isar reference
2011-11-08, by bulwahn
adding a minimal documentation about the code_pred command to the isar reference
2011-11-08, by bulwahn
more specific treatment of defines/assumes -- avoid normalizing defs by themselves (NB: locale specifications and Local_Theory.define may lead to arbitrary mixture);
2011-11-08, by wenzelm
clarified Local_Defs.export: avoid costly still_fixed test, return all defs;
2011-11-08, by wenzelm
eliminated obsolete tuning (NB: Thm.eta_conversion/Envir.eta_contract based on Same.operation);
2011-11-08, by wenzelm
tuned;
2011-11-08, by wenzelm
tuned;
2011-11-08, by wenzelm
tweaked comment
2011-11-08, by blanchet
made SML/NJ happy
2011-11-08, by blanchet
merged;
2011-11-08, by wenzelm
added FIXME comment
2011-11-07, by blanchet
avoid infinite recursion in peephole optimizer function -- this had a debilitating effect on rationals and reals
2011-11-07, by blanchet
revived Refute in Mutabelle
2011-11-07, by blanchet
tuned;
2011-11-07, by wenzelm
more scalable zero_var_indexes, depending on canonical order within table;
2011-11-07, by wenzelm
more benchmarks;
2011-11-07, by wenzelm
try different alternatives in discharging extra assumptions when schematic theorems obtained from lambda-lifting can be instantiated in different ways
2011-11-07, by boehmes
replace higher-order matching against schematic theorem with dedicated reconstruction method
2011-11-07, by boehmes
less
more
|
(0)
-30000
-10000
-3000
-1000
-224
+224
+1000
+3000
+10000
+30000
tip