Mercurial
Mercurial
>
repos
>
isabelle
/ graph
summary
|
shortlog
|
changelog
| graph |
tags
|
bookmarks
|
branches
|
files
|
gz
|
help
less
more
|
(0)
-30000
-10000
-3000
-1000
-960
+960
+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.
added signature
2012-11-28, by smolkas
moved thms_of_name to Sledgehammer_Util and removed copies, updated references
2012-11-28, by smolkas
removed duplicate decleration
2012-11-28, by smolkas
made use of sledgehammer_util
2012-11-28, by smolkas
renamed sledgehammer_isar_reconstruct to sledgehammer_proof
2012-11-28, by smolkas
added comments to new source files
2012-11-28, by smolkas
fixed problem with fact names
2012-11-28, by smolkas
remove hack and generalize code slightly
2012-11-28, by smolkas
simplified isar_qualifiers and qs merging
2012-11-28, by smolkas
put shrink in own structure
2012-11-28, by smolkas
put annotate in own structure
2012-11-28, by smolkas
support assumptions as facts for preplaying
2012-11-28, by smolkas
some minor improvements in shrink_proof
2012-11-28, by smolkas
some support for ML runtime statistics;
2012-11-28, by wenzelm
prefer tight Markup.print_int/parse_int for property values;
2012-11-28, by wenzelm
clarified new identifier syntax: exclude \<^isup>, include subscripted prime (to allow imitating full identifier here);
2012-11-28, by wenzelm
eliminated slightly odd identifiers;
2012-11-28, by wenzelm
tuned syntax, potentially more robust;
2012-11-28, by wenzelm
smarter list layout;
2012-11-28, by wenzelm
repaired text following 491c5c81c2e8;
2012-11-27, by wenzelm
merged
2012-11-27, by wenzelm
introduce filter_lim as a generatlization of tendsto
2012-11-27, by hoelzl
merged
2012-11-27, by wenzelm
based countable topological basis on Countable_Set
2012-11-27, by immler
qualified interpretation of sigma_algebra, to avoid name clashes
2012-11-27, by immler
eliminated finite_set_sequence with countable set
2012-11-22, by immler
support for sub-structured identifier syntax (inactive);
2012-11-27, by wenzelm
eliminated some improper identifiers;
2012-11-27, by wenzelm
add upper bounds for factorial and binomial; add equation for binomial using nat-division (both from AFP/Girth_Chromatic)
2012-11-27, by hoelzl
tuned signature;
2012-11-26, by wenzelm
more uniform Symbol.is_ascii_identifier in ML/Scala;
2012-11-26, by wenzelm
tuned;
2012-11-26, by wenzelm
clarified Symbol.scan_ascii_id;
2012-11-26, by wenzelm
tuned;
2012-11-26, by wenzelm
convenience operations for table as set;
2012-11-26, by wenzelm
removed remains of Oheimb's double-space (cf. 0a5af667dc75);
2012-11-26, by wenzelm
tuned;
2012-11-26, by wenzelm
merged
2012-11-26, by wenzelm
updated two components
2012-11-26, by blanchet
simplify code slightly
2012-11-26, by blanchet
avoid non-ASCII sign
2012-11-26, by blanchet
generate a parameterized correspondence relation
2012-11-26, by kuncar
quot_thm_crel
2012-11-26, by kuncar
add option_fold
2012-11-26, by kuncar
add binomial_ge_n_over_k_pow_k
2012-11-26, by hoelzl
removed tool that was never finished
2012-11-26, by blanchet
added file headers
2012-11-26, by blanchet
updated MaSh doc
2012-11-26, by blanchet
moved MaSh's Python code into Isabelle
2012-11-26, by blanchet
updated NEWS etc.
2012-11-26, by blanchet
distinguish declated tfrees from other tfrees -- only the later can be optimized away
2012-11-26, by blanchet
clarified status of Legacy_XML_Syntax, despite lack of Proofterm_XML;
2012-11-26, by wenzelm
reset active areas on content update;
2012-11-26, by wenzelm
more general sendback properties;
2012-11-26, by wenzelm
tuned command descriptions;
2012-11-26, by wenzelm
refined outer syntax 'help' command;
2012-11-26, by wenzelm
tuned signature;
2012-11-26, by wenzelm
always reset active areas;
2012-11-26, by wenzelm
no special treatment of control_reset, in accordance to other control styles;
2012-11-26, by wenzelm
tuned signature;
2012-11-25, by wenzelm
tuned signature;
2012-11-25, by wenzelm
tuned signature;
2012-11-25, by wenzelm
tuned signature;
2012-11-25, by wenzelm
renamed main plugin object to PIDE;
2012-11-25, by wenzelm
tuned signature -- avoid intrusion of module Path in generic PIDE concepts;
2012-11-25, by wenzelm
explicit module UTF8;
2012-11-25, by wenzelm
tuned file name;
2012-11-25, by wenzelm
Isabelle-specific implementation of quasi-abstract markup elements -- back to module arrangement before d83797ef0d2d;
2012-11-25, by wenzelm
prefer strict error;
2012-11-25, by wenzelm
quasi-abstract module Rendering, with Isabelle-specific implementation;
2012-11-25, by wenzelm
added convenience actions isabelle.increase-font-size and isabelle.decrease-font-size;
2012-11-25, by wenzelm
eval PDF_VIEWER/DVI_VIEWER command line, which allows additional quotes for program name, for example;
2012-11-25, by wenzelm
retain hidden_color (i.e. transparent white) instead of replacing it by semantic text color, to make control symbols more hidden and avoid "dirty" lines with some fonts;
2012-11-24, by wenzelm
prefer buffer_edit combinator over Java-style boilerplate;
2012-11-24, by wenzelm
more robust font for control symbols, to ensure these obscure codepoints are properly rendered;
2012-11-24, by wenzelm
tuned symbol groups;
2012-11-24, by wenzelm
tuned -- Symbol.groups already sorted;
2012-11-24, by wenzelm
more robust default font -- user might have switched jEdit TextArea to another font that lacks glyphs;
2012-11-24, by wenzelm
added option jedit_symbols_search_limit;
2012-11-24, by wenzelm
avoid empty tooltip;
2012-11-24, by wenzelm
tuned symbol groups;
2012-11-24, by wenzelm
special handling of control symbols in Symbols dockable;
2012-11-24, by wenzelm
recovered some tooltip wrapping from e2762f962042, with multi-line support via HTML.encode;
2012-11-24, by wenzelm
avoid showing semantic aspects of Unicode -- Isabelle/Scala merely (ab)uses the low-level rendering model (codepoint + font);
2012-11-24, by wenzelm
more NEWS/CONTRIBUTORS;
2012-11-24, by wenzelm
improved editing support for control styles;
2012-11-24, by wenzelm
added ISABELLE_PLATFORM_FAMILY;
2012-11-24, by wenzelm
merged
2012-11-23, by nipkow
moved lemma
2012-11-23, by nipkow
timeout in proper place (HOL-Quickcheck_Examples approx. 1min, HOL-Quickcheck_Benchmark approx. 1h);
2012-11-23, by wenzelm
add quotient_of_div
2012-11-23, by hoelzl
generate correct names
2012-11-23, by kuncar
simplified code
2012-11-23, by kuncar
generate correct correspondence relation name
2012-11-23, by kuncar
more uniform title, follow-up to 928cb8b35e6e;
2012-11-23, by wenzelm
tuned
2012-11-23, by nipkow
defer interpretation of markup via implicit print mode;
2012-11-22, by wenzelm
merged
2012-11-22, by wenzelm
made SML/NJ happier
2012-11-22, by traytel
pack window before accessing its geometry;
2012-11-22, by wenzelm
always refresh font metrics, to help window size calculation (amending 2585c81d840a);
2012-11-22, by wenzelm
more precise tooltip window size;
2012-11-22, by wenzelm
take component width as indication if it is already visible/layed-out, to avoid multiple formatting with minimal margin;
2012-11-22, by wenzelm
reset active area for outdated snapshot (again?);
2012-11-22, by wenzelm
some support for implicit senback, meaning that it uses the caret position instead of explicit command exec_id;
2012-11-22, by wenzelm
more abstract Sendback operations, with explicit id/exec_id properties;
2012-11-22, by wenzelm
some support for breakable text and paragraphs;
2012-11-22, by wenzelm
tuned names
2012-11-22, by nipkow
tuned comment;
2012-11-21, by wenzelm
clarified symbol groups, despite this traditional arrangement in X-symbol grid;
2012-11-21, by wenzelm
always retain message positions, in order to allow Isabelle_Rendering.sendback retrieve the exec_id, even in tooltip or detached window;
2012-11-21, by wenzelm
tuned whitespace;
2012-11-21, by wenzelm
merged
2012-11-21, by immler
included abbrev in tooltip
2012-11-21, by immler
removed (unicode) tooltips: can not adjust font in basic swing tooltip
2012-11-21, by immler
delayed search to improve reactivity
2012-11-21, by immler
respect font property for symbols
2012-11-21, by immler
capitalize lowercase groups;
2012-11-21, by immler
merged
2012-11-21, by wenzelm
more generous timeout for SML/NJ, which is approx. 40-80 times slower than Poly/ML;
2012-11-21, by wenzelm
Countable_Set: tuned lemma names; more generic lemmas
2012-11-21, by hoelzl
enable Symbols dockable by default;
2012-11-21, by wenzelm
tuned;
2012-11-21, by wenzelm
accomodate scala-2.10.0-RC2 with its slight reform on for-syntax;
2012-11-21, by wenzelm
renamed BNF/Countable_Set to Countable_Type and moved its generic stuff to Library/Countable_Set
2012-11-21, by hoelzl
dockable with buttons for symbols, grouped and sorted in tabs according to ~~/etc/symbols;
2012-11-21, by immler
CONTRIBUTION: add fabians work
2012-11-21, by hoelzl
NEWS: document changes in HOL-Probability
2012-11-21, by hoelzl
NEWS (changeset 13211e07d931): add Countable_Set
2012-11-21, by hoelzl
NEWS (changeset 69b35a75caf3): document changes in FuncSet
2012-11-21, by hoelzl
new theory of immutable arrays
2012-11-21, by nipkow
some grouping of Isabelle symbols, based on X-Symbol grid in PG-3.7.1.1 and a proposal by Fabian Immler;
2012-11-20, by wenzelm
support for symbol groups, retaining original order of declarations;
2012-11-20, by wenzelm
tuned;
2012-11-20, by wenzelm
add Countable_Set theory
2012-11-20, by hoelzl
tuned proof
2012-11-20, by nipkow
simplified command line of "isabelle install";
2012-11-20, by wenzelm
known problems with Mac OS X are back -- Java 7u6 is not the last word (cf. ce37d4f8b4f4);
2012-11-20, by wenzelm
some documentation for "algebra" in HOL;
2012-11-20, by wenzelm
global default for session timeout;
2012-11-20, by wenzelm
alternative completion for outer syntax keywords;
2012-11-19, by wenzelm
init options on startup as well;
2012-11-19, by wenzelm
theorem status about oracles/futures is no longer printed by default;
2012-11-19, by wenzelm
tuned: use induction rule sigma_sets_induct_disjoint
2012-11-19, by hoelzl
tuned FinMap
2012-11-19, by hoelzl
merge extensional dependent function space from FuncSet with the one in Finite_Product_Measure
2012-11-19, by hoelzl
more refs;
2012-11-19, by wenzelm
isabelle build no longer supports document_dump/document_dump_mode (no INCOMPATIBILITY, since it was never in official release);
2012-11-18, by wenzelm
proper jvmpath for windows;
2012-11-18, by wenzelm
more generous tracing_limit, with explicit system option;
2012-11-18, by wenzelm
adjust max_threads_value to capabilities of Poly/ML 5.5 and current hardware;
2012-11-18, by wenzelm
update options via protocol;
2012-11-18, by wenzelm
more accurate pixel_range -- do not round offset here;
2012-11-18, by wenzelm
tuned signature;
2012-11-18, by wenzelm
prefer absolute default $USER_HOME/Scratch.thy;
2012-11-17, by wenzelm
more portable process exit;
2012-11-17, by wenzelm
tuned -- eliminate pointless ML method definition;
2012-11-17, by wenzelm
tuned;
2012-11-17, by wenzelm
NEWS;
2012-11-17, by wenzelm
tuned structure of Isabelle/HOL;
2012-11-17, by wenzelm
method setup for Classical steps;
2012-11-17, by wenzelm
tuned signature;
2012-11-17, by wenzelm
updated keywords;
2012-11-17, by wenzelm
moved (b)choice_iff(') to Hilbert_Choice
2012-11-16, by hoelzl
move theorems to be more generally useable
2012-11-16, by hoelzl
merged
2012-11-16, by wenzelm
made SML/NJ happy;
2012-11-16, by wenzelm
renamed prob_space to proj_prob_space as it clashed with Probability_Measure.prob_space
2012-11-16, by hoelzl
renamed measurable_compose -> measurable_finmap_compose, clashed with Sigma_Algebra.measurable_compose
2012-11-16, by hoelzl
measurability for nat_case and comb_seq
2012-11-16, by hoelzl
rules for AE and prob
2012-11-16, by hoelzl
rules for intergration: integrating nat-functions, integrals on finite measures, constant multiplication
2012-11-16, by hoelzl
more measurability rules
2012-11-16, by hoelzl
renamed to more appropriate lim_P for projective limit
2012-11-16, by immler
allow arbitrary enumerations of basis in locale for generation of borel sets
2012-11-16, by immler
repaired slip accidentally introduced in 57209cfbf16b
2012-11-15, by haftmann
prefer implementation in HOL;
2012-11-15, by haftmann
corrected headers
2012-11-15, by immler
hide constants of auxiliary type finmap
2012-11-15, by immler
generalized to copy of countable types instead of instantiation of nat for discrete topology
2012-11-15, by immler
added projective limit;
2012-11-15, by immler
regularity of measures, therefore:
2012-11-15, by immler
tuned -- eliminated obsolete citation of isabelle-ref;
2012-11-15, by wenzelm
updated basic equality rules;
2012-11-12, by wenzelm
removed somewhat pointless historic material;
2012-11-12, by wenzelm
updated unification options;
2012-11-11, by wenzelm
removed some historic material that is obsolete or rarely used;
2012-11-11, by wenzelm
tuned;
2012-11-11, by wenzelm
updated section on ordered rewriting;
2012-11-11, by wenzelm
updated subgoaler/solver/looper;
2012-11-10, by wenzelm
removed somewhat pointless historic material;
2012-11-08, by wenzelm
tuned;
2012-11-08, by wenzelm
updated explanation of rewrite rules;
2012-11-08, by wenzelm
(re)moved old material about Simplifier;
2012-11-07, by wenzelm
some coverage of "resolution without lifting", which should be normally avoided;
2012-11-07, by wenzelm
removed somewhat pointless historic material;
2012-11-07, by wenzelm
updated biresolve_tac, bimatch_tac;
2012-11-07, by wenzelm
moved classical wrappers to IsarRef;
2012-11-07, by wenzelm
avoid clash of terminology wrt. "semi-automated" in the sense of Isar (e.g. method "rule");
2012-11-04, by wenzelm
updated citations;
2012-11-04, by wenzelm
tuned;
2012-11-04, by wenzelm
removed junk;
2012-11-04, by wenzelm
removed pointless historic material;
2012-11-04, by wenzelm
more on Simplifier rules, based on old material;
2012-11-04, by wenzelm
refurbished Simplifier examples;
2012-11-04, by wenzelm
more on the Simplifier, based on old material;
2012-11-03, by wenzelm
more concise/precise documentation;
2012-11-03, by wenzelm
tuned text
2012-11-14, by nipkow
replaced relation by function - simplifies development
2012-11-14, by nipkow
made SMLNJ happier
2012-11-13, by traytel
import Sublist rather than PrefixOrder to avoid unnecessary class instantiation
2012-11-13, by traytel
prefer explicit Random.seed
2012-11-13, by haftmann
dropped dead code
2012-11-12, by haftmann
tuned import order
2012-11-12, by haftmann
tuned layout
2012-11-12, by nipkow
fixed detection of tautologies -- things like "a = b" in a structured proof, where a and b are Frees, shouldn't be discarted as tautologies
2012-11-12, by blanchet
create temp directory if not already created
2012-11-12, by blanchet
merged
2012-11-12, by nipkow
new theory IMP/Finite_Reachable
2012-11-12, by nipkow
avoid messing too much with output of "string_of_term", so that it doesn't break the yxml encoding for jEdit
2012-11-12, by blanchet
centralized term printing code
2012-11-12, by blanchet
thread context correctly when printing backquoted facts
2012-11-12, by blanchet
dropped dead code;
2012-11-11, by haftmann
modernized, simplified and compacted oracle and proof method glue code;
2012-11-11, by haftmann
merged
2012-11-09, by nipkow
fixed underscores
2012-11-09, by nipkow
moved lemmas into projective_family; added header for theory Projective_Family
2012-11-09, by immler
removed redundant/unnecessary assumptions from projective_family
2012-11-09, by immler
assume probability spaces; allow empty index set
2012-11-07, by immler
added projective_family; generalized generator in product_prob_space to projective_family
2012-11-07, by immler
moved lemmas further up
2012-11-06, by immler
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
add induction rules for simple functions and for Borel measurable functions
2012-10-10, by hoelzl
introduce induction rules for simple functions and for Borel measurable functions
2012-10-10, by hoelzl
joint distribution of independent variables
2012-10-10, by hoelzl
indep_vars does not need sigma-sets
2012-10-10, by hoelzl
simplified definitions
2012-10-10, by hoelzl
remove unnecessary assumption from conditional_entropy_eq
2012-10-10, by hoelzl
alternative definition of conditional entropy
2012-10-10, by hoelzl
remove unneeded assumption from conditional_entropy_generic_eq
2012-10-10, by hoelzl
add induction rule for intersection-stable sigma-sets
2012-10-10, by hoelzl
show and use distributed_swap and distributed_jointI
2012-10-10, by hoelzl
rule to show that conditional mutual information is non-negative in the continuous case
2012-10-10, by hoelzl
continuous version of entropy_le
2012-10-10, by hoelzl
simplified entropy_uniform
2012-10-10, by hoelzl
remove incseq assumption from measure_eqI_generator_eq
2012-10-10, by hoelzl
generalize from prob_space to finite_measure
2012-10-10, by hoelzl
add measurable_compose
2012-10-10, by hoelzl
simplified assumptions for kolmogorov_0_1_law
2012-10-10, by hoelzl
merge should operate on pairs
2012-10-10, by hoelzl
remove incseq assumption from sigma_prod_algebra_sigma_eq
2012-10-10, by hoelzl
sigma_finite_iff_density_finite does not require a positive density function
2012-10-10, by hoelzl
tuned Lebesgue measure proofs
2012-10-10, by hoelzl
tuned product measurability
2012-10-10, by hoelzl
remove some unneeded positivity assumptions; generalize some assumptions to AE; tuned proofs
2012-10-10, by hoelzl
use continuity to show Borel-measurability
2012-10-10, by hoelzl
tuned measurable_If; moved countably_additive equalities to Measure_Space; tuned proofs
2012-10-10, by hoelzl
rename terminal_events to tail_event
2012-10-10, by hoelzl
merged
2012-10-10, by Andreas Lochbihler
efficient construction of red black trees from sorted associative lists
2012-10-10, by Andreas Lochbihler
more explicit code equations
2012-10-10, by haftmann
adding necessary syntactic functions in set_comprehension_pointfree simproc as a first step to integrate an improved simproc
2012-10-10, by bulwahn
special code setup for step function in IMP is redundant as definition was tuned (cf. c54d901d2946)
2012-10-10, by bulwahn
test case for set_comprehension_pointfree simproc succeeds now
2012-10-10, by bulwahn
unfolding bounded existential quantifiers as first step in the set_comprehension_pointfree simproc
2012-10-10, by bulwahn
moving simproc from Finite_Set to more appropriate Product_Type theory
2012-10-10, by bulwahn
generalizing set_comprehension_pointfree simproc to work for arbitrary predicates (and not just the finite predicate)
2012-10-10, by bulwahn
adding some example that motivates some of the current changes in the set_comprehension_pointfree simproc
2012-10-10, by bulwahn
set_comprehension_pointfree also handles terms where the equation is not at the first position, which is a necessary generalisation to eventually handle bounded existentials; tuned
2012-10-10, by bulwahn
more consistent error messages on malformed code equations
2012-10-10, by haftmann
removed support for set constant definitions in HOLCF {cpo,pcpo,domain}def commands;
2012-10-09, by huffman
use Set.filter instead of Finite_Set.filter, which is removed then
2012-10-09, by kuncar
rename Set.project to Set.filter - more appropriate name
2012-10-09, by kuncar
added some ad-hoc namespace prefixes to avoid duplicate facts;
2012-10-10, by wenzelm
avoid duplicate facts;
2012-10-10, by wenzelm
more explicit namespace prefix for 'statespace' -- duplicate facts;
2012-10-10, by wenzelm
eliminated spurious fact duplicates;
2012-10-10, by wenzelm
modernized dynamic "rules" -- avoid rebinding of static facts;
2012-10-10, by wenzelm
removed redundant lemma, cf. class zero_neq_one in HOL/Rings.thy;
2012-10-09, by wenzelm
clarified Element.init vs. Element.activate: refrain from hard-wiring Thm.def_binding_optional to avoid duplicate facts;
2012-10-09, by wenzelm
tuned;
2012-10-09, by wenzelm
clarified Local_Defs.add_def(s): refrain from hard-wiring Thm.def_binding_optional;
2012-10-09, by wenzelm
more explicit flags for facts table;
2012-10-09, by wenzelm
minor tuning;
2012-10-09, by wenzelm
more conventional Double constants;
2012-10-09, by wenzelm
tuned source structure;
2012-10-09, by wenzelm
tuned;
2012-10-09, by wenzelm
tuned;
2012-10-09, by wenzelm
merged
2012-10-09, by wenzelm
added type annotations to generated Isar proofs -- code by Steffen Smolka
2012-10-09, by blanchet
consolidated names of theorems on composition;
2012-10-08, by haftmann
corrected NEWS
2012-10-08, by haftmann
avoid somewhat heavy rebuilding of SortedMap via map where plain iteration is sufficient;
2012-10-08, by wenzelm
clarified long_names -- conform to usual Isabelle practice of not analysing internal names;
2012-10-08, by wenzelm
more precise repaint and revalidate -- the latter is important to keep in sync with content update;
2012-10-08, by wenzelm
tuned;
2012-10-08, by wenzelm
prefer synchronous Mutator_Event.Bus on Swing_Thread;
2012-10-08, by wenzelm
more direct tooltip content;
2012-10-08, by wenzelm
tuned;
2012-10-08, by wenzelm
use Pretty_Tooltip for Graphview_Panel;
2012-10-08, by wenzelm
more basic tooltips;
2012-10-08, by wenzelm
close tooltips more thoroughly;
2012-10-07, by wenzelm
make buttons closer to original mouse position;
2012-10-07, by wenzelm
detach tooltip as dockable window;
2012-10-07, by wenzelm
explicit close button;
2012-10-07, by wenzelm
congruence rule for Finite_Set.fold
2012-10-06, by haftmann
alternative simplification of ^^ to the righthand side;
2012-10-06, by haftmann
eliminated obsolete tooltip delay -- bypassed by Pretty_Tooltip;
2012-10-05, by wenzelm
merged
2012-10-05, by wenzelm
newer versions of Z3 call it "Bool" not "bool"
2012-10-05, by blanchet
simplified type of msetprod;
2012-10-04, by haftmann
tuned proof
2012-10-04, by haftmann
default simp rule for image under identity
2012-10-04, by haftmann
dropped duplicate facts; tuned syntax
2012-10-04, by haftmann
more facts on setsum and setprod
2012-10-04, by haftmann
made SML/NJ happier
2012-10-04, by traytel
do not expose details of internal data structures for composition of BNFs
2012-10-04, by traytel
further support for nested tooltips;
2012-10-05, by wenzelm
tuned proofs;
2012-10-05, by wenzelm
refer to parent frame -- relevant for floating dockables in particular;
2012-10-05, by wenzelm
tuned window position to fit on screen;
2012-10-05, by wenzelm
tuned window position;
2012-10-05, by wenzelm
determine window size from content;
2012-10-05, by wenzelm
tuned color and font size;
2012-10-05, by wenzelm
close tooltip window on escape;
2012-10-05, by wenzelm
proper message markup for output;
2012-10-05, by wenzelm
some re-ordering of initialization to ensure proper formatting;
2012-10-04, by wenzelm
separate module Pretty_Tooltip;
2012-10-04, by wenzelm
refined rich tooltip options;
2012-10-04, by wenzelm
Rich_Text_Area tooltips via nested Pretty_Text_Area, based on some techniques of FoldViewer plugin;
2012-10-04, by wenzelm
some documentation of show_markup;
2012-10-04, by wenzelm
tuned proofs;
2012-10-04, by wenzelm
option to bypass potentially slow text overview;
2012-10-04, by wenzelm
tuned signature;
2012-10-04, by wenzelm
clarified platform dependency;
2012-10-04, by wenzelm
updated crontab and afp-poly settings
2012-10-04, by Gerwin Klein
thread the right local theory through + reenable parallel proofs for previously problematic theories
2012-10-03, by blanchet
made code more conform to rest of BNF package
2012-10-03, by blanchet
more error positions;
2012-10-03, by wenzelm
more explicit show_type_constraint, show_sort_constraint;
2012-10-03, by wenzelm
recovered print translation after 'a => bool to 'a set change;
2012-10-03, by wenzelm
tuned;
2012-10-03, by wenzelm
use explicit Type.strip_sorts_dummy to suppress sort constraints in output;
2012-10-03, by wenzelm
printed "_ofsort" is subject to show_markup as well;
2012-10-03, by wenzelm
allow position constraints to coexist with 0 or 1 sort constraints;
2012-10-03, by wenzelm
made tactic more robust (less usage of stac)
2012-10-02, by traytel
continued changing type of corec type
2012-10-02, by blanchet
removed dead params and dead code
2012-10-02, by blanchet
changed type of corecursor for the nested recursion case
2012-10-02, by blanchet
made (co)rec tactic more robust when the simplifier succeeds early
2012-10-02, by blanchet
tuned;
2012-10-01, by wenzelm
removed unused module Blob;
2012-10-01, by wenzelm
more direct message header: eliminated historic encoding via single letter;
2012-10-01, by wenzelm
tuned whitespace;
2012-10-01, by wenzelm
tuned proofs;
2012-10-01, by wenzelm
report sort assignment of visible type variables;
2012-10-01, by wenzelm
more robust File.eq, and thus File.copy of "~~/lib/logo/isabelle.gif";
2012-10-01, by wenzelm
fixed recursor definition for datatypes with inner products (e.g. "'a trm" from the lambda-term example)
2012-10-01, by blanchet
tweaked corecursor/coiterator tactic
2012-10-01, by blanchet
changed the type of the recursor for nested recursion
2012-10-01, by blanchet
fixed quick-and-dirty mode
2012-09-30, by blanchet
tuning
2012-09-30, by blanchet
use Thm.close_derivation in theorems proved using Skip_Proof.prove; tuned signature;
2012-09-30, by traytel
got rid of subst_tac alias
2012-09-30, by traytel
tuned tactic
2012-09-30, by traytel
tuned proofs;
2012-09-29, by wenzelm
tuned proofs;
2012-09-29, by wenzelm
proper handling of constraints stemming from idtyp_ast_tr';
2012-09-29, by wenzelm
enable show_markup by default (approx. double output size);
2012-09-29, by wenzelm
more explicit Syntax_Trans.mark_bound_abs/mark_bound_body: preserve type information for show_markup;
2012-09-29, by wenzelm
explicit show_types takes preferenced over show_markup;
2012-09-29, by wenzelm
ignore wrapped markup elements in Proof General;
2012-09-29, by wenzelm
turn constraints into Isabelle_Markup.typing, depending on show_markup options;
2012-09-29, by wenzelm
treat wrapped markup elements as raw markup delimiters;
2012-09-29, by wenzelm
tuned signature;
2012-09-29, by wenzelm
tuned proofs;
2012-09-28, by wenzelm
tuned proofs;
2012-09-28, by wenzelm
tuned proofs;
2012-09-28, by wenzelm
tuned;
2012-09-28, by wenzelm
support for wrapped XML elements, which allows to preserve full markup tree information in to_XML/from_XML conversion;
2012-09-28, by wenzelm
merged
2012-09-28, by wenzelm
eliminated dead code;
2012-09-28, by wenzelm
smarter handling of tracing messages;
2012-09-28, by wenzelm
display number of tracing messages;
2012-09-28, by wenzelm
tuned signature;
2012-09-28, by wenzelm
tuned proofs;
2012-09-28, by wenzelm
simplified simpset
2012-09-28, by blanchet
fixed simplification of prod and sum relators to avoid issues with e.g. codata ('a, 'b) k = K "'a + 'b"
2012-09-28, by blanchet
tuned tactic
2012-09-28, by traytel
updated keywords using proper "isabelle update_keywords";
2012-09-28, by wenzelm
tuned tactic
2012-09-28, by traytel
tuned tactic
2012-09-28, by traytel
merge
2012-09-28, by blanchet
renamed ML file in preparation for next step
2012-09-28, by blanchet
killed temporary "data_raw" and "codata_raw" now that the examples have been ported to "data" and "codata"
2012-09-28, by blanchet
modernized example, exploiting "rep_compat" option
2012-09-28, by blanchet
compatibility option to use "rep_datatype"
2012-09-28, by blanchet
tuned message
2012-09-28, by blanchet
modernized example
2012-09-28, by blanchet
tuned tactics
2012-09-28, by traytel
second usage of const_typ
2012-09-28, by nipkow
new antiquotation const_typ
2012-09-28, by nipkow
tuned printing of _ in latex
2012-09-28, by nipkow
mk_readable_rsp_thm_eq is more robust now
2012-09-27, by kuncar
new get function for non-symmetric relator_eq & tuned
2012-09-27, by kuncar
merged
2012-09-27, by wenzelm
tuned tactic; got rid of substs_tac alias
2012-09-27, by traytel
use a nicer scheme to indexify names
2012-09-27, by blanchet
tuned tactic
2012-09-27, by traytel
type of the bound of a BNF depends at most on dead type variables
2012-09-27, by traytel
repaired signature
2012-09-27, by blanchet
lower the defaults for the number of bits, based on an example by Lukas Bulwahn
2012-09-27, by blanchet
modernized examples
2012-09-27, by blanchet
merged
2012-09-27, by nipkow
tuned
2012-09-27, by nipkow
operations to turn markup into XML;
2012-09-27, by wenzelm
removed obsolete org.w3c.dom operations;
2012-09-27, by wenzelm
eliminated obsolete HTML/CSS functionality;
2012-09-27, by wenzelm
removed obsolete Output1 dockable;
2012-09-27, by wenzelm
physical File.eq in conformance to Isabelle/ML;
2012-09-27, by wenzelm
tuned proofs;
2012-09-27, by wenzelm
tuned;
2012-09-27, by wenzelm
updated to consolidated SortedMap in scala-2.9.x;
2012-09-27, by wenzelm
partly ported "TreeFI" example to new syntax
2012-09-27, by blanchet
avoid another brand of trivial "disc_rel" theorems (which made the simplifier loop for all single-constructor types)
2012-09-27, by blanchet
tuned
2012-09-27, by nipkow
tuned
2012-09-27, by nipkow
merge
2012-09-27, by blanchet
modernized examples;
2012-09-27, by blanchet
some support for jEdit warmstart;
2012-09-26, by wenzelm
discontinued XML.cache experiment -- Poly/ML 5.5.0 RTS does online sharing better;
2012-09-26, by wenzelm
tuned message;
2012-09-26, by wenzelm
merged
2012-09-26, by wenzelm
disable parallel proofs for two big examples -- speeds up things and eliminates spurious Interrupt exceptions (to be investigated)
2012-09-26, by blanchet
got rid of other instance of shaky "Thm.generalize"
2012-09-26, by blanchet
tweaked theorem names (in particular, dropped s's)
2012-09-26, by blanchet
get rid of shaky "Thm.generalize"
2012-09-26, by blanchet
fixed "rels" + split them into injectivity and distinctness
2012-09-26, by blanchet
generate high-level "coinduct" and "strong_coinduct" properties
2012-09-26, by blanchet
added coinduction tactic
2012-09-26, by blanchet
generalized tactic a bit
2012-09-26, by blanchet
export "dtor_map_coinduct" theorems, since they're used in one example
2012-09-26, by blanchet
name tuning
2012-09-26, by blanchet
parameterized "subst_tac"
2012-09-26, by blanchet
generate high-level "maps", "sets", and "rels" properties
2012-09-26, by blanchet
use singular since there is always only one theorem
2012-09-26, by blanchet
nicer type var names
2012-09-26, by blanchet
renamed "dtor_rel_coinduct" etc. to "dtor_coinduct"
2012-09-26, by blanchet
renamed "dtor_coinduct" etc. to "dtor_map_coinduct"
2012-09-26, by blanchet
leave out some internal theorems unless "bnf_note_all" is set
2012-09-26, by blanchet
tuned
2012-09-26, by nipkow
added counterexamples
2012-09-26, by nipkow
tuned
2012-09-26, by nipkow
tuned
2012-09-25, by nipkow
more uniform graphview terminology;
2012-09-26, by wenzelm
proper Symbol.decode -- especially relevant for Proof General;
2012-09-26, by wenzelm
suppress empty tooltips;
2012-09-26, by wenzelm
obsolete;
2012-09-26, by wenzelm
updated keywords;
2012-09-26, by wenzelm
more uniform graphview terminology;
2012-09-26, by wenzelm
tuned pretty_locale/print_locale, with more basic pretty_locale_deps based on that;
2012-09-26, by wenzelm
proper install_fonts;
2012-09-26, by wenzelm
proper jvmpath for Windows;
2012-09-25, by wenzelm
basic integration of graphview into document model;
2012-09-25, by wenzelm
ML support for generic graph display, with browser and graphview backends (via print modes);
2012-09-25, by wenzelm
tuned;
2012-09-25, by wenzelm
more complete build;
2012-09-25, by wenzelm
proper error message;
2012-09-25, by wenzelm
separate module Graph_Display;
2012-09-25, by wenzelm
added graph encode/decode operations;
2012-09-25, by wenzelm
tuned;
2012-09-25, by wenzelm
minimal component and build setup for graphview;
2012-09-24, by wenzelm
added Graphview tool, based on Isabelle/Scala and Swing/Graphics2D;
2012-09-24, by Markus Kaiser
made smlnj even happier
2012-09-24, by haftmann
tuned proofs;
2012-09-24, by wenzelm
more explicit keyword1/keyword2 markup -- avoid potential conflict with input token markup produced by Token_Marker;
2012-09-24, by wenzelm
updated checksum, which appears to have changed accidentally;
2012-09-24, by wenzelm
updated to exec_process-1.0.2;
2012-09-24, by wenzelm
search bash via PATH as usual (this is no longer restricted to Cygwin with its known file-system layout);
2012-09-24, by wenzelm
discontinued futile attempt to hardwire build options into the image, sequential mode is enabled more robustly at runtime (cf. 3b0a60eee56e);
2012-09-24, by wenzelm
Mirabelle appears to work better in single-threaded mode;
2012-09-24, by wenzelm
generalized types
2012-09-24, by nipkow
tuned termination proof
2012-09-24, by nipkow
adapted examples to new names
2012-09-23, by blanchet
renamed coinduction principles to have "dtor" in the name
2012-09-23, by blanchet
renamed "set_incl" etc. to have "ctor" or "dtor" in the name
2012-09-23, by blanchet
renamed low-level "map_unique" to have "ctor" or "dtor" in the name
2012-09-23, by blanchet
renamed low-level "set_simps" and "set_induct" to have "ctor" or "dtor" in the name
2012-09-23, by blanchet
renamed "map_simps" to "{c,d}tor_maps"
2012-09-23, by blanchet
took out accidentally submitted "tracing" calls
2012-09-23, by blanchet
fixed bug in "fold" tactic with nested products (beyond the sum of product corresponding to constructors)
2012-09-23, by blanchet
simplified fact policies
2012-09-23, by blanchet
generate "rel_as_srel" and "rel_flip" properties
2012-09-23, by blanchet
started work on generation of "rel" theorems
2012-09-23, by blanchet
make smlnj happy
2012-09-23, by haftmann
more strict typscheme_equiv check: must fix variables of more specific type;
2012-09-22, by haftmann
cache should not contain material from descendant theory
2012-09-22, by haftmann
some PIDE NEWS from this summer;
2012-09-22, by wenzelm
tuned whitespace;
2012-09-22, by wenzelm
tuned;
2012-09-22, by wenzelm
tuned proofs;
2012-09-22, by wenzelm
report proper binding positions only -- avoid swamping document model with unspecific information;
2012-09-22, by wenzelm
accumulate under exec_id as well;
2012-09-22, by wenzelm
more restrictive pattern, to avoid malformed positions intruding the command range (cf. d7a1973b063c);
2012-09-22, by wenzelm
misc tuning;
2012-09-22, by wenzelm
Thy_Syntax.consolidate_spans is subject to editor_reparse_limit, for improved experience of unbalanced comments etc.;
2012-09-22, by wenzelm
tuned signature;
2012-09-22, by wenzelm
tuned proofs;
2012-09-21, by wenzelm
misc tuning;
2012-09-21, by wenzelm
tighten margin for TextArea instead of Lobo;
2012-09-21, by wenzelm
misc tuning;
2012-09-21, by wenzelm
renamed LFP low-level rel property to have ctor not dtor in its name
2012-09-21, by blanchet
changed base session for "HOL-BNF" for faster building in the typical case
2012-09-21, by blanchet
renamed "rel_simp" to "dtor_rel" and similarly for "srel"
2012-09-21, by blanchet
fixed a few names that escaped the renaming
2012-09-21, by blanchet
tuned whitespace
2012-09-21, by blanchet
merged
2012-09-21, by wenzelm
clean up lemmas used for composition
2012-09-21, by blanchet
created separate session "HOL-BNF-LFP" as a step towards eventual integration in "HOL" in the middle term
2012-09-21, by blanchet
renamed "Codatatype" directory "BNF" (and corresponding session) -- this opens the door to no-nonsense session names like "HOL-BNF-LFP"
2012-09-21, by blanchet
renamed top-level theory from "Codatatype" to "BNF"
2012-09-21, by blanchet
adapted examples to renamings
2012-09-21, by blanchet
renamed "pred" to "rel" (relator)
2012-09-21, by blanchet
renamed "rel" to "srel"
2012-09-21, by blanchet
fixed bug introduced by fold/unfold renaming
2012-09-21, by blanchet
renamed "iter"/"coiter" to "fold"/"unfold" (cf. Wadler)
2012-09-21, by blanchet
simplified code
2012-09-21, by blanchet
tuned a few ML names
2012-09-21, by blanchet
renamed "fld"/"unf" to "ctor"/"dtor"
2012-09-21, by blanchet
tuning
2012-09-21, by blanchet
renamed "upto" coinduction "strong"
2012-09-21, by blanchet
tuned variable names
2012-09-21, by blanchet
tuned names
2012-09-21, by nipkow
more termination proofs
2012-09-21, by nipkow
rel_Gr does not depend on map_wpull
2012-09-21, by traytel
renamed Output to Output1 and Output2 to Output, and thus make the new version the default;
2012-09-21, by wenzelm
more realistic sendback: pick exec_id from message position and text from buffer;
2012-09-21, by wenzelm
some support for hovering and sendback area;
2012-09-21, by wenzelm
merged
2012-09-21, by wenzelm
tuned antiquotations
2012-09-21, by traytel
merged
2012-09-21, by wenzelm
use iffD* instead of (s)subst instantiated with identity; tuned antiquotations;
2012-09-21, by traytel
conected CS to big-step
2012-09-21, by nipkow
generate "expand" property
2012-09-21, by blanchet
merge
2012-09-20, by blanchet
finished "disc_coiter_iff" etc. generation
2012-09-20, by blanchet
the Codatatype package currently needs all of Cardinals (temporary -- because of countable sets)
2012-09-20, by blanchet
generate coiter_iff and corec_iff theorems
2012-09-20, by blanchet
NEWS and CONTRIBUTORS for a5377f6d9f14 and f0ecc1550998
2012-09-20, by Andreas Lochbihler
more efficient code setup
2012-09-20, by Andreas Lochbihler
added "simp"s to coiter/corec theorems + export under "simps" name
2012-09-20, by blanchet
tuning
2012-09-20, by blanchet
tuned
2012-09-20, by nipkow
less rendering (cf. 28bd0709443a) -- avoid conflict with static token markup of different keyword kinds;
2012-09-21, by wenzelm
tuned painter;
2012-09-20, by wenzelm
clarified message background;
2012-09-20, by wenzelm
tuned rendering;
2012-09-20, by wenzelm
no caret painting;
2012-09-20, by wenzelm
text_rendering as managed task, with cancellation;
2012-09-20, by wenzelm
more management of Invoke_Scala tasks;
2012-09-20, by wenzelm
more direct Markup_Tree.from_XML;
2012-09-20, by wenzelm
tuned signature;
2012-09-20, by wenzelm
more direct Markup_Tree.from_XML;
2012-09-20, by wenzelm
tuned signature;
2012-09-20, by wenzelm
tuned;
2012-09-20, by wenzelm
removed lpfp and proved least pfp thm
2012-09-20, by nipkow
provide predicator, define relator
2012-09-20, by blanchet
tuning
2012-09-20, by blanchet
adapting "More_BNFs" to new relators/predicators
2012-09-20, by blanchet
fixed infinite loop with trivial rel_O_Gr + tuning
2012-09-20, by blanchet
adapted FP code to new relator approach
2012-09-20, by blanchet
tuning
2012-09-20, by blanchet
renamed "bnf_fp_util.ML" to "bnf_fp.ML"
2012-09-20, by blanchet
adapted BNF composition to new relator approach
2012-09-20, by blanchet
don't define relators unless necessary
2012-09-20, by blanchet
moved predicator definition before after_qed
2012-09-20, by blanchet
add rel as first-class citizen of BNF
2012-09-20, by blanchet
renamed "rel_def" to "rel_O_Gr"
2012-09-20, by blanchet
renamed "sum_setl" to "setl" and similarly for r
2012-09-20, by blanchet
tuned ID/DEADID setup
2012-09-20, by blanchet
JavaFX is inactive by default;
2012-09-19, by wenzelm
reactivate HOL-Mirabelle-ex with increased chances that it works most of the time (cf. bec1add86e79, a93d920707bb, be27a453aacc);
2012-09-19, by wenzelm
universal component exec_process -- avoids special Admin/components/windows and might actually improve stability of forked processes (without using perl);
2012-09-19, by wenzelm
more direct GUI component;
2012-09-19, by wenzelm
earlier treatment of embedded report/no_report messages (see also 4110cc1b8f9f);
2012-09-19, by wenzelm
made SML/NJ happy;
2012-09-19, by wenzelm
tuned;
2012-09-19, by wenzelm
merged
2012-09-19, by wenzelm
recording elapsed time in mutabelle for more detailed evaluation
2012-09-19, by bulwahn
Added missing predicators (for multisets and countable sets)
2012-09-18, by popescua
added top-level theory for Cardinals
2012-09-18, by popescua
group "simps" together
2012-09-18, by blanchet
register induct attributes
2012-09-18, by blanchet
further tuned simpset
2012-09-18, by blanchet
bnf_note_all mode for "pre_"-BNFs
2012-09-18, by traytel
separated registration of BNFs from bnf_def (BNFs are now stored only for bnf_def and (co)data commands)
2012-09-18, by traytel
tuned
2012-09-18, by nipkow
beautified names
2012-09-18, by nipkow
proved all upper bounds
2012-09-18, by nipkow
tuned simpset
2012-09-17, by blanchet
cleaner way of dealing with the set functions of sums and products
2012-09-17, by blanchet
handle the general case with more than two levels of nesting when discharging induction prem prems
2012-09-17, by blanchet
clean unfolding of prod and sum sets
2012-09-17, by blanchet
got rid of one "auto" in induction tactic
2012-09-17, by blanchet
cleaned up internal naming scheme for bnfs
2012-09-17, by traytel
more robust GUI component handlers;
2012-09-19, by wenzelm
more rendering;
2012-09-18, by wenzelm
minimal clipboard support (similar to org.lobobrowser.html.gui.HtmlBlockPanel);
2012-09-18, by wenzelm
output is read-only;
2012-09-18, by wenzelm
token marker for extended syntax styles;
2012-09-18, by wenzelm
pass base_snapshot to enable hyperlinks into other nodes;
2012-09-18, by wenzelm
more explicit message markup and rendering;
2012-09-18, by wenzelm
recover order of stacked markup;
2012-09-18, by wenzelm
some actual rich text markup via XML.content_markup;
2012-09-18, by wenzelm
proper separation of output messages;
2012-09-18, by wenzelm
some support for inital command markup;
2012-09-18, by wenzelm
more static rendering state;
2012-09-18, by wenzelm
Pretty_Text_Area is based on Rich_Text_Area;
2012-09-18, by wenzelm
renamed Text_Area_Painter to Rich_Text_Area;
2012-09-17, by wenzelm
tuned signature -- more general Text_Area_Painter operations;
2012-09-17, by wenzelm
tuned signature;
2012-09-17, by wenzelm
tuned signature;
2012-09-17, by wenzelm
tuned signature;
2012-09-17, by wenzelm
somewhat more general JEdit_Lib;
2012-09-17, by wenzelm
prefer official polyml-5.5.0;
2012-09-17, by wenzelm
bypass HOL-Mirabelle-ex in regular test, until its tendency to "hang" has been resolved;
2012-09-17, by wenzelm
merged
2012-09-17, by wenzelm
tuned
2012-09-17, by nipkow
updated to polyml-5.5.0;
2012-09-17, by wenzelm
some updates for polyml-5.5.0;
2012-09-17, by wenzelm
tuned
2012-09-17, by nipkow
alternative output panel, based on Pretty_Text_Area, based on JEditEmbeddedTextArea;
2012-09-16, by wenzelm
got rid of ad-hoc lift function
2012-09-16, by nipkow
converted wt into a set, tuned names
2012-09-16, by nipkow
use strip_typeN in bnf_def (instead of repairing strip_type)
2012-09-16, by traytel
removing find_theorems commands that were left in the developments accidently
2012-09-16, by bulwahn
tuning
2012-09-15, by blanchet
tuned code to avoid special case for "fun"
2012-09-15, by blanchet
tuned induction tactic
2012-09-15, by blanchet
tuned error message
2012-09-15, by blanchet
tuning
2012-09-15, by blanchet
typeclass formalising bounded subtraction
2012-09-15, by haftmann
dropped some unused identifiers
2012-09-15, by haftmann
export rel_mono theorem
2012-09-15, by traytel
merged two unfold steps
2012-09-14, by blanchet
took out one rotate_tac
2012-09-14, by blanchet
killed spurious rotate_tac; use auto instead of blast
2012-09-14, by blanchet
moved blast tactic to where it is actually needed
2012-09-14, by blanchet
fixed bug in "mk_map" for the "fun" case
2012-09-14, by blanchet
correct generalization to 3 or more mutually recursive datatypes
2012-09-14, by blanchet
provide more guidance, exploiting our knowledge of the goal
2012-09-14, by blanchet
fixed issue with bound variables in prem prems + tuning
2012-09-14, by blanchet
use right version of "mk_UnIN"
2012-09-14, by blanchet
select the right premise in "mk_induct_discharge_prem_prems_tac" instead of relying on backtracking
2012-09-14, by blanchet
tuned code before fixing "mk_induct_discharge_prem_prems_tac"
2012-09-14, by blanchet
tuned proofs;
2012-09-14, by wenzelm
merged
2012-09-14, by wenzelm
polished the induction
2012-09-14, by blanchet
put the flat at the right place (to avoid exceptions)
2012-09-14, by blanchet
fixed variable exporting problem
2012-09-14, by blanchet
compile
2012-09-14, by blanchet
added induct tactic
2012-09-14, by blanchet
tuning
2012-09-14, by blanchet
renamed "mk_UnN" to "mk_UnIN"
2012-09-14, by blanchet
merged two commands
2012-09-14, by blanchet
allow default values to refer to selector arguments -- this is useful, e.g. for tllist: ttl (TNil x) = TNil x (example by Andreas Lochbihler)
2012-09-14, by blanchet
distinguish between nested and nesting BNFs
2012-09-14, by blanchet
make tactic more robust in the case where "asm_simp_tac" already finishes the job
2012-09-14, by blanchet
derive induction via backward proof, to ensure that the premises are in the right order for constructors like "X x y x" where x and y are mutually recursive
2012-09-14, by blanchet
no longer react on global_settings (cf. 34ac36642a31);
2012-09-14, by wenzelm
refined output panel: more value-oriented approach to update and caret focus;
2012-09-14, by wenzelm
clarified markup names;
2012-09-14, by wenzelm
more general Document_Model.point_range;
2012-09-14, by wenzelm
more static handling of rendering options;
2012-09-14, by wenzelm
tuned options (again);
2012-09-14, by wenzelm
more scalable option-group;
2012-09-14, by wenzelm
tuned
2012-09-14, by nipkow
merged
2012-09-13, by wenzelm
tuned proofs;
2012-09-13, by wenzelm
remove theory Real_Integration, not needed since 44e42d392c6e when Euclidean spaces where introduced
2012-09-13, by hoelzl
workaround for HOL-Mirabelle-ex oddities;
2012-09-13, by wenzelm
instructions for quick start in 20min;
2012-09-13, by wenzelm
more liberal init_components: base dir may get created later when resolving missing components;
2012-09-13, by wenzelm
more efficient painting based on cached result;
2012-09-13, by wenzelm
more standard init_components -- particularly important to pick up correct jdk/scala version;
2012-09-13, by wenzelm
tuned
2012-09-13, by nipkow
merged
2012-09-12, by wenzelm
rough and ready induction
2012-09-12, by blanchet
nicer error message, indicating which type is empty (relying on metatheoretical completeness proof here)
2012-09-12, by blanchet
observe context more carefully when producing "fresh" variables -- for increased chances that method "subst" works in local context (including that of forked proofs);
2012-09-12, by wenzelm
eliminated some old material that is unused in the visible universe;
2012-09-12, by wenzelm
tuning
2012-09-12, by blanchet
set up things for (co)induction sugar
2012-09-12, by blanchet
tuning
2012-09-12, by blanchet
added sumEN_tupled_balanced
2012-09-12, by blanchet
load fonts into JavaFX as well;
2012-09-12, by wenzelm
some support for actual HTML rendering;
2012-09-12, by wenzelm
merged
2012-09-12, by wenzelm
free variable name tuning
2012-09-12, by blanchet
reuse generated names (they look better + slightly more efficient)
2012-09-12, by blanchet
desambiguate grammar (e.g. for Nil's mixfix ("[]"))
2012-09-12, by blanchet
avoided duplicate lemma
2012-09-12, by blanchet
put an underscore between names, for compatibility with old package (and also because it makes sense)
2012-09-12, by blanchet
got rid of metis calls
2012-09-12, by blanchet
tuning
2012-09-12, by blanchet
removed obsolete argument "int" and thus made SML/NJ happy (cf. 03bee3a6a1b7);
2012-09-12, by wenzelm
standardized ML aliases;
2012-09-12, by wenzelm
tuned headers;
2012-09-12, by wenzelm
avoid spaces in markup names, which might cause problems in boundary situations (e.g. HTML class);
2012-09-12, by wenzelm
discontinued experiment with literal replacement text in PDF (cf. b646316f8b3c, 2ff10e613689);
2012-09-12, by wenzelm
more robust interrupt handling;
2012-09-12, by wenzelm
some attempts to synchronize ROOT/files and document/build;
2012-09-12, by wenzelm
tuned error;
2012-09-12, by wenzelm
option_pred characterization
2012-09-12, by traytel
true vs. True in pattern matching
2012-09-12, by traytel
reduced theory dependencies
2012-09-12, by blanchet
tuning
2012-09-12, by blanchet
moved theorems closer to where they are used
2012-09-12, by blanchet
tuning
2012-09-12, by blanchet
renamed "Ordinals_and_Cardinals" to "Cardinals"
2012-09-12, by blanchet
split basic BNFs into really basic ones and others, and added Andreas Lochbihler's "option" BNF
2012-09-12, by blanchet
less
more
|
(0)
-30000
-10000
-3000
-1000
-960
+960
+1000
+3000
+10000
+30000
tip