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.
Thm.add_axiom/add_def: return internal name of foundational axiom;
2010-04-11, by wenzelm
modernized datatype constructors;
2010-04-11, by wenzelm
of_sort_derivation: weaken bypasses derivation for identical sort -- accomodate proof terms by krauss/schropp, for example;
2010-04-11, by wenzelm
tuned;
2010-04-11, by wenzelm
of_sort_derivation: pass-through full type information -- following the version by krauss/schropp;
2010-04-11, by wenzelm
include JEDIT_APPLE_PROPERTIES by default;
2010-04-09, by wenzelm
isatest: more uniform setup for Unix vs. Cygwin;
2010-04-09, by wenzelm
added missing case: meta universal quantifier
2010-04-08, by boehmes
added imperative SAT checker; improved headers of example files; adopted IsaMakefile
2010-04-08, by bulwahn
Merged.
2010-04-07, by ballarin
Merged resolving conflicts NEWS and locale.ML.
2010-04-07, by ballarin
Proper inheritance of mixins for activated facts and locale dependencies.
2010-04-02, by ballarin
Removed obsolete function.
2010-02-15, by ballarin
Graceful treatment of non-locale subgoals by methods unfold_locales and intro_locales.
2010-02-15, by ballarin
Tuned interpretation proofs.
2010-02-15, by ballarin
A rough implementation of full mixin inheritance; additional unit tests.
2010-02-11, by ballarin
Clarified invariant; tuned.
2010-02-02, by ballarin
More mixin tests.
2010-02-01, by ballarin
Use serial to be more debug friendly.
2010-02-01, by ballarin
buffered output (faster than direct output)
2010-04-07, by boehmes
simplified Cache_IO interface (input is just a string and not already stored in a file)
2010-04-07, by boehmes
shortened interface (do not export unused options and functions)
2010-04-07, by boehmes
always unfold definitions of specific constants (including special binders)
2010-04-07, by boehmes
shorten the code by conditional function application
2010-04-07, by boehmes
fail for problems containg the universal sort (as those problems cannot be atomized)
2010-04-07, by boehmes
renamed "smt_record" to "smt_fixed" (somewhat more expressive) and inverted its semantics
2010-04-07, by boehmes
Added Information theory and Example: dining cryptographers
2010-04-07, by hoelzl
simplified induction case in finite_psubset_induct; tuned the proof that uses this induction principle
2010-04-07, by Christian Urban
removed (latex output) notation which is sometimes very ugly
2010-04-06, by krauss
merged
2010-04-06, by boehmes
added missing mult_1_left to linarith simp rules
2010-04-06, by boehmes
tuned proof (no induction needed); removed unused lemma and fuzzy comment
2010-04-06, by krauss
isatest: basic setup for cygwin-poly on atbroy102;
2010-04-02, by wenzelm
slightly more standard dependencies;
2010-04-01, by wenzelm
merged
2010-04-01, by nipkow
tuned many proofs a bit
2010-04-01, by nipkow
merged
2010-04-01, by nipkow
documented [[trace_simp=true]]
2010-03-29, by nipkow
add missing goal argument
2010-04-01, by blanchet
adapt syntax of Sledgehammer options in examples
2010-04-01, by blanchet
merged
2010-04-01, by blanchet
fixed layout of Sledgehammer output
2010-04-01, by blanchet
added "modulus" and "sorts" options to control Sledgehammer's Isar proof output
2010-03-29, by blanchet
make Sledgehammer output "by" vs. "apply", "qed" vs. "next", and any necessary "prefer"
2010-03-29, by blanchet
get rid of Polyhash, since it's no longer used
2010-03-29, by blanchet
remove use of Polyhash;
2010-03-29, by blanchet
reintroduce efficient set structure to collect "no_atp" theorems
2010-03-29, by blanchet
made "theory_const" a Sledgehammer option;
2010-03-29, by blanchet
added "respect_no_atp" and "convergence" options to Sledgehammer;
2010-03-29, by blanchet
adding MREC induction rule in Imperative HOL
2010-03-31, by bulwahn
made smlnj happy
2010-03-31, by bulwahn
adding examples of function predicate replacement and arithmetic examples for the predicate compiler; tuned
2010-03-31, by bulwahn
adopting specialisation examples to moving the alternative defs in the library
2010-03-31, by bulwahn
adding setup for handling arithmetic of natural numbers and integers precisely and more efficiently in the predicate compiler; changed alternative size_list definition for predicate compiler
2010-03-31, by bulwahn
no specialisation for predicates without introduction rules in the predicate compiler
2010-03-31, by bulwahn
improving lookup function to handle overloaded constants more correctly in the function flattening of the predicate compiler
2010-03-31, by bulwahn
activating the signature of Predicate_Compile again which was deactivated in changeset d93a3cb55068 for debugging purposes
2010-03-31, by bulwahn
adding iterate_upto interface in compilations and iterate_upto functions in Isabelle theories for arithmetic setup of the predicate compiler
2010-03-31, by bulwahn
clarifying the Predicate_Compile_Core signature
2010-03-31, by bulwahn
adding signature to Predicate_Compile_Aux; tuning Predicate_Compile_Aux structure
2010-03-31, by bulwahn
putting compilation setup of predicate compiler in a separate file
2010-03-31, by bulwahn
simplify fold_graph proofs
2010-03-30, by huffman
NEWS
2010-03-30, by krauss
removed dead code; fixed typo
2010-03-30, by krauss
switched PThm/PAxm etc. to use canonical order of type variables (term variables unchanged)
2010-03-30, by krauss
merged
2010-03-30, by wenzelm
adding skip_proof in the examples because proof procedure cannot handle alternative compilations yet
2010-03-29, by bulwahn
tuned
2010-03-29, by bulwahn
generalized alternative functions to alternative compilation to handle arithmetic functions better
2010-03-29, by bulwahn
correcting alternative functions with tuples
2010-03-29, by bulwahn
no specialisation for patterns with only tuples in the predicate compiler
2010-03-29, by bulwahn
adding registration of functions in the function flattening
2010-03-29, by bulwahn
added book-keeping, registration and compilation with alternative functions for predicates in the predicate compiler
2010-03-29, by bulwahn
adding specialisation examples of the predicate compiler
2010-03-29, by bulwahn
adding specialisation of predicates to the predicate compiler
2010-03-29, by bulwahn
returning an more understandable user error message in the values command
2010-03-29, by bulwahn
adding Lazy_Sequences with explicit depth-bound
2010-03-29, by bulwahn
removing fishing for split thm in the predicate compiler
2010-03-29, by bulwahn
prefer recursive calls before others in the mode inference
2010-03-29, by bulwahn
added statistics to values command for random generation
2010-03-29, by bulwahn
adopting Predicate_Compile_Quickcheck
2010-03-29, by bulwahn
made quickcheck generic with respect to which compilation; added random compilation to quickcheck
2010-03-29, by bulwahn
removed yieldn in Lazy_Sequence and put in the ML structure; corrects behaviour of values command
2010-03-29, by bulwahn
adding a hook for experiments in the predicate compilation process
2010-03-29, by bulwahn
removing simple equalities in introduction rules in the predicate compiler
2010-03-29, by bulwahn
adopting Predicate_Compile
2010-03-29, by bulwahn
adding values command for new monad; added new random monad compilation to predicate_compile_quickcheck
2010-03-29, by bulwahn
generalizing the compilation process of the predicate compiler
2010-03-29, by bulwahn
added new compilation to predicate_compiler
2010-03-29, by bulwahn
adding new depth-limited and new random monad for the predicate compiler
2010-03-29, by bulwahn
recovered StringBuilder functionality after subtle change of + and ++ in Scala 2.8.0 Beta 1;
2010-03-30, by wenzelm
adapted to Scala 2.8.0 Beta 1;
2010-03-30, by wenzelm
auto update by Netbeans 6.8;
2010-03-30, by wenzelm
adapted to Netbeans 6.8 and Scala for Netbeans 6.8v1.1;
2010-03-30, by wenzelm
replaced some deprecated methods;
2010-03-29, by wenzelm
adapted to Scala 2.8.0 Beta1 -- with notable changes to scala.collection;
2010-03-29, by wenzelm
merged
2010-03-29, by huffman
use lattice theorems to prove set theorems
2010-03-28, by huffman
add/change some lemmas about lattices
2010-03-28, by huffman
cleaned up some proofs
2010-03-28, by huffman
the configuration option 'trace_simp' now uses the reference of the ProofGeneral settings menu as (dynamic) default value
2010-03-29, by boehmes
merged
2010-03-28, by wenzelm
implicit checkpoint in Local_Theory.theory as well -- no longer export Local_Theory.checkpoint;
2010-03-28, by wenzelm
make SML/NJ happy
2010-03-28, by blanchet
pass raw Context.generic, to avoid wasteful Context.proof_of -- Config.get_thy is often used in performance critical spots like unify.ML;
2010-03-28, by wenzelm
static defaults for configuration options;
2010-03-28, by wenzelm
configuration options admit dynamic default values;
2010-03-28, by wenzelm
tuned;
2010-03-28, by wenzelm
do not export Attrib.register_config, to make it harder to use low-level Config.declare after the bootstrap phase;
2010-03-28, by wenzelm
use regular Attrib.config instead of low-level Config.declare/Attrib.register_config;
2010-03-28, by wenzelm
merged
2010-03-27, by wenzelm
re-introduce reference to control simplifier tracing (needed for ProofGeneral settings menu) (cf. 12bb31230550)
2010-03-27, by boehmes
Typedef.info: separate global and local part, only the latter is transformed by morphisms;
2010-03-27, by wenzelm
merged
2010-03-27, by nipkow
added reference to Trace Simp Depth.
2010-03-27, by nipkow
merged
2010-03-27, by wenzelm
Automated lifting can be restricted to specific quotient types
2010-03-27, by Cezary Kaliszyk
moved Primitive_Defs.mk_defpair to OldGoals.mk_defpair;
2010-03-27, by wenzelm
disallow premises in primitive Theory.add_def -- handle in Thm.add_def;
2010-03-27, by wenzelm
disallow sort constraints in primitive Theory.add_axiom/add_def -- handled in Thm.add_axiom/add_def;
2010-03-27, by wenzelm
less
more
|
(0)
-30000
-10000
-3000
-1000
-120
+120
+1000
+3000
+10000
+30000
tip