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
2012-04-12, by krauss
distributivity of * over Un and UNION
2012-04-12, by krauss
Set_Algebras: removed syntax \<oplus> and \<otimes>, in favour of plain + and *
2012-04-12, by krauss
removed "setsum_set", now subsumed by generic setsum
2012-04-12, by krauss
backported Set_Algebras to use type classes (basically reverting b3e8d5ec721d from 2008)
2012-04-12, by krauss
tuned README;
2012-04-12, by wenzelm
direct scala toplevel tools to ISABELLE_JDK_HOME;
2012-04-12, by wenzelm
simplified component structure;
2012-04-12, by wenzelm
merged
2012-04-12, by wenzelm
merged
2012-04-12, by Andreas Lochbihler
generalise case certificates to allow ignored parameters
2012-04-12, by Andreas Lochbihler
merged
2012-04-12, by bulwahn
manual merge
2012-04-04, by griff
dropped abbreviation "pred_comp"; introduced infix notation "P OO Q" for "relcompp P Q"
2012-04-03, by griff
renamed "rel_comp" to "relcomp" (to be consistent with, e.g., "relpow")
2012-04-03, by griff
more standard method setup;
2012-04-12, by wenzelm
more precise declaration of goal_tfrees in forked proof state;
2012-04-12, by wenzelm
partial revert of 8a179a0493e3 -- expose failure status of result (potentially via group) instead of isolated interrupt;
2012-04-12, by wenzelm
multiset operations are defined with lift_definitions;
2012-04-12, by bulwahn
remove outdated comment
2012-04-12, by huffman
rule composition via attribute "OF" (or ML functions OF/MRS) is more tolerant against multiple unifiers;
2012-04-11, by wenzelm
standardized ML aliases;
2012-04-11, by wenzelm
clarified proof_result: finish proof formally via head tr, not end_tr;
2012-04-11, by wenzelm
tuned;
2012-04-11, by wenzelm
more robust Future.fulfill wrt. duplicate assignment and interrupt;
2012-04-11, by wenzelm
tuned message;
2012-04-11, by wenzelm
always signal after cancel_group: passive tasks may have become active;
2012-04-11, by wenzelm
just one dedicated execution per document version -- NB: non-monotonicity of cancel always requires fresh update;
2012-04-11, by wenzelm
merged
2012-04-10, by wenzelm
moved lift_raw_const wrapper out of the Quotient-package into Nominal2
2012-04-10, by Christian Urban
misc tuning and simplification;
2012-04-10, by wenzelm
static relevance of proof via syntax keywords;
2012-04-10, by wenzelm
tuned future priorities: print 0, goal ~1, execute ~2;
2012-04-10, by wenzelm
updated for Poly/ML SVN 1476;
2012-04-10, by wenzelm
some coverage of HOL/TPTP;
2012-04-10, by wenzelm
added graph-conversion utility for TPTP files
2012-04-10, by sultana
moved non-interpret-specific code to different module
2012-04-10, by sultana
disable parallel proofs (again) -- still suffering from instabilites wrt. interrupts;
2012-04-09, by wenzelm
tuned proofs;
2012-04-09, by wenzelm
slightly faster default compilation of Isabelle/Scala;
2012-04-09, by wenzelm
more explicit last exec result;
2012-04-09, by wenzelm
dynamic propagation of node "updated" status, which is required to propagate edits and re-assigments and allow direct memo_result;
2012-04-09, by wenzelm
tuned;
2012-04-09, by wenzelm
simplified Future.cancel/cancel_group (again) -- running threads only;
2012-04-09, by wenzelm
added ML pretty-printing;
2012-04-09, by wenzelm
merged
2012-04-07, by wenzelm
merged
2012-04-07, by wenzelm
explicit constructor Nat leaves nat_of as conversion
2012-04-07, by haftmann
abandoned almost redundant *_foldr lemmas
2012-04-06, by haftmann
tuned
2012-04-06, by haftmann
no preference wrt. fold(l/r); prefer fold rather than foldr for iterating over lists in generated code
2012-04-06, by haftmann
enable parallel proofs (cf. e8552cba702d), only affects packages so far;
2012-04-07, by wenzelm
added static command status markup, to emphasize accepted but unassigned/unparsed commands (notably in overview panel);
2012-04-07, by wenzelm
tuned proofs;
2012-04-07, by wenzelm
more robust update_perspective, e.g. required after reload of buffer that is not at start position;
2012-04-07, by wenzelm
tuned imports;
2012-04-07, by wenzelm
updated header keywords;
2012-04-07, by wenzelm
init message not bad;
2012-04-07, by wenzelm
explicit checks stable_finished_theory/stable_command allow parallel asynchronous command transactions;
2012-04-07, by wenzelm
discontinued obsolete last_execs (cf. cd3ab7625519);
2012-04-06, by wenzelm
remove now-unnecessary type annotations from lift_definition commands
2012-04-06, by huffman
more robust generation of quotient rules using tactics
2012-04-06, by huffman
merged
2012-04-06, by huffman
add function dest_Quotient
2012-04-06, by huffman
standardized alias;
2012-04-06, by wenzelm
fixed document;
2012-04-06, by wenzelm
merged
2012-04-06, by wenzelm
correct plumbing of proof contexts, so that force_rty_type won't generalize more type variables than it should
2012-04-06, by huffman
detect incorrect situations; better error messages; sanity check for quot_thm in setup_lifting_infr
2012-04-05, by kuncar
make Quotient_Def.lift_raw_const working again
2012-04-05, by kuncar
use standard quotient lemmas to generate transfer rules
2012-04-05, by huffman
add transfer lemmas for quotients
2012-04-05, by huffman
define reflp directly, in the manner of symp and transp
2012-04-05, by huffman
set up and use lift_definition for word operations
2012-04-05, by huffman
lift_definition declares transfer_rule attribute
2012-04-05, by huffman
configure transfer method for 'a word -> int
2012-04-05, by huffman
added timestamps to logging of named thms
2012-04-05, by krauss
merged
2012-04-05, by huffman
merged
2012-04-04, by huffman
add lemmas for generating transfer rules for typedefs
2012-04-04, by huffman
tuned;
2012-04-05, by sultana
improved import_tptp to use standard TPTP directory structure; extended the TPTP testing theory to include an example of using the import_tptp command;
2012-04-04, by sultana
merge
2012-04-04, by Cezary Kaliszyk
HOL/Import more precise map types
2012-04-04, by Cezary Kaliszyk
HOL/Import typed matches against Isabelle typedef result
2012-04-04, by Cezary Kaliszyk
connect the Quotient package to the Lifting package
2012-04-04, by kuncar
support non-open typedefs; define cr_rel in terms of a rep function for typedefs
2012-04-04, by kuncar
tuned;
2012-04-04, by sultana
added interpretation for formula conditional;
2012-04-04, by sultana
refactored tptp lex;
2012-04-04, by sultana
refactored tptp yacc to bring close to official spec;
2012-04-04, by sultana
transfer method generalizes over free variables in goal
2012-04-04, by huffman
add bounded quantifier constant transfer_bforall, whose definition is unfolded after transfer
2012-04-04, by huffman
update keywords file
2012-04-04, by huffman
merged
2012-04-04, by huffman
fix typos
2012-04-04, by huffman
lift_definition command generates transfer rule
2012-04-04, by huffman
prove_quot_theorem fixes types
2012-04-04, by huffman
documenting options quickcheck_locale; adjusting IsarRef documentation of Quotient predicate; NEWS
2012-04-04, by bulwahn
added option quickcheck_locale to allow different behaviours for handling locales in Quickcheck;
2012-04-04, by bulwahn
stop node execution at first unassigned exec;
2012-04-06, by wenzelm
discontinued Document.update_perspective side-entry (cf. 546adfa8a6fc) -- NB: re-assignment is always necessary due to non-monotonic cancel_execution;
2012-04-06, by wenzelm
more scalable execute/update: avoid redundant traversal of invisible/finished nodes;
2012-04-05, by wenzelm
less ambitious memo_eval, since memo_result is still not robust here;
2012-04-05, by wenzelm
less aggressive discontinue_execution before document update, to avoid unstable execs that need to be re-assigned;
2012-04-05, by wenzelm
more explicit memo_eval vs. memo_result, to enforce bottom-up execution;
2012-04-05, by wenzelm
Command.memo including physical interrupts (unlike Lazy.lazy);
2012-04-05, by wenzelm
tuned;
2012-04-05, by wenzelm
tuned -- NB: get_theory still needs to apply Lazy.force due to interrupt instabilities;
2012-04-04, by wenzelm
proper signature constraint;
2012-04-04, by wenzelm
tuned comments;
2012-04-04, by wenzelm
separate module for prover command execution;
2012-04-04, by wenzelm
tuned;
2012-04-04, by wenzelm
fix typo in ML structure name
2012-04-04, by huffman
removed obsolete isar-overview manual;
2012-04-04, by wenzelm
dealing with SMLNJ errors 'value type in structure doesn't match signature spec' (which originated from lack of type generalisation) and 'unresolved flex record' wrt tptp_interpret
2012-04-04, by sultana
merged
2012-04-04, by bulwahn
rudimentary handling of products in finitize_functions in Quickcheck-Narrowing
2012-04-04, by bulwahn
improved equality check for modes in predicate compiler
2012-04-04, by bulwahn
rename ML structure to avoid shadowing earlier name
2012-04-04, by huffman
less
more
|
(0)
-30000
-10000
-3000
-1000
-120
+120
+1000
+3000
+10000
+30000
tip