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.
clarified @{const_name} vs. @{const_abbrev};
2010-02-27, by wenzelm
clarified @{const_name} (only logical consts) vs. @{const_abbrev};
2010-02-27, by wenzelm
type/const name: explicitly allow abbreviations as well;
2010-02-27, by wenzelm
clarified ProofContext.read_const(_proper)/Args.const(_proper) wrt. strict logical consts;
2010-02-27, by wenzelm
added at-poly-test, which is intended for performance tests of Poly/ML itself;
2010-02-27, by wenzelm
more precise syntax antiquotations;
2010-02-27, by wenzelm
ML antiquotations for type classes;
2010-02-27, by wenzelm
read_class: perform actual read, with source position;
2010-02-27, by wenzelm
parallel brute-force disambiguation;
2010-02-27, by wenzelm
degrade gracefully in CRITICAL section;
2010-02-27, by wenzelm
gen_dest_case: recovered @{const_name} from c8a6fae0ad0c, because of separate Syntax.mark_const in case_tr' -- avoid extra syntax markers in output;
2010-02-26, by wenzelm
tuned;
2010-02-26, by wenzelm
use simplified Syntax.escape;
2010-02-26, by wenzelm
tuned hyp_subst_tac';
2010-02-26, by wenzelm
use SAT4J for "Tests_Nits.thy" for safety (this should solve the Isatest failures) + minor changes
2010-02-26, by blanchet
merged
2010-02-26, by blanchet
more work on the new monotonicity stuff in Nitpick
2010-02-26, by blanchet
improved precision of infinite "shallow" datatypes in Nitpick;
2010-02-25, by blanchet
cosmetics
2010-02-25, by blanchet
merged
2010-02-26, by bulwahn
merged
2010-02-26, by bulwahn
adding no_topmost_reordering as new option to the code_pred command
2010-02-25, by bulwahn
adopting Mutabelle to quickcheck reporting; improving quickcheck reporting
2010-02-25, by bulwahn
added quiet option to quickcheck command
2010-02-25, by bulwahn
added basic reporting of test cases to quickcheck
2010-02-25, by bulwahn
merged
2010-02-26, by haftmann
use abstract code cerficates for bare code theorems
2010-02-26, by haftmann
implement quotient_of for odl SML code generator
2010-02-26, by haftmann
adjusted to cs. e4a7947e02b8
2010-02-26, by haftmann
bound argument for abstype proposition
2010-02-24, by haftmann
renamed theory Rational to Rat
2010-02-24, by haftmann
tuned whitespace
2010-02-24, by haftmann
more precise exception handler
2010-02-24, by haftmann
more general case and induct rules; normalize and quotient_of; abstract code generation
2010-02-24, by haftmann
crossproduct coprimality lemmas
2010-02-24, by haftmann
lemma div_mult_swap, dvd_div_eq_mult, dvd_div_div_eq_mult
2010-02-24, by haftmann
evaluation for abstypes
2010-02-24, by haftmann
modernized structure Split_Rule;
2010-02-25, by wenzelm
more antiquotations;
2010-02-25, by wenzelm
explicit @{type_syntax} markup;
2010-02-25, by wenzelm
explicit @{type_syntax} markup;
2010-02-25, by wenzelm
more orthogonal antiquotations for type constructors;
2010-02-25, by wenzelm
clarified ProofContext.read_type_name/Args.type_name wrt strict logical constructors;
2010-02-25, by wenzelm
provide direct access to the different kinds of type declarations;
2010-02-25, by wenzelm
use mixfix syntax for Boogie types
2010-02-25, by boehmes
merged
2010-02-24, by wenzelm
added variant of boogie_vc to prove a single assertion: keep premises (i.e. the trace up this assertion) as facts in the context (and not as part of the goal) to increase performance when dealing with large goals
2010-02-24, by boehmes
modernized syntax declarations, and make them actually work with authentic syntax;
2010-02-24, by wenzelm
observe standard convention for syntax consts;
2010-02-24, by wenzelm
proper type syntax (cf. 7425aece4ee3);
2010-02-24, by wenzelm
observe standard convention for syntax consts;
2010-02-24, by wenzelm
allow general mixfix syntax for type constructors;
2010-02-24, by wenzelm
merged
2010-02-24, by huffman
merged
2010-02-23, by huffman
remove redundant lemma realpow_increasing
2010-02-23, by huffman
remove redundant simp rules from RealPow.thy
2010-02-23, by huffman
adapt to new realpow rules
2010-02-23, by huffman
adapt to changes in simpset
2010-02-23, by huffman
moved some lemmas from RealPow to RealDef; changed orientation of real_of_int_power
2010-02-23, by huffman
move float syntax from RealPow to Rational
2010-02-23, by huffman
compile
2010-02-24, by blanchet
merged
2010-02-24, by blanchet
compile
2010-02-24, by blanchet
make example compile
2010-02-24, by blanchet
got rid of "axclass", apparently
2010-02-24, by blanchet
merged
2010-02-24, by blanchet
cosmetics
2010-02-24, by blanchet
support local definitions in Nitpick
2010-02-23, by blanchet
show Kodkod warning message even in non-verbose mode
2010-02-23, by blanchet
distinguish between Kodkodi warnings and errors in Nitpick;
2010-02-23, by blanchet
optimized multisets in Nitpick by fishing "finite"
2010-02-23, by blanchet
document Quickcheck's "no_assms" option
2010-02-23, by blanchet
tuned comment
2010-02-24, by haftmann
merged
2010-02-23, by hoelzl
Moved old Integration to examples.
2010-02-23, by hoelzl
merged
2010-02-23, by bulwahn
merged
2010-02-23, by bulwahn
adding ROOT.ML to HOL-Mutabelle session; uncommenting HOL.induct constants in Mutabelle session
2010-02-23, by bulwahn
adopting mutabelle and quickcheck to return timing information; exporting make_case_combs in datatype package for predicate compiler; adding Spec_Rules declaration for tail recursive functions; improving the predicate compiler and function flattening
2010-02-23, by bulwahn
separated narrowing timeouts for intermediate and final steps
2010-02-23, by boehmes
merged
2010-02-23, by haftmann
merged
2010-02-23, by haftmann
dropped axclass; dropped Id; session theory Hoare.thy
2010-02-23, by haftmann
dropped session W0; c.f. MiniML in AFP
2010-02-23, by haftmann
dropped axclass, going back to purely syntactic type classes
2010-02-23, by haftmann
dropped axclass; dropped Id
2010-02-23, by haftmann
dropped axclass; dropped Id; session theory Hoare.thy
2010-02-23, by haftmann
dropped axclass
2010-02-23, by haftmann
export prs_rules and rsp_rules attributes
2010-02-23, by Cezary Kaliszyk
merge
2010-02-23, by blanchet
improved precision of small sets in Nitpick
2010-02-23, by blanchet
improved Nitpick's support for quotient types
2010-02-23, by blanchet
Forgot to check NSA in changeset e4a431b6d9b7 ; Removed import of Integration
2010-02-23, by hoelzl
catch IO errors in Nitpick's "kodkodi" invocation + shorten execution time of "Manual_Nits" example
2010-02-23, by blanchet
mind the "s"
2010-02-23, by haftmann
merged
2010-02-23, by haftmann
NEWS
2010-02-22, by haftmann
added missing separator
2010-02-22, by haftmann
more accurate when registering new types
2010-02-22, by haftmann
added Dlist
2010-02-22, by haftmann
tuned text
2010-02-22, by haftmann
distributed theory Algebras to theories Groups and Lattices
2010-02-22, by haftmann
merged
2010-02-22, by haftmann
proper distinction of code datatypes and abstypes
2010-02-22, by haftmann
merged
2010-02-22, by haftmann
merged
2010-02-22, by haftmann
merged
2010-02-22, by haftmann
lemma distinct_insert
2010-02-20, by haftmann
proper header and subsection headings
2010-02-22, by huffman
remove unneeded premise from rat_floor_lemma and floor_Fract
2010-02-22, by huffman
Replaced Integration by Multivariate-Analysis/Real_Integration
2010-02-22, by hoelzl
Support for one-dimensional integration in Multivariate-Analysis
2010-02-22, by himmelma
Equivalence between DERIV and one-dimensional derivation in Multivariate-Analysis
2010-02-18, by himmelma
merged
2010-02-22, by huffman
add mixfix field to type Domain_Library.cons
2010-02-22, by huffman
remove unnecessary local
2010-02-22, by huffman
update to use fixrec package
2010-02-21, by huffman
merge
2010-02-22, by blanchet
enabled Nitpick's support for quotient types + shortened the Nitpick tests a bit
2010-02-22, by blanchet
filter out trivial definitions in Nitpick (e.g. "Topology.topo" from AFP)
2010-02-22, by blanchet
less
more
|
(0)
-30000
-10000
-3000
-1000
-120
+120
+1000
+3000
+10000
+30000
tip