Mercurial
Mercurial
>
repos
>
isabelle
/ graph
summary
|
shortlog
|
changelog
| graph |
tags
|
bookmarks
|
branches
|
files
|
gz
|
help
less
more
|
(0)
-30000
-10000
-3000
-1000
-120
+120
+1000
+3000
+10000
+30000
tip
Find changesets by keywords (author, files, the commit message), revision number or hash, or
revset expression
.
The revision graph only works with JavaScript-enabled browsers.
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
less
more
|
(0)
-30000
-10000
-3000
-1000
-120
+120
+1000
+3000
+10000
+30000
tip