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
+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.
merged
2011-09-07, by bulwahn
removing previously used function locally_monomorphic in the code generator
2011-09-07, by bulwahn
setting const_sorts to false in the type inference of the code generator
2011-09-07, by bulwahn
adapting Imperative HOL serializer to changes of the iterm datatype in the code generator
2011-09-07, by bulwahn
removing previous crude approximation to add type annotations to disambiguate types
2011-09-07, by bulwahn
adding minimalistic implementation for printing the type annotations
2011-09-07, by bulwahn
adding call to disambiguation annotations
2011-09-07, by bulwahn
adding type inference for disambiguation annotations in code equation
2011-09-07, by bulwahn
adding the body type as well to the code generation for constants as it is required for type annotations of constants
2011-09-07, by bulwahn
changing const type to pass along if typing annotations are necessary for disambigous terms
2011-09-07, by bulwahn
fixed THF type constructor syntax
2011-09-07, by blanchet
tweaking polymorphic TFF and THF output
2011-09-07, by blanchet
parse new experimental '@' encodings
2011-09-07, by blanchet
tuning
2011-09-07, by blanchet
tuning
2011-09-07, by blanchet
tuning
2011-09-07, by blanchet
clarified import;
2011-09-07, by wenzelm
tuned/simplified proofs;
2011-09-07, by wenzelm
tuned proofs;
2011-09-07, by wenzelm
deactivate unfinished charset provider for now, to avoid user confusion;
2011-09-07, by wenzelm
more NEWS;
2011-09-07, by wenzelm
added "check" button: adhoc change to full buffer perspective;
2011-09-07, by wenzelm
added "cancel" button based on cancel_execution, not interrupt (cf. 156be0e43336);
2011-09-07, by wenzelm
separate mangling, which can (and should) be done before the formulas are first-orderized, and type arg filtering, which must be done after once the min arities have been computed
2011-09-07, by blanchet
perform mangling before computing symbol arity, to avoid needless "hAPP"s and "hBOOL"s
2011-09-07, by blanchet
tuning
2011-09-07, by blanchet
make mangling sound w.r.t. type arguments
2011-09-07, by blanchet
make "filter_type_args" more robust if the actual arity is higher than the declared one
2011-09-07, by blanchet
updated Sledgehammer documentation
2011-09-07, by blanchet
rationalize uniform encodings
2011-09-07, by blanchet
merged
2011-09-06, by huffman
avoid using legacy theorem names
2011-09-06, by huffman
merged
2011-09-06, by huffman
remove redundant lemmas i_mult_eq and i_mult_eq2 in favor of i_squared
2011-09-06, by huffman
HOL/Import: Update HOL4 generated files to current Isabelle.
2011-09-07, by Cezary Kaliszyk
tuned proofs;
2011-09-07, by wenzelm
remove some unnecessary simp rules from simpset
2011-09-06, by huffman
some Isabelle/jEdit NEWS;
2011-09-06, by wenzelm
more README;
2011-09-06, by wenzelm
merged
2011-09-06, by wenzelm
merged
2011-09-06, by huffman
simplify proof of tan_half, removing unused assumptions
2011-09-06, by huffman
convert some proofs to Isar-style
2011-09-06, by huffman
added dummy polymorphic THF system
2011-09-06, by blanchet
added some examples for pattern and weight annotations
2011-09-06, by boehmes
merged
2011-09-06, by bulwahn
avoid "Code" as structure name (cf. 3bc39cfe27fe)
2011-09-06, by bulwahn
remove duplicate copy of lemma sqrt_add_le_add_sqrt
2011-09-06, by huffman
remove redundant lemma real_sum_squared_expand in favor of power2_sum
2011-09-06, by huffman
remove redundant lemma LIMSEQ_Complex in favor of tendsto_Complex
2011-09-06, by huffman
merged
2011-09-06, by huffman
add lemmas about arctan;
2011-09-05, by huffman
convert lemma cos_total to Isar-style proof
2011-09-05, by huffman
added new lemmas
2011-09-06, by nipkow
updated Sledgehammer's docs
2011-09-06, by blanchet
cleanup "simple" type encodings
2011-09-06, by blanchet
merge
2011-09-06, by Cezary Kaliszyk
HOL/Import: Make HOL4 Import work with current Isabelle. Updated constant maps, added bool type map, and tuned compat theorem.
2011-09-06, by Cezary Kaliszyk
tuning
2011-09-06, by blanchet
drop more type arguments soundly, when they can be deduced from the arg types
2011-09-06, by blanchet
bulk reports for improved message throughput;
2011-09-06, by wenzelm
bulk reports for improved message throughput;
2011-09-06, by wenzelm
tuned signature;
2011-09-06, by wenzelm
more specific message channels to avoid potential bottle-neck of raw_messages;
2011-09-06, by wenzelm
buffer prover messages to prevent overloading of session_actor input channel -- which is critical due to synchronous messages wrt. GUI thread;
2011-09-06, by wenzelm
more abstract receiver interface;
2011-09-06, by wenzelm
flush after Output.raw_message (and init message) for reduced latency of important protocol events;
2011-09-06, by wenzelm
convert lemma cos_is_zero to Isar-style
2011-09-05, by huffman
merged
2011-09-05, by huffman
convert lemma sin_gt_zero to Isar style;
2011-09-05, by huffman
modify lemma sums_group, and shorten proofs that use it
2011-09-05, by huffman
generalize some lemmas
2011-09-05, by huffman
add lemmas cos_arctan and sin_arctan
2011-09-05, by huffman
tuned indentation
2011-09-05, by huffman
more visible outdated_color;
2011-09-05, by wenzelm
commands_change_delay within main actor -- prevents overloading of commands_change_buffer input channel;
2011-09-05, by wenzelm
tuned imports;
2011-09-05, by wenzelm
fixed handling of "sledgehammer_params", so that "sledgehammer_params [e]" is really the same as "sledgehammer_params [provers = e]"
2011-09-05, by blanchet
tuned
2011-09-05, by boehmes
tuned
2011-09-05, by boehmes
filter out all schematic theorems if the problem contains no ground constants
2011-09-05, by boehmes
merged
2011-09-04, by huffman
tuned comments
2011-09-04, by huffman
simplify proof of Bseq_mono_convergent
2011-09-04, by huffman
merged
2011-09-04, by wenzelm
replace lemma expi_imaginary with reoriented lemma cis_conv_exp
2011-09-04, by huffman
remove redundant lemmas expi_add and expi_zero
2011-09-04, by huffman
remove redundant lemmas about LIMSEQ
2011-09-04, by huffman
introduce abbreviation 'int' earlier in Int.thy
2011-09-04, by huffman
remove unused assumptions from natceiling lemmas
2011-09-04, by huffman
move lemmas nat_le_iff and nat_mono into Int.thy
2011-09-04, by huffman
eliminated markup for plain identifiers (frequent but insignificant);
2011-09-04, by wenzelm
simplified signatures;
2011-09-04, by wenzelm
synchronous XML.Cache without actor -- potentially more efficient on machines with few cores;
2011-09-04, by wenzelm
tuned document;
2011-09-04, by wenzelm
improved handling of extended styles and hard tabs when prover is inactive;
2011-09-04, by wenzelm
mark hard tabs as single chunks, as required by jEdit;
2011-09-04, by wenzelm
updated READMEs;
2011-09-04, by wenzelm
property "tooltip-dismiss-delay" is edited in ms, not seconds;
2011-09-04, by wenzelm
moved XML/YXML to src/Pure/PIDE;
2011-09-04, by wenzelm
pass raw messages through xml_cache actor, which is important to retain ordering of results (e.g. read_command reports before assign, cf. 383c9d758a56);
2011-09-04, by wenzelm
pseudo-definition for perms on sets; tuned
2011-09-04, by haftmann
remove duplicate lemma nat_zero in favor of nat_0
2011-09-03, by huffman
merged
2011-09-03, by huffman
merged
2011-09-03, by huffman
modify nominal packages to better respect set/pred distinction
2011-09-03, by huffman
merged
2011-09-03, by huffman
remove unused assumption from lemma posreal_complete
2011-09-03, by huffman
tuned specifications
2011-09-03, by haftmann
merged
2011-09-03, by haftmann
tuned proof
2011-09-03, by haftmann
merged
2011-09-03, by haftmann
assert Pure equations for theorem references; avoid dynamic reference to fact
2011-09-03, by haftmann
assert Pure equations for theorem references; tuned
2011-09-03, by haftmann
tuned specifications and proofs
2011-09-03, by haftmann
merged
2011-09-03, by wenzelm
remove duplicate lemma finite_choice in favor of finite_set_choice
2011-09-03, by huffman
simplify proof
2011-09-03, by huffman
shorten some proofs
2011-09-03, by huffman
remove redundant simp rules ceiling_floor and floor_ceiling
2011-09-02, by huffman
less
more
|
(0)
-30000
-10000
-3000
-1000
-120
+120
+1000
+3000
+10000
+30000
tip