hoelzl [Wed, 07 Apr 2010 17:24:44 +0200] rev 36080
Added Information theory and Example: dining cryptographers
Christian Urban <urbanc@in.tum.de> [Wed, 07 Apr 2010 11:05:11 +0200] rev 36079
simplified induction case in finite_psubset_induct; tuned the proof that uses this induction principle
krauss [Tue, 06 Apr 2010 11:00:57 +0200] rev 36078
removed (latex output) notation which is sometimes very ugly
boehmes [Tue, 06 Apr 2010 10:48:16 +0200] rev 36077
merged
boehmes [Tue, 06 Apr 2010 10:46:28 +0200] rev 36076
added missing mult_1_left to linarith simp rules
krauss [Tue, 06 Apr 2010 09:27:03 +0200] rev 36075
tuned proof (no induction needed); removed unused lemma and fuzzy comment
wenzelm [Fri, 02 Apr 2010 17:20:43 +0200] rev 36074
isatest: basic setup for cygwin-poly on atbroy102;
wenzelm [Thu, 01 Apr 2010 15:37:30 +0200] rev 36073
slightly more standard dependencies;
nipkow [Thu, 01 Apr 2010 12:19:37 +0200] rev 36072
merged
nipkow [Thu, 01 Apr 2010 12:19:20 +0200] rev 36071
tuned many proofs a bit
nipkow [Thu, 01 Apr 2010 09:31:58 +0200] rev 36070
merged
nipkow [Mon, 29 Mar 2010 09:47:21 +0200] rev 36069
documented [[trace_simp=true]]
blanchet [Thu, 01 Apr 2010 11:12:08 +0200] rev 36068
add missing goal argument
blanchet [Thu, 01 Apr 2010 10:54:21 +0200] rev 36067
adapt syntax of Sledgehammer options in examples
blanchet [Thu, 01 Apr 2010 10:27:06 +0200] rev 36066
merged
blanchet [Thu, 01 Apr 2010 10:26:45 +0200] rev 36065
fixed layout of Sledgehammer output
blanchet [Mon, 29 Mar 2010 19:49:57 +0200] rev 36064
added "modulus" and "sorts" options to control Sledgehammer's Isar proof output
blanchet [Mon, 29 Mar 2010 18:44:24 +0200] rev 36063
make Sledgehammer output "by" vs. "apply", "qed" vs. "next", and any necessary "prefer"
blanchet [Mon, 29 Mar 2010 15:50:18 +0200] rev 36062
get rid of Polyhash, since it's no longer used
blanchet [Mon, 29 Mar 2010 15:26:19 +0200] rev 36061
remove use of Polyhash;
the new code is slightly faster. Also, "subtract_cls" now has canonical argument ordering.
blanchet [Mon, 29 Mar 2010 14:49:53 +0200] rev 36060
reintroduce efficient set structure to collect "no_atp" theorems
blanchet [Mon, 29 Mar 2010 12:21:51 +0200] rev 36059
made "theory_const" a Sledgehammer option;
by default, it's true for SPASS and false for the others. This eliminates the need for the "spass_no_tc" ATP, which can be obtained by passing "no_theory_const" instead.
blanchet [Mon, 29 Mar 2010 12:01:00 +0200] rev 36058
added "respect_no_atp" and "convergence" options to Sledgehammer;
these were previously hard-coded in "sledgehammer_fact_filter.ML"
bulwahn [Wed, 31 Mar 2010 16:44:41 +0200] rev 36057
adding MREC induction rule in Imperative HOL
bulwahn [Wed, 31 Mar 2010 16:44:41 +0200] rev 36056
made smlnj happy
bulwahn [Wed, 31 Mar 2010 16:44:41 +0200] rev 36055
adding examples of function predicate replacement and arithmetic examples for the predicate compiler; tuned
bulwahn [Wed, 31 Mar 2010 16:44:41 +0200] rev 36054
adopting specialisation examples to moving the alternative defs in the library
bulwahn [Wed, 31 Mar 2010 16:44:41 +0200] rev 36053
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
bulwahn [Wed, 31 Mar 2010 16:44:41 +0200] rev 36052
no specialisation for predicates without introduction rules in the predicate compiler
bulwahn [Wed, 31 Mar 2010 16:44:41 +0200] rev 36051
improving lookup function to handle overloaded constants more correctly in the function flattening of the predicate compiler
bulwahn [Wed, 31 Mar 2010 16:44:41 +0200] rev 36050
activating the signature of Predicate_Compile again which was deactivated in changeset d93a3cb55068 for debugging purposes
bulwahn [Wed, 31 Mar 2010 16:44:41 +0200] rev 36049
adding iterate_upto interface in compilations and iterate_upto functions in Isabelle theories for arithmetic setup of the predicate compiler
bulwahn [Wed, 31 Mar 2010 16:44:41 +0200] rev 36048
clarifying the Predicate_Compile_Core signature
bulwahn [Wed, 31 Mar 2010 16:44:41 +0200] rev 36047
adding signature to Predicate_Compile_Aux; tuning Predicate_Compile_Aux structure
bulwahn [Wed, 31 Mar 2010 16:44:41 +0200] rev 36046
putting compilation setup of predicate compiler in a separate file
huffman [Tue, 30 Mar 2010 15:46:50 -0700] rev 36045
simplify fold_graph proofs
krauss [Tue, 30 Mar 2010 23:12:55 +0200] rev 36044
NEWS
krauss [Tue, 30 Mar 2010 15:25:35 +0200] rev 36043
removed dead code; fixed typo
krauss [Tue, 30 Mar 2010 15:25:30 +0200] rev 36042
switched PThm/PAxm etc. to use canonical order of type variables (term variables unchanged)
wenzelm [Tue, 30 Mar 2010 12:47:39 +0200] rev 36041
merged
bulwahn [Mon, 29 Mar 2010 17:30:56 +0200] rev 36040
adding skip_proof in the examples because proof procedure cannot handle alternative compilations yet
bulwahn [Mon, 29 Mar 2010 17:30:55 +0200] rev 36039
tuned
bulwahn [Mon, 29 Mar 2010 17:30:54 +0200] rev 36038
generalized alternative functions to alternative compilation to handle arithmetic functions better
bulwahn [Mon, 29 Mar 2010 17:30:54 +0200] rev 36037
correcting alternative functions with tuples
bulwahn [Mon, 29 Mar 2010 17:30:53 +0200] rev 36036
no specialisation for patterns with only tuples in the predicate compiler
bulwahn [Mon, 29 Mar 2010 17:30:53 +0200] rev 36035
adding registration of functions in the function flattening
bulwahn [Mon, 29 Mar 2010 17:30:53 +0200] rev 36034
added book-keeping, registration and compilation with alternative functions for predicates in the predicate compiler
bulwahn [Mon, 29 Mar 2010 17:30:52 +0200] rev 36033
adding specialisation examples of the predicate compiler
bulwahn [Mon, 29 Mar 2010 17:30:52 +0200] rev 36032
adding specialisation of predicates to the predicate compiler
bulwahn [Mon, 29 Mar 2010 17:30:50 +0200] rev 36031
returning an more understandable user error message in the values command
bulwahn [Mon, 29 Mar 2010 17:30:49 +0200] rev 36030
adding Lazy_Sequences with explicit depth-bound
bulwahn [Mon, 29 Mar 2010 17:30:48 +0200] rev 36029
removing fishing for split thm in the predicate compiler
bulwahn [Mon, 29 Mar 2010 17:30:46 +0200] rev 36028
prefer recursive calls before others in the mode inference
bulwahn [Mon, 29 Mar 2010 17:30:45 +0200] rev 36027
added statistics to values command for random generation
bulwahn [Mon, 29 Mar 2010 17:30:43 +0200] rev 36026
adopting Predicate_Compile_Quickcheck
bulwahn [Mon, 29 Mar 2010 17:30:43 +0200] rev 36025
made quickcheck generic with respect to which compilation; added random compilation to quickcheck
bulwahn [Mon, 29 Mar 2010 17:30:41 +0200] rev 36024
removed yieldn in Lazy_Sequence and put in the ML structure; corrects behaviour of values command
bulwahn [Mon, 29 Mar 2010 17:30:40 +0200] rev 36023
adding a hook for experiments in the predicate compilation process
bulwahn [Mon, 29 Mar 2010 17:30:40 +0200] rev 36022
removing simple equalities in introduction rules in the predicate compiler
bulwahn [Mon, 29 Mar 2010 17:30:39 +0200] rev 36021
adopting Predicate_Compile
bulwahn [Mon, 29 Mar 2010 17:30:38 +0200] rev 36020
adding values command for new monad; added new random monad compilation to predicate_compile_quickcheck
bulwahn [Mon, 29 Mar 2010 17:30:36 +0200] rev 36019
generalizing the compilation process of the predicate compiler
bulwahn [Mon, 29 Mar 2010 17:30:36 +0200] rev 36018
added new compilation to predicate_compiler
bulwahn [Mon, 29 Mar 2010 17:30:34 +0200] rev 36017
adding new depth-limited and new random monad for the predicate compiler
wenzelm [Tue, 30 Mar 2010 00:47:52 +0200] rev 36016
recovered StringBuilder functionality after subtle change of + and ++ in Scala 2.8.0 Beta 1;
wenzelm [Tue, 30 Mar 2010 00:13:27 +0200] rev 36015
adapted to Scala 2.8.0 Beta 1;
wenzelm [Tue, 30 Mar 2010 00:12:42 +0200] rev 36014
auto update by Netbeans 6.8;
wenzelm [Tue, 30 Mar 2010 00:11:41 +0200] rev 36013
adapted to Netbeans 6.8 and Scala for Netbeans 6.8v1.1;
wenzelm [Mon, 29 Mar 2010 22:55:57 +0200] rev 36012
replaced some deprecated methods;
wenzelm [Mon, 29 Mar 2010 22:43:56 +0200] rev 36011
adapted to Scala 2.8.0 Beta1 -- with notable changes to scala.collection;
huffman [Mon, 29 Mar 2010 01:07:01 -0700] rev 36010
merged
huffman [Sun, 28 Mar 2010 12:50:38 -0700] rev 36009
use lattice theorems to prove set theorems
huffman [Sun, 28 Mar 2010 12:49:14 -0700] rev 36008
add/change some lemmas about lattices
huffman [Sun, 28 Mar 2010 10:34:02 -0700] rev 36007
cleaned up some proofs
boehmes [Mon, 29 Mar 2010 09:06:34 +0200] rev 36006
the configuration option 'trace_simp' now uses the reference of the ProofGeneral settings menu as (dynamic) default value
wenzelm [Sun, 28 Mar 2010 19:34:08 +0200] rev 36005
merged
wenzelm [Sun, 28 Mar 2010 19:20:52 +0200] rev 36004
implicit checkpoint in Local_Theory.theory as well -- no longer export Local_Theory.checkpoint;
blanchet [Sun, 28 Mar 2010 18:39:27 +0200] rev 36003
make SML/NJ happy
wenzelm [Sun, 28 Mar 2010 17:43:09 +0200] rev 36002
pass raw Context.generic, to avoid wasteful Context.proof_of -- Config.get_thy is often used in performance critical spots like unify.ML;
wenzelm [Sun, 28 Mar 2010 16:59:06 +0200] rev 36001
static defaults for configuration options;
wenzelm [Sun, 28 Mar 2010 16:13:29 +0200] rev 36000
configuration options admit dynamic default values;
wenzelm [Sun, 28 Mar 2010 16:29:51 +0200] rev 35999
tuned;
wenzelm [Sun, 28 Mar 2010 15:38:07 +0200] rev 35998
do not export Attrib.register_config, to make it harder to use low-level Config.declare after the bootstrap phase;
wenzelm [Sun, 28 Mar 2010 15:13:19 +0200] rev 35997
use regular Attrib.config instead of low-level Config.declare/Attrib.register_config;
wenzelm [Sat, 27 Mar 2010 21:46:10 +0100] rev 35996
merged
boehmes [Sat, 27 Mar 2010 21:34:28 +0100] rev 35995
re-introduce reference to control simplifier tracing (needed for ProofGeneral settings menu) (cf. 12bb31230550)
wenzelm [Sat, 27 Mar 2010 21:38:38 +0100] rev 35994
Typedef.info: separate global and local part, only the latter is transformed by morphisms;
nipkow [Sat, 27 Mar 2010 18:43:11 +0100] rev 35993
merged
nipkow [Sat, 27 Mar 2010 18:42:27 +0100] rev 35992
added reference to Trace Simp Depth.
wenzelm [Sat, 27 Mar 2010 18:12:02 +0100] rev 35991
merged
Cezary Kaliszyk <kaliszyk@in.tum.de> [Sat, 27 Mar 2010 14:48:46 +0100] rev 35990
Automated lifting can be restricted to specific quotient types
wenzelm [Sat, 27 Mar 2010 18:07:21 +0100] rev 35989
moved Primitive_Defs.mk_defpair to OldGoals.mk_defpair;
wenzelm [Sat, 27 Mar 2010 17:36:32 +0100] rev 35988
disallow premises in primitive Theory.add_def -- handle in Thm.add_def;
eliminated obsolete Sign.cert_def;
misc tuning and clarification;
wenzelm [Sat, 27 Mar 2010 16:01:45 +0100] rev 35987
disallow sort constraints in primitive Theory.add_axiom/add_def -- handled in Thm.add_axiom/add_def;
wenzelm [Sat, 27 Mar 2010 15:47:57 +0100] rev 35986
added Term.fold_atyps_sorts convenience;
wenzelm [Sat, 27 Mar 2010 15:20:31 +0100] rev 35985
moved Drule.forall_intr_frees to Thm.forall_intr_frees (in more_thm.ML, which is loaded before pure_thy.ML);
discontinued old-style Theory.add_defs(_i) in favour of more basic Theory.add_def;
modernized PureThy.add_defs etc. -- refer to high-level Thm.add_def;