src/HOL/Tools/Function/lexicographic_order.ML
Mon, 13 May 2013 12:40:17 +0200 wenzelm retain goal display options when printing error messages, to avoid breakdown for huge goals;
Thu, 18 Apr 2013 17:07:01 +0200 wenzelm simplifier uses proper Proof.context instead of historic type simpset;
Mon, 15 Oct 2012 15:43:12 +0200 wenzelm tuned message -- avoid extra blank lines;
Sat, 13 Oct 2012 19:53:04 +0200 wenzelm some attempts to unify/simplify pretty_goal;
Thu, 12 Apr 2012 18:39:19 +0200 wenzelm more standard method setup;
Fri, 02 Dec 2011 14:54:25 +0100 wenzelm more antiquotations;
Fri, 13 May 2011 23:58:40 +0200 wenzelm clarified map_simpset versus Simplifier.map_simpset_global;
Fri, 13 May 2011 22:55:00 +0200 wenzelm proper Proof.context for classical tactics;
Thu, 12 May 2011 22:46:21 +0200 wenzelm prefer plain simpset operations;
Sat, 16 Apr 2011 16:15:37 +0200 wenzelm modernized structure Proof_Context;
Thu, 13 Jan 2011 21:50:13 +0100 wenzelm more precise pretty printing -- to accomodate Scala message layout;
Wed, 03 Nov 2010 11:11:49 +0100 wenzelm replaced ancient sys_error by raise Fail, assuming that the latter is not handled specifically by the environment;
Tue, 05 Oct 2010 18:09:31 +0200 krauss tuned
Tue, 05 Oct 2010 18:09:29 +0200 krauss force less agressively
Tue, 05 Oct 2010 16:33:16 +0200 krauss lexicographic_order: replace parallel map with laziness to avoid wasting cycles on proofs that are not needed
Fri, 03 Sep 2010 21:13:53 +0200 wenzelm pretty_goals: turned some global references and function arguments into configuration options (goals_limit = 10, goals_total = true, show_main_goal = false) depending on the context;
Wed, 28 Apr 2010 11:52:04 +0200 krauss default termination prover as plain tactic
Sat, 27 Feb 2010 20:57:08 +0100 wenzelm clarified @{const_name} vs. @{const_abbrev};
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
Sat, 02 Jan 2010 23:18:58 +0100 krauss new year's resolution: reindented code in function package
Mon, 23 Nov 2009 15:05:59 +0100 krauss eliminated dead code and some unused bindings, reported by polyml
Mon, 02 Nov 2009 23:06:06 +0100 krauss lexicographic order: run local descent proofs in parallel
Fri, 30 Oct 2009 01:32:06 +0100 krauss less verbose termination tactics
Fri, 23 Oct 2009 16:22:10 +0200 krauss function package: more standard names for structures and files
Thu, 15 Oct 2009 23:28:10 +0200 wenzelm replaced String.concat by implode;
Fri, 18 Sep 2009 09:07:50 +0200 haftmann tuned const_name antiquotations
Sat, 25 Jul 2009 10:31:27 +0200 wenzelm renamed structure Display_Goal to Goal_Display;
Fri, 24 Jul 2009 11:50:35 +0200 wenzelm Display_Goal.pretty_goals: always Markup.subgoal, clarified options;
Thu, 23 Jul 2009 18:44:09 +0200 wenzelm renamed simpset_of to global_simpset_of, and local_simpset_of to simpset_of -- same for claset and clasimpset;
Thu, 23 Jul 2009 16:52:16 +0200 wenzelm clarified pretty_goals, pretty_thm_aux: plain context;
Mon, 20 Jul 2009 21:20:09 +0200 wenzelm moved pretty_goals etc. to Display_Goal (required by tracing tacticals);
Thu, 02 Jul 2009 17:34:14 +0200 wenzelm renamed NamedThmsFun to Named_Thms;
Tue, 23 Jun 2009 12:09:30 +0200 haftmann uniformly capitialized names for subdirectories
less more (0) tip