src/HOL/Tools/refute.ML
Wed, 04 May 2011 19:35:48 +0200 blanchet exploit inferred monotonicity
Sat, 16 Apr 2011 18:11:20 +0200 wenzelm eliminated old List.nth;
Sat, 16 Apr 2011 16:15:37 +0200 wenzelm modernized structure Proof_Context;
Sun, 27 Mar 2011 16:56:16 +0200 krauss avoid *** in normal output, which usually marks errors in logs
Sat, 08 Jan 2011 17:14:48 +0100 wenzelm misc tuning and comments based on review of Theory_Data, Proof_Data, Generic_Data usage;
Sat, 08 Jan 2011 16:01:51 +0100 wenzelm modernized structure Prop_Logic;
Fri, 26 Nov 2010 21:31:46 +0100 wenzelm explicit use of unprefix;
Sat, 20 Nov 2010 00:53:26 +0100 wenzelm renamed raw "explode" function to "raw_explode" to emphasize its meaning;
Mon, 25 Oct 2010 21:06:56 +0200 wenzelm renamed Output.priority to Output.urgent_message to emphasize its special role more clearly;
Fri, 01 Oct 2010 10:25:36 +0200 haftmann chop_while replace drop_while and take_while
Thu, 30 Sep 2010 18:37:29 +0200 haftmann take_while, drop_while
Fri, 03 Sep 2010 11:21:58 +0200 wenzelm turned show_consts into proper configuration option;
Fri, 03 Sep 2010 10:58:11 +0200 wenzelm prefer regular Proof.context over background theory;
Thu, 02 Sep 2010 17:12:16 +0200 wenzelm just one refute.ML;
Thu, 02 Sep 2010 16:45:21 +0200 wenzelm use existing Integer.pow, despite its slightly odd argument order;
Thu, 02 Sep 2010 16:31:50 +0200 wenzelm tuned whitespace and indentation, emphasizing the logical structure of this long text;
Sat, 28 Aug 2010 16:14:32 +0200 haftmann formerly unnamed infix equality now named HOL.eq
Fri, 27 Aug 2010 10:56:46 +0200 haftmann formerly unnamed infix conjunction and disjunction now named HOL.conj and HOL.disj
Thu, 26 Aug 2010 20:51:17 +0200 haftmann formerly unnamed infix impliciation now named HOL.implies
Thu, 19 Aug 2010 12:11:57 +0200 haftmann use HOLogic.boolT and @{typ bool} more pervasively
Thu, 01 Jul 2010 16:54:42 +0200 haftmann qualified constants Set.member and Set.Collect
Mon, 28 Jun 2010 15:32:25 +0200 haftmann avoid List.all
Fri, 11 Jun 2010 17:14:01 +0200 haftmann avoid references to old constdefs
Thu, 10 Jun 2010 12:24:03 +0200 haftmann tuned quotes, antiquotations and whitespace
Tue, 08 Jun 2010 16:37:22 +0200 haftmann tuned quotes, antiquotations and whitespace
Mon, 31 May 2010 18:49:32 +0200 blanchet move SAT solver warning from every invocation of SAT solver to the tool, Refute, that uses it;
Tue, 25 May 2010 20:28:16 +0200 wenzelm eliminated various catch-all exception patterns, guessing at the concrete exeptions that are intended here;
Wed, 05 May 2010 18:25:34 +0200 haftmann farewell to old-style mem infixes -- type inference in situations with mem_int and mem_string should provide enough information to resolve the type of (op =)
Thu, 29 Apr 2010 01:17:14 +0200 blanchet expand combinators in Isar proofs constructed by Sledgehammer;
Fri, 23 Apr 2010 16:59:48 +0200 blanchet remove debugging code
Tue, 13 Apr 2010 15:16:54 +0200 blanchet commented out unsound "lfp"/"gfp" handling + fixed set output syntax;
Sat, 13 Mar 2010 15:12:56 +0100 wenzelm more antiquotations;
Fri, 19 Feb 2010 14:47:01 +0100 haftmann moved remaning class operations from Algebras.thy to Groups.thy
Wed, 10 Feb 2010 14:12:04 +0100 haftmann moved less_eq, less to Orderings.thy; moved abs, sgn to Groups.thy
Thu, 28 Jan 2010 11:48:49 +0100 haftmann new theory Algebras.thy for generic algebraic structures
Mon, 14 Dec 2009 12:14:12 +0100 blanchet added "no_assms" option to Refute, and include structured proof assumptions by default;
Mon, 07 Dec 2009 11:44:49 +0100 blanchet better error message in Refute when specifying a non-existing SAT solver
Mon, 30 Nov 2009 11:42:49 +0100 haftmann modernized structures and tuned headers of datatype package modules; joined former datatype.ML and datatype_rep_proofs.ML
Tue, 24 Nov 2009 17:28:25 +0100 haftmann curried take/drop
Sun, 08 Nov 2009 18:43:42 +0100 wenzelm adapted Theory_Data;
Thu, 29 Oct 2009 23:56:33 +0100 wenzelm eliminated some old folds;
Thu, 29 Oct 2009 17:58:26 +0100 wenzelm standardized filter/filter_out;
Tue, 27 Oct 2009 22:57:23 +0100 wenzelm eliminated some old folds;
Tue, 27 Oct 2009 17:34:00 +0100 wenzelm normalized basic type abbreviations;
Thu, 22 Oct 2009 13:48:06 +0200 haftmann map_range (and map_index) combinator
Wed, 21 Oct 2009 16:57:57 +0200 blanchet merged
Wed, 21 Oct 2009 16:54:04 +0200 blanchet fixed the "expect" mechanism of Refute in the face of timeouts
Wed, 21 Oct 2009 12:02:56 +0200 haftmann curried union as canonical list operation
Wed, 21 Oct 2009 08:16:25 +0200 haftmann merged
Wed, 21 Oct 2009 08:14:38 +0200 haftmann dropped redundant gen_ prefix
Tue, 20 Oct 2009 16:13:01 +0200 haftmann replaced old_style infixes eq_set, subset, union, inter and variants by generic versions
Wed, 21 Oct 2009 00:36:12 +0200 wenzelm standardized basic operations on type option;
Mon, 19 Oct 2009 21:54:57 +0200 wenzelm uniform use of Integer.add/mult/sum/prod;
Thu, 15 Oct 2009 23:28:10 +0200 wenzelm replaced String.concat by implode;
Thu, 15 Oct 2009 21:28:39 +0200 wenzelm normalized aliases of Output operations;
Fri, 02 Oct 2009 21:41:57 +0200 wenzelm Refute.refute_goal: canonical goal addresses from 1 (renamed from refute_subgoal to clarify change in semantics);
Fri, 10 Jul 2009 07:59:27 +0200 haftmann dropped find_index_eq
Mon, 06 Jul 2009 19:58:52 +0200 wenzelm renamed inclass/Inclass to of_class/OfClass, in accordance to of_sort;
Tue, 23 Jun 2009 16:27:12 +0200 haftmann tuned interfaces of datatype module
Sun, 21 Jun 2009 08:38:58 +0200 haftmann simplified names of common datatype types
Fri, 19 Jun 2009 17:23:21 +0200 haftmann discontinued ancient tradition to suffix certain ML module names with "_package"
Wed, 11 Mar 2009 15:56:51 +0100 haftmann HOLogic.mk_set, HOLogic.dest_set
Sat, 07 Mar 2009 16:47:36 +0100 blanchet Added a second timeout mechanism to Refute.
Sat, 07 Mar 2009 12:26:56 +0100 blanchet Refute: Distinguish between "genuine" and "potential" in the newly added "expect" option.
Fri, 06 Mar 2009 19:37:31 +0100 blanchet Added "expect" option to Refute, like in Nitpick, that allows to write regression tests.
Fri, 06 Mar 2009 17:21:17 +0100 blanchet Fix remaining occurrences of "'a set" in Refute, by using "'a => bool" instead.
Fri, 06 Mar 2009 11:10:57 +0100 haftmann merged
Thu, 05 Mar 2009 08:24:28 +0100 haftmann merged
Thu, 05 Mar 2009 08:23:11 +0100 haftmann set operations Int, Un, INTER, UNION, Inter, Union, empty, UNIV are now proper qualified constants with authentic syntax
Thu, 05 Mar 2009 10:19:51 +0100 blanchet Reintroduced previous changes: Made "Refute.norm_rhs" public and simplified the configuration of the BerkMin and zChaff SAT solvers.
Wed, 04 Mar 2009 11:05:29 +0100 blanchet Merge.
Wed, 04 Mar 2009 10:45:52 +0100 blanchet Merge.
Wed, 04 Mar 2009 10:43:39 +0100 blanchet Made Refute.norm_rhs public, so I can use it in Nitpick.
Sun, 01 Mar 2009 23:36:12 +0100 wenzelm use long names for old-style fold combinators;
Tue, 17 Feb 2009 14:01:54 +0100 blanchet Reintroduce set_interpreter for Collect and op :.
Fri, 06 Feb 2009 13:43:19 +0100 blanchet Rearrange Refute/SAT theory dependencies so as to use even more antiquotations in refute.ML +
Wed, 04 Feb 2009 18:10:07 +0100 blanchet Make some Refute functions public so I can use them in Nitpick,
Thu, 01 Jan 2009 14:23:39 +0100 wenzelm avoid polymorphic equality;
Wed, 31 Dec 2008 18:53:17 +0100 wenzelm use regular Term.add_XXX etc.;
Wed, 31 Dec 2008 00:08:13 +0100 wenzelm moved old add_term_vars, add_term_frees etc. to structure OldTerm;
Fri, 05 Dec 2008 18:42:37 +0100 haftmann removed Table.extend, NameSpace.extend_table
Tue, 07 Oct 2008 16:07:50 +0200 haftmann arbitrary is undefined
Sun, 18 May 2008 17:03:20 +0200 wenzelm eliminated theory CPure;
Sun, 18 May 2008 15:04:09 +0200 wenzelm moved global pretty/string_of functions from Sign to Syntax;
Sat, 17 May 2008 15:31:42 +0200 wenzelm cat_lines;
Thu, 27 Mar 2008 14:41:07 +0100 wenzelm removed Display.raw_string_of_XXX (use regular Sign.string_of_XXX);
Wed, 19 Mar 2008 07:20:32 +0100 haftmann Type.lookup now curried
Wed, 05 Dec 2007 14:16:05 +0100 haftmann map_product and fold_product
Mon, 15 Oct 2007 01:57:50 +0200 webertj interpreter for List.append added again
Fri, 12 Oct 2007 22:00:47 +0200 webertj significant code overhaul, bugfix for inductive data types
Tue, 09 Oct 2007 17:10:38 +0200 wenzelm renamed AxClass.get_definition to AxClass.get_info (again);
Mon, 24 Sep 2007 13:52:50 +0200 wenzelm replaced interrupt_timeout by TimeLimit.timeLimit (available on SML/NJ and Poly/ML 5.1);
Fri, 20 Jul 2007 14:28:25 +0200 haftmann moved class ord from Orderings.thy to HOL.thy
Sat, 19 May 2007 11:33:57 +0200 haftmann constant op @ now named append
Thu, 17 May 2007 19:49:40 +0200 haftmann canonical prefixing of class constants
Mon, 07 May 2007 00:49:59 +0200 wenzelm simplified DataFun interfaces;
Wed, 04 Apr 2007 00:11:10 +0200 wenzelm cleaned-up Output functions;
Tue, 03 Apr 2007 19:24:11 +0200 wenzelm removed assert/deny (avoid clash with Alice keywords and confusion due to strict evaluation);
Fri, 19 Jan 2007 22:04:22 +0100 webertj interpreter for Finite_Set.finite added
Fri, 19 Jan 2007 21:20:10 +0100 webertj reformatted to 80 chars/line
Wed, 10 Jan 2007 19:19:24 +0100 webertj tuned
Fri, 05 Jan 2007 15:33:05 +0100 webertj reverted to v1.60 (PolyML 4.1.3 still has the wrong signature for Array.modifyi)
Thu, 04 Jan 2007 17:52:28 +0100 webertj using Array.modifyi (no functional change)
Thu, 04 Jan 2007 15:29:44 +0100 webertj obsolete sign_of calls removed
Thu, 04 Jan 2007 00:12:30 +0100 webertj constants are unfolded, universal quantifiers are stripped, some minor changes
Fri, 29 Dec 2006 17:24:41 +0100 wenzelm replaced Sign.classes by Sign.all_classes (topologically sorted);
Mon, 27 Nov 2006 14:33:18 +0100 webertj outermost universal quantifiers are stripped
Thu, 09 Nov 2006 18:48:45 +0100 webertj interpreters for fst and snd added
Mon, 23 Oct 2006 16:49:21 +0200 haftmann switched merge_alists'' to AList.merge'' whenever appropriate
Fri, 20 Oct 2006 17:07:26 +0200 haftmann slight cleanup
Fri, 20 Oct 2006 10:44:33 +0200 haftmann Symtab.foldl replaced by Symtab.fold
Wed, 04 Oct 2006 14:17:38 +0200 haftmann insert replacing ins ins_int ins_string
Fri, 15 Sep 2006 22:56:13 +0200 wenzelm renamed Term.map_term_types to Term.map_types (cf. Term.fold_types);
Fri, 15 Sep 2006 18:06:51 +0200 webertj trivial whitespace change
Tue, 11 Jul 2006 12:16:58 +0200 wenzelm removed obsolete mem_term;
Tue, 16 May 2006 13:01:24 +0200 wenzelm more abstract interface to classes/arities;
Thu, 06 Apr 2006 16:10:46 +0200 haftmann cleanup in datatype package
Fri, 17 Mar 2006 09:34:23 +0100 haftmann renamed op < <= to Orderings.less(_eq)
Fri, 10 Mar 2006 15:33:48 +0100 haftmann renamed HOL + - * etc. to HOL.plus HOL.minus HOL.times etc.
Mon, 06 Feb 2006 20:58:59 +0100 wenzelm Logic.const_of_class/class_of_const;
less more (0) -120 tip