Mercurial
Mercurial
>
repos
>
isabelle
/ graph
summary
|
shortlog
|
changelog
| graph |
tags
|
bookmarks
|
branches
|
files
|
gz
|
help
less
more
|
(0)
-30000
-10000
-3000
-1000
-300
-100
-96
+96
+100
+300
+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.
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
add type annotations to make SML happy (cf. ec6187036495)
2012-04-04, by huffman
merged
2012-04-03, by huffman
new transfer proof method
2012-04-03, by huffman
renamed Tools/transfer.ML to Tools/legacy_transfer.ML
2012-04-03, by huffman
prefer prog-prove, suppress isar-overview;
2012-04-03, by wenzelm
merged
2012-04-03, by wenzelm
merged
2012-04-03, by wenzelm
formal integration of "prog-prove" manual;
2012-04-03, by wenzelm
prefer static dependencies;
2012-04-03, by wenzelm
merged
2012-04-03, by huffman
modernized obsolete old-style theory name with proper new-style underscore
2012-04-03, by huffman
removed use of CharVector in generated parser, to make SMLNJ happy
2012-04-03, by sultana
avoid duplicate PIDE markup;
2012-04-03, by wenzelm
less intrusive visibility;
2012-04-03, by wenzelm
more robust re-import wrt. non-HHF assumptions;
2012-04-03, by wenzelm
consider polyml-5.3.0 as "experimental" since it chokes on HOL-Codegenerator_Test, while 5.2.1 happens to work;
2012-04-03, by wenzelm
close context elements via Expression.cert/read_declaration;
2012-04-03, by wenzelm
merged
2012-04-03, by wenzelm
added me to isatest email list
2012-04-03, by sultana
new package Lifting - initial commit
2012-04-03, by kuncar
add floor/ceiling lemmas suggested by René Thiemann
2012-04-03, by huffman
made sure that " is shown in tutorial text
2012-04-03, by nipkow
merged
2012-04-02, by Christian Urban
tuned proofs
2012-04-02, by Christian Urban
merged
2012-04-02, by nipkow
towards showing " in the tutorial
2012-04-02, by nipkow
tuned proof in order to avoid warning message
2012-04-02, by Christian Urban
remove unnecessary qualifiers on names
2012-04-02, by huffman
add lemma Suc_1
2012-04-02, by huffman
merged
2012-04-02, by berghofe
Require "For" keyword to be followed by at least one whitespace, to avoid that
2012-04-02, by berghofe
normalize defs (again, cf. 008b7858f3c0);
2012-04-03, by wenzelm
some context examples;
2012-04-03, by wenzelm
retain literal non-HHF assumptions, to facilitate re-import in Generic_Target.import_export_proof;
2012-04-03, by wenzelm
another attempt to avoid duplication of global vs. local syntax (reminiscent of old fork_mixfix);
2012-04-03, by wenzelm
export into target context (again), to retain its 'defines' (e.g. abbreviation lcoeff in theory HOL/Algebra/UnivPoly);
2012-04-03, by wenzelm
better drop background syntax if entity depends on parameters;
2012-04-03, by wenzelm
more uniform abbrev vs. define;
2012-04-03, by wenzelm
tuned;
2012-04-03, by wenzelm
clarified generic_const vs. close_schematic_term;
2012-04-03, by wenzelm
tuned;
2012-04-03, by wenzelm
more uniform theory_abbrev with const_declaration;
2012-04-03, by wenzelm
avoid const_declaration in aux. context (cf. locale_foundation);
2012-04-03, by wenzelm
clarified background_foundation vs. theory_foundation (with const_declaration);
2012-04-03, by wenzelm
tuned;
2012-04-03, by wenzelm
more general standard_declaration;
2012-04-02, by wenzelm
better restore after close_target;
2012-04-02, by wenzelm
tuned;
2012-04-02, by wenzelm
clarified standard_declaration vs. theory_declaration;
2012-04-02, by wenzelm
smarter generic_const: plain alias for non-dependent case (e.g. prospective datatype or record syntax);
2012-04-02, by wenzelm
tuned;
2012-04-02, by wenzelm
tuned;
2012-04-02, by wenzelm
tuned signature;
2012-04-02, by wenzelm
misc tuning and simplification;
2012-04-02, by wenzelm
better restore to first target, not last target;
2012-04-02, by wenzelm
refined define/abbrev: allow extra fixes in aux. context vs. bottom target (NB: export_term expands defined variables, leaving fixed ones);
2012-04-02, by wenzelm
more general Local_Theory.restore, allow any nesting level;
2012-04-02, by wenzelm
new tutorial
2012-04-02, by nipkow
New manual Programming and Proving in Isabelle/HOL
2012-04-02, by nipkow
add simp rules for dvd on negative numerals
2012-04-02, by huffman
merged, manually resolving conflicts due to session renaming (cf. 6488c5efec49)
2012-04-01, by krauss
clarified terminology; added reference to bundle component
2012-04-01, by krauss
less modest NEWS; CONTRIBUTORS
2012-04-01, by krauss
renamed import session back to Import, conforming to directory name; NEWS
2012-04-01, by krauss
more precise IsaMakefile (eg. see HOL-Algebra);
2012-04-01, by wenzelm
more keywords;
2012-04-01, by wenzelm
less
more
|
(0)
-30000
-10000
-3000
-1000
-300
-100
-96
+96
+100
+300
+1000
+3000
+10000
+30000
tip