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.
updated docs
2011-12-21, by blanchet
killed "guard@?" encodings -- they were found to be unsound
2011-12-21, by blanchet
extend previous optimizations to guard-based encodings
2011-12-21, by blanchet
treat polymorphic constructors specially in @? encodings
2011-12-21, by blanchet
tuning
2011-12-21, by blanchet
no need for type arguments for monomorphic constructors of polymorphic datatypes (e.g. "Nil")
2011-12-21, by blanchet
added some basic documentation about method induction_schema extracted from old NEWS
2011-12-21, by bulwahn
adding documentation about the quickcheck_generator command in the IsarRef
2011-12-21, by bulwahn
extending quickcheck example
2011-12-21, by bulwahn
NEWS
2011-12-21, by bulwahn
quickcheck_generator command also creates random generators
2011-12-21, by bulwahn
don't try to avoid SPASS keywords; instead, just suffix an underscore to all generated identifiers
2011-12-20, by blanchet
one more SPASS identifier
2011-12-20, by blanchet
tuning
2011-12-20, by blanchet
merged
2011-12-20, by noschinl
meaningful error message on failing merges of coercion tables
2011-12-17, by traytel
add simp rules for enat and ereal
2011-12-20, by noschinl
add lemmas
2011-12-19, by noschinl
add lemmas
2011-12-19, by noschinl
weaken preconditions on lemmas
2011-12-19, by noschinl
add lemmas
2011-12-19, by noschinl
removing some debug output in quotient_definition
2011-12-20, by bulwahn
adding quickcheck generators in some HOL-Library theories
2011-12-20, by bulwahn
adding quickcheck generator for distinct lists; adding examples
2011-12-20, by bulwahn
added keywords
2011-12-20, by bulwahn
quickcheck generators for abstract types; tuned
2011-12-20, by bulwahn
exporting instantiation functions in quickcheck for their usage in abstract generators
2011-12-20, by bulwahn
generalize ensure_sort_datatype to ensure_sort in quickcheck_common to allow generators for abstract types;
2011-12-20, by bulwahn
tuned
2011-12-20, by bulwahn
tuned
2011-12-20, by bulwahn
ensure TPTP FOF/TFF/THF formulas are close
2011-12-20, by blanchet
tuned
2011-12-20, by nipkow
merged
2011-12-19, by nipkow
added old chestnut
2011-12-19, by nipkow
isarfied proof; add log to DERIV_intros
2011-12-19, by hoelzl
tendsto lemmas for ln and powr
2011-12-15, by huffman
tuned settings;
2011-12-18, by wenzelm
updated jedit_build component;
2011-12-17, by wenzelm
updated version information;
2011-12-17, by wenzelm
patch for Lobo/Cobra 0.98.4 to make it work with Java 1.7 (see also http://sourceforge.net/tracker/index.php?func=detail&aid=2991043&group_id=139023&atid=742262);
2011-12-17, by wenzelm
eliminated Drule.export_without_context which is not really required here;
2011-12-17, by wenzelm
tuned signature;
2011-12-17, by wenzelm
enforce short hostname on all platforms (especially macbroy2);
2011-12-17, by wenzelm
clarified modules that contribute to datatype package;
2011-12-17, by wenzelm
tuned signature;
2011-12-17, by wenzelm
merged
2011-12-16, by wenzelm
merged
2011-12-16, by nipkow
improved indexed complete lattice
2011-12-16, by nipkow
more elementary defs;
2011-12-16, by wenzelm
eliminated old-fashioned Global_Theory.add_thms(s);
2011-12-16, by wenzelm
prefer sorting from Scala library;
2011-12-16, by wenzelm
prefer Name.context operations;
2011-12-16, by wenzelm
tuned;
2011-12-16, by wenzelm
clarified modules that contribute to datatype package;
2011-12-16, by wenzelm
tuned signature;
2011-12-16, by wenzelm
merged;
2011-12-15, by wenzelm
tuned;
2011-12-15, by wenzelm
add complementary lemmas for {min,max}_least
2011-12-15, by noschinl
add lemmas about limits
2011-12-15, by noschinl
clarified module dependencies: Datatype_Data, Datatype_Case, Rep_Datatype;
2011-12-15, by wenzelm
separate rep_datatype.ML;
2011-12-15, by wenzelm
misc tuning and simplification;
2011-12-15, by wenzelm
more stats;
2011-12-15, by wenzelm
made SML/NJ happier
2011-12-15, by blanchet
merged
2011-12-15, by nipkow
tuned
2011-12-15, by nipkow
hiding the precious name map_entry in AList_Impl
2011-12-15, by bulwahn
killed dead code
2011-12-14, by blanchet
use new redirection algorithm in Sledgehammer
2011-12-14, by blanchet
fixed parsing of TPTP atoms
2011-12-14, by blanchet
tuned signature;
2011-12-14, by wenzelm
avoid fragile Sign.intern_const -- pass internal names directly;
2011-12-14, by wenzelm
tuned;
2011-12-14, by wenzelm
added new proof redirection code
2011-12-14, by blanchet
SPASS is incomplete because of the -Splits and -FullRed options, not just because of -SOS=1 -- don't pretend the opposite
2011-12-14, by blanchet
make sure that all symbols are declared in untyped SPASS DFG output (broken since 3b8606fba2dd)
2011-12-14, by blanchet
NEWS
2011-12-14, by bulwahn
correcting dependencies after renaming
2011-12-14, by bulwahn
tuned header after renaming
2011-12-14, by bulwahn
moving AList theory to AList_Impl to make space for the association lists with invariant
2011-12-14, by bulwahn
merged
2011-12-14, by bulwahn
adding map_entry to AList theory
2011-12-14, by bulwahn
adding map_default to AList theory
2011-12-14, by bulwahn
fixed typo in theorem name in AList theory
2011-12-14, by bulwahn
adding code attribute to enable evaluation of equality on multisets
2011-12-14, by bulwahn
merged
2011-12-14, by wenzelm
updated Sledgehammer/SMT docs
2011-12-14, by blanchet
tuned signature;
2011-12-14, by wenzelm
eliminated dead code;
2011-12-14, by wenzelm
some full isatest runs, which include benchmark targets;
2011-12-14, by wenzelm
more visible benchmarks;
2011-12-14, by wenzelm
fixed Nitpick definition of "<" on "real"s
2011-12-14, by blanchet
replace 'lemmas' with 'lemma'
2011-12-14, by huffman
merged
2011-12-14, by huffman
more simp rules for sbintrunc
2011-12-13, by huffman
add simp rules for sbintrunc applied to numerals
2011-12-13, by huffman
replace many uses of 'lemmas' with explicit 'lemma'
2011-12-13, by huffman
add lemma bin_nth_zero
2011-12-13, by huffman
add simp rules for bintrunc applied to numerals
2011-12-13, by huffman
add simp rules for bin_rest and bin_last applied to numerals
2011-12-13, by huffman
add simp rules for bin_sign applied to numerals
2011-12-13, by huffman
add simp rules for BIT applied to numerals
2011-12-13, by huffman
declare BIT_eq_iff [iff]; remove unneeded lemmas
2011-12-13, by huffman
towards removing BIT_simps from the simpset
2011-12-13, by huffman
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
reporting random compilation also catches match exceptions internally
2011-12-01, by bulwahn
the narrowing also indicates if counterexample is potentially spurious
2011-12-01, by bulwahn
the simple exhaustive compilation also indicates if counterexample is potentially spurious;
2011-12-01, by bulwahn
quickcheck-random compilation also indicates if the counterexample is potentially spurious or not
2011-12-01, by bulwahn
changing the exhaustive generator signatures;
2011-12-01, by bulwahn
quickcheck's compilation returns if it is genuine counterexample or a counterexample due to a match exception
2011-12-01, by bulwahn
adding examples for quickcheck-random
2011-12-01, by bulwahn
removing exception handling now that is caught at some other point;
2011-12-01, by bulwahn
quickcheck random can also find potential counterexamples;
2011-12-01, by bulwahn
merged
2011-12-01, by wenzelm
merged IMP/Util into IMP/Vars
2011-12-01, by nipkow
use list theorems in Dining Cryptographers and Koepf Duermuth Countermeasure
2011-12-01, by hoelzl
cardinality of sets of lists
2011-12-01, by hoelzl
do not import examples Probability theory
2011-12-01, by hoelzl
moved theorems about distribution to the definition; removed oopsed-lemma
2011-12-01, by hoelzl
rename finite_prob_space.setsum_distribution, it collides with prob_space.setsum_distribution
2011-12-01, by hoelzl
less
more
|
(0)
-30000
-10000
-3000
-1000
-240
+240
+1000
+3000
+10000
+30000
tip