src/HOL/Relation.thy
Sat, 17 Mar 2012 11:35:18 +0100 spelt out missing colemmas
Sat, 17 Mar 2012 08:00:18 +0100 generalized INF_INT_eq, SUP_UN_eq
Mon, 12 Mar 2012 21:41:11 +0100 tuned proofs
Mon, 12 Mar 2012 15:12:22 +0100 tuned pred_set_conv lemmas. Skipped lemmas changing the lemmas generated by inductive_set
Mon, 12 Mar 2012 15:11:24 +0100 tuned simpset
Wed, 07 Mar 2012 21:34:36 +0100 tuned syntax; more candidates
Fri, 02 Mar 2012 21:45:45 +0100 more fundamental pred-to-set conversions for range and domain by means of inductive_set
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)
Sun, 26 Feb 2012 21:44:12 +0100 restored accidental omission
Sun, 26 Feb 2012 21:26:28 +0100 tuned structure
Sun, 26 Feb 2012 20:43:33 +0100 tuned structure; dropped already existing syntax declarations
Sun, 26 Feb 2012 20:10:14 +0100 tuned syntax declarations; tuned structure
Sun, 26 Feb 2012 15:28:48 +0100 marked candidates for rule declarations
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
Fri, 24 Feb 2012 08:49:36 +0100 explicit remove of lattice notation
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 21:49:41 +0100 added "'a rel"
Sun, 01 Jan 2012 11:28:45 +0100 cleanup of code declarations
Sat, 24 Dec 2011 15:53:09 +0100 dropped obsolete code equation for Id
Thu, 13 Oct 2011 23:02:59 +0200 moved acyclic predicate up in hierarchy
Thu, 13 Oct 2011 22:56:19 +0200 modernized definitions
Tue, 20 Sep 2011 21:47:52 +0200 tuned specification and lemma distribution among theories; tuned proofs
Tue, 13 Sep 2011 17:07:33 -0700 tuned proofs
Thu, 18 Aug 2011 13:55:26 +0200 observe distinction between sets and predicates more properly
Mon, 21 Feb 2011 10:44:19 +0100 renamed "nitpick\_def" to "nitpick_unfold" to reflect its new semantics
Tue, 07 Dec 2010 13:33:28 +0100 adding a definition for refl_on which is friendly for quickcheck and nitpick
Fri, 03 Dec 2010 08:40:47 +0100 adding a nice definition of Id_on for quickcheck and nitpick
Sun, 09 May 2010 12:00:43 +0200 added lemmas rel_comp_UNION_distrib(2)
Fri, 07 May 2010 15:03:57 +0200 removed semicolons
Fri, 07 May 2010 15:03:53 +0200 rule subrelI (for nice Isar proofs of relation inequalities)
Thu, 18 Mar 2010 12:58:52 +0100 now use "Named_Thms" for "noatp", and renamed "noatp" to "no_atp"
Mon, 26 Oct 2009 23:27:24 +0100 lemma converse_inv_image
Mon, 05 Oct 2009 16:41:06 +0100 New facts about domain and range in
Thu, 01 Oct 2009 17:11:48 +0200 proper merge of interpretation equations
Mon, 31 Aug 2009 20:34:48 +0200 moved lemma Wellfounded.in_inv_image to Relation.thy
Mon, 27 Jul 2009 21:47:41 +0200 "more standard" argument order of relation composition (op O)
Tue, 28 Apr 2009 13:34:48 +0200 ephermal enforcement of import order to circumvent current problem in merging interpretation morphisms
Mon, 02 Mar 2009 16:53:55 +0100 name changes
Wed, 11 Feb 2009 10:51:07 +0100 Moved Order_Relation into Library and moved some of it into Relation.
Wed, 21 Jan 2009 23:40:23 +0100 changed import hierarchy
Tue, 26 Aug 2008 18:59:52 +0200 added distributivity of relation composition over union [simp]
Mon, 17 Mar 2008 16:47:24 +0100 added lemmas
Fri, 14 Mar 2008 19:57:12 +0100 Added lemmas
Mon, 08 Oct 2007 22:03:25 +0200 integrated FixedPoint into Inductive
Wed, 15 Aug 2007 12:52:56 +0200 ATP blacklisting is now in theory data, attribute noatp
Tue, 10 Jul 2007 17:30:50 +0200 moved lfp_induct2 here
Fri, 01 Jun 2007 15:12:56 +0200 Added simp-rules: "R O {} = {}" and "{} O R = {}"
Wed, 24 Jan 2007 17:10:50 +0100 some new lemmas
Fri, 17 Nov 2006 02:20:03 +0100 more robust syntax for definition/abbreviation/notation;
Tue, 07 Nov 2006 11:47:57 +0100 renamed 'const_syntax' to 'notation';
Tue, 26 Sep 2006 17:33:04 +0200 Changed precedence of "op O" (relation composition) from 60 to 75.
Tue, 16 May 2006 21:33:01 +0200 tuned concrete syntax -- abbreviation/const_syntax;
Sat, 08 Apr 2006 22:51:06 +0200 refined 'abbreviation';
Thu, 23 Mar 2006 20:03:53 +0100 Converted translations to abbbreviations.
Fri, 10 Mar 2006 00:53:28 +0100 added many simple lemmas
Thu, 22 Sep 2005 23:56:15 +0200 renamed rules to iprover
Fri, 03 Sep 2004 10:27:05 +0200 new theorem symD
Wed, 18 Aug 2004 11:09:40 +0200 import -> imports
Mon, 16 Aug 2004 14:22:27 +0200 New theory header syntax.