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.
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
remove duplicate theorem setsum_real_distribution
2011-12-01, by hoelzl
clarified modules (again) -- NB: both Document and Protocol are specific to this particular prover;
2011-12-01, by wenzelm
updated Sledgehammer docs with new/renamed options
2011-12-01, by blanchet
added "minimize" option for more control over automatic minimization
2011-12-01, by blanchet
renamed "slicing" to "slice"
2011-12-01, by blanchet
tuning
2011-12-01, by blanchet
minor example tweak
2011-12-01, by blanchet
renamed inner syntax categories "num" to "num_token" and "xnum" to "xnum_token";
2011-12-01, by wenzelm
updated markup conforming to ML side;
2011-12-01, by wenzelm
discontinued obsolete datatype "alt_names";
2011-11-30, by wenzelm
misc tuning;
2011-11-30, by wenzelm
merged
2011-11-30, by wenzelm
removed outdated comment moved back and updated (at the direct request of Christian Urban)
2011-11-30, by kuncar
more stable introduction of the internally used unknown term
2011-11-30, by bulwahn
prefer typedef without alternative name;
2011-11-30, by wenzelm
prefer cpodef without extra definition;
2011-11-30, by wenzelm
prefer typedef without extra definition and alternative name;
2011-11-30, by wenzelm
tuned layout;
2011-11-30, by wenzelm
tuned header;
2011-11-30, by wenzelm
updated version information;
2011-11-30, by wenzelm
removed outdated comment
2011-11-30, by kuncar
adding examples for the potential counterexamples in the simple scheme
2011-11-30, by bulwahn
also potential counterexamples in the simple exhaustive testing in quickcheck
2011-11-30, by bulwahn
quickcheck does not show evaluation terms of equations if they are simply free variables to avoid duplicated output; tuned
2011-11-30, by bulwahn
adding more verbose messages to exhaustive quickcheck
2011-11-30, by bulwahn
quickcheck narrowing also shows potential counterexamples
2011-11-30, by bulwahn
adding a exception-safe term reification step in quickcheck; adding examples
2011-11-30, by bulwahn
quickcheck returns counterexamples that are potentially spurious due to underspecified code equations and match exceptions
2011-11-30, by bulwahn
adding parsing of potential configuration to quickcheck command
2011-11-30, by bulwahn
adding quickcheck's potential configuration
2011-11-30, by bulwahn
more conventional file name;
2011-11-29, by wenzelm
merged
2011-11-29, by wenzelm
updated documentation for the quotient package
2011-11-29, by kuncar
merged
2011-11-29, by kuncar
alternative names of morphisms in the definition of a quotient type can be specified
2011-11-29, by kuncar
adjusting antiquote_setup (cf. d83797ef0d2d)
2011-11-29, by bulwahn
clarified Time vs. Timing;
2011-11-29, by wenzelm
separate compilation of PIDE vs. Pure sources, which enables independent Scala library;
2011-11-29, by wenzelm
clarified modules;
2011-11-29, by wenzelm
tuned proofs;
2011-11-29, by wenzelm
rearranged files;
2011-11-29, by wenzelm
merged
2011-11-29, by huffman
use HOL_basic_ss instead of HOL_ss for internal simproc proofs (cf. b36eedcd1633)
2011-11-28, by huffman
explicit indication of modules for independent Scala library;
2011-11-28, by wenzelm
separate module for concrete Isabelle markup;
2011-11-28, by wenzelm
renamed Isabelle_Markup to Isabelle_Rendering to emphasize its meaning and make room for Pure Isabelle_Markup module;
2011-11-28, by wenzelm
tuned signature (according to ML version);
2011-11-28, by wenzelm
merged
2011-11-28, by nipkow
Hide Product_Type.Times - too precious an identifier
2011-11-28, by nipkow
more antiquotations;
2011-11-28, by wenzelm
tuned messages;
2011-11-28, by wenzelm
avoid stepping outside of context -- plain zero_var_indexes should be sufficient;
2011-11-28, by wenzelm
increasing timeout to avoid test failures
2011-11-28, by bulwahn
merged
2011-11-27, by wenzelm
merged
2011-11-27, by nipkow
simplified Collecting1 and renamed: step -> step', step_cs -> step
2011-11-27, by nipkow
more antiquotations;
2011-11-27, by wenzelm
tuned proof;
2011-11-27, by wenzelm
permissive update for improved "tool compliance";
2011-11-27, by wenzelm
just one data slot per module;
2011-11-27, by wenzelm
tuned;
2011-11-27, by wenzelm
tuned;
2011-11-27, by wenzelm
more antiquotations;
2011-11-27, by wenzelm
misc tuning;
2011-11-27, by wenzelm
refined "literal" document style, with some correspondence to actual text source;
2011-11-27, by wenzelm
modernized section about congruence rules;
2011-11-27, by wenzelm
sharing of token source with span source;
2011-11-26, by wenzelm
memoing of forked proofs;
2011-11-26, by wenzelm
tuned;
2011-11-26, by wenzelm
removed obsolete argument (cf. 954e9d6782ea);
2011-11-25, by wenzelm
merged
2011-11-25, by wenzelm
removed obsolete uses of Local_Theory.restore -- package composition P1 #> P2 no longer requires them due to 57def0b39696: P2 finds the results of P1 in the auxiliary context
2011-11-25, by krauss
merged
2011-11-25, by nipkow
tuned
2011-11-25, by nipkow
increased stack limits (again, cf. d9cf3520083c and 77c3e74bd954);
2011-11-25, by wenzelm
explicit change_parser thread, which avoids undirected Future.fork with its tendency towards hundreds of worker threads;
2011-11-25, by wenzelm
tuned proofs;
2011-11-25, by wenzelm
retain stderr and include it in syslog, which is buffered and thus increases the chance that users see remains from crashes etc.;
2011-11-25, by wenzelm
prefer Parser.make_gram over Parser.merge_gram, to approximate n-ary merges on theory import;
2011-11-25, by wenzelm
recovered structural equality from 9d97bd3c086a, otherwise update_perspective might be issued over and over again, canceling a pending/slow execution;
2011-11-25, by wenzelm
proper intro? declarations -- NB: elim? indexes on major premise, which is too flexible here and easily leads to inefficiences (cf. a0336f8b6558);
2011-11-25, by wenzelm
improved example to only use quotient_definitions; added lemmas to serve as possible replacement for the existing RBT theory
2011-11-25, by bulwahn
in a local context, also the free variable case needs to be analysed default tip
2011-11-25, by Christian Urban
speed-up proof;
2011-11-24, by wenzelm
more abstract datatype stamp, which avoids pointless allocation of mutable cells;
2011-11-24, by wenzelm
modernized some old-style infix operations, which were left over from the time of ML proof scripts;
2011-11-24, by wenzelm
simplified -- empty_ss already contains minimal mksimps;
2011-11-24, by wenzelm
Abstract interpretation is now based uniformly on annotated programs,
2011-11-24, by nipkow
tuned;
2011-11-23, by wenzelm
tuned;
2011-11-23, by wenzelm
modernized some old-style infix operations, which were left over from the time of ML proof scripts;
2011-11-23, by wenzelm
tuned;
2011-11-23, by wenzelm
updated according to bdcaa3f3a2f4;
2011-11-23, by wenzelm
updated proof;
2011-11-23, by wenzelm
tuned
2011-11-23, by nipkow
remove outdated comment
2011-11-23, by huffman
NEWS;
2011-11-21, by wenzelm
simplified read_instantiate -- no longer need to assign values, since rule attributes are now static;
2011-11-21, by wenzelm
drop vacuous decls;
2011-11-21, by wenzelm
tuned;
2011-11-21, by wenzelm
tuned header;
2011-11-21, by wenzelm
misspelled name
2011-11-21, by kuncar
eliminated obsolete "standard";
2011-11-20, by wenzelm
eliminated obsolete "standard";
2011-11-20, by wenzelm
less
more
|
(0)
-30000
-10000
-3000
-1000
-240
+240
+1000
+3000
+10000
+30000
tip