src/HOL/Decision_Procs/Parametric_Ferrante_Rackoff.thy
Wed, 31 Oct 2018 14:47:59 +0100 wenzelm tuned;
Thu, 14 Jun 2018 15:45:53 +0200 nipkow tuned
Wed, 10 Jan 2018 15:25:09 +0100 nipkow ran isabelle update_op on all sources
Sun, 03 Dec 2017 22:28:19 +0100 wenzelm misc tuning and modernization;
Sun, 08 Oct 2017 22:28:21 +0200 haftmann replaced recdef were easy to replace
Fri, 18 Aug 2017 20:47:47 +0200 wenzelm session-qualified theory imports: isabelle imports -U -i -d '~~/src/Benchmarks' -a;
Sun, 16 Oct 2016 09:31:04 +0200 haftmann more standardized names
Thu, 05 Nov 2015 10:39:59 +0100 wenzelm isabelle update_cartouches -c -t;
Tue, 13 Oct 2015 09:21:15 +0200 haftmann prod_case as canonical name for product type eliminator
Sat, 18 Jul 2015 20:54:56 +0200 wenzelm prefer tactics with explicit context;
Wed, 24 Jun 2015 23:03:55 +0200 wenzelm tuned proofs -- less digits;
Tue, 23 Jun 2015 17:20:16 +0200 wenzelm tuned proofs;
Mon, 22 Jun 2015 23:19:48 +0200 wenzelm tuned proofs;
Sat, 20 Jun 2015 16:31:44 +0200 wenzelm isabelle update_cartouches;
Mon, 01 Jun 2015 18:59:21 +0200 haftmann separate class for division operator, with particular syntax added in more specific classes
Tue, 31 Mar 2015 21:54:32 +0200 haftmann given up separate type classes demanding `inverse 0 = 0`
Fri, 06 Mar 2015 15:58:56 +0100 wenzelm Thm.cterm_of and Thm.ctyp_of operate on local context;
Wed, 04 Mar 2015 19:53:18 +0100 wenzelm tuned signature -- prefer qualified names;
Tue, 03 Mar 2015 19:08:04 +0100 traytel eliminated some clones of Proof_Context.cterm_of
Wed, 26 Nov 2014 20:05:34 +0100 wenzelm renamed "pairself" to "apply2", in accordance to @{apply 2};
Sun, 02 Nov 2014 18:21:45 +0100 wenzelm modernized header uniformly as section;
Thu, 11 Sep 2014 19:32:36 +0200 blanchet updated news
Tue, 09 Sep 2014 20:51:36 +0200 blanchet ported Decision_Procs to new datatypes
Tue, 09 Sep 2014 20:51:36 +0200 blanchet use 'datatype_new' (soon to be renamed 'datatype') in Isabelle's libraries
Fri, 04 Jul 2014 20:18:47 +0200 haftmann reduced name variants for assoc and commute on plus and mult
Wed, 09 Apr 2014 09:37:47 +0200 hoelzl revert c1bbd3e22226, a14831ac3023, and 36489d77c484: divide_minus_left/right are again simp rules
Fri, 04 Apr 2014 17:58:25 +0100 paulson divide_minus_left divide_minus_right are in field_simps but are not default simprules
Wed, 26 Feb 2014 17:12:07 +0100 wenzelm tuned specifications and proofs;
Tue, 25 Feb 2014 23:12:48 +0100 wenzelm tuned specifications and proofs;
Wed, 12 Feb 2014 08:37:28 +0100 blanchet compile
Wed, 12 Feb 2014 08:37:06 +0100 blanchet adapted to 'xxx_{case,rec}' renaming, to new theorem names, and to new variable names in theorems
Sat, 14 Dec 2013 17:28:05 +0100 wenzelm proper context for basic Simplifier operations: rewrite_rule, rewrite_goals_rule, rewrite_goals_tac etc.;
Fri, 01 Nov 2013 18:51:14 +0100 haftmann more simplification rules on unary and binary minus
Tue, 03 Sep 2013 01:12:40 +0200 wenzelm tuned proofs -- clarified flow of facts wrt. calculation;
Fri, 15 Feb 2013 08:31:31 +0100 haftmann two target language numeral types: integer and natural, as replacement for code_numeral;
Thu, 29 Nov 2012 14:05:53 +0100 wenzelm more robust syntax that survives collapse of \<^isub> and \<^sub>;
Sun, 11 Nov 2012 19:24:01 +0100 haftmann modernized, simplified and compacted oracle and proof method glue code;
Fri, 19 Oct 2012 15:12:52 +0200 webertj Renamed {left,right}_distrib to distrib_{right,left}.
Fri, 27 Jul 2012 19:57:23 +0200 wenzelm tuned proofs -- avoid odd situations of polymorphic Frees in goal state;
Sun, 25 Mar 2012 20:15:39 +0200 huffman merged fork with new numeral representation (see NEWS)
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, 08 Aug 2011 09:52:09 -0700 huffman moved division ring stuff from Rings.thy to Fields.thy
Tue, 02 Aug 2011 10:36:50 +0200 krauss moved recdef package to HOL/Library/Old_Recdef.thy
Sun, 15 May 2011 17:45:53 +0200 wenzelm simplified/unified method_setup/attribute_setup;
Sat, 16 Apr 2011 20:49:48 +0200 wenzelm proper subgoal addressing via SUBGOAL/CSUBGOAL -- assuming these tactics did not handle Subscript in any special way;
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;
Fri, 08 Apr 2011 13:31:16 +0200 wenzelm explicit structure Syntax_Trans;
Fri, 25 Feb 2011 20:07:48 +0100 nipkow Some cleaning up
Fri, 25 Feb 2011 14:25:41 +0100 nipkow added simp lemma nth_Cons_pos to List
Thu, 24 Feb 2011 20:52:05 +0100 krauss removed unused lemma
Wed, 23 Feb 2011 11:16:56 +0100 krauss eliminated remdps in favor of List.remdups
Wed, 23 Feb 2011 11:15:06 +0100 krauss recdef -> fun
Wed, 23 Feb 2011 10:48:57 +0100 krauss recdef -> fun
Mon, 21 Feb 2011 23:54:53 +0100 wenzelm merged, resolving spurious conflicts and giving up Reflected_Multivariate_Polynomial.thy from ab5d2d81f9fb;
Mon, 21 Feb 2011 23:14:36 +0100 krauss removed duplicate declarations
Mon, 21 Feb 2011 23:47:19 +0100 wenzelm tuned proofs -- eliminated prems;
Wed, 29 Dec 2010 17:34:41 +0100 wenzelm explicit file specifications -- avoid secondary load path;
Wed, 08 Sep 2010 19:21:46 +0200 haftmann modernized primrec
Sat, 28 Aug 2010 16:14:32 +0200 haftmann formerly unnamed infix equality now named HOL.eq
less more (0) -60 tip