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.
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
less
more
|
(0)
-30000
-10000
-3000
-1000
-120
+120
+1000
+3000
+10000
+30000
tip