Thu, 05 Nov 2009 17:02:43 +0100 wenzelm made SML/NJ happy;
Thu, 05 Nov 2009 16:10:49 +0100 wenzelm eliminated funny record patterns and made SML/NJ happy;
Thu, 05 Nov 2009 14:47:27 +0100 wenzelm proper header;
Thu, 05 Nov 2009 14:37:39 +0100 wenzelm more accurate dependencies;
Thu, 05 Nov 2009 13:57:56 +0100 wenzelm merged
Wed, 04 Nov 2009 17:17:30 +0100 krauss added Tree23 to IsaMakefile
Wed, 04 Nov 2009 16:54:22 +0100 nipkow New
Wed, 04 Nov 2009 10:17:58 +0100 nipkow merged
Wed, 04 Nov 2009 10:17:43 +0100 nipkow fixed order of parameters in induction rules
Wed, 04 Nov 2009 09:43:25 +0100 krauss added bulwahn to isatest mailings
Wed, 04 Nov 2009 09:18:46 +0100 nipkow merged
Wed, 04 Nov 2009 09:18:03 +0100 nipkow Completely overhauled
Tue, 03 Nov 2009 19:01:06 -0800 huffman better error handling for fixrec_simp
Tue, 03 Nov 2009 18:33:16 -0800 huffman add more fixrec_simp rules
Tue, 03 Nov 2009 18:32:56 -0800 huffman fixrec examples use fixrec_simp instead of fixpat
Tue, 03 Nov 2009 18:32:30 -0800 huffman domain package registers fixrec_simp lemmas
Tue, 03 Nov 2009 17:09:27 -0800 huffman merged
Tue, 03 Nov 2009 17:03:21 -0800 huffman add fixrec_simp attribute and method (eventually to replace fixpat)
Tue, 03 Nov 2009 23:44:16 +0100 boehmes proper and unique case names for the split_vc method,
Tue, 03 Nov 2009 19:32:08 +0100 haftmann merged
Tue, 03 Nov 2009 17:08:57 +0100 haftmann merged
Tue, 03 Nov 2009 17:06:35 +0100 haftmann always be qualified -- suspected smartness in fact never worked as expected
Tue, 03 Nov 2009 17:06:08 +0100 haftmann pretty name for ==>
Tue, 03 Nov 2009 17:54:24 +0100 boehmes added HOL-Boogie
Tue, 03 Nov 2009 14:51:55 +0100 boehmes added a specific SMT exception captured by smt_tac (prevents the SMT method from failing with an exception),
Tue, 03 Nov 2009 14:07:38 +0100 boehmes ignore parsing errors, return empty assignment instead
Thu, 05 Nov 2009 13:16:22 +0100 wenzelm scheduler: clarified interrupt attributes and handling;
Thu, 05 Nov 2009 13:01:11 +0100 wenzelm worker_next: plain signalling via work_available only, not scheduler_event;
Thu, 05 Nov 2009 00:13:00 +0100 wenzelm revert fulfill_proof_future tuning (actually a bit slower due to granularity issues?);
Wed, 04 Nov 2009 21:22:35 +0100 wenzelm avoid broadcast work_available, use daisy-chained signal instead;
Wed, 04 Nov 2009 21:21:05 +0100 wenzelm fulfill_proof_future: tuned important special case of singleton promise;
Wed, 04 Nov 2009 20:31:36 +0100 wenzelm worker_next: treat wait for work_available as Sleeping, not Waiting;
Wed, 04 Nov 2009 11:58:29 +0100 wenzelm worker activity: distinguish between waiting (formerly active) and sleeping;
Wed, 04 Nov 2009 11:37:06 +0100 wenzelm tuned;
Wed, 04 Nov 2009 11:30:22 +0100 wenzelm tuned thread data;
Wed, 04 Nov 2009 00:29:58 +0100 wenzelm worker_next: ensure that work_available is passed on before sleeping (was occasionally lost when worker configuration changed, causing scheduler deadlock);
Tue, 03 Nov 2009 19:52:09 +0100 wenzelm slightly leaner and more direct control of worker activity etc.;
Tue, 03 Nov 2009 10:36:20 +0100 bulwahn adding testcases for code inlining, sets and numerals to the example files of the predicate compiler and its quickcheck prototype; disabling length example
Tue, 03 Nov 2009 10:24:06 +0100 bulwahn adapted the inlining in the predicate compiler
Tue, 03 Nov 2009 10:24:05 +0100 bulwahn recursively replacing abstractions by new definitions in the predicate compiler
Mon, 02 Nov 2009 18:49:53 -0800 huffman merge
Mon, 02 Nov 2009 18:39:41 -0800 huffman add fixrec support for HOL pair constructor patterns
Mon, 02 Nov 2009 17:29:34 -0800 huffman define cprod_fun using Pair instead of cpair
Mon, 02 Nov 2009 17:19:49 -0800 huffman add (LAM (x, y). t) syntax and lemma csplit_Pair
Mon, 02 Nov 2009 23:06:06 +0100 krauss lexicographic order: run local descent proofs in parallel
Mon, 02 Nov 2009 13:43:50 -0800 huffman merged
Mon, 02 Nov 2009 12:26:23 -0800 huffman domain package no longer uses cfst/csnd/cpair
Mon, 02 Nov 2009 22:24:03 +0100 krauss conceal partial rules depending on config flag (i.e. when called via "fun")
Mon, 02 Nov 2009 22:24:00 +0100 krauss conceal "termination" rule, used only by special tools
Mon, 02 Nov 2009 22:23:57 +0100 krauss do not use Binding.empty: conceal flag gets lost in Thm.def_binding_optional
Mon, 02 Nov 2009 21:07:10 +0100 wenzelm modernized structure XML_Syntax;
Mon, 02 Nov 2009 21:05:47 +0100 wenzelm structure Thm_Deps;
Mon, 02 Nov 2009 21:03:41 +0100 wenzelm modernized structure Proof_Node;
Mon, 02 Nov 2009 20:57:48 +0100 wenzelm modernized structure Proof_Display;
Mon, 02 Nov 2009 20:50:48 +0100 wenzelm modernized structure Proof_Syntax;
Mon, 02 Nov 2009 20:48:08 +0100 wenzelm modernized structure Local_Syntax;
Mon, 02 Nov 2009 20:45:23 +0100 wenzelm modernized structure AutoBind;
Mon, 02 Nov 2009 20:38:46 +0100 wenzelm modernized structure Primitive_Defs;
Mon, 02 Nov 2009 20:34:59 +0100 wenzelm modernized structure Simple_Syntax;
Mon, 02 Nov 2009 20:30:40 +0100 wenzelm modernized structure Context_Position;
Mon, 02 Nov 2009 19:56:06 +0100 wenzelm observe usual naming conventions;
Mon, 02 Nov 2009 16:44:18 +0100 krauss find_theorems: respect conceal flag
Mon, 02 Nov 2009 17:30:38 +0100 wenzelm DEEPEN: all tracing is subject to trace_DEEPEN (NB: Proof General tends to "popup" tracing output);
Mon, 02 Nov 2009 17:29:48 +0100 wenzelm back to warning -- Proof General tends to "popup" tracing output;
Mon, 02 Nov 2009 15:49:59 +0100 boehmes split parsing of counterexamples from translation into terms (avoids Term.dummyT and ill-typed terms)
Mon, 02 Nov 2009 09:01:18 +0100 bulwahn merged
Sat, 31 Oct 2009 10:02:37 +0100 bulwahn predicate compiler creates code equations for predicates with full mode
Fri, 30 Oct 2009 09:55:15 +0100 bulwahn renamed rpred to random
Sun, 01 Nov 2009 21:42:27 +0100 wenzelm Rules that characterize functional/relational specifications.
Sun, 01 Nov 2009 20:59:34 +0100 wenzelm adapted Item_Net;
Sun, 01 Nov 2009 20:55:39 +0100 wenzelm allow multi-index;
Sun, 01 Nov 2009 20:55:14 +0100 wenzelm added insert_safe, delete_safe variants;
Sun, 01 Nov 2009 16:23:31 +0100 wenzelm tuned signature;
Sun, 01 Nov 2009 15:44:26 +0100 wenzelm modernized structure Context_Rules;
Sun, 01 Nov 2009 15:24:45 +0100 wenzelm modernized structure Rule_Cases;
Fri, 30 Oct 2009 18:33:21 +0100 haftmann merged
Fri, 30 Oct 2009 18:33:07 +0100 haftmann dedicated theory for loading numeral simprocs
Fri, 30 Oct 2009 18:32:41 +0100 haftmann set Pure theory name properly
Fri, 30 Oct 2009 18:32:40 +0100 haftmann tuned code setup
Fri, 30 Oct 2009 14:52:14 +0100 wenzelm some notes on SPASS 3.0 distribution;
Fri, 30 Oct 2009 14:02:42 +0100 haftmann merged
Fri, 30 Oct 2009 14:00:43 +0100 haftmann combined former theories Divides and IntDiv to one theory Divides
Fri, 30 Oct 2009 13:59:52 +0100 haftmann tuned variable names of bindings; conceal predicate constants
Fri, 30 Oct 2009 13:59:51 +0100 haftmann dedicated theory for loading numeral simprocs
Fri, 30 Oct 2009 13:59:51 +0100 haftmann moved some div/mod lemmas to theory Divides
Fri, 30 Oct 2009 13:59:50 +0100 haftmann tuned proof
Fri, 30 Oct 2009 13:59:49 +0100 haftmann moved Commutative_Ring into session Decision_Procs
Fri, 30 Oct 2009 11:31:34 +0100 boehmes abstract over variables in reversed order (application uses given order)
Fri, 30 Oct 2009 11:27:47 +0100 boehmes disable printing of unparsed counterexamples for CVC3 and Yices
Fri, 30 Oct 2009 11:26:38 +0100 boehmes pattern are separated only by spaces (no comma)
Fri, 30 Oct 2009 10:42:39 +0100 wenzelm back to polyml-svn -- performance impact is minimal, slowdown was caused by accumulated cruft of long-running Mac OS;
Fri, 30 Oct 2009 01:32:06 +0100 krauss less verbose termination tactics
Fri, 30 Oct 2009 01:32:06 +0100 krauss less verbose inductive invocation
Fri, 30 Oct 2009 01:32:06 +0100 krauss tuned
Fri, 30 Oct 2009 01:32:06 +0100 krauss absorbed inductive_wrap function into Function_Core; more conventional argument order; tuned
Thu, 29 Oct 2009 23:58:15 +0100 wenzelm merged
Thu, 29 Oct 2009 23:17:35 +0100 wenzelm recovered from 7a1f597f454e, simplified imports;
Thu, 29 Oct 2009 22:29:51 +0100 wenzelm merged
Thu, 29 Oct 2009 22:16:58 +0100 haftmann merged
Thu, 29 Oct 2009 22:16:40 +0100 haftmann adjusted to changes in theory Divides
Thu, 29 Oct 2009 22:16:12 +0100 haftmann moved some lemmas to theory Int
Thu, 29 Oct 2009 22:13:11 +0100 haftmann moved some dvd [int] facts to Int
Thu, 29 Oct 2009 22:13:09 +0100 haftmann moved Nat_Transfer before Divides; distributed Nat_Transfer setup accordingly
Thu, 29 Oct 2009 23:56:33 +0100 wenzelm eliminated some old folds;
Thu, 29 Oct 2009 23:49:55 +0100 wenzelm eliminated some old folds;
Thu, 29 Oct 2009 23:48:56 +0100 wenzelm eliminated some old folds;
Thu, 29 Oct 2009 20:53:24 +0100 wenzelm less aggressive tracing;
Thu, 29 Oct 2009 20:35:47 +0100 wenzelm DEEPEN: less aggressive tracing, subject to trace_DEEPEN;
Thu, 29 Oct 2009 18:53:58 +0100 wenzelm merged
Thu, 29 Oct 2009 18:17:26 +0100 wenzelm merged
Thu, 29 Oct 2009 14:06:49 +0100 bulwahn removing ancient predicate compiler files
Thu, 29 Oct 2009 14:03:55 +0100 bulwahn merged
Thu, 29 Oct 2009 13:59:37 +0100 bulwahn encapsulating records with datatype constructors and adding type annotations to make SML/NJ happy
Wed, 28 Oct 2009 12:29:03 +0100 bulwahn improved mode parser; added mode annotations to examples
Wed, 28 Oct 2009 12:29:02 +0100 bulwahn moved datatype mode and string functions to the auxillary structure
Wed, 28 Oct 2009 12:29:01 +0100 bulwahn improving mode parsing in the predicate compiler
Wed, 28 Oct 2009 12:29:00 +0100 bulwahn improved handling of alternative rules; added test cases for alternative rules; normalized tracing in the predicate compiler
Thu, 29 Oct 2009 16:22:14 +0000 paulson merged
Thu, 29 Oct 2009 16:21:43 +0000 paulson Tidied up some very ugly proofs
Thu, 29 Oct 2009 15:47:03 +0100 nipkow small fixes
(0) -30000 -10000 -3000 -1000 -120 +120 +1000 +3000 +10000 +30000 tip