src/HOL/Tools/Function/lexicographic_order.ML
Sat, 25 Jul 2015 23:41:53 +0200 wenzelm updated to infer_instantiate;
Sat, 18 Jul 2015 20:47:08 +0200 wenzelm prefer tactics with explicit context;
Tue, 07 Jul 2015 18:37:24 +0200 blanchet have the installed termination prover take a 'quiet' flag
Mon, 01 Jun 2015 13:35:16 +0200 wenzelm clarified context;
Fri, 06 Mar 2015 15:58:56 +0100 wenzelm Thm.cterm_of and Thm.ctyp_of operate on local context;
Fri, 06 Mar 2015 13:39:34 +0100 wenzelm clarified context;
Wed, 04 Mar 2015 19:53:18 +0100 wenzelm tuned signature -- prefer qualified names;
Fri, 19 Dec 2014 23:01:46 +0100 wenzelm just one data slot per program unit;
Wed, 29 Oct 2014 14:14:36 +0100 wenzelm modernized setup;
Sat, 16 Aug 2014 19:20:11 +0200 wenzelm updated to named_theorems;
Thu, 20 Mar 2014 21:07:57 +0100 wenzelm enforce subgoal boundaries via SUBGOAL/SUBGOAL_CASES -- clean tactical failure if out-of-range;
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
less more (0) -30 tip