Fri, 18 Nov 2011 11:47:12 +0100 blanchet minor textual improvement
Fri, 18 Nov 2011 11:47:12 +0100 blanchet pull variables (Var) out of lambdas, so that the Isabelle theorems closely mirror the Metis lambda-lifted ones
Fri, 18 Nov 2011 11:47:12 +0100 blanchet wrap lambdas earlier, to get more control over beta/eta
Fri, 18 Nov 2011 11:47:12 +0100 blanchet move eta-contraction to before translation to Metis, to ensure everything stays in sync
Fri, 18 Nov 2011 11:47:12 +0100 blanchet avoid that var names get changed by resolution in Metis lambda-lifting
Fri, 18 Nov 2011 11:47:12 +0100 blanchet better threading of type encodings between Sledgehammer and "metis"
Fri, 18 Nov 2011 11:47:12 +0100 blanchet fixed bugs in lambda-lifting code -- ensure distinct names for variables
Fri, 18 Nov 2011 11:47:12 +0100 blanchet protect prefix against variant mutations
Fri, 18 Nov 2011 11:47:12 +0100 blanchet example cleanup
Fri, 18 Nov 2011 11:47:12 +0100 blanchet example cleanup
Fri, 18 Nov 2011 11:47:12 +0100 blanchet don't propagate user-set "type_enc" or "lam_trans" to Metis calls
Fri, 18 Nov 2011 11:47:12 +0100 blanchet don't needlessly pass "lam_lifted" option to "metis" call for SMT proof
Fri, 18 Nov 2011 11:47:12 +0100 blanchet avoid spurious messages in "lam_lifting" mode
Fri, 18 Nov 2011 11:47:12 +0100 blanchet eta-contract to avoid needless "lambda" wrappers
Fri, 18 Nov 2011 11:47:12 +0100 blanchet quiet down SMT
Fri, 18 Nov 2011 11:47:12 +0100 blanchet more aggressive lambda hiding (if we anyway need to pass an option to Metis)
Fri, 18 Nov 2011 11:47:12 +0100 blanchet updated Sledgehammer docs
Fri, 18 Nov 2011 11:47:12 +0100 blanchet don't pass "lam_lifted" option to "metis" unless there's a good reason
Fri, 18 Nov 2011 11:47:12 +0100 blanchet no needless reconstructors
Fri, 18 Nov 2011 11:47:12 +0100 blanchet removed more clutter
Fri, 18 Nov 2011 11:47:12 +0100 blanchet removed needless baggage
Fri, 18 Nov 2011 06:50:05 +0100 huffman Word.thy: reduce usage of numeral-representation-dependent thms like number_of_is_id in proofs
Fri, 18 Nov 2011 04:56:35 +0100 huffman merged
Thu, 17 Nov 2011 18:31:00 +0100 huffman Groups.thy: generalize several lemmas from class ab_group_add to class group_add
Thu, 17 Nov 2011 15:07:46 +0100 huffman HOL-Word: removed more duplicate theorems
Thu, 17 Nov 2011 14:52:05 +0100 huffman HOL-Word: removed many duplicate theorems (see NEWS)
Thu, 17 Nov 2011 14:24:10 +0100 huffman Word.thy: rearrange to instantiate arithmetic classes together with arithmetic operations
Thu, 17 Nov 2011 12:38:03 +0100 huffman move definitions of bitwise operators into appropriate document section
Thu, 17 Nov 2011 12:29:48 +0100 huffman HOL-Word: add simp rules for bin_rest, bin_last; shorten several proofs
Thu, 17 Nov 2011 08:07:54 +0100 huffman HOL-NSA: add number_semiring instance, reformulate several lemmas using '2' instead of '1+1'
Thu, 17 Nov 2011 07:55:09 +0100 huffman simplify implementation of approx_reorient_simproc
Thu, 17 Nov 2011 07:31:37 +0100 huffman name simp theorems st_0 and st_1
Thu, 17 Nov 2011 07:15:30 +0100 huffman remove redundant simp rules plus_enat_0
Thu, 17 Nov 2011 21:58:10 +0100 wenzelm eliminated slightly odd Rep' with dynamically-scoped [simplified];
Thu, 17 Nov 2011 21:31:29 +0100 wenzelm partial evaluation in invisible context;
Thu, 17 Nov 2011 19:01:05 +0100 bulwahn adding a preliminary example to show how the quotient_definition package can be generalized
Thu, 17 Nov 2011 18:44:56 +0100 bulwahn tuned header
Thu, 17 Nov 2011 14:35:32 +0100 bulwahn adding database of abs and rep terms to the quotient package; registering abs and rep terms in quotient_type and using them in quotient_definition
Thu, 17 Nov 2011 06:04:59 +0100 huffman simplify some proofs
Thu, 17 Nov 2011 06:01:47 +0100 huffman Int.thy: remove duplicate lemmas double_less_0_iff and odd_less_0, use {even,odd}_less_0_iff instead
Thu, 17 Nov 2011 05:27:45 +0100 huffman merged
Wed, 16 Nov 2011 15:20:27 +0100 huffman rewrite integer numeral div/mod simprocs to not return conditional rewrites; add regression tests
Wed, 16 Nov 2011 13:58:31 +0100 huffman remove redundant lemmas bin_last_mod and bin_rest_div, use bin_last_def and bin_rest_def instead
Wed, 16 Nov 2011 12:29:50 +0100 huffman simplify proof of word_of_int; remove several now-unused lemmas about Rep_Integ
Wed, 16 Nov 2011 23:09:46 +0100 wenzelm retain mixed attributes as dynamic theorem expression, but disallow subsequent static rules;
Wed, 16 Nov 2011 21:16:36 +0100 wenzelm clarified Attrib.partial_evaluation;
Wed, 16 Nov 2011 20:56:21 +0100 wenzelm tagging is not stable under morphisms and need to be replayed dynamically (mixed_attribute);
Wed, 16 Nov 2011 17:59:58 +0100 blanchet compile
Wed, 16 Nov 2011 17:26:42 +0100 blanchet compile
Wed, 16 Nov 2011 17:19:08 +0100 blanchet compile
Wed, 16 Nov 2011 17:06:14 +0100 blanchet give each time slice its own lambda translation
Wed, 16 Nov 2011 16:35:19 +0100 blanchet thread in additional options to minimizer
Wed, 16 Nov 2011 13:22:36 +0100 blanchet make metis reconstruction handling more flexible
Wed, 16 Nov 2011 11:16:23 +0100 blanchet document metis options better
Wed, 16 Nov 2011 10:44:36 +0100 blanchet fixed typo
Wed, 16 Nov 2011 10:34:08 +0100 blanchet document "lam_trans" option
Wed, 16 Nov 2011 10:09:44 +0100 blanchet nicer bullets
Wed, 16 Nov 2011 09:42:27 +0100 blanchet parse lambda translation option in Metis
Tue, 15 Nov 2011 22:20:58 +0100 blanchet rename the lambda translation schemes, so that they are understandable out of context
Tue, 15 Nov 2011 22:15:51 +0100 blanchet rename configuration option to more reasonable length
Tue, 15 Nov 2011 22:13:39 +0100 blanchet continued implementation of lambda-lifting in Metis
Tue, 15 Nov 2011 22:13:39 +0100 blanchet disable debugging output
Tue, 15 Nov 2011 22:13:39 +0100 blanchet use consts, not frees, for lambda-lifting
Tue, 15 Nov 2011 22:13:39 +0100 blanchet started implementing lambda-lifting in Metis
Tue, 15 Nov 2011 15:38:50 +0100 bulwahn improved generators for rational numbers to generate negative numbers;
Tue, 15 Nov 2011 15:38:49 +0100 bulwahn tuned
Tue, 15 Nov 2011 12:51:14 +0100 huffman remove one more old-style semicolon
Tue, 15 Nov 2011 12:49:05 +0100 huffman Metis_Examples/Big_O.thy: add number_ring class constraints, adapt proofs to use cancellation simprocs
Tue, 15 Nov 2011 12:39:49 +0100 huffman remove old-style semicolons
Tue, 15 Nov 2011 12:39:29 +0100 huffman avoid theorem references like 'semiring_norm(111)'
Tue, 15 Nov 2011 09:22:19 +0100 huffman merged
Mon, 14 Nov 2011 19:35:41 +0100 huffman merged
Mon, 14 Nov 2011 19:35:05 +0100 huffman Parametric_Ferrante_Rackoff.thy: restrict to class number_ring, replace '1+1' with '2' everywhere
Mon, 14 Nov 2011 09:49:05 +0100 huffman avoid numeral-representation-specific rules in metis proof
Mon, 14 Nov 2011 23:13:23 +0100 wenzelm merged
Mon, 14 Nov 2011 21:11:31 +0100 hoelzl remove sorry, otherwise it breaks the testboard
Mon, 14 Nov 2011 18:36:31 +0100 hoelzl cleaned up float theories; removed duplicate definitions and theorems
Mon, 14 Nov 2011 12:28:34 +0100 hoelzl enforce quick_and_dirty in Code_Real_Approx_By_Float
Mon, 14 Nov 2011 23:00:56 +0100 wenzelm some support for partial evaluation of attributed facts;
Mon, 14 Nov 2011 20:25:22 +0100 wenzelm tuned;
Mon, 14 Nov 2011 19:27:42 +0100 wenzelm eliminated dead code;
Mon, 14 Nov 2011 17:48:26 +0100 wenzelm inner syntax positions for string literals;
Mon, 14 Nov 2011 17:47:59 +0100 wenzelm less confusion subexpression markup;
Mon, 14 Nov 2011 16:52:19 +0100 wenzelm pass positions for named targets, for formal links in the document model;
Mon, 14 Nov 2011 16:24:50 +0100 wenzelm simplified Runtime.exn_messages: always print detailed version of low-level exeptions, which should not occur in regular user errors anyway;
Mon, 14 Nov 2011 16:16:49 +0100 wenzelm more detailed exception_trace: in Poly/ML 5.4.x intermediate handlers reset the trace (cf. Poly/ML SVN 1110);
Mon, 14 Nov 2011 12:29:19 +0100 bulwahn merged
Mon, 14 Nov 2011 11:14:06 +0100 bulwahn setting up exhaustive generators which are used for the smart generators
Mon, 14 Nov 2011 11:50:52 +0100 hoelzl add Code_Real_Approx_By_Float
Mon, 14 Nov 2011 09:25:05 +0100 huffman merged
Sun, 13 Nov 2011 19:30:35 +0100 huffman remove lemma float_remove_real_numeral, which duplicated Float.float_number_of
Sun, 13 Nov 2011 19:26:53 +0100 huffman remove unnecessary number-representation-specific rules from metis calls;
Sun, 13 Nov 2011 20:28:22 +0100 blanchet avoid confusing selector output
Sun, 13 Nov 2011 20:28:22 +0100 blanchet remove unsound line in Nitpick's "rat" setup
Sat, 12 Nov 2011 21:10:56 +0100 wenzelm tuned proofs;
Sat, 12 Nov 2011 20:14:09 +0100 wenzelm merged
Sat, 12 Nov 2011 13:01:56 +0100 huffman removed some old-style semicolons
Sat, 12 Nov 2011 19:44:56 +0100 wenzelm index markup elements for more efficient cumulate/select operations;
Sat, 12 Nov 2011 18:56:49 +0100 wenzelm tuned;
Sat, 12 Nov 2011 18:05:31 +0100 wenzelm tuned markup -- prefer user-perspective;
Sat, 12 Nov 2011 17:53:48 +0100 wenzelm tuned specifications and proofs;
Sat, 12 Nov 2011 17:52:28 +0100 wenzelm more precise type;
Sat, 12 Nov 2011 17:01:58 +0100 wenzelm refined Markup_Tree implementation: stacked markup within each entry;
Sat, 12 Nov 2011 12:21:42 +0100 wenzelm tuned signature;
Sat, 12 Nov 2011 11:45:49 +0100 wenzelm tuned signature;
Fri, 11 Nov 2011 22:09:07 +0100 wenzelm merged
Fri, 11 Nov 2011 12:31:00 +0100 huffman merged
Fri, 11 Nov 2011 12:30:28 +0100 huffman abel_cancel.ML: avoid canceling zeros, which would cause the simproc to return a trivial rewrite;
Fri, 11 Nov 2011 11:30:31 +0100 huffman use simproc_setup for the remaining nat_numeral simprocs
Fri, 11 Nov 2011 11:11:03 +0100 huffman use simproc_setup for more nat_numeral simprocs; add simproc tests
Fri, 11 Nov 2011 12:10:49 +0100 bulwahn using more conventional names for monad plus operations
Fri, 11 Nov 2011 22:05:18 +0100 wenzelm more tooltip content;
Fri, 11 Nov 2011 21:45:52 +0100 wenzelm added markup_cumulate operator;
Fri, 11 Nov 2011 16:25:32 +0100 wenzelm depth-first proof forking for improved locality (wrt. cancellation and overall memory usage);
Fri, 11 Nov 2011 16:06:26 +0100 wenzelm tuned;
Fri, 11 Nov 2011 15:25:22 +0100 wenzelm more abstract Markup_Tree;
Fri, 11 Nov 2011 14:24:38 +0100 wenzelm prefer statically typed Text.Markup;
Fri, 11 Nov 2011 14:07:20 +0100 wenzelm discontinued entity text color, notably historic red for classes;
Fri, 11 Nov 2011 12:52:57 +0100 wenzelm more scalable Proof_Context.prepare_sorts;
Fri, 11 Nov 2011 10:40:36 +0100 bulwahn increasing values_timeout to avoid failures of isatest with HOL-IMP
Fri, 11 Nov 2011 08:32:48 +0100 bulwahn renaming example invocations: tester predicate_compile is renamed to smart_exhaustive
Fri, 11 Nov 2011 08:32:45 +0100 bulwahn adding CPS compilation to predicate compiler;
Fri, 11 Nov 2011 08:32:44 +0100 bulwahn adding option allow_function_inversion to quickcheck options
Thu, 10 Nov 2011 23:30:50 +0100 wenzelm more efficient prepare_sorts -- bypass encoded positions;
Thu, 10 Nov 2011 22:54:15 +0100 wenzelm suppress irrelevant positions;
Thu, 10 Nov 2011 22:39:32 +0100 wenzelm more generous margin;
Thu, 10 Nov 2011 22:32:10 +0100 wenzelm pass term positions into check phase, where resulting types are reported accordingly, and eventually shown as tooltips;
Thu, 10 Nov 2011 17:47:25 +0100 wenzelm tuned signature;
(0) -30000 -10000 -3000 -1000 -128 +128 +1000 +3000 +10000 +30000 tip