Fri, 27 Apr 2012 15:24:37 +0200 blanchet thread theory cleanly and use "smt" method rather than Sledgehammer for Z3 (because of obscure debilitating bug)
Fri, 27 Apr 2012 15:24:37 +0200 blanchet move LEO-II closer to the top, for testing
Fri, 27 Apr 2012 15:24:37 +0200 blanchet get rid of old CASC setup and move the arithmetic part to a new theory
Fri, 27 Apr 2012 15:24:37 +0200 blanchet smaller batches, to play safe
Fri, 27 Apr 2012 15:24:37 +0200 blanchet move file to where it belongs
Fri, 27 Apr 2012 14:07:31 +0200 huffman implement transfer tactic with more scalable forward proof methods
Fri, 27 Apr 2012 13:19:21 +0200 blanchet tuning
Fri, 27 Apr 2012 13:18:55 +0200 blanchet tweak LEO-II setup
Fri, 27 Apr 2012 12:16:10 +0200 blanchet eta-expand unapplied equalities in THF rather than using a proxy
Fri, 27 Apr 2012 12:16:10 +0200 blanchet more tweaking of TPTP/CASC setup
Thu, 26 Apr 2012 21:58:16 +0200 kuncar added a basic sanity check for quot_map
Thu, 26 Apr 2012 20:22:39 +0200 wenzelm tuned comment;
Thu, 26 Apr 2012 20:09:38 +0200 blanchet fixed bug in handling of new numerals -- the left-hand side of "Numeral1 = 1" should be left alone and not translated to a built-in Kodkod numeral in the specification of the "numeral" function
Thu, 26 Apr 2012 19:44:18 +0200 wenzelm merged
Thu, 26 Apr 2012 14:42:50 +0200 hoelzl add code equation for real_of_float
Thu, 26 Apr 2012 14:11:13 +0200 kuncar tuned; don't generate abs code if quotient_type is used
Thu, 26 Apr 2012 12:03:11 +0200 kuncar support Quotient map theorems with invariant parameters
Thu, 26 Apr 2012 12:01:58 +0200 kuncar use a quot_map theorem attribute instead of the complicated map attribute
Thu, 26 Apr 2012 01:05:06 +0200 blanchet further tweaking for Satallax, so that TPTP problems before parsing and after generation are as similar as possible/practical
Thu, 26 Apr 2012 00:33:47 +0200 blanchet put Satallax first, at least for now (useful for experiments)
Thu, 26 Apr 2012 00:33:23 +0200 blanchet tuning
Thu, 26 Apr 2012 00:33:00 +0200 blanchet tuning
Thu, 26 Apr 2012 00:29:46 +0200 blanchet tentatively tag hypotheses as definition -- this sometimes help the "tptp_sledgehammer" tool (e.g. SEU466^1.p)
Thu, 26 Apr 2012 00:28:06 +0200 blanchet tuning; no need for relevance filter
Wed, 25 Apr 2012 23:39:19 +0200 blanchet tuning
Wed, 25 Apr 2012 22:00:33 +0200 blanchet don't extensionalize formulas for higher-order provers -- Satallax in particular will only expand definitions of the form "constant = ..."
Wed, 25 Apr 2012 22:00:33 +0200 blanchet don't use the native choice operator if the type encoding isn't higher-order
Wed, 25 Apr 2012 22:00:33 +0200 blanchet tuning
Wed, 25 Apr 2012 22:00:33 +0200 blanchet more work on TPTP Isabelle and Sledgehammer tactics
Wed, 25 Apr 2012 22:00:33 +0200 blanchet more work on CASC setup
Wed, 25 Apr 2012 22:53:35 +0200 wenzelm more direct bash process group invocation on Cygwin, bypassing extra sh.exe and perl.exe which tend to crash;
Wed, 25 Apr 2012 20:08:33 +0200 wenzelm mingw is windows (still inactive);
Wed, 25 Apr 2012 19:26:27 +0200 hoelzl add Caratheodories theorem for semi-rings of sets
Wed, 25 Apr 2012 19:26:00 +0200 hoelzl moved lemmas to appropriate places
Wed, 25 Apr 2012 17:15:10 +0200 wenzelm register polyml executables so that Cygwin rebaseall will see them;
Wed, 25 Apr 2012 15:54:36 +0200 wenzelm merged
Wed, 25 Apr 2012 15:44:26 +0200 wenzelm smarter PDF_VIEWER defaults, based on hints by Lars Noschinski;
Wed, 25 Apr 2012 15:09:18 +0200 hoelzl equate positive Lebesgue integral and MV-Analysis' Gauge integral
Wed, 25 Apr 2012 15:06:59 +0200 hoelzl correct lemma name
Wed, 25 Apr 2012 14:33:21 +0200 blanchet tweak TPTP Nitpick's output
Wed, 25 Apr 2012 14:33:21 +0200 blanchet remove too aggressive skolemization optimization (prevented discovery of a model in SYN994^1)
Wed, 25 Apr 2012 14:33:21 +0200 blanchet improve precision (noticed on SEV296^5.thy) -- the exception for "bool" used to be necessary because of a hack where "opt" meant two different things
Wed, 25 Apr 2012 14:33:21 +0200 blanchet output SZS status as early as possible
Wed, 25 Apr 2012 14:28:13 +0200 hoelzl sorted lemma list in NEWS
Wed, 25 Apr 2012 15:14:57 +0200 wenzelm merged
Wed, 25 Apr 2012 15:13:40 +0200 wenzelm reactivated ListCellRenderer for Java 6 (cf. b9e2ed4b1579, 0ddac15782e4, de249b5ae6e2);
Wed, 25 Apr 2012 15:13:03 +0200 wenzelm enforce our JAVA_HOME to avoid potential conflicts with other Java installations by the user;
Wed, 25 Apr 2012 14:30:42 +0200 wenzelm updated README;
Wed, 25 Apr 2012 14:29:15 +0200 wenzelm include generated application wrapper;
Wed, 25 Apr 2012 14:24:27 +0200 wenzelm back to mature jdk1.6.0_31, to avoid issues like Sidekick TAB completion and generic ListCellRenderer;
Wed, 25 Apr 2012 14:19:53 +0200 wenzelm ISABELLE_JDK_HOME is already provided by isatest shell environment;
Wed, 25 Apr 2012 11:29:55 +0200 wenzelm added splash screen, to reduce confusion when waiting for main application to start up;
Wed, 25 Apr 2012 10:59:06 +0200 wenzelm move polyml within Cygwin /usr/local to simplify its rebasing;
Wed, 25 Apr 2012 10:24:41 +0200 wenzelm improved spelling;
Wed, 25 Apr 2012 00:57:41 +0200 blanchet added "no_atp"s for extremely prolific, useless facts for ATPs
Tue, 24 Apr 2012 23:22:40 +0200 wenzelm tuned;
Tue, 24 Apr 2012 23:03:59 +0200 wenzelm merged
Tue, 24 Apr 2012 20:55:09 +0200 blanchet made "split_last" more robust in the face of obscure low-level errors
Tue, 24 Apr 2012 20:55:09 +0200 blanchet removed confusing error
Tue, 24 Apr 2012 19:14:03 +0200 wenzelm some friendly message;
Tue, 24 Apr 2012 16:09:17 +0200 wenzelm merged
Tue, 24 Apr 2012 16:06:12 +0200 wenzelm merged
Tue, 24 Apr 2012 14:13:04 +0100 sultana merged
Tue, 24 Apr 2012 14:06:38 +0100 sultana merged
Tue, 24 Apr 2012 13:59:29 +0100 sultana reversed Tools to Actions Mirabelle renaming;
Tue, 24 Apr 2012 13:55:02 +0100 sultana tuned;
Tue, 24 Apr 2012 13:56:13 +0200 blanchet reintroduce file offsets in Mirabelle output, but make sure they are not influenced by the length of the path
Tue, 24 Apr 2012 12:36:27 +0200 nipkow doc update
Tue, 24 Apr 2012 15:56:09 +0200 wenzelm prefer evince over old xpdf -- NB: x86-cygwin bundles its own application;
Tue, 24 Apr 2012 15:23:12 +0200 wenzelm cold-start HOME is user.home, in accordance with Cygwin-Terminal.bat;
Tue, 24 Apr 2012 15:07:49 +0200 wenzelm chmod -x;
Tue, 24 Apr 2012 13:33:10 +0200 wenzelm augment Isabelle home directory more systematically;
Tue, 24 Apr 2012 12:24:52 +0200 wenzelm Cygwin setup via the quasi-mirror isabelle.in.tum.de, which serves a fixed (downgraded) version;
Tue, 24 Apr 2012 12:23:19 +0200 wenzelm prevent change of directory, by pretending we are the "Command Here" utility;
Tue, 24 Apr 2012 11:07:50 +0200 nipkow typo
Tue, 24 Apr 2012 10:44:04 +0200 nipkow the perennial doc problem of how to define lists a second time
Tue, 24 Apr 2012 09:47:40 +0200 blanchet smoother handling of conjecture, so that its Skolem constants get displayed in countermodels
Tue, 24 Apr 2012 09:47:40 +0200 blanchet updated doc
Tue, 24 Apr 2012 09:47:40 +0200 blanchet add a timeout on the monotonicity check
Tue, 24 Apr 2012 09:47:40 +0200 blanchet handle TPTP definitions as definitions in Nitpick rather than as axioms
Tue, 24 Apr 2012 09:47:40 +0200 blanchet get rid of old parser, hopefully for good
Tue, 24 Apr 2012 09:47:40 +0200 blanchet fix handling of atomizable conjectures without a top-level "Trueprop" (e.g. "x == (y::nat)")
Tue, 24 Apr 2012 09:47:40 +0200 blanchet run Mirabelle in quick and dirty mode
Tue, 24 Apr 2012 09:09:55 +0200 nipkow doc update
Mon, 23 Apr 2012 23:55:06 +0200 wenzelm scrollable text;
Mon, 23 Apr 2012 23:50:27 +0200 wenzelm bundle Cygwin-Terminal.bat;
Mon, 23 Apr 2012 23:38:35 +0200 wenzelm basic Cygwin-Terminal for main Isabelle directory;
Mon, 23 Apr 2012 22:26:22 +0200 wenzelm moved to ~isatest/.bashrc to accomodate AFP;
Mon, 23 Apr 2012 22:22:57 +0200 wenzelm merged
Mon, 23 Apr 2012 21:46:52 +0200 nipkow merged
Mon, 23 Apr 2012 21:46:37 +0200 nipkow doc update
Mon, 23 Apr 2012 21:31:52 +0200 krauss NEWS
Mon, 23 Apr 2012 21:53:43 +0200 wenzelm typedef with implicit set definition is considered legacy;
Mon, 23 Apr 2012 21:44:36 +0200 wenzelm more standard method setup;
Mon, 23 Apr 2012 18:42:05 +0200 kuncar CONTRIBUTORS
Mon, 23 Apr 2012 18:42:03 +0200 kuncar added useful Trueprop_conv
Mon, 23 Apr 2012 17:18:18 +0200 kuncar move MRSL to a separate file
Mon, 23 Apr 2012 16:30:43 +0200 wenzelm avoid conflict of Isabelle vs. Isabelle.exe on Cygwin;
Mon, 23 Apr 2012 16:05:18 +0200 wenzelm more notes on Cygwin, notably for downgrading to 1.7.9 to avoid multi-threading instabilities starting with 1.7.10 early 2012;
Mon, 23 Apr 2012 13:40:02 +0200 hoelzl CONTRIBUTORS
Mon, 23 Apr 2012 12:14:35 +0200 hoelzl reworked Probability theory
Mon, 23 Apr 2012 12:23:23 +0100 sultana updated test;
Mon, 23 Apr 2012 12:23:23 +0100 sultana improved non-interpretation of constants and numbers;
Mon, 23 Apr 2012 12:23:23 +0100 sultana improved interpreting conditionals;
Mon, 23 Apr 2012 12:23:23 +0100 sultana disabled interpreting arithmetic;
Mon, 23 Apr 2012 12:23:23 +0100 sultana improved handling of single-quoted names;
Mon, 23 Apr 2012 12:23:23 +0100 sultana disabled exception packaging in tptp;
Mon, 23 Apr 2012 12:23:23 +0100 sultana moved function for testing problem-name parsing;
Mon, 23 Apr 2012 12:23:23 +0100 sultana removed redundant function;
Sun, 22 Apr 2012 23:08:53 +0200 wenzelm bundle Isabelle.exe;
Sun, 22 Apr 2012 21:32:35 +0200 huffman tuned precedence order of transfer rules
Sun, 22 Apr 2012 22:02:52 +0200 wenzelm updated generated files;
Sun, 22 Apr 2012 22:01:45 +0200 wenzelm updated const "relcomp";
Sun, 22 Apr 2012 21:47:32 +0200 wenzelm merged
Sun, 22 Apr 2012 20:16:30 +0200 huffman add transfer rule for set difference
Sun, 22 Apr 2012 21:43:57 +0200 wenzelm support Cygwin cold-start via Isabelle.exe, assuming layout of bundle;
Sun, 22 Apr 2012 19:44:40 +0200 wenzelm merged
Sun, 22 Apr 2012 19:18:26 +0200 huffman merged
Sun, 22 Apr 2012 17:54:47 +0200 huffman adapt to changes in generated transfer rules (cf. 4483c004499a)
Sun, 22 Apr 2012 16:53:24 +0200 huffman fix bug caused by misunderstanding of operator precedences (cf. cb44d09d9d22)
Sun, 22 Apr 2012 19:04:30 +0200 wenzelm more robust handling of PATH vs PATH_JVM -- required for cold start of Cygwin from Windows (e.g. Isabelle.exe);
Sun, 22 Apr 2012 16:33:41 +0200 wenzelm merged
Sun, 22 Apr 2012 14:16:46 +0200 blanchet fixed typos
Sun, 22 Apr 2012 14:16:46 +0200 blanchet tried harder to make SML/NJ happy
Sun, 22 Apr 2012 14:16:46 +0200 blanchet added timeout argument to TPTP tools
Sun, 22 Apr 2012 14:16:46 +0200 blanchet fix bug where "==" was used instead of "HOL.eq"
Sun, 22 Apr 2012 14:16:46 +0200 blanchet more meaningful default value
Sun, 22 Apr 2012 14:16:45 +0200 blanchet handle exception (needed to solve TPTP problem SEU880^5)
Sun, 22 Apr 2012 16:32:26 +0200 wenzelm pretend jedit is up-to-date if this is not a repository -- avoid accidental build attempts after touching files etc.;
Sun, 22 Apr 2012 16:08:10 +0200 wenzelm refer to isabelle.Main application wrapper;
Sun, 22 Apr 2012 15:55:13 +0200 wenzelm display return code like Isabelle.app on Mac OS;
Sun, 22 Apr 2012 15:50:29 +0200 wenzelm default Isabelle application wrapper -- JVM entry point for Isabelle.exe;
Sun, 22 Apr 2012 15:19:46 +0200 wenzelm updated Isabelle.exe specification, assuming layout of bundle;
Sun, 22 Apr 2012 14:30:18 +0200 wenzelm USER_HOME settings variable points to cross-platform user home directory;
Sun, 22 Apr 2012 11:05:04 +0200 huffman new example theory for quotient/transfer
Sat, 21 Apr 2012 21:38:08 +0200 huffman update NEWS for transfer/quotient
Sat, 21 Apr 2012 20:52:33 +0200 huffman enable variant of transfer method that proves an implication instead of an equivalence
Thu, 19 Apr 2012 19:36:24 +0200 haftmann moved modules with only vague relation to the code generator to theory HOL rather than theory Code_Generator
Sat, 21 Apr 2012 15:26:05 +0200 wenzelm merged
Sat, 21 Apr 2012 13:54:29 +0200 huffman NEWS for transfer, lifting, and quotient
Sat, 21 Apr 2012 13:49:31 +0200 huffman new example theory for transfer package
Sat, 21 Apr 2012 14:53:04 +0200 wenzelm some builtin session timing;
Sat, 21 Apr 2012 13:12:27 +0200 huffman move alternative definition lemmas into Lifting.thy;
Sat, 21 Apr 2012 13:06:22 +0200 huffman tuned proofs
Sat, 21 Apr 2012 11:21:23 +0200 huffman add transfer rule for List.set
Sat, 21 Apr 2012 11:04:21 +0200 huffman remove duplicate of lemma id_transfer
Sat, 21 Apr 2012 11:02:01 +0200 huffman added covariant relator set_rel, with transfer rules for set operations
Sat, 21 Apr 2012 10:59:52 +0200 huffman renamed contravariant relator set_rel to vset_rel, to make room for new covariant relator
Sat, 21 Apr 2012 11:15:49 +0200 blanchet tried to make SML/NJ happy
Sat, 21 Apr 2012 11:15:49 +0200 blanchet tuned "max_relevant" defaults for SMT solvers based on Judgment Day
Sat, 21 Apr 2012 11:15:49 +0200 blanchet prepend PWD to relative paths
Sat, 21 Apr 2012 11:15:49 +0200 blanchet reintroduced old FOF and CNF parsers, to work around TPTP_Parser failures
Sat, 21 Apr 2012 11:15:49 +0200 blanchet swap out Satallax, pull in E-SInE again -- it's not clear yet how useful Satallax is after proof reconstruction, whereas E-SInE performed surprisingly well on latest evaluations
Sat, 21 Apr 2012 07:33:47 +0200 huffman new transfer package rules and lifting setup for lists
Sat, 21 Apr 2012 06:49:04 +0200 huffman strengthen rule list_all2_induct
Fri, 20 Apr 2012 23:57:29 +0200 wenzelm more standard Theory_Data setup;
Fri, 20 Apr 2012 23:34:03 +0200 wenzelm merged
Fri, 20 Apr 2012 22:05:07 +0200 huffman add transfer rule for nat_case
Fri, 20 Apr 2012 22:54:13 +0200 huffman uniform naming scheme for transfer rules
Fri, 20 Apr 2012 22:49:40 +0200 huffman rename 'correspondence' method to 'transfer_prover'
Fri, 20 Apr 2012 18:29:21 +0200 kuncar hide the invariant constant for relators: invariant_commute infrastracture
Fri, 20 Apr 2012 23:16:46 +0200 wenzelm improved interleaving of start_execution vs. cancel_execution of the next update;
Fri, 20 Apr 2012 23:15:44 +0200 wenzelm tuned proofs;
Fri, 20 Apr 2012 22:48:48 +0200 wenzelm always revisit nodes independently of "required" flag, which may change during editing -- avoid "bloodbath effect" when changing perspective while loading;
Fri, 20 Apr 2012 22:51:06 +0200 wenzelm tuned;
Fri, 20 Apr 2012 20:29:44 +0200 wenzelm simplified internal actor protocol;
Fri, 20 Apr 2012 20:21:22 +0200 wenzelm builtin timing for main operations;
Fri, 20 Apr 2012 15:49:45 +0200 huffman add secondary transfer rule for universal quantifiers on non-bi-total relations
Fri, 20 Apr 2012 15:34:33 +0200 huffman move definition of set_rel into Library/Quotient_Set.thy
Fri, 20 Apr 2012 15:30:13 +0200 huffman add transfer rule for 'id'
Fri, 20 Apr 2012 14:57:19 +0200 huffman add new transfer rules and setup for lifting package
Fri, 20 Apr 2012 10:37:00 +0200 huffman setup_lifting preprocesses forall_transfer rule by unfolding mem_Collect_eq
Fri, 20 Apr 2012 11:17:01 +0200 hoelzl NEWS
Fri, 20 Apr 2012 11:14:39 +0200 hoelzl hide code generation facts in the Float theory, they are only exported for Approximation
Fri, 20 Apr 2012 10:47:04 +0200 nipkow merged
Fri, 20 Apr 2012 10:46:55 +0200 nipkow forgot to add file
Fri, 20 Apr 2012 10:18:08 +0200 huffman make correspondence tactic more robust by replacing lhs with schematic variable before applying intro rules
Thu, 19 Apr 2012 23:18:47 +0200 wenzelm merged
Thu, 19 Apr 2012 22:21:15 +0200 hoelzl NEWS
Thu, 19 Apr 2012 22:13:46 +0200 hoelzl transfer now handles Let
Thu, 19 Apr 2012 20:19:24 +0200 nipkow merged
Thu, 19 Apr 2012 20:19:13 +0200 nipkow added revised version of Abs_Int
Thu, 19 Apr 2012 19:36:09 +0200 huffman add transfer rule for Let
Thu, 19 Apr 2012 19:32:30 +0200 huffman add code lemmas for word operations
Thu, 19 Apr 2012 19:18:47 +0200 haftmann tuned whitespace
Thu, 19 Apr 2012 19:18:11 +0200 haftmann dropped dead code
Thu, 19 Apr 2012 18:24:40 +0200 kuncar rename no_code to no_abs_code - more appropriate name
Thu, 19 Apr 2012 17:31:34 +0200 kuncar use tnames for bound variables in rsp thms
Thu, 19 Apr 2012 17:49:08 +0200 blanchet true delayed evaluation of "SPASS_VERSION" environment variable
Thu, 19 Apr 2012 17:49:02 +0200 blanchet merged
Thu, 19 Apr 2012 11:14:57 +0200 blanchet use latest Z3
Thu, 19 Apr 2012 17:32:35 +0200 nipkow merged
Thu, 19 Apr 2012 17:32:30 +0200 nipkow reorganised IMP
Thu, 19 Apr 2012 11:55:30 +0200 hoelzl use real :: float => real as lifting-morphism so we can directlry use the rep_eq theorems
Wed, 18 Apr 2012 14:29:22 +0200 hoelzl use lifting to introduce floating point numbers
Wed, 18 Apr 2012 14:29:21 +0200 hoelzl replace the float datatype by a type with unique representation
Wed, 18 Apr 2012 14:29:20 +0200 hoelzl add lemmas to remove real conversions when compared to power of numerals
Wed, 18 Apr 2012 14:29:20 +0200 hoelzl add simp rules to rewrite comparisons of 1 and real
Wed, 18 Apr 2012 14:29:19 +0200 hoelzl add lemma to equate floor and div
Wed, 18 Apr 2012 14:29:18 +0200 hoelzl add powr_inj
Wed, 18 Apr 2012 14:29:17 +0200 hoelzl add lemmas to rewrite powr to power
Wed, 18 Apr 2012 14:29:16 +0200 hoelzl add lemmas to compare log with 0 and 1
Wed, 18 Apr 2012 14:29:05 +0200 hoelzl add ceiling_diff_floor_le_1
Thu, 19 Apr 2012 23:15:58 +0200 wenzelm display Java 7 only code for now (cf. b9e2ed4b1579);
Thu, 19 Apr 2012 21:53:24 +0200 wenzelm some sidekick options for more advanced completion;
Thu, 19 Apr 2012 21:47:50 +0200 wenzelm custom ListCellRenderer with text area font ensures that symbols are displayed reliably;
Thu, 19 Apr 2012 21:42:24 +0200 wenzelm tuned imports;
Thu, 19 Apr 2012 19:54:48 +0200 wenzelm more robust wrt. exceptions;
Thu, 19 Apr 2012 15:47:32 +0200 wenzelm accomodate digits within Isar command names, notably 'try0';
Thu, 19 Apr 2012 15:02:13 +0200 wenzelm more robust Sledgehammer in Prover IDE;
Thu, 19 Apr 2012 14:59:17 +0200 wenzelm test with jdk-7u3 that is also bundled;
Thu, 19 Apr 2012 12:28:10 +0200 kuncar create thm names correctly
Thu, 19 Apr 2012 13:19:57 +0200 wenzelm updated components according to tentative bundle;
Thu, 19 Apr 2012 13:15:06 +0200 wenzelm back to isatest with official polyml-5.4.1 (cf. ffa6e10df091);
Thu, 19 Apr 2012 11:52:07 +0200 huffman use simpler method for preserving bound variable names in transfer tactic
Thu, 19 Apr 2012 10:49:47 +0200 huffman tuned lemmas (v)image_id;
Thu, 19 Apr 2012 11:10:03 +0200 blanchet use latest SPASS
Thu, 19 Apr 2012 11:00:12 +0200 blanchet doc update
Thu, 19 Apr 2012 10:16:51 +0200 haftmann dropped dead code;
Thu, 19 Apr 2012 08:45:13 +0200 huffman generate abs_induct rules for quotient types
Thu, 19 Apr 2012 09:58:54 +0200 haftmann tuned
Thu, 19 Apr 2012 09:45:49 +0200 haftmann corrected Nbe.static_value: ignore cached compilations;
Thu, 19 Apr 2012 09:31:36 +0200 haftmann tuned heading
Wed, 18 Apr 2012 21:47:26 +0200 haftmann tuned name
Thu, 19 Apr 2012 07:25:44 +0100 sultana improved threading of thy-values through interpret functions;
Thu, 19 Apr 2012 07:25:41 +0100 sultana exceptions related to interpreting tptp problems now mention the relevant position in the tptp file;
Wed, 18 Apr 2012 17:44:39 +0200 huffman add option to transfer method for specifying variables not to generalize over
Tue, 17 Apr 2012 16:21:47 +1000 Thomas Sewell New tactic "word_bitwise" expands word equalities/inequalities into logic.
Wed, 18 Apr 2012 23:57:44 +0200 kuncar setup_lifting: no_code switch and supoport for quotient theorems
Wed, 18 Apr 2012 23:13:11 +0200 blanchet remove old TPTP CNF/FOF parser; always use Nik's new parser
Wed, 18 Apr 2012 23:13:10 +0200 blanchet more standard SZS output
Wed, 18 Apr 2012 22:40:25 +0200 blanchet Sledgehammer NEWS and CONTRIBUTORS
Wed, 18 Apr 2012 22:40:25 +0200 blanchet tuned SZS status output
Wed, 18 Apr 2012 22:40:25 +0200 blanchet update documentation (mostly based on feedback by Makarius)
Wed, 18 Apr 2012 22:40:25 +0200 blanchet added SZS status wrappers in TPTP mode
Wed, 18 Apr 2012 22:40:25 +0200 blanchet fixed Auto Nitpick's output
Wed, 18 Apr 2012 22:39:35 +0200 blanchet phase out "$TPTP_PROBLEMS_PATH"; prefer "$TPTP" for consistency with CASC setup
Wed, 18 Apr 2012 22:16:05 +0200 blanchet started integrating Nik's parser into TPTP command-line tools
Wed, 18 Apr 2012 21:28:49 +0200 wenzelm merged
Wed, 18 Apr 2012 21:11:50 +0200 haftmann tuned
(0) -30000 -10000 -3000 -1000 -240 +240 +1000 +3000 +10000 +30000 tip