src/HOL/Set.thy
Mon, 09 Nov 2009 15:50:15 +0000 paulson New theory Probability/Borel.thy, and some associated lemmas
Wed, 21 Oct 2009 11:19:11 +0100 paulson merged
Tue, 20 Oct 2009 16:32:51 +0100 paulson Some new lemmas concerning sets
Wed, 21 Oct 2009 08:16:25 +0200 haftmann merged
Wed, 21 Oct 2009 08:14:38 +0200 haftmann dropped redundant gen_ prefix
Tue, 20 Oct 2009 16:13:01 +0200 haftmann replaced old_style infixes eq_set, subset, union, inter and variants by generic versions
Tue, 20 Oct 2009 15:02:48 +0100 paulson Removal of the unused atpset concept, the atp attribute and some related code.
Wed, 07 Oct 2009 14:01:26 +0200 haftmann tuned proofs
Sat, 19 Sep 2009 07:38:03 +0200 haftmann inter and union are mere abbreviations for inf and sup
Mon, 31 Aug 2009 14:09:42 +0200 nipkow tuned the simp rules for Int involving insert and intervals.
Tue, 28 Jul 2009 13:37:09 +0200 haftmann Set.UNIV and Set.empty are mere abbreviations for top and bot
Wed, 22 Jul 2009 18:02:10 +0200 haftmann moved complete_lattice &c. into separate theory
Wed, 22 Jul 2009 14:20:32 +0200 haftmann set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
Tue, 21 Jul 2009 14:38:07 +0200 haftmann attempt for more concise setup of non-etacontracting binders
Tue, 21 Jul 2009 11:09:50 +0200 haftmann Set.thy: prefer = over == where possible; tuned ML setup; dropped (moved) ML legacy
Tue, 21 Jul 2009 07:54:44 +0200 haftmann swapped bootstrap order of UNION/Union and INTER/Inter in theory Set
Mon, 20 Jul 2009 15:24:15 +0200 haftmann less digestible
Mon, 20 Jul 2009 11:47:17 +0200 haftmann refined outline structure
Mon, 20 Jul 2009 09:52:09 +0200 haftmann merged
Mon, 20 Jul 2009 08:31:12 +0200 haftmann closer relation of sets and complete lattices; corresponding consts, defs and syntax at similar places in theory text
Mon, 20 Jul 2009 08:32:07 +0200 haftmann merged
Tue, 14 Jul 2009 15:54:19 +0200 haftmann refinement of lattice classes
Wed, 15 Jul 2009 23:48:21 +0200 wenzelm more antiquotations;
Sat, 11 Jul 2009 21:33:01 +0200 haftmann added boolean_algebra type class; tuned lattice duals
Mon, 06 Jul 2009 21:24:30 +0200 wenzelm structure Thm: less pervasive names;
Mon, 15 Jun 2009 16:13:19 +0200 haftmann authentic syntax for Pow and image
Fri, 05 Jun 2009 08:06:03 +0200 haftmann merged
Thu, 04 Jun 2009 15:28:59 +0200 haftmann insert now qualified and with authentic syntax
Thu, 04 Jun 2009 19:44:06 +0200 nipkow finite lemmas
Mon, 18 May 2009 23:15:38 +0200 nipkow fine-tuned elimination of comprehensions involving x=t.
Sat, 16 May 2009 11:28:02 +0200 nipkow "{x. P x & x=t & Q x}" is now rewritten to "if P t & Q t then {t} else {}"
Tue, 31 Mar 2009 13:23:39 +0200 wenzelm tuned;
Thu, 19 Mar 2009 14:08:41 +0100 haftmann tuned some theorem and attribute bindings
Sat, 14 Mar 2009 12:50:29 +0100 haftmann reverted to old version of Set.thy -- strange effects have to be traced first
Sat, 07 Mar 2009 15:20:32 +0100 haftmann restructured theory Set.thy
Thu, 05 Mar 2009 08:23:11 +0100 haftmann set operations Int, Un, INTER, UNION, Inter, Union, empty, UNIV are now proper qualified constants with authentic syntax
Fri, 13 Feb 2009 23:55:04 +0100 nipkow finiteness lemmas
Thu, 29 Jan 2009 22:28:03 +0100 berghofe Added strong congruence rule for UN.
Fri, 10 Oct 2008 06:45:53 +0200 haftmann `code func` now just `code`
Mon, 11 Aug 2008 14:50:00 +0200 haftmann rudimentary code setup for set operations
Tue, 01 Jul 2008 06:51:59 +0200 huffman remove simp attribute from range_composition
Tue, 10 Jun 2008 15:30:56 +0200 haftmann removed some dubious code lemmas
Wed, 07 May 2008 10:56:43 +0200 berghofe - Now uses Orderings as parent theory
Tue, 22 Apr 2008 08:33:16 +0200 haftmann constant HOL.eq now qualified
Wed, 02 Apr 2008 15:58:32 +0200 haftmann explicit class "eq" for operational equality
Sat, 29 Mar 2008 19:14:00 +0100 wenzelm replaced 'ML_setup' by 'ML';
Wed, 19 Mar 2008 22:47:35 +0100 wenzelm eliminated change_claset/simpset;
Tue, 26 Feb 2008 20:38:15 +0100 haftmann moved some set lemmas from Set.thy here
Fri, 25 Jan 2008 14:54:41 +0100 haftmann improved code theorem setup
Wed, 02 Jan 2008 15:14:02 +0100 haftmann splitted class uminus from class minus
Fri, 30 Nov 2007 20:13:03 +0100 haftmann adjustions to due to instance target
Thu, 29 Nov 2007 17:08:26 +0100 haftmann instance command as rudimentary class target
Fri, 23 Nov 2007 21:09:33 +0100 haftmann interpretation of typedecls: instantiation to class type
Fri, 09 Nov 2007 13:41:27 +0100 krauss avoid name clashes when generating code for union, inter
Mon, 05 Nov 2007 18:18:39 +0100 nipkow added lemmas
Wed, 26 Sep 2007 20:27:58 +0200 haftmann convenient obtain rule for sets
Thu, 20 Sep 2007 16:37:30 +0200 haftmann clarified code lemmas
Fri, 24 Aug 2007 14:14:16 +0200 haftmann made sets executable
Sun, 19 Aug 2007 21:21:37 +0200 nipkow Made UN_Un simp
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
Wed, 15 Aug 2007 08:57:39 +0200 haftmann updated code generator setup
Fri, 20 Jul 2007 14:27:56 +0200 haftmann simplified HOL bootstrap
Thu, 19 Jul 2007 21:47:44 +0200 haftmann code lemma for contents
Sun, 06 May 2007 21:50:17 +0200 haftmann changed code generator invocation syntax
Fri, 20 Apr 2007 11:21:42 +0200 haftmann Isar definitions are now added explicitly to code theorem table
Tue, 20 Mar 2007 08:27:23 +0100 haftmann fixed typo
Fri, 16 Mar 2007 21:32:11 +0100 haftmann added instance of sets as distributive lattices
Mon, 12 Mar 2007 19:23:49 +0100 wenzelm syntax: proper body priorty for derived binders;
Wed, 28 Feb 2007 22:05:43 +0100 wenzelm tuned ML setup;
Wed, 24 Jan 2007 17:10:50 +0100 paulson some new lemmas
Sat, 20 Jan 2007 14:09:27 +0100 wenzelm tuned ML setup;
Wed, 13 Dec 2006 20:38:17 +0100 haftmann dropped FIXME comment
Wed, 13 Dec 2006 15:45:30 +0100 haftmann fixed syntax for bounded quantification
Wed, 06 Dec 2006 01:12:36 +0100 wenzelm removed legacy ML bindings;
Mon, 27 Nov 2006 13:42:42 +0100 haftmann restructured some proofs
Sun, 26 Nov 2006 18:07:16 +0100 wenzelm updated (binder) syntax/notation;
Fri, 17 Nov 2006 02:20:03 +0100 wenzelm more robust syntax for definition/abbreviation/notation;
Wed, 15 Nov 2006 17:05:43 +0100 haftmann moved transitivity rules to Orderings.thy
Mon, 13 Nov 2006 15:43:11 +0100 haftmann dropped LOrder dependency
Sun, 12 Nov 2006 21:31:52 +0100 nipkow image_constant_conv no longer [simp]
Sun, 12 Nov 2006 19:22:10 +0100 nipkow started reorgnization of lattice theories
Tue, 07 Nov 2006 11:47:57 +0100 wenzelm renamed 'const_syntax' to 'notation';
Mon, 14 Aug 2006 13:46:06 +0200 haftmann simplified code generator setup
Wed, 26 Jul 2006 19:23:04 +0200 webertj linear arithmetic splits certain operators (e.g. min, max, abs)
Tue, 13 Jun 2006 15:07:58 +0200 paulson new results
Tue, 16 May 2006 21:33:01 +0200 wenzelm tuned concrete syntax -- abbreviation/const_syntax;
Sat, 13 May 2006 21:13:25 +0200 wenzelm reactivated translations for less/less_eq;
Sat, 08 Apr 2006 22:51:06 +0200 wenzelm refined 'abbreviation';
Thu, 23 Mar 2006 20:03:53 +0100 nipkow Converted translations to abbbreviations.
Mon, 20 Mar 2006 17:38:22 +0100 paulson subsetI is often necessary
Fri, 17 Mar 2006 09:34:23 +0100 haftmann renamed op < <= to Orderings.less(_eq)
Fri, 10 Mar 2006 15:33:48 +0100 haftmann renamed HOL + - * etc. to HOL.plus HOL.minus HOL.times etc.
Thu, 02 Mar 2006 18:50:43 +0100 paulson subset_refl now included using the atp attribute
Mon, 30 Jan 2006 08:20:56 +0100 haftmann adaptions to codegen_package
Sun, 29 Jan 2006 19:23:38 +0100 wenzelm declare 'defn' rules;
Fri, 13 Jan 2006 14:43:09 +0100 nipkow *** empty log message ***
Wed, 21 Dec 2005 12:02:57 +0100 paulson removed or modified some instances of [iff]
Fri, 16 Dec 2005 16:59:32 +0100 nipkow new lemmas
Thu, 15 Dec 2005 19:42:00 +0100 wenzelm removed obsolete/unused setup_induction;
Thu, 01 Dec 2005 22:04:27 +0100 wenzelm simprocs: static evaluation of simpset;
Thu, 01 Dec 2005 15:45:54 +0100 paulson restoring the old status of subset_refl
Thu, 10 Nov 2005 17:33:14 +0100 paulson duplicate axioms in ATP linkup, and general fixes
Mon, 17 Oct 2005 23:10:10 +0200 wenzelm change_claset/simpset;
Fri, 07 Oct 2005 22:59:22 +0200 wenzelm Term.absdummy;
Thu, 29 Sep 2005 12:43:40 +0200 paulson a name for empty_not_insert
Thu, 29 Sep 2005 00:58:55 +0200 wenzelm more finalconsts;
Thu, 22 Sep 2005 23:56:15 +0200 nipkow renamed rules to iprover
Tue, 20 Sep 2005 14:03:37 +0200 wenzelm tuned theory dependencies;
Tue, 16 Aug 2005 18:53:11 +0200 paulson more simprules now have names
Tue, 16 Aug 2005 15:36:28 +0200 paulson classical rules must have names for ATP integration
Tue, 02 Aug 2005 19:47:12 +0200 wenzelm simprocs: Simplifier.inherit_bounds;
Tue, 12 Jul 2005 12:49:00 +0200 paulson tweaked
Fri, 01 Jul 2005 13:57:53 +0200 berghofe Added strong_ball_cong and strong_bex_cong (these are now the standard
Wed, 11 May 2005 09:50:33 +0200 nipkow Added thms by Brian Huffmann
Tue, 01 Mar 2005 18:48:52 +0100 nipkow integrated Jeremy's FiniteLib
Fri, 18 Feb 2005 11:48:42 +0100 nipkow tuning
Thu, 10 Feb 2005 18:51:12 +0100 nipkow Moved oderings from HOL into the new Orderings.thy
Mon, 27 Sep 2004 10:27:34 +0200 ballarin Modified locales: improved implementation of "includes".
Wed, 18 Aug 2004 11:09:40 +0200 nipkow import -> imports
less more (0) -120 tip