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.
type signature for bin_sign
2011-12-13, by huffman
remove some unwanted numeral-representation-specific simp rules
2011-12-13, by huffman
remove redundant lemmas
2011-12-13, by huffman
reorder some definitions and proofs, in preparation for new numeral representation
2011-12-13, by huffman
merged
2011-12-13, by wenzelm
added lemmas
2011-12-13, by noschinl
added concrete syntax
2011-12-13, by nipkow
'datatype' specifications allow explicit sort constraints;
2011-12-13, by wenzelm
do not open ML structures;
2011-12-13, by wenzelm
tuned;
2011-12-13, by wenzelm
removed dead code;
2011-12-13, by wenzelm
comment;
2011-12-13, by wenzelm
connect while_option with lfp
2011-12-13, by nipkow
lemmas about Kleene iteration
2011-12-13, by nipkow
merged
2011-12-13, by wenzelm
avoid multiple type decls in TFF (improves on cef82dc1462d)
2011-12-13, by blanchet
added missing quantifier
2011-12-13, by blanchet
remove needless declaration in TFF1 problems
2011-12-13, by blanchet
correctly declare implicit TFF1 types that appear first as type arguments with "$tType" and not "$i
2011-12-13, by blanchet
modernized specifications;
2011-12-13, by wenzelm
support phantom types as quotient types
2011-12-13, by kuncar
merged
2011-12-12, by wenzelm
merged
2011-12-12, by nipkow
tuned
2011-12-12, by nipkow
datatype dtyp with explicit sort information;
2011-12-12, by wenzelm
tuned;
2011-12-12, by wenzelm
updated generated file;
2011-12-12, by wenzelm
tuned quickcheck's response
2011-12-12, by bulwahn
hiding constants and facts in the Quickcheck_Exhaustive and Quickcheck_Narrowing theory;
2011-12-12, by bulwahn
merged
2011-12-12, by huffman
replace more uses of 'lemmas' with explicit 'lemma';
2011-12-12, by huffman
Add Quotient_Rat: an example of using the quotient package with partial equivalence relations, defining rational numbers.
2011-12-12, by Cezary Kaliszyk
fix spelling
2011-12-11, by huffman
fix spelling
2011-12-11, by huffman
added IMP/Live_True.thy
2011-12-11, by nipkow
replace many uses of 'lemmas' with 'lemma';
2011-12-11, by huffman
prove class instances without extra lemmas
2011-12-10, by huffman
finite class instance for word type; remove unused lemmas
2011-12-10, by huffman
remove unused lemmas
2011-12-10, by huffman
generalize some lemmas
2011-12-10, by huffman
merged
2011-12-10, by huffman
tidied Word.thy;
2011-12-10, by huffman
remove redundant lemma word_diff_minus
2011-12-09, by huffman
remove some duplicate lemmas, simplify some proofs
2011-12-09, by huffman
Quotient_Info stores only relation maps
2011-12-09, by kuncar
hiding definitional facts in Quickcheck; introducing catch_match more honestly
2011-12-09, by bulwahn
added dependencies
2011-12-09, by kuncar
added an example file with lifting of constants with contravariant and co/contravariant types
2011-12-09, by kuncar
merged
2011-12-09, by kuncar
make ctxt the first parameter
2011-12-09, by kuncar
context/theory parametres tuned
2011-12-09, by kuncar
maps are taken from enriched type infrastracture, rewritten lifting of constants, now we can lift even contravariant and co/contravariant types
2011-12-09, by kuncar
add induction rule for list_all2
2011-12-09, by huffman
deactivating quickcheck_narrowing if Efficient_Nat theory is loaded
2011-12-09, by bulwahn
tuned quickcheck's response
2011-12-09, by bulwahn
more systematic lemma name
2011-12-09, by noschinl
adding examples for quickcheck narrowing about partial functions
2011-12-08, by bulwahn
removing special code generator setup for hd and last function because this causes problems with quickcheck narrowing as the Haskell Prelude functions throw errors that cannot be caught instead of PatternFail exceptions
2011-12-08, by bulwahn
HOLCF/ex/Letrec.thy: keep class 'domain' as default sort
2011-12-08, by huffman
more error checking for fixrec
2011-12-08, by huffman
reinstate old functions cfst and csnd as abbreviations
2011-12-08, by huffman
merged
2011-12-08, by nipkow
tuned
2011-12-08, by nipkow
merged
2011-12-07, by Christian Urban
added a specific tactic and method that deal with partial equivalence relations
2011-12-07, by Christian Urban
use same order of facts for preplay as for actual reconstruction -- Metis sometimes exhibits very different timings depending on the order of the facts
2011-12-07, by blanchet
avoid multiple TFF1 declarations
2011-12-07, by blanchet
updated TFF1 support
2011-12-07, by blanchet
updated Metis to 20110926 version
2011-12-07, by blanchet
remove unnecessary sublocale instantiations in HOL-Probability (for clarity and speedup); remove Infinite_Product_Measure.product_prob_space which was a duplicate of Probability_Measure.product_prob_space
2011-12-07, by hoelzl
remove mem_(c)ball_0 and centre_in_(c)ball from simpset, as rules mem_(c)ball always match instead
2011-12-05, by huffman
add cancellation simprocs for type enat
2011-12-07, by huffman
tuned
2011-12-07, by nipkow
increasing quickcheck's timeout in the example theory to avoid failures on the testing infrastructure
2011-12-06, by bulwahn
tuned proofs
2011-12-06, by hoelzl
added lemmas
2011-12-06, by nipkow
tuned proof
2011-12-05, by nipkow
real is better supported than real_of_nat, use it in the nat => ereal coercion
2011-12-05, by hoelzl
merged
2011-12-05, by kuncar
the note about morphisms moved in the description part
2011-12-05, by kuncar
updating documentation about quiet and verbose options in quickcheck
2011-12-05, by bulwahn
making the default behaviour of quickcheck a little bit less verbose;
2011-12-05, by bulwahn
adding verbose configuration to quickcheck
2011-12-05, by bulwahn
random reporting compilation returns if counterexample is genuine or potentially spurious, and takes genuine_only option as argument
2011-12-05, by bulwahn
the reporting random testing also returns if the counterexample is genuine or potentially spurious
2011-12-05, by bulwahn
exhaustive returns if a counterexample is genuine or potentially spurious in the presence of assumptions more correctly
2011-12-05, by bulwahn
inverted flag potential to genuine_only in the quickcheck narrowing Haskell code
2011-12-05, by bulwahn
NEWS
2011-12-05, by bulwahn
documenting the genuine_only option in quickcheck;
2011-12-05, by bulwahn
renaming potential flag to genuine_only flag with an inverse semantics
2011-12-05, by bulwahn
quickcheck narrowing continues searching after found a potentially spurious counterexample
2011-12-05, by bulwahn
outputing the potentially spurious counterexample and continue search
2011-12-05, by bulwahn
dynamic genuine_flag in compilation of random and exhaustive
2011-12-05, by bulwahn
indicating where the restart should occur; making safe_if dynamic
2011-12-05, by bulwahn
merged
2011-12-05, by nipkow
enforce parantheses around SKIP {_}
2011-12-05, by nipkow
adding genuine flag to predicate_compile_quickcheck and prolog_quickcheck (cf. 5e46c225370e);
2011-12-04, by bulwahn
merged
2011-12-04, by huffman
remove Library/Diagonalize.thy, because Library/Nat_Bijection.thy includes all the same functionality
2011-12-04, by huffman
missing dependency
2011-12-04, by nipkow
improved var names
2011-12-04, by nipkow
invariant holds before loop
2011-12-03, by nipkow
caret_range based on BreakIterator, which handles combined unicode characters as well;
2011-12-03, by wenzelm
misc tuning;
2011-12-02, by wenzelm
some localization;
2011-12-02, by wenzelm
eliminated some legacy operations;
2011-12-02, by wenzelm
more antiquotations;
2011-12-02, by wenzelm
tuned whitespace;
2011-12-02, by wenzelm
eliminated some legacy operations;
2011-12-02, by wenzelm
removed dead code, which has never been active in recorded history;
2011-12-02, by wenzelm
do not open ML structures;
2011-12-02, by wenzelm
tuned signature;
2011-12-02, by wenzelm
hide quickcheck constants Abs_cfun and Rep_cfun, to avoid clash with HOLCF
2011-12-02, by huffman
hiding internal constants and facts more properly
2011-12-01, by bulwahn
removing catch_match' now that catch_match is polymorphic
2011-12-01, by bulwahn
adapting exhaustive generators in record package
2011-12-01, by bulwahn
outputing if counterexample is potentially spurious or not
2011-12-01, by bulwahn
making catch_match polymorphic
2011-12-01, by bulwahn
compilations return genuine flag to quickcheck framework
2011-12-01, by bulwahn
extending quickcheck's result by the genuine flag
2011-12-01, by bulwahn
less
more
|
(0)
-30000
-10000
-3000
-1000
-120
+120
+1000
+3000
+10000
+30000
tip