Mercurial
Mercurial
>
repos
>
isabelle
/ graph
summary
|
shortlog
|
changelog
| graph |
tags
|
bookmarks
|
branches
|
files
|
gz
|
help
less
more
|
(0)
-30000
-10000
-3000
-1000
-192
+192
+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.
simpler argument
2010-06-25, by blanchet
got rid of "respect_no_atp" option, which even I don't use
2010-06-25, by blanchet
reorder ML files
2010-06-25, by blanchet
renamed "Sledgehammer_FOL_Clauses" to "Metis_Clauses", so that Metis doesn't depend on Sledgehammer
2010-06-25, by blanchet
merge "Sledgehammer_{F,H}OL_Clause", as requested by a FIXME
2010-06-25, by blanchet
get rid of type alias
2010-06-25, by blanchet
exploit "Name.desymbolize" to remove some dependencies
2010-06-25, by blanchet
renamed "Sledgehammer_Fact_Preprocessor" to "Clausifier";
2010-06-25, by blanchet
fewer dependencies
2010-06-25, by blanchet
more intra-module dependency cleanup + merge "const" and "type_const" tables, since this is safe
2010-06-25, by blanchet
more moving around of ML files in "Sledgehammer.thy"
2010-06-25, by blanchet
got rid of needless exception
2010-06-25, by blanchet
move "MESON" up;
2010-06-25, by blanchet
remove junk
2010-06-25, by blanchet
further reduce dependencies on "sledgehammer_fact_filter.ML"
2010-06-25, by blanchet
move "prepare_clauses" from "sledgehammer_fact_filter.ML" to "sledgehammer_hol_clause.ML";
2010-06-25, by blanchet
merged
2010-06-28, by wenzelm
Quotient package reverse lifting
2010-06-28, by Cezary Kaliszyk
Add reverse lifting flag to automated theorem derivation
2010-06-28, by Cezary Kaliszyk
Restrict quotient definitions to constants
2010-06-28, by Cezary Kaliszyk
mixfix can be given for automatically lifted constants
2010-06-27, by Christian Urban
streamlined the generation of quotient theorems out of raw theorems
2010-06-26, by Christian Urban
merged
2010-06-25, by haftmann
avoid REPEAT after THEN_ALL_NEW
2010-06-25, by haftmann
refresh Isabelle token marker after buffer properties changed, e.g. when fold mode is switched;
2010-06-26, by wenzelm
treat alternative newline symbols as in Isabelle/ML;
2010-06-26, by wenzelm
simplified text_area_painter, with more precise treatment of visible line end;
2010-06-26, by wenzelm
merged
2010-06-25, by wenzelm
merged
2010-06-25, by blanchet
eta-expand
2010-06-25, by blanchet
improve the natural formula relevance filter code, so that it behaves more like the CNF one
2010-06-25, by blanchet
split SPASS time slot between SOS and non-SOS, in case SOS times out
2010-06-25, by blanchet
yields ill-typed ATP/metis proofs -- raus!
2010-06-24, by blanchet
make sure "metisFT" is tried upon "metis" failure in "resolve_inc_tyvars"
2010-06-24, by blanchet
merged
2010-06-25, by haftmann
more direct definition simplifies proofs
2010-06-24, by haftmann
merged
2010-06-24, by haftmann
more precise tactic: do not escape to a different goal branch (REPEAT is still problematic, though)
2010-06-24, by haftmann
a76ace919f1c wasn't quite right; second try
2010-06-24, by blanchet
merge
2010-06-24, by blanchet
never include anything from the Sledgehammer theory in the relevant facts + killed two obsolete facts
2010-06-24, by blanchet
better eta-expansion in Sledgehammer's clausification;
2010-06-24, by blanchet
cosmetics
2010-06-24, by blanchet
make sure that theorems passed using "add:" to Sledgehammer are not eliminated on heuristic grounds
2010-06-24, by blanchet
improve the new "natural formula" fact filter
2010-06-23, by blanchet
explicit treatment of UTF8 sequences as Isabelle symbols;
2010-06-25, by wenzelm
ML pretty printing of type string according to (quasi-abstract) YXML markup and symbols (including UTF8);
2010-06-24, by wenzelm
escape UTF8 symbols for the ML compiler;
2010-06-24, by wenzelm
explicit treatment of UTF8 character sequences as Isabelle symbols;
2010-06-24, by wenzelm
slight cleaning and simplification of the automatic wrapper for quotient definitions
2010-06-24, by Christian Urban
merged
2010-06-24, by wenzelm
export of proper information in the ML-interface of the quotient package
2010-06-24, by Christian Urban
treat Pretty.T as strictly abstract type;
2010-06-24, by wenzelm
slightly more standard data merge: Symtax.merge (K true) avoids equality on abstract type Pretty.T and gracefully accepts overriding, Symtab.join prefers first entry as usual;
2010-06-24, by wenzelm
avoid equality on abstract type Pretty.T;
2010-06-24, by wenzelm
notes on packaging;
2010-06-24, by wenzelm
misc tuning;
2010-06-24, by wenzelm
tuned auxiliary structures;
2010-06-24, by wenzelm
Net.encode_type;
2010-06-24, by wenzelm
more accurate dependencies;
2010-06-24, by wenzelm
made smlnj happy
2010-06-24, by haftmann
fix syntax bug in the TPTP output, by ensuring that "hBOOL" is correctly used for n-ary predicates even if (n + k)-ary occurrences of the same predicate, but with a different type, occur in the same problem
2010-06-23, by blanchet
renamed for easier grep
2010-06-23, by blanchet
use Skolem inlining also in the nonpolymorphic case, as a step toward simplifying the source code
2010-06-23, by blanchet
steal some of http://isabelle.in.tum.de/sledgehammer.html and add it to the docs
2010-06-23, by blanchet
have "metis" method and "metis_tac" fall back on "metisFT" upon failure, following a suggestion by Larry
2010-06-23, by blanchet
fix bug with "skolem_id" + sort facts for increased readability
2010-06-23, by blanchet
if SPASS fails at finding a proof with the SOS option turned on, turn it off and try again
2010-06-23, by blanchet
merged
2010-06-23, by blanchet
this looks like the most appropriate place to do the beta-eta-contraction
2010-06-23, by blanchet
killed legacy "neg_clausify" and "clausify"
2010-06-23, by blanchet
merged
2010-06-22, by blanchet
factor out TPTP format output into file of its own, to facilitate further changes
2010-06-22, by blanchet
merged
2010-06-22, by blanchet
turn on "natural form" filtering in the Mirabelle tests, to see how it performs
2010-06-22, by blanchet
missing "Unsynchronized" + make exception take a unit
2010-06-22, by blanchet
added code to optionally perform fact filtering on the original (non-CNF) formulas
2010-06-22, by blanchet
more cosmetics
2010-06-22, by blanchet
cosmetics + prevent consideration of inlined Skolem terms in relevance filter
2010-06-22, by blanchet
canonical argument order
2010-06-22, by blanchet
leverage new data structure for handling "add:" and "del:"
2010-06-22, by blanchet
thread original theorem along with CNF theorem, as a step toward killing the Skolem cache
2010-06-22, by blanchet
merge "generic_prover" and "generic_tptp_prover"
2010-06-22, by blanchet
removed Sledgehammer's support for the DFG syntax;
2010-06-22, by blanchet
distinguish between "unknown" and "no Kodkodi installed" errors
2010-06-22, by blanchet
reintroduce new Sledgehammer polymorphic handling code;
2010-06-22, by blanchet
make the Nitpick_Example theory processable even when Kodkodi is not installed;
2010-06-22, by blanchet
Make latex happy
2010-06-23, by hoelzl
Quotient package now uses Partial Equivalence instead place of equivalence
2010-06-23, by Cezary Kaliszyk
Replace 'list_rel' by 'list_all2'; they are equivalent.
2010-06-23, by Cezary Kaliszyk
Proper treatment of non-inherited mixins.
2010-06-22, by ballarin
merged
2010-06-22, by hoelzl
Introduce a type class for euclidean spaces, port most lemmas from real^'n to this type class.
2010-06-21, by hoelzl
reredisable new polymorphic code
2010-06-22, by blanchet
merged
2010-06-21, by blanchet
beta-eta was too much, because it transformed SOME x. P x into Eps P, which caused problems later;
2010-06-21, by blanchet
back to post-release mode;
2010-06-21, by wenzelm
merged, resolving conflicts in doc-src/IsarRef/Thy/HOL_Specific.thy;
2010-06-21, by wenzelm
make Nitpick's unsound mode a bit more unsound
2010-06-21, by blanchet
sort cases on the proper key
2010-06-21, by blanchet
compile
2010-06-21, by blanchet
thread "full_types"
2010-06-21, by blanchet
try to improve Sledgehammer/Metis's behavior in full_types mode, e.g. by handing True, False, and If better
2010-06-21, by blanchet
clean up after fcc768dc9dd0
2010-06-21, by blanchet
adjusted Nitpick examples to latest changes + make them slightly faster
2010-06-21, by blanchet
optimized code generated for datatype cases + more;
2010-06-21, by blanchet
activated Scala code generator test
2010-06-21, by haftmann
added bot instances; tuned
2010-06-21, by haftmann
extensionality rule fset_eqI
2010-06-21, by haftmann
merged
2010-06-20, by haftmann
separate section for diagnostic commands
2010-06-20, by haftmann
more binding; avoid arcane Rep and Abs prefixes
2010-06-19, by haftmann
cleanup of typecopy package
2010-06-19, by haftmann
quickcheck for fsets
2010-06-19, by haftmann
merged
2010-06-18, by nipkow
added pigeonhole lemmas
2010-06-18, by nipkow
merged
2010-06-18, by haftmann
tuned whitespace; dropped dead code
2010-06-18, by haftmann
code_simp: only succeed on real progress
2010-06-18, by haftmann
prefer fold over foldl
2010-06-18, by haftmann
conclude simplification with default simpset
2010-06-18, by haftmann
drop subsumed default equations (requires a little bit unfortunate laziness)
2010-06-18, by haftmann
avoid Scala legacy operations
2010-06-18, by haftmann
prefer fold over foldl
2010-06-18, by haftmann
made List.thy a join point in the theory graph
2010-06-18, by haftmann
tuned set_replicate lemmas
2010-06-18, by nipkow
merged
2010-06-18, by nipkow
added lemmas
2010-06-18, by nipkow
dropped dead code
2010-06-18, by haftmann
replaced unreliable metis proof
2010-06-17, by haftmann
rev is reverse in Haskell
2010-06-17, by haftmann
first serious draft of a scala code generator
2010-06-17, by haftmann
more precise code
2010-06-17, by haftmann
explicit type variable arguments for constructors
2010-06-17, by haftmann
transitive superclasses were also only a misunderstanding
2010-06-17, by haftmann
formal introduction of transitive superclasses
2010-06-17, by haftmann
dropped obscure type argument weakening mapping -- was only a misunderstanding
2010-06-17, by haftmann
added simp evaluator
2010-06-17, by haftmann
merged
2010-06-17, by haftmann
added code_simp infrastructure
2010-06-15, by haftmann
tuned whitespace
2010-06-15, by haftmann
maintain cong rules for case combinators; more precise permissiveness
2010-06-15, by haftmann
drop function definitions of combinators
2010-06-15, by haftmann
maintain cong rules for case combinators
2010-06-15, by haftmann
formal introduction of case cong
2010-06-15, by haftmann
found missing beta-eta-contraction
2010-06-15, by blanchet
added missing Umlaut
2010-06-15, by blanchet
make example run a bit faster (might help atbroy102)
2010-06-15, by blanchet
merged
2010-06-15, by haftmann
tuned documents
2010-06-15, by haftmann
teaked naming of superclass projections
2010-06-14, by haftmann
added lemma funpow_mult
2010-06-14, by haftmann
extended bib
2010-06-14, by haftmann
updated generated code
2010-06-14, by haftmann
added reference
2010-06-14, by haftmann
subsection on locale interpretation
2010-06-14, by haftmann
explicitly name and note equations for class eq
2010-06-14, by haftmann
use various predefined Haskell operations when generating code
2010-06-14, by haftmann
NEWS
2010-06-14, by haftmann
tuned internal order
2010-06-14, by haftmann
dropped unused bindings
2010-06-14, by haftmann
corrected syntax diagram
2010-06-14, by haftmann
turn off new polymorphism code again -- a new issue popped up
2010-06-14, by blanchet
missing case
2010-06-14, by blanchet
A function called "untyped_aconv" shouldn't look at the bound names!
2010-06-14, by blanchet
no point in introducing combinators for inlined Skolem functions
2010-06-14, by blanchet
better error reporting for Vampire
2010-06-14, by blanchet
expect SPASS 3.7, and give a friendly warning if an older version is used
2010-06-14, by blanchet
improve ATP-specific error messages
2010-06-14, by blanchet
merged
2010-06-14, by haftmann
removed simplifier congruence rule of "prod_case"
2010-06-14, by haftmann
adjusted the polymorphism handling of Skolem constants so that proof reconstruction doesn't fail in "equality_inf"
2010-06-14, by blanchet
merged
2010-06-12, by haftmann
declare lexn.simps [code del]
2010-06-12, by haftmann
declare lex_prod_def [code del]
2010-06-11, by haftmann
modernized specifications
2010-06-11, by haftmann
avoid references to old constdefs
2010-06-11, by haftmann
merged
2010-06-12, by blanchet
disable new polymorphic code for now, until remaining issues in "equality_inf" are resolved
2010-06-12, by blanchet
"raise Fail" for internal errors + one new internal error (instead of "Match")
2010-06-12, by blanchet
make test work again (broken since 09467cdfa198?)
2010-06-11, by blanchet
adjust Nitpick example to follow latest wave of renamings
2010-06-11, by blanchet
proper polymorphic Skolemization of uncached facts + synchronization of caching and relevance filter
2010-06-11, by blanchet
beta-eta-contract, to respect "first_order_match"'s specification;
2010-06-11, by blanchet
adjust Nitpick's handling of "<" on "rat"s and "reals"
2010-06-11, by blanchet
remove needless variables
2010-06-11, by blanchet
hide sum explicitly
2010-06-11, by haftmann
merged
2010-06-10, by haftmann
adjust popular symbolic type constructors
2010-06-10, by haftmann
tailored set of code equations manually
2010-06-10, by haftmann
tuned quotes, antiquotations and whitespace
2010-06-10, by haftmann
moved inductive_codegen to place where product type is available; tuned structure name
2010-06-10, by haftmann
less
more
|
(0)
-30000
-10000
-3000
-1000
-192
+192
+1000
+3000
+10000
+30000
tip