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.
tuned proofs
2012-11-08, by bulwahn
using hyp_subst_tac that allows to pass the current simpset to avoid the renamed bound variable warning in the simplifier
2012-11-08, by bulwahn
hyp_subst_tac allows to pass an optional simpset to the internal simplifier call to avoid renamed bound variable warnings in the simplifier call
2012-11-08, by bulwahn
NEWS
2012-11-08, by bulwahn
rewriting with the simpset that is passed to the simproc
2012-11-08, by bulwahn
handling x : S y pattern with the default mechanism instead of raising an exception in the set_comprehension_pointfree simproc
2012-11-08, by bulwahn
tuned
2012-11-08, by bulwahn
syntactic tuning and restructuring of set_comprehension_pointfree simproc
2012-11-08, by bulwahn
using more proper simpset in tactic of set_comprehension_pointfree simproc to avoid renamed bound variable warnings in recursive simplifier calls
2012-11-08, by bulwahn
improving the extension of sets in case of more than one bound variable; rearranging the tactic to prefer simpler steps before more involved ones
2012-11-08, by bulwahn
adjusting proofs as the set_comprehension_pointfree simproc breaks some existing proofs
2012-11-08, by bulwahn
importing term with schematic type variables properly before passing it to the tactic in the set_comprehension_pointfree simproc
2012-11-08, by bulwahn
handling arbitrary terms in the set comprehension and more general merging of patterns possible in the set_comprehension_pointfree simproc
2012-11-08, by bulwahn
simplified structure of patterns in set_comprehension_simproc
2012-11-08, by bulwahn
refined stack of library theories implementing int and/or nat by target language numerals
2012-11-08, by haftmann
restored SML code check which got unintentionally broken: must explicitly check for error during compilation;
2012-11-07, by haftmann
add support for function application to measurability prover
2012-11-06, by hoelzl
renamed Sledgehammer option
2012-11-06, by blanchet
always show timing for structured proofs
2012-11-06, by blanchet
use implications rather than disjunctions to improve readability
2012-11-06, by blanchet
avoid name clashes
2012-11-06, by blanchet
fixed more "Trueprop" issues
2012-11-06, by blanchet
removed needless sort
2012-11-06, by blanchet
avoid double "Trueprop"s
2012-11-06, by blanchet
use original formulas for hypotheses and conclusion to avoid mismatches
2012-11-06, by blanchet
track formula roles in proofs and use that to determine whether the conjecture should be negated or not
2012-11-06, by blanchet
correct parsing of E dependencies
2012-11-06, by blanchet
proper handling of assumptions arising from the goal's being expressed in rule format, for Isar proof construction
2012-11-06, by blanchet
tuned
2012-11-05, by nipkow
code for while directly, not via while_option
2012-11-04, by nipkow
executable true liveness analysis incl an approximating version
2012-11-04, by nipkow
now that sets are executable again, no more special treatment of variable sets
2012-11-04, by nipkow
handle non-unit clauses gracefully
2012-11-02, by blanchet
several improvements to Isar proof reconstruction, by Steffen Smolka (step merging in case splits, time measurements, etc.)
2012-11-02, by blanchet
use measurability prover
2012-11-02, by hoelzl
add measurability prover; add support for Borel sets
2012-11-02, by hoelzl
add syntax and a.e.-rules for (conditional) probability on predicates
2012-11-02, by hoelzl
infinite product measure is invariant under adding prefixes
2012-11-02, by hoelzl
for the product measure it is enough if only one measure is sigma-finite
2012-11-02, by hoelzl
Allow parentheses around left-hand sides of array associations
2012-11-02, by berghofe
made MaSh more robust in the face of duplicate "nicknames" (which can happen e.g. if you have a lemma called foo(1) and another called foo_1 in the same theory)
2012-11-01, by blanchet
regenerated SMT certificates
2012-11-01, by blanchet
regenerated "SMT_Examples" certificates after soft-timeout change + removed a few needless oracles
2012-11-01, by blanchet
fixed bool vs. prop mismatch
2012-10-31, by blanchet
removed "refute" command from Isar manual, now that it has been moved outside "Main"
2012-10-31, by blanchet
repaired "Mutabelle" after Refute move
2012-10-31, by blanchet
less verbose -- the warning will reach the users anyway by other means
2012-10-31, by blanchet
tuned messages
2012-10-31, by blanchet
moved "SAT" before "FunDef" and moved back all SAT-related ML files to where they belong
2012-10-31, by blanchet
fixes related to Refute's move
2012-10-31, by blanchet
added a timeout around script that relies on the network
2012-10-31, by blanchet
took out "using only ..." comments in Sledgehammer generated metis/smt calls, until these can be generated soundly
2012-10-31, by blanchet
moved Refute to "HOL/Library" to speed up building "Main" even more
2012-10-31, by blanchet
tuning
2012-10-31, by blanchet
use metaquantification when possible in Isar proofs
2012-10-31, by blanchet
tuned code
2012-10-31, by blanchet
tuning
2012-10-31, by blanchet
soft SMT timeout
2012-10-31, by blanchet
added function store_termination_rule to the signature, as it is used in Nominal2
2012-10-28, by Christian Urban
longer log, to accomodate final status line of isabelle build;
2012-10-27, by wenzelm
transfer package: error message if preprocessing goal to object-logic formula fails
2012-10-24, by huffman
transfer package: add test to prevent trying to make cterms from open terms
2012-10-24, by huffman
transfer package: more flexible handling of equality relations using is_equality predicate
2012-10-24, by huffman
ensured that rewr_conv rule t = "t == u" literally not just modulo beta-eta
2012-10-24, by nipkow
new theorems
2012-10-22, by kuncar
incorporated constant chars into instantiation proof for enum;
2012-10-22, by haftmann
close code theorems explicitly after preprocessing
2012-10-22, by haftmann
tuned proofs;
2012-10-22, by wenzelm
further attempts to cope with large files via option jedit_text_overview_limit;
2012-10-22, by wenzelm
more detailed Prover IDE NEWS;
2012-10-22, by wenzelm
recovered explicit error message, which was lost in b8570ea1ce25;
2012-10-21, by wenzelm
removed dead code;
2012-10-21, by wenzelm
proper signatures;
2012-10-21, by wenzelm
tuned;
2012-10-21, by wenzelm
merged
2012-10-21, by webertj
Renamed {left,right}_distrib to distrib_{right,left}.
2012-10-19, by webertj
Tuned.
2012-10-19, by webertj
more conventional argument order;
2012-10-21, by haftmann
another refinement in the comprehension conversion
2012-10-21, by bulwahn
refined simplifier call in comprehension_conv
2012-10-21, by bulwahn
passing around the simpset instead of the context; rewriting tactics to avoid the 'renamed bound variable' warnings in nested simplifier calls
2012-10-21, by bulwahn
avoid STIX font, which tends to render badly;
2012-10-20, by wenzelm
extra jar for scala-2.10.0-RC1;
2012-10-20, by wenzelm
more explicit auxiliary classes to avoid warning "reflective access of structural type member method" of scala-2.10.0-RC1;
2012-10-20, by wenzelm
avoid duplicate build of jars_fresh;
2012-10-20, by wenzelm
obsolete, cf. README_REPOSITORY;
2012-10-20, by wenzelm
accomodate scala-2.10.0-RC1;
2012-10-20, by wenzelm
tailored enum specification towards simple instantiation;
2012-10-20, by haftmann
refined internal structure of Enum.thy
2012-10-20, by haftmann
moved quite generic material from theory Enum to more appropriate places
2012-10-20, by haftmann
adding another test case for the set_comprehension_simproc to the theory in HOL/ex
2012-10-20, by bulwahn
improving tactic in setcomprehension_simproc
2012-10-20, by bulwahn
adjusting proofs
2012-10-20, by bulwahn
tuned tactic in set_comprehension_pointfree simproc to handle composition of negation and vimage
2012-10-20, by bulwahn
passing names and types of all bounds around in the simproc
2012-10-20, by bulwahn
locally inverting previously applied simplifications with ex_simps in set_comprehension_pointfree
2012-10-18, by bulwahn
more precise pixel_range: avoid popup when pointing into empty space after actual end-of-line;
2012-10-19, by wenzelm
merged
2012-10-19, by wenzelm
don't include Quotient_Option - workaround to a transfer bug
2012-10-19, by kuncar
ignore old stuff and thus speed up the script greatly;
2012-10-19, by wenzelm
proper find -mtime (file data) instead of -ctime (meta data);
2012-10-19, by wenzelm
made SML/NJ happy;
2012-10-19, by wenzelm
clarified Future.map (again): finished value is mapped in-place, which saves task structures and changes error behaviour slightly (tolerance against canceled group of old value etc.);
2012-10-19, by wenzelm
back to polyml-5.4.1 (cf. b3110dec1a32) -- no cause of spurious interrupts;
2012-10-18, by wenzelm
merged
2012-10-18, by wenzelm
back to parallel HOL-BNF-Examples, which seems to have suffered from Future.map on canceled persistent futures;
2012-10-18, by wenzelm
more basic Goal.reset_futures as snapshot of implicit state;
2012-10-18, by wenzelm
tuned proof;
2012-10-18, by wenzelm
update RBT_Mapping, AList_Mapping and Mapping to use lifting/transfer
2012-10-18, by kuncar
tuned proofs
2012-10-18, by kuncar
new theorem
2012-10-18, by kuncar
merged
2012-10-18, by wenzelm
merged
2012-10-18, by wenzelm
merged
2012-10-18, by wenzelm
merged
2012-10-18, by wenzelm
fixed proof (cf. a81f95693c68);
2012-10-18, by wenzelm
tuned Isar output
2012-10-18, by blanchet
tuned
2012-10-18, by nipkow
updated docs
2012-10-18, by blanchet
renamed Isar-proof related options + changed semantics of Isar shrinking
2012-10-18, by blanchet
tuning
2012-10-18, by blanchet
fixed theorem lookup code in Isar proof reconstruction
2012-10-18, by blanchet
tuning
2012-10-18, by blanchet
refactor code
2012-10-18, by blanchet
tuning
2012-10-18, by blanchet
more robust future_proof result with specific error message (e.g. relevant for incomplete proof of non-registered theorem);
2012-10-18, by wenzelm
collective errors from use_thys and Session.finish/Goal.finish_futures -- avoid uninformative interrupts stemming from failure of goal forks that are not registered in the theory (e.g. unnamed theorems);
2012-10-18, by wenzelm
more uniform group for map_future, which is relevant for cancel in worker_task vs. future_job -- prefer peer group despite 81d03a29980c;
2012-10-18, by wenzelm
tuned message;
2012-10-18, by wenzelm
tuned comment;
2012-10-18, by wenzelm
avoid spurious "bad" markup for show/test_proof;
2012-10-18, by wenzelm
more official Future.terminate;
2012-10-18, by wenzelm
simp results for simplification results of Inf/Sup expressions on bool;
2012-10-18, by haftmann
no sort constraints on datatype constructors in internal bookkeeping
2012-10-18, by haftmann
HOL-BNF-Examples is sequential for now, due to spurious interrupts (again);
2012-10-17, by wenzelm
merged
2012-10-17, by wenzelm
comprehension conversion reuses suggested names for bound variables instead of invented fresh ones; tuned tactic
2012-10-17, by bulwahn
checking for bound variables in the set expression; handling negation more generally
2012-10-17, by bulwahn
set_comprehension_pointfree simproc now handles the complicated test case; tuned
2012-10-17, by bulwahn
refined conversion to only react on proper set comprehensions; tuned
2012-10-17, by bulwahn
moving Pair_inject from legacy and duplicate section to general section, as Pair_inject was considered a duplicate in e8400e31528a by mistake (cf. communication on dev mailing list)
2012-10-17, by bulwahn
employing a preprocessing conversion that rewrites {(x1, ..., xn). P x1 ... xn} to {(x1, ..., xn) | x1 ... xn. P x1 ... xn} in set_comprehension_pointfree simproc
2012-10-17, by bulwahn
another Future.shutdown after Future.cancel_groups (cf. 0d4106850eb2);
2012-10-17, by wenzelm
more robust cancel_now: avoid shooting yourself in the foot;
2012-10-17, by wenzelm
more robust Session.finish (batch mode): use Goal.finish_futures to exhibit remaining failures of disconnected goal forks (e.g. from unnamed theorems) and Goal.cancel_futures the purge the persistent state;
2012-10-17, by wenzelm
proper 'oops' to force sequential checking here, and avoid spurious *** Interrupt stemming from crash of forked outer syntax element;
2012-10-17, by wenzelm
added Output "Detach" button;
2012-10-17, by wenzelm
skipped proofs appear as "bad" without counting as error;
2012-10-17, by wenzelm
more method position information, notably finished_pos after end of previous text;
2012-10-17, by wenzelm
more formal markup;
2012-10-17, by wenzelm
tuned signature;
2012-10-17, by wenzelm
more formal markup;
2012-10-17, by wenzelm
don't be so aggressive when expanding a transfer rule relation; rewrite only the relational part of the rule
2012-10-17, by kuncar
merged
2012-10-16, by wenzelm
added missing file
2012-10-16, by blanchet
tuned for document output
2012-10-16, by traytel
added proof minimization code from Steffen Smolka
2012-10-16, by blanchet
tuned blank lines
2012-10-16, by traytel
tuned whitespace
2012-10-16, by traytel
a few notations changed in HOL/BNF/Examples/Derivation_Trees
2012-10-16, by popescua
ported HOL/BNF/Examples/Derivation_Trees to the latest status of the codatatype package
2012-10-16, by popescua
adding test cases for f x y : S patterns in set_comprehension_pointfree simproc
2012-10-16, by bulwahn
tactic of set_comprehension_pointfree simproc handles f x y : S patterns with Set.vimage
2012-10-16, by bulwahn
term construction of set_comprehension_pointfree simproc handles f x y : S patterns with Set.vimage
2012-10-16, by bulwahn
extending preprocessing of simproc to rewrite subset inequality into membership of powerset
2012-10-16, by bulwahn
update ROOT with teh directory change in BNF
2012-10-16, by popescua
changed name of BNF/Example directory from Infinite_Derivation_Trees to Derivation_Trees
2012-10-16, by popescua
retain info dockable state via educated guess on window focus;
2012-10-16, by wenzelm
support for more informative errors in lazy enumerations;
2012-10-16, by wenzelm
more informative errors for 'also' and 'finally';
2012-10-16, by wenzelm
tuned messages;
2012-10-16, by wenzelm
more proof method text position information;
2012-10-16, by wenzelm
clarified defer/prefer: more specific errors;
2012-10-16, by wenzelm
updated Toplevel.proofs;
2012-10-16, by wenzelm
more informative errors for 'proof' and 'apply' steps;
2012-10-16, by wenzelm
more friendly handling of Pure.thy bootstrap errors;
2012-10-16, by wenzelm
more informative error for stand-alone 'qed';
2012-10-16, by wenzelm
further attempts to unify/simplify goal output;
2012-10-16, by wenzelm
more informative error messages of initial/terminal proof methods;
2012-10-16, by wenzelm
merged
2012-10-15, by wenzelm
setcomprehension_pointfree simproc also works for set comprehension without an equation
2012-10-15, by bulwahn
tuned message -- avoid extra blank lines;
2012-10-15, by wenzelm
updated to polyml-5.5.0 which reduces chance of HOL-IMP failure (although it is hard to reproduce anyway);
2012-10-15, by wenzelm
store colors after build
2012-10-14, by Markus Kaiser
adding further test cases for the set_comprehension_pointfree simproc
2012-10-14, by bulwahn
refined tactic in set_comprehension_pointfree simproc
2012-10-14, by bulwahn
adding further test cases to check new functionality of the simproc; strengthened test cases to check the success of the simproc more faithfully
2012-10-14, by bulwahn
adding postprocessing of computed pointfree expression in set_comprehension_pointfree simproc
2012-10-14, by bulwahn
extending the setcomprehension_pointfree simproc to handle nesting disjunctions, conjunctions and negations (with contributions from Rafal Kolanski, NICTA); tuned
2012-10-14, by bulwahn
more informative error of initial/terminal proof steps;
2012-10-13, by wenzelm
some attempts to unify/simplify pretty_goal;
2012-10-13, by wenzelm
refined Proof.the_finished_goal with more informative error;
2012-10-13, by wenzelm
tuned signature;
2012-10-13, by wenzelm
improved adhoc height for small fonts;
2012-10-13, by wenzelm
further refinement of jEdit line range, avoiding lack of final \n;
2012-10-12, by wenzelm
more uniform tooltip color;
2012-10-12, by wenzelm
more NEWS;
2012-10-12, by wenzelm
merged
2012-10-12, by wenzelm
disambiguated grammar
2012-10-12, by traytel
tuned proofs
2012-10-12, by traytel
tuned
2012-10-12, by nipkow
simplified 'typedef' specifications: discontinued implicit set definition and alternative name;
2012-10-12, by wenzelm
discontinued typedef with alternative name;
2012-10-12, by wenzelm
discontinued obsolete typedef (open) syntax;
2012-10-12, by wenzelm
discontinued typedef with implicit set_def;
2012-10-12, by wenzelm
merged
2012-10-12, by wenzelm
increading indexes to avoid clashes in the set_comprehension_pointfree simproc
2012-10-12, by bulwahn
no special treatment of errors inside goal forks without transaction id, to avoid duplication in plain build with sequential log, for example;
2012-10-12, by wenzelm
do not treat interrupt as error here, to avoid confusion in log etc.;
2012-10-12, by wenzelm
more basic ML compiler messages -- avoid conflict of 638cefe3ee99 and cb7264721c91 concerning Protocol.message_positions;
2012-10-12, by wenzelm
refined separator: FBreak needs to be free for proper breaking, extra space at end helps to work around last-line oddity in jEdit;
2012-10-11, by wenzelm
merged
2012-10-11, by wenzelm
cleanup borel_measurable_positive_integral_(fst|snd)
2012-10-11, by hoelzl
msetprod based directly on Multiset.fold;
2012-10-11, by haftmann
avoid global interpretation
2012-10-11, by haftmann
simplified construction of fold combinator on multisets;
2012-10-11, by haftmann
clarified output token markup (see also bc22daeed49e);
2012-10-11, by wenzelm
refined aprop_tr' -- retain entity information by using type slot as adhoc marker;
2012-10-11, by wenzelm
refrain from quantifying outer fixes, to enable nesting of contexts like "context fixes x context assumes A x";
2012-10-11, by wenzelm
tuned;
2012-10-11, by wenzelm
tuned;
2012-10-11, by wenzelm
more position information for hyperlink and placement of message;
2012-10-11, by wenzelm
tuned;
2012-10-11, by wenzelm
mira: discontinued special settings for lxbroy10, which are probably made obsolete by newer polyml
2012-10-11, by krauss
removed unused legacy material from mira.py
2012-10-10, by krauss
eliminated some remaining uses of typedef with implicit set definition;
2012-10-10, by wenzelm
merged
2012-10-10, by Andreas Lochbihler
fix code equation for RBT_Impl.fold
2012-10-10, by Andreas Lochbihler
merged
2012-10-10, by Andreas Lochbihler
tail-recursive implementation for length
2012-10-10, by Andreas Lochbihler
correct definition for skip_black
2012-10-10, by Andreas Lochbihler
merged
2012-10-10, by wenzelm
merged
2012-10-10, by hoelzl
infprod generator works also with empty index set
2012-10-10, by hoelzl
add finite entropy
2012-10-10, by hoelzl
continuous version of mutual_information_eq_entropy_conditional_entropy
2012-10-10, by hoelzl
add induction for real Borel measurable functions
2012-10-10, by hoelzl
induction prove for positive_integral_fst
2012-10-10, by hoelzl
strong nonnegativ (instead of ae nn) for induction rule
2012-10-10, by hoelzl
induction prove for positive_integral_density
2012-10-10, by hoelzl
less
more
|
(0)
-30000
-10000
-3000
-1000
-240
+240
+1000
+3000
+10000
+30000
tip