Mercurial
Mercurial
>
repos
>
isabelle
/ graph
summary
|
shortlog
|
changelog
| graph |
tags
|
bookmarks
|
branches
|
files
|
gz
|
help
less
more
|
(0)
-30000
-10000
-3000
-1000
-240
+240
+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.
update Sledgehammer docs
2011-09-07, by blanchet
added new tagged encodings to Metis tests
2011-09-07, by blanchet
also implemented ghost version of the tagged encodings
2011-09-07, by blanchet
added new guards encoding to test
2011-09-07, by blanchet
smarter explicit apply business
2011-09-07, by blanchet
started work on ghost type arg encoding
2011-09-07, by blanchet
stricted type encoding parsing
2011-09-07, by blanchet
more substructural sharing to gain significant compression;
2011-09-08, by wenzelm
XML.cache for partial sharing (strings only);
2011-09-07, by wenzelm
platform-specific look and feel;
2011-09-07, by wenzelm
more README;
2011-09-07, by wenzelm
clarified terminology;
2011-09-07, by wenzelm
no print_state for final proof commands, which return to theory state;
2011-09-07, by wenzelm
NEWS on IsabelleText font;
2011-09-07, by wenzelm
explicit join_syntax ensures command transaction integrity of 'theory';
2011-09-07, by wenzelm
some updates for release;
2011-09-07, by wenzelm
some tuning for release;
2011-09-07, by wenzelm
updated file locations;
2011-09-07, by wenzelm
merged
2011-09-07, by wenzelm
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
misc tuning and simplification of proofs;
2011-09-03, by wenzelm
Document.removed_versions on Scala side;
2011-09-03, by wenzelm
discontinued predefined empty command (obsolete!?);
2011-09-03, by wenzelm
discontinued global execs: store exec value directly within entries;
2011-09-03, by wenzelm
Document.remove_versions on ML side;
2011-09-03, by wenzelm
some support to prune_history;
2011-09-03, by wenzelm
merged
2011-09-02, by huffman
speed up extremely slow metis proof of Sup_real_iff
2011-09-02, by huffman
remove redundant lemma reals_complete2 in favor of complete_real
2011-09-02, by huffman
simplify proof of Rats_dense_in_real;
2011-09-02, by huffman
remove unused, unnecessary lemmas
2011-09-02, by huffman
remove more duplicate lemmas
2011-09-02, by huffman
merged
2011-09-02, by wenzelm
merged
2011-09-02, by haftmann
avoid "Code" as structure name
2011-09-02, by haftmann
more robust chunk painting wrt. hard tabs, when chunk.str == null;
2011-09-02, by wenzelm
raw message function "assign_execs" avoids full overhead of decoding and caching message body;
2011-09-02, by wenzelm
less agressive parsing of commands (priority ~1);
2011-09-02, by wenzelm
tuned;
2011-09-02, by wenzelm
more direct Token.range_pos and Outer_Syntax.read_command, bypassing Thy_Syntax.span;
2011-09-02, by wenzelm
merged
2011-09-02, by nipkow
Added Abstract Interpretation theories
2011-09-02, by nipkow
tuned proofs;
2011-09-02, by wenzelm
proper config option linarith_trace;
2011-09-02, by wenzelm
discontinued slightly odd "Defining record ..." message and corresponding quiet_mode;
2011-09-02, by wenzelm
merged
2011-09-02, by wenzelm
renamed "Metis_Tactics" to "Metis_Tactic", now that there is only one Metis tactic ("metisFT" is legacy)
2011-09-02, by blanchet
use new syntax for Pi binder in TFF1 output
2011-09-02, by blanchet
fewer TPTP important messages
2011-09-02, by blanchet
simplify some proofs about uniform continuity, and add some new ones;
2011-09-01, by huffman
modernize lemmas about 'continuous' and 'continuous_on';
2011-09-01, by huffman
add lemma tendsto_infnorm
2011-09-01, by huffman
more precise iterate_entries_after if start refers to last entry;
2011-09-02, by wenzelm
clarified define_command: store name as structural information;
2011-09-02, by wenzelm
amended last_common, if that happens to the very last entry (important to load HOL/Auth, for example);
2011-09-01, by wenzelm
more redable Document.Node.toString;
2011-09-01, by wenzelm
sort wrt. theory name;
2011-09-01, by wenzelm
modernized theory name;
2011-09-01, by wenzelm
repaired benchmarks;
2011-09-01, by wenzelm
merged
2011-09-01, by wenzelm
tuning
2011-09-01, by blanchet
always measure time for ATPs -- auto minimization relies on it
2011-09-01, by blanchet
added two lemmas about "distinct" to help Sledgehammer
2011-09-01, by blanchet
make "sound" sound and "unsound" more sound, based on evaluation
2011-09-01, by blanchet
HOL/Import: observe distinction between sets and predicates (where possible)
2011-09-01, by Cezary Kaliszyk
simplify/generalize some proofs
2011-08-31, by huffman
generalize lemma isCont_vec_nth
2011-08-31, by huffman
convert proof to Isar-style
2011-08-31, by huffman
remove redundant lemma card_enum
2011-08-31, by huffman
move lemmas from Topology_Euclidean_Space to Euclidean_Space
2011-08-31, by huffman
convert to Isar-style proof
2011-08-31, by huffman
make SML/NJ happy
2011-08-31, by blanchet
more tuning
2011-08-31, by blanchet
more tuning
2011-08-31, by blanchet
tuning
2011-08-31, by blanchet
avoid relying on dubious TFF1 feature
2011-08-31, by blanchet
killed FIXME (the ATP exporter outputs TPTP FOF, which is first-order)
2011-08-31, by blanchet
fixed explicit declaration of TFF1 types
2011-08-31, by blanchet
adding list_size_append (thanks to Rene Thiemann)
2011-08-30, by bulwahn
strengthening list_size_pointwise (thanks to Rene Thiemann)
2011-08-30, by bulwahn
more flexible sorting;
2011-09-01, by wenzelm
tuned signature;
2011-09-01, by wenzelm
more abstract Document.Node.Name;
2011-09-01, by wenzelm
more careful treatment of interrupts, to retain them within forked/joined boundary of command transactions;
2011-09-01, by wenzelm
crude display of node status;
2011-08-31, by wenzelm
explicit cancel_execution before queueing new edits -- potential performance improvement for machines with few cores;
2011-08-31, by wenzelm
explicit running_color;
2011-08-31, by wenzelm
tuned join_commands: avoid traversing cumulative table;
2011-08-31, by wenzelm
some support for theory status overview;
2011-08-31, by wenzelm
tuned Commands_Changed: cover nodes as well;
2011-08-31, by wenzelm
maintain name of *the* enclosing node as part of command -- avoid full document traversal;
2011-08-31, by wenzelm
improved auto loading: selectable file list;
2011-08-31, by wenzelm
tuned document;
2011-08-30, by wenzelm
tuned import;
2011-08-30, by wenzelm
tuned document;
2011-08-30, by wenzelm
tuned color for Mac OS X (very light color profile?);
2011-08-30, by wenzelm
tuned document;
2011-08-30, by wenzelm
merged;
2011-08-30, by wenzelm
fixed just introduced silly bug
2011-08-30, by blanchet
"simple" was renamed "mono_simple" and there's now "poly_simple" as well -- but they are not needed here since for Metis they amount to the same as guards
2011-08-30, by blanchet
tuning
2011-08-30, by blanchet
cleaner "pff" dummy TFF0 prover
2011-08-30, by blanchet
generate properly typed TFF1 (PFF) problems in the presence of type class predicates
2011-08-30, by blanchet
added type abstractions (for declaring polymorphic constants) to TFF syntax
2011-08-30, by blanchet
implement more of the polymorphic simply typed format TFF(1)
2011-08-30, by blanchet
flip logic of boolean option so it's off by default
2011-08-30, by blanchet
extended simple types with polymorphism -- the implementation still needs some work though
2011-08-30, by blanchet
added dummy PFF prover, for debugging purposes
2011-08-30, by blanchet
first step towards polymorphic TFF + changed defaults for Vampire
2011-08-30, by blanchet
tuning
2011-08-30, by blanchet
removed explicit reliance on Hilbert_Choice.Eps
2011-08-30, by nik
improved handling of induction rules in Sledgehammer
2011-08-30, by nik
added generation of induction rules
2011-08-30, by nik
simplify some proofs
2011-08-29, by huffman
restrict perspective to actual buffer_range, to avoid spurious edits due to faulty last_exec_offset (NB: jEdit screenlines may be silently extended by trailing newline);
2011-08-30, by wenzelm
tuned signature;
2011-08-30, by wenzelm
dynamic exec state lookup for implicit position information (e.g. 'definition' without binding);
2011-08-30, by wenzelm
some support for hyperlinks between different buffers;
2011-08-30, by wenzelm
tuned colors -- more distance between outdated_color and quoted_color;
2011-08-30, by wenzelm
do not normalized extra file dependencies for now -- still loaded by prover process;
2011-08-30, by wenzelm
separate module for jEdit primitives for loading theory files;
2011-08-30, by wenzelm
less
more
|
(0)
-30000
-10000
-3000
-1000
-240
+240
+1000
+3000
+10000
+30000
tip