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.
more Nitpick doc updates
2012-01-04, by blanchet
reenable Kodkodi in Mira now that Nitpick has been ported to 'a set constructor
2012-01-04, by blanchet
reenable Kodkodi in Isatest now that Nitpick has been ported to 'a set constructor
2012-01-04, by blanchet
fixed bisimilarity axiom -- avoid "insert" with wrong type
2012-01-03, by blanchet
tuning
2012-01-03, by blanchet
updated Nitpick docs after "set" reintroduction
2012-01-03, by blanchet
no abuse of notation
2012-01-03, by blanchet
always treat "unit" as a deep datatype, so that we get a good interaction with the record syntax (2.7 of the Nitpick manual)
2012-01-03, by blanchet
more robust destruction of "set Collect" idiom
2012-01-03, by blanchet
handle starred predicates correctly w.r.t. "set"
2012-01-03, by blanchet
handle "Id" gracefully w.r.t. "set"
2012-01-03, by blanchet
reintroduced 'refute' calls taken out after reintroducing the "set" constructor, and use "expect" feature
2012-01-03, by blanchet
handle "set" correctly in Refute -- inspired by old code from Isabelle2007
2012-01-03, by blanchet
create consts with proper "set" types
2012-01-03, by blanchet
tuned Refute
2012-01-03, by blanchet
lower cardinality for faster testing
2012-01-03, by blanchet
simplify mem Collect
2012-01-03, by blanchet
tuning
2012-01-03, by blanchet
ported Minipick to "set"
2012-01-03, by blanchet
fixed set extensionality code
2012-01-03, by blanchet
tuned import
2012-01-03, by blanchet
construct correct "set" type for wf goal
2012-01-03, by blanchet
fixed Nitpick's typedef handling w.r.t. "set"
2012-01-03, by blanchet
fixed type annotations
2012-01-03, by blanchet
rationalized output (a bit)
2012-01-03, by blanchet
fixed a few more bugs in \Nitpick's new "set" support
2012-01-03, by blanchet
regenerate SMT example certificates, to reflect "set" type constructor
2012-01-03, by blanchet
port part of Nitpick to "set" type constructor
2012-01-03, by blanchet
reintroduced failing examples now that they work again, after reintroduction of "set"
2012-01-03, by blanchet
ported mono calculus to handle "set" type constructors
2012-01-03, by blanchet
fixed spurious catch-all patterns
2012-01-03, by blanchet
more benchmarks;
2012-01-03, by wenzelm
tuned
2012-01-02, by nipkow
ported "Sets" example to "set" type constructor
2012-01-02, by blanchet
ported a dozen of proofs to the "set" type constructor
2012-01-02, by blanchet
reintroduced "metis" call taken out after reintroducing "set" as a constructor, and added two "metis" calls that used to be too slow
2012-01-02, by blanchet
update docs to reflect "Manual_Nits"
2012-01-02, by blanchet
removed special handling for set constants in relevance filter
2012-01-02, by blanchet
reintroduced Sledgehammer call taken out by 9bc924006136, with some hints to guide the naive relevance filter
2012-01-02, by blanchet
killed unfold_set_const option that makes no sense now that set is a type constructor again
2012-01-02, by blanchet
tuned
2012-01-02, by nipkow
removed unnecessary lemmas
2012-01-02, by nipkow
tuned proofs
2012-01-02, by nipkow
tuned var names
2012-01-01, by nipkow
tuned argument order
2012-01-01, by nipkow
merged
2012-01-01, by huffman
add simp rules for bitwise word operations with 1
2011-12-30, by huffman
tuned types
2011-12-31, by nipkow
disabled failing sledgehammer unit test (collateral damage of 184d36538e51)
2011-12-31, by krauss
disabled kodkodi in mira runs as well (cf. 493d9c4d7ed5)
2011-12-31, by krauss
merged
2011-12-30, by berghofe
Made gen_dest_case more robust against eta contraction
2011-12-30, by berghofe
merged
2011-12-30, by wenzelm
remove unnecessary intermediate lemmas
2011-12-30, by huffman
tuned;
2011-12-30, by wenzelm
eliminated old-fashioned Global_Theory.add_thms;
2011-12-30, by wenzelm
simplified proof -- avoid res_inst_tac, afford plain asm_full_simp_tac;
2011-12-30, by wenzelm
simplified proof;
2011-12-30, by wenzelm
simplified proof;
2011-12-30, by wenzelm
simplified proof;
2011-12-30, by wenzelm
more parallelism;
2011-12-30, by wenzelm
tuned;
2011-12-30, by wenzelm
merged
2011-12-29, by wenzelm
tuned -- afford slightly larger simpset in simp_defs_tac;
2011-12-29, by wenzelm
tuned -- standard proofs by default;
2011-12-29, by wenzelm
do not fork skipped proofs;
2011-12-29, by wenzelm
clarified timeit_msg;
2011-12-29, by wenzelm
tuned;
2011-12-29, by wenzelm
comments;
2011-12-29, by wenzelm
remove constant 'ccpo.lub', re-use constant 'Sup' instead
2011-12-29, by huffman
merged
2011-12-29, by nipkow
tuned
2011-12-29, by nipkow
conversions from sets to predicates and vice versa; extensionality on predicates
2011-12-29, by haftmann
added implementation of pred_of_set
2011-12-29, by haftmann
fundamental theorems on Set.bind
2011-12-29, by haftmann
updated generated files;
2011-12-29, by wenzelm
qualified Finite_Set.fold
2011-12-29, by haftmann
qualified Finite_Set.fold
2011-12-29, by haftmann
dropped redundant setup
2011-12-29, by haftmann
tuned declaration
2011-12-29, by haftmann
attribute code_abbrev superseedes code_unfold_post; tuned text
2011-12-29, by haftmann
attribute code_abbrev superseedes code_unfold_post; tuned names and spacing
2011-12-29, by haftmann
attribute code_abbrev superseedes code_unfold_post
2011-12-29, by haftmann
semiring_numeral_0_eq_0, semiring_numeral_1_eq_1 now [simp], superseeding corresponding simp rules on type nat; attribute code_abbrev superseedes code_unfold_post
2011-12-29, by haftmann
semiring_numeral_0_eq_0, semiring_numeral_1_eq_1 now [simp], superseeding corresponding simp rules on type nat
2011-12-29, by haftmann
merged
2011-12-28, by wenzelm
merged
2011-12-28, by huffman
restate some lemmas to respect int/bin distinction
2011-12-28, by huffman
simplify some proofs
2011-12-28, by huffman
add lemma word_eq_iff
2011-12-28, by huffman
restate lemma word_1_no in terms of Numeral1
2011-12-28, by huffman
remove recursion combinator bin_rec;
2011-12-28, by huffman
simplify definition of XOR for type int;
2011-12-28, by huffman
simplify definition of OR for type int;
2011-12-28, by huffman
simplify definition of NOT for type int
2011-12-28, by huffman
add several new tests, most of which don't work yet
2011-12-28, by huffman
fix typos
2011-12-28, by huffman
remove some duplicate lemmas
2011-12-28, by huffman
simplify proof
2011-12-28, by huffman
replace 'lemmas' with explicit 'lemma'
2011-12-28, by huffman
add section headings
2011-12-28, by huffman
remove duplicate lemma lists
2011-12-27, by huffman
reverted some changes for set->predicate transition, according to "hg log -u berghofe -r Isabelle2007:Isabelle2008";
2011-12-28, by wenzelm
disable kodkodi for now to prevent isatest failure of HOL-Nitpick_Examples due to 'a set constructor;
2011-12-28, by wenzelm
updated platform information;
2011-12-28, by wenzelm
discontinued broken macbroy5 and thus the obsolete ppc-darwin platform;
2011-12-28, by wenzelm
more selective target "full" -- avoid failure of HOL-Datatype_Benchmark on 32bit platforms;
2011-12-28, by wenzelm
print case syntax depending on "show_cases" configuration option;
2011-12-28, by wenzelm
merged
2011-12-27, by huffman
redefine some binary operations on integers work on abstract numerals instead of Int.Pls and Int.Min
2011-12-27, by huffman
remove some uses of Int.succ and Int.pred
2011-12-27, by huffman
removed unused lemmas
2011-12-27, by huffman
remove redundant syntax declaration
2011-12-27, by huffman
use 'induct arbitrary' instead of 'rule_format' attribute
2011-12-27, by huffman
declare simp rules immediately, instead of using 'declare' commands
2011-12-27, by huffman
declare word_of_int_{0,1} [simp], for consistency with word_of_int_bin
2011-12-27, by huffman
be explicit about Finite_Set.fold
2011-12-27, by haftmann
dropped fact whose names clash with corresponding facts on canonical fold
2011-12-27, by haftmann
prefer canonical fold on lists
2011-12-27, by haftmann
be explicit about Finite_Set.fold
2011-12-27, by haftmann
less
more
|
(0)
-30000
-10000
-3000
-1000
-120
+120
+1000
+3000
+10000
+30000
tip