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
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.
repaired 'if' logic
2014-03-13, by blanchet
killed a few 'metis' calls
2014-03-13, by blanchet
honor the fact that the new Z3 can generate Isar proofs
2014-03-13, by blanchet
have Sledgehammer generate Isar proofs from Z3 proofs
2014-03-13, by blanchet
tuned ML interface
2014-03-13, by blanchet
integrate SMT2 with Sledgehammer
2014-03-13, by blanchet
removed tracing output
2014-03-13, by blanchet
use 'smt2' in SMT examples as much as currently possible
2014-03-13, by blanchet
moved 'SMT2' (SMT-LIB-2-based SMT module) into Isabelle
2014-03-13, by blanchet
tuned proofs
2014-03-13, by haftmann
dropped redundant theorems
2014-03-13, by haftmann
tuned
2014-03-13, by haftmann
monotonicity in complete lattices
2014-03-13, by haftmann
enhanced simplifier solver for preconditions of rewrite rule, can now deal with conjunctions
2014-03-13, by nipkow
tuned signature -- clarified module name;
2014-03-12, by wenzelm
added ML antiquotation @{here};
2014-03-12, by wenzelm
ML_Context.check_antiquotation still required;
2014-03-12, by wenzelm
simplified programming interface to define ML antiquotations -- NB: the transformed context ignores updates of the context parser;
2014-03-12, by wenzelm
proper base comparison;
2014-03-12, by wenzelm
tuned;
2014-03-12, by wenzelm
tuned proofs;
2014-03-12, by wenzelm
more explicit markup and explanation of the improper status of 'back', following the AFP style-guide;
2014-03-12, by wenzelm
clarified Markup.operator vs. Markup.delimiter;
2014-03-12, by wenzelm
more explicit markup for Token.Literal;
2014-03-12, by wenzelm
tuned signature;
2014-03-12, by wenzelm
modernized setup;
2014-03-12, by wenzelm
tuned;
2014-03-12, by wenzelm
some document antiquotations for Isabelle/jEdit elements;
2014-03-12, by wenzelm
merged
2014-03-12, by wenzelm
more explicit Sign.change_check -- detect structural mistakes where they emerge, not at later theory merges;
2014-03-12, by wenzelm
more efficient local theory operations, by imposing a linear change discipline on the main types/consts tables, in order to speed-up Proof_Context.transfer_syntax required for Local_Theory.raw_theory_result;
2014-03-11, by wenzelm
slightly more rubust (and opportunistic) exit for old-fashioned theory_to_proof, which is used by global 'sublocale' with Named_Target.init but without proper exit;
2014-03-11, by wenzelm
more standard internal data integrity;
2014-03-11, by wenzelm
tables with changes relative to some common base version -- support for efficient join/merge of big global tables with small local updates;
2014-03-11, by wenzelm
tuned signature;
2014-03-11, by wenzelm
tuned comment;
2014-03-11, by wenzelm
minor performance tuning via fast matching filter;
2014-03-11, by wenzelm
added missing theorems to unfolding set
2014-03-11, by blanchet
moved 'Quickcheck_Narrowing' further down the theory graph
2014-03-11, by blanchet
make it possible to load Quickcheck exhaustive & narrowing in parallel
2014-03-11, by blanchet
full path
2014-03-11, by blanchet
measurable_lfp/gfp: indirection not necessary
2014-03-11, by hoelzl
merged
2014-03-10, by wenzelm
tuned proofs;
2014-03-10, by wenzelm
proper Char comparison, despite weakly-typed Scala (cf. 5ff5208de089);
2014-03-10, by wenzelm
tuned message;
2014-03-10, by wenzelm
tuned message;
2014-03-10, by wenzelm
include long identifiers in the reckoning of words (e.g. "integer.lifting" vs. 'lifting_update');
2014-03-10, by wenzelm
tuned messages -- in accordance to Isabelle/Scala;
2014-03-10, by wenzelm
tuned;
2014-03-10, by wenzelm
enabled test in PIDE interaction;
2014-03-10, by wenzelm
proper Args.syntax for slightly odd bundle trickery;
2014-03-10, by wenzelm
some Markup.language_path to prevent completion of symbols (notably "~") -- always "delimited" for simplicity in contrast to 42ac3cfb89f6;
2014-03-10, by wenzelm
more markup;
2014-03-10, by wenzelm
clarified Args.check_src: retain name space information for error output;
2014-03-10, by wenzelm
tuned;
2014-03-10, by wenzelm
modernized data managed via Name_Space.table;
2014-03-10, by wenzelm
clarified Args.src: more abstract type, position refers to name only;
2014-03-10, by wenzelm
tuned signature;
2014-03-10, by wenzelm
prefer Name_Space.pretty with its builtin markup;
2014-03-10, by wenzelm
tuned signature -- prefer Name_Space.get with its builtin error;
2014-03-10, by wenzelm
abstract type Name_Space.table;
2014-03-10, by wenzelm
more structured order;
2014-03-10, by wenzelm
more direct Long_Name.qualification;
2014-03-10, by wenzelm
more restrictive completion: intern/extern stability;
2014-03-10, by wenzelm
add measurability rule for (co)inductive predicates
2014-03-10, by hoelzl
introduced antimono; incseq, decseq are now abbreviations for mono and antimono; renamed Library/Continuity to Library/Order_Continuity; removed up_cont; renamed down_cont to down_continuity and generalized to complete_lattices
2014-03-10, by hoelzl
hide implementation details
2014-03-10, by kuncar
copy-paste typo
2014-03-10, by traytel
tuned tactic
2014-03-10, by traytel
unfold intermediate definitions after sealing the bnf
2014-03-10, by traytel
bootstrap fundamental Fun theory immediately after Set theory, without dependency on complete lattices
2014-03-09, by haftmann
tuned;
2014-03-09, by haftmann
more careful unfolding of internal constants
2014-03-09, by traytel
made typedef for the type of the bound optional (size-based)
2014-03-09, by traytel
made natLe{q,ss} constants (yields smaller terms in composition)
2014-03-07, by traytel
removed junk
2014-03-07, by traytel
tuned proofs;
2014-03-09, by wenzelm
unused;
2014-03-09, by wenzelm
tuned;
2014-03-09, by wenzelm
more formal read_root;
2014-03-09, by wenzelm
simplified / modernized hide commands: proper outer parsers and PIDE markup via check;
2014-03-09, by wenzelm
removed dead code;
2014-03-09, by wenzelm
check fact names with PIDE markup;
2014-03-09, by wenzelm
tuned signature;
2014-03-09, by wenzelm
do allow replacement of words where this is appropriate, notably symbol abbrevs and keyword templates (see also 1c42ebdb3a58);
2014-03-09, by wenzelm
tuned proofs;
2014-03-08, by wenzelm
tuned proofs;
2014-03-08, by wenzelm
keep current context visibility for PIDE markup and completion (in contrast to 8e3e004f1c31): Attrib.check_src of 9dc5ce83202c should intern/report attributes once, which happens for local_theory in the (visible) auxiliary context;
2014-03-08, by wenzelm
modernized Attrib.check_name/check_src similar to methods (see also a989bdaf8121);
2014-03-08, by wenzelm
allow suffix of underscores for words (notably keywords), similar to semantic completion;
2014-03-08, by wenzelm
back to polyml-svn, with more threads to avoid problems with HOL-Proofs (see f376f18fd0b7);
2014-03-08, by wenzelm
no completion for complete keywords, to avoid confusion of 'assume' ~> 'assumes' etc.;
2014-03-08, by wenzelm
clarified description;
2014-03-08, by wenzelm
tuned;
2014-03-08, by wenzelm
tuned proofs;
2014-03-07, by wenzelm
more antiquotations;
2014-03-07, by wenzelm
ignore special names that are treated differently for various sub-languages (main wild-card is identifier "__");
2014-03-07, by wenzelm
merged
2014-03-07, by wenzelm
misc tuning;
2014-03-07, by wenzelm
more strict discrimination: symbols vs. keywords could overlap;
2014-03-07, by wenzelm
tuned;
2014-03-07, by wenzelm
more accurate description;
2014-03-07, by wenzelm
misc tuning and clarification;
2014-03-07, by wenzelm
more accurate description;
2014-03-07, by wenzelm
tuned proofs;
2014-03-07, by wenzelm
tuned;
2014-03-07, by wenzelm
tuned message: reveal ambiguity where Syntax_Phases.decode_term fails and thus reduces proper_results beforehand, e.g. term "f(x := y)" in ~~/src/HOL/Hoare/Hoare_Logic.thy;
2014-03-07, by wenzelm
tuned description and its rendering;
2014-03-07, by wenzelm
more detailed description of completion items;
2014-03-07, by wenzelm
more basic const report (without completion) for known Const within syntax tree, which usually refers to special syntax (without proper @{const_syntax} markers);
2014-03-07, by wenzelm
no completion of concealed names;
2014-03-07, by wenzelm
more official const syntax: avoid educated guessing by Syntax_Phases.decode_term;
2014-03-07, by wenzelm
tuned whitespace;
2014-03-07, by wenzelm
removed dead code;
2014-03-07, by wenzelm
modernized theory setup;
2014-03-07, by wenzelm
Some new proofs. Tidying up, esp to remove "apply rule".
2014-03-07, by paulson
use balanced tuples in 'primcorec'
2014-03-07, by blanchet
tuning
2014-03-07, by blanchet
a few new lemmas
2014-03-07, by paulson
balance tuples that represent curried functions
2014-03-07, by blanchet
merged
2014-03-06, by wenzelm
tuned proofs;
2014-03-06, by wenzelm
some NEWS;
2014-03-06, by wenzelm
special identifier "__" (i.e. empty name with internal suffix) serves as wild-card for completion;
2014-03-06, by wenzelm
completion is part of error (not report) and thus not subject to context visibility -- e.g. relevant for 'fixes' in long statements;
2014-03-06, by wenzelm
proper position for decode_pos, which is relevant for completion;
2014-03-06, by wenzelm
more decisive commitment to get_free vs. the_const;
2014-03-06, by wenzelm
more rigid const demands, based on educated guesses about the tools involved here;
2014-03-06, by wenzelm
more compact Markup.markup_report: message body may consist of multiple elements;
2014-03-06, by wenzelm
reject internal term names outright, and complete consts instead;
2014-03-06, by wenzelm
eliminated odd type constraint for read_const (see also 79c1d2bbe5a9);
2014-03-06, by wenzelm
more uniform check_const/read_const;
2014-03-06, by wenzelm
tuned;
2014-03-06, by wenzelm
more rigid type_name demands, based on educated guesses about the tools involved here;
2014-03-06, by wenzelm
tuned signature -- more uniform check_type_name/read_type_name;
2014-03-06, by wenzelm
clarified treatment of consts -- prefer value-oriented reports;
2014-03-06, by wenzelm
clarified check of internal names;
2014-03-06, by wenzelm
tuned signature;
2014-03-06, by wenzelm
tuned;
2014-03-06, by wenzelm
tuned
2014-03-06, by Lars Hupel
renamed 'fun_rel' to 'rel_fun'
2014-03-06, by blanchet
renamed 'prod_rel' to 'rel_prod'
2014-03-06, by blanchet
renamed 'sum_rel' to 'rel_sum'
2014-03-06, by blanchet
renamed 'filter_rel' to 'rel_filter'
2014-03-06, by blanchet
renamed 'endofun_rel' to 'rel_endofun'
2014-03-06, by blanchet
renamed 'vset_rel' to 'rel_vset'
2014-03-06, by blanchet
fixed NEWS
2014-03-06, by blanchet
renamed 'set_rel' to 'rel_set'
2014-03-06, by blanchet
tuned
2014-03-06, by traytel
rationalized imports
2014-03-06, by traytel
move special BNFs used for composition only to BNF_Comp;
2014-03-06, by traytel
renamed 'cset_rel' to 'rel_cset'
2014-03-06, by blanchet
renamed 'fset_rel' to 'rel_fset'
2014-03-06, by blanchet
renamed 'map_pair' to 'map_prod'
2014-03-06, by blanchet
renamed 'map_sum' to 'sum_map'
2014-03-06, by blanchet
more careful simplification of sets (cf. abf91ebd0820)---yields smaller terms
2014-03-06, by traytel
remove lemmas in favor of more general ones: convex(_hull)_set_{plus,setsum}
2014-03-05, by huffman
generalize lemma closure_sum
2014-03-05, by huffman
generalize lemmas
2014-03-05, by huffman
more symbols;
2014-03-05, by wenzelm
tuned proofs;
2014-03-05, by wenzelm
tuned color (cf. jEdit FUNCTION);
2014-03-05, by wenzelm
tuned;
2014-03-05, by wenzelm
more markup for inner syntax class/type names (notably for completion);
2014-03-05, by wenzelm
tuned proofs;
2014-03-05, by wenzelm
back to stable polyml-5.5.1, due to problems with Poly/ML SVN 1913 and HOL-Proofs (Fail "Insufficient memory");
2014-03-05, by wenzelm
more explicit quasi_keyword markup, for Args.$$$ material, which is somewhere in between of outer and inner syntax;
2014-03-05, by wenzelm
unused;
2014-03-05, by wenzelm
special treatment of method combinators like Args.$$$ keywords, although parsed via Parse.$$$;
2014-03-05, by wenzelm
more thorough (potentially duplicate) markup, e.g. relevant for embedded Args syntax within antiquotations;
2014-03-05, by wenzelm
suppress short abbreviations more uniformly, for outer and quasi-outer syntax;
2014-03-05, by wenzelm
clarified init_assignable: make double-sure that initial values are reset;
2014-03-05, by wenzelm
proper UTF-8;
2014-03-05, by wenzelm
fix typo
2014-03-04, by huffman
remove simp rules made redundant by the replacement of neg_numeral with negated numerals
2014-03-04, by huffman
tuned proof
2014-03-04, by huffman
tuned proof script
2014-03-04, by huffman
no 'sorry' so that the schematic variable gets instantiated
2014-03-04, by blanchet
removed junk
2014-03-04, by blanchet
simplify sets in BNF composition
2014-03-04, by blanchet
tuning
2014-03-04, by blanchet
more caching in composition pipeline
2014-03-04, by blanchet
register relator equations as spec rules only for datatypes -- for codatatypes they underspecify the function and are therefore dangerous (e.g. to Nitpick)
2014-03-04, by blanchet
updated docs
2014-03-04, by blanchet
renamed a pair of low-level theorems to have c/dtor in their names (like the others)
2014-03-04, by blanchet
propagate the exception that is expected later on
2014-03-04, by traytel
N2M does not use the low-level 'fold'; removed the latter from the fp_result interface;
2014-03-04, by traytel
merge
2014-03-04, by blanchet
removed debugging leftover
2014-03-04, by blanchet
minor doc fix
2014-03-04, by blanchet
added contributor
2014-03-04, by nipkow
simplified N2M code now that 'fold' is no longer used by the sugar layer + use right context in all 'force_typ' calls
2014-03-03, by blanchet
fixed handling of 'case_prod' and other 'case' functions for interpreted types
2014-03-03, by blanchet
updated docs
2014-03-03, by blanchet
support 'datatype_new'-defined datatypes in Nitpick + better support for 'codatatype's
2014-03-03, by blanchet
tuned ML names
2014-03-03, by blanchet
tuned code
2014-03-03, by blanchet
removed nonstandard models from Nitpick
2014-03-03, by blanchet
more code lemmas by Rene Thiemann
2014-03-03, by nipkow
merged;
2014-03-03, by wenzelm
tuned proofs;
2014-03-03, by wenzelm
tuned signature -- emphasize symbol positions (prover) vs. decoded text offsets (editor);
2014-03-03, by wenzelm
recovered position hyperlinks from 65c9968286d5 (NB: "def" position vs. regular one);
2014-03-03, by wenzelm
tuned messages and markup;
2014-03-03, by wenzelm
test polyml-svn;
2014-03-03, by wenzelm
README is optional in test compilations;
2014-03-03, by wenzelm
clarified path checks: avoid crash of rendering due to spurious errors;
2014-03-03, by wenzelm
more precise navigation within open files;
2014-03-03, by wenzelm
tuned signature;
2014-03-03, by wenzelm
tuned signature;
2014-03-03, by wenzelm
updated NEWS
2014-03-03, by blanchet
guard against unsound cases that arise when people peek into 'int' and similar types that are handled specially by Nitpick
2014-03-03, by blanchet
adapted example
2014-03-03, by blanchet
removed obsolete, harmful step in tactic
2014-03-03, by blanchet
removed (co)iterators from documentation
2014-03-03, by blanchet
avoid duplicate 'disc_iff' theorems
2014-03-03, by blanchet
rationalized internals
2014-03-03, by blanchet
rationalized internals
2014-03-03, by blanchet
rationalized internals
2014-03-03, by blanchet
life without 'metis'
2014-03-03, by blanchet
rationalized internals
2014-03-03, by blanchet
rationalized internals
2014-03-03, by blanchet
rationalize internals
2014-03-03, by blanchet
optimized simple non-recursive datatypes by reusing 'case' for 'rec' constant
2014-03-03, by blanchet
compile
2014-03-03, by blanchet
make 'diff_iff' a simp rule if available
2014-03-03, by blanchet
less aggressive resolving
2014-03-03, by blanchet
repaired argument list to corecursor
2014-03-03, by blanchet
adapted to absence of 'unfold'
2014-03-03, by blanchet
got rid of automatically generated fold constant and theorems (to reduce overhead)
2014-03-03, by blanchet
use same identity function for abs and rep (doesn't seem to confuse any proofs)
2014-03-03, by blanchet
make 'typedef' optional, depending on size of original type
2014-03-03, by blanchet
use aconv to compare terms (for cleanliness)
2014-03-03, by blanchet
tuning
2014-03-03, by blanchet
optimize cardinal bounds involving natLeq (omega)
2014-03-03, by blanchet
no extend_word for now, it is in conflict with manual reformatting of sources via TAB (e.g. accidental replacement of 'assume' by 'assumes');
2014-03-03, by wenzelm
merged
2014-03-02, by wenzelm
more standard module name;
2014-03-02, by wenzelm
silence warning due to addsimps @{thms dnf_simps}: duplicate not_not rule via simp_thms and nnf_simps;
2014-03-02, by wenzelm
less
more
|
(0)
-30000
-10000
-3000
-1000
-240
+240
+1000
+3000
+10000
tip