src/HOL/Transitive_Closure.thy
Mon, 16 Apr 2012 17:22:51 +0200 duplicate "relpow" facts for "relpowp" (to emphasize that both worlds exist and obtain better search results with "find_theorems")
Tue, 03 Apr 2012 17:26:30 +0900 renamed "rel_comp" to "relcomp" (to be consistent with, e.g., "relpow")
Fri, 30 Mar 2012 09:04:29 +0200 power on predicate relations
Thu, 01 Mar 2012 19:34:52 +0100 more fundamental pred-to-set conversions, particularly by means of inductive_set; associated consolidation of some theorem names (c.f. NEWS)
Fri, 24 Feb 2012 22:46:44 +0100 moved predicate relations and conversion rules between set and predicate relations from Predicate.thy to Relation.thy; moved Predicate.thy upwards in theory hierarchy
Fri, 24 Feb 2012 09:40:02 +0100 given up disfruitful branch
Thu, 23 Feb 2012 21:25:59 +0100 moved predicate relations and conversion rules between set and predicate relations from Predicate.thy to Relation.thy; moved Predicate.thy upwards in theory hierarchy
Mon, 30 Jan 2012 13:55:26 +0100 renaming all lemmas with name rel_pow to relpow
Mon, 30 Jan 2012 13:55:23 +0100 adding code generation for relpow by copying the ideas for code generation of funpow
Fri, 27 Jan 2012 17:22:05 +0100 new code equation for ntrancl that allows computation of the transitive closure of sets on infinite types as well
Sun, 01 Jan 2012 11:28:45 +0100 cleanup of code declarations
Sat, 24 Dec 2011 15:53:12 +0100 tuned layout
Sun, 20 Nov 2011 21:07:10 +0100 eliminated obsolete "standard";
Sun, 16 Oct 2011 14:48:00 +0200 tuned type annnotation
Thu, 13 Oct 2011 23:35:15 +0200 avoid very specific code equation for card; corrected spelling
Thu, 13 Oct 2011 23:27:46 +0200 bouned transitive closure
Thu, 13 Oct 2011 23:02:59 +0200 moved acyclic predicate up in hierarchy
Thu, 13 Oct 2011 22:56:19 +0200 modernized definitions
Mon, 03 Oct 2011 14:43:13 +0200 adding lemma about rel_pow in Transitive_Closure for executable equation of the (refl) transitive closure
Tue, 13 Sep 2011 17:07:33 -0700 tuned proofs
Mon, 12 Sep 2011 07:55:43 +0200 new fastforce replacing fastsimp - less confusing name
Wed, 29 Jun 2011 20:39:41 +0200 simplified/unified Simplifier.mk_solver;
Fri, 13 May 2011 23:58:40 +0200 clarified map_simpset versus Simplifier.map_simpset_global;
Wed, 16 Mar 2011 19:50:56 +0100 added lemmas
Mon, 21 Feb 2011 10:44:19 +0100 renamed "nitpick\_def" to "nitpick_unfold" to reflect its new semantics
Mon, 13 Sep 2010 11:13:15 +0200 renamed lemmas: ext_iff -> fun_eq_iff, set_ext_iff -> set_eq_iff, set_ext -> set_eqI
Tue, 07 Sep 2010 10:05:19 +0200 expand_fun_eq -> ext_iff
Thu, 01 Jul 2010 16:54:42 +0200 qualified constants Set.member and Set.Collect
Thu, 10 Jun 2010 12:24:03 +0200 tuned quotes, antiquotations and whitespace
Thu, 18 Feb 2010 14:21:44 -0800 get rid of many duplicate simp rule warnings
Wed, 27 Jan 2010 14:02:53 +0100 lemma Image_closed_trancl
Sun, 10 Jan 2010 18:06:30 +0100 Tuned some proofs; nicer case names for some of the induction / cases rules.
Tue, 24 Nov 2009 10:31:01 +0100 removed "nitpick_def" attributes from (r)trancl(p), since "Nitpick.thy" overrides these
Fri, 13 Nov 2009 14:03:24 +0100 a few lemmas for point-free reasoning about transitive closure
Fri, 09 Oct 2009 13:40:34 +0200 simplified proof
Tue, 06 Oct 2009 18:44:06 +0200 inf/sup1/2_iff are mere duplicates of underlying definitions: dropped
Fri, 18 Sep 2009 09:07:48 +0200 be more cautious wrt. simp rules: sup1_iff, sup2_iff, inf1_iff, inf2_iff, SUP1_iff, SUP2_iff, INF1_iff, INF2_iff are no longer simp by default
Mon, 27 Jul 2009 21:47:41 +0200 "more standard" argument order of relation composition (op O)
Sun, 26 Jul 2009 22:28:31 +0200 replaced old METAHYPS by FOCUS;
Thu, 09 Jul 2009 17:34:59 +0200 move rel_pow_commute: "R O R ^^ n = R ^^ n O R" to Transitive_Closure
Wed, 17 Jun 2009 15:41:49 +0200 rtrancl lemmas
Thu, 11 Jun 2009 23:13:02 +0200 added lemma
Thu, 11 Jun 2009 22:17:13 +0200 added lemma
Mon, 01 Jun 2009 10:02:01 +0200 new lemma
Fri, 24 Apr 2009 17:45:15 +0200 funpow and relpow with shared "^^" syntax
Mon, 20 Apr 2009 09:32:40 +0200 power operation on functions in theory Nat; power operation on relations in theory Transitive_Closure
Mon, 16 Mar 2009 18:24:30 +0100 simplified method setup;
Fri, 13 Mar 2009 19:58:26 +0100 unified type Proof.method and pervasive METHOD combinators;
Wed, 04 Mar 2009 11:05:29 +0100 Merge.
Wed, 04 Mar 2009 10:45:52 +0100 Merge.
Mon, 02 Mar 2009 16:53:55 +0100 name changes
Thu, 26 Feb 2009 16:32:46 +0100 Fixed nonexhaustive match problem in decomp, to make it fail more gracefully
Wed, 21 Jan 2009 23:40:23 +0100 changed import hierarchy
Wed, 07 May 2008 10:56:49 +0200 - Function dec in Trancl_Tac must eta-contract relation before calling
Wed, 19 Mar 2008 22:47:38 +0100 more antiquotations;
Fri, 14 Mar 2008 19:57:12 +0100 Added lemmas
Thu, 28 Feb 2008 15:54:37 +0100 rtranclp_induct, tranclp_induct: added case_names;
Thu, 28 Feb 2008 12:56:28 +0100 rtranclE, tranclE: tuned statement, added case_names;
Tue, 13 Nov 2007 11:02:55 +0100 Removed some case_names and consumes attributes that are now no longer
Mon, 05 Nov 2007 22:48:37 +0100 tranclD2 (tranclD at the other end) + trancl_power