src/HOL/Finite_Set.thy
Thu, 11 Dec 2008 18:30:26 +0100 ballarin Conversion of HOL-Main and ZF to new locales.
Tue, 09 Dec 2008 15:31:38 -0800 huffman move lemmas from Numeral_Type.thy to other theories
Wed, 19 Nov 2008 17:54:55 +0100 nipkow Added new fold operator and renamed the old oe to fold_image.
Mon, 17 Nov 2008 17:00:55 +0100 haftmann tuned unfold_locales invocation
Sun, 24 Aug 2008 14:42:22 +0200 haftmann tuned import order
Tue, 15 Jul 2008 16:50:09 +0200 ballarin Removed uses of context element includes.
Tue, 01 Jul 2008 20:26:48 +0200 huffman prove lemma finite in context of finite class
Tue, 01 Jul 2008 06:51:59 +0200 huffman remove simp attribute from range_composition
Thu, 12 Jun 2008 14:10:41 +0200 nipkow Hid swap
Wed, 07 May 2008 10:56:34 +0200 berghofe - Deleted code setup for finite and card
Mon, 28 Apr 2008 20:21:11 +0200 haftmann thms Max_ge, Min_le: dropped superfluous premise
Fri, 25 Apr 2008 15:30:33 +0200 krauss Merged theories about wellfoundedness into one: Wellfounded.thy
Fri, 28 Mar 2008 22:00:59 +0100 haftmann only invoke interpret
Thu, 27 Mar 2008 19:04:35 +0100 haftmann no "attach UNIV" any more
Tue, 26 Feb 2008 20:38:10 +0100 haftmann tuned proofs
Wed, 06 Feb 2008 08:34:32 +0100 haftmann locales ACf, ACIf, ACIfSL and ACIfSLlin have been abandoned in favour of the existing algebraic classes ab_semigroup_mult, ab_semigroup_idem_mult, lower_semilattice (resp. uper_semilattice) and linorder
Fri, 07 Dec 2007 15:07:59 +0100 haftmann instantiation target rather than legacy instance
Thu, 29 Nov 2007 17:08:26 +0100 haftmann instance command as rudimentary class target
Fri, 23 Nov 2007 21:09:32 +0100 haftmann deleted card definition as code lemma; authentic syntax for card
Tue, 06 Nov 2007 08:47:25 +0100 haftmann renamed lordered_*_* to lordered_*_add_*; further localization
Fri, 26 Oct 2007 21:22:16 +0200 haftmann dropped "brown" syntax
Tue, 23 Oct 2007 23:27:23 +0200 nipkow went back to >0
Tue, 16 Oct 2007 23:12:45 +0200 haftmann global class syntax
Mon, 15 Oct 2007 15:29:39 +0200 haftmann explicit parameter for class finite
Mon, 08 Oct 2007 08:04:26 +0200 haftmann clarified
Fri, 05 Oct 2007 08:38:09 +0200 nipkow added lemmas
Sat, 29 Sep 2007 08:58:51 +0200 haftmann proper syntax during class specification
Wed, 26 Sep 2007 20:27:55 +0200 haftmann moved Finite_Set before Datatype
Thu, 20 Sep 2007 16:37:28 +0200 haftmann code lemmas for cardinality
Sat, 15 Sep 2007 19:27:41 +0200 haftmann added lemmas for finiteness
Fri, 24 Aug 2007 14:21:33 +0200 paulson revised blacklisting for ATP linkup
Tue, 21 Aug 2007 13:30:36 +0200 haftmann moved ordered_ab_semigroup_add to OrderedGroup.thy
Mon, 20 Aug 2007 18:07:25 +0200 haftmann conciliated Inf/Inf_fin
Fri, 17 Aug 2007 13:58:57 +0200 haftmann dropped junk
Wed, 15 Aug 2007 12:52:56 +0200 paulson ATP blacklisting is now in theory data, attribute noatp
Tue, 14 Aug 2007 23:04:27 +0200 huffman minimize imports
Tue, 14 Aug 2007 23:03:42 +0200 huffman rename lemmas finite->finite_UNIV, finite_set->finite; declare finite[simp]
Thu, 09 Aug 2007 15:52:42 +0200 haftmann re-eliminated Option.thy
Tue, 07 Aug 2007 09:38:46 +0200 haftmann simplified proofs
Tue, 24 Jul 2007 15:20:47 +0200 haftmann using interpretation with derived concepts
Fri, 20 Jul 2007 14:27:56 +0200 haftmann simplified HOL bootstrap
Wed, 11 Jul 2007 11:00:46 +0200 berghofe Renamed inductive2 to inductive.
Tue, 10 Jul 2007 17:30:45 +0200 haftmann moved some finite lemmas here
Sat, 23 Jun 2007 19:33:22 +0200 nipkow tuned and renamed group_eq_simps and ring_eq_simps
Sun, 17 Jun 2007 18:47:03 +0200 nipkow tuned laws for cancellation in divisions for fields.
Fri, 15 Jun 2007 15:10:32 +0200 nipkow made divide_self a simp rule
Thu, 14 Jun 2007 18:33:31 +0200 wenzelm tuned proofs: avoid implicit prems;
Wed, 06 Jun 2007 17:01:33 +0200 huffman generalize class constraints on some lemmas
Mon, 04 Jun 2007 15:43:30 +0200 haftmann tuned comments
Thu, 24 May 2007 08:37:39 +0200 haftmann rudimentary class target implementation
Sat, 19 May 2007 11:33:22 +0200 haftmann no special treatment in naming of locale predicates stemming form classes
Fri, 11 May 2007 20:47:30 +0200 nipkow *** empty log message ***
Fri, 11 May 2007 03:31:12 +0200 huffman generalize setsum lemmas from semiring_0_cancel to semiring_0
Thu, 10 May 2007 10:21:46 +0200 haftmann localized Min/Max
Mon, 09 Apr 2007 21:28:24 +0200 huffman generalized type of lemma setsum_product
Tue, 20 Mar 2007 08:27:15 +0100 haftmann explizit "type" superclass
Fri, 16 Mar 2007 21:32:07 +0100 haftmann added FIXME hints
Fri, 09 Mar 2007 08:45:57 +0100 haftmann moved order on functions here
Sat, 03 Mar 2007 09:26:58 +0100 haftmann moved instance option :: finite here
Fri, 02 Mar 2007 15:43:19 +0100 haftmann added code theorems for UNIV
less more (0) -100 -60 tip