src/HOL/Multivariate_Analysis/Topology_Euclidean_Space.thy
Wed, 17 Aug 2011 11:07:32 -0700 huffman Topology_Euclidean_Space.thy: simplify some proofs
Wed, 17 Aug 2011 09:59:10 -0700 huffman simplify proofs of lemmas open_interval, closed_interval
Tue, 16 Aug 2011 09:31:23 -0700 huffman add simp rules for isCont
Mon, 15 Aug 2011 18:35:36 -0700 huffman generalize lemmas open_Collect_less, closed_Collect_le, closed_Collect_eq to class topological_space
Mon, 15 Aug 2011 15:11:55 -0700 huffman generalized lemma closed_Collect_eq
Mon, 15 Aug 2011 14:09:39 -0700 huffman add lemmas open_Collect_less, closed_Collect_le, closed_Collect_eq;
Mon, 15 Aug 2011 12:18:34 -0700 huffman generalize lemma continuous_uniform_limit to class metric_space
Mon, 15 Aug 2011 12:13:46 -0700 huffman remove duplicate lemmas eventually_conjI, eventually_and, eventually_false
Mon, 15 Aug 2011 10:49:48 -0700 huffman Topology_Euclidean_Space.thy: organize section headings
Sun, 14 Aug 2011 11:44:12 -0700 huffman locale-ize some definitions, so perfect_space and heine_borel can inherit from the proper superclasses
Fri, 12 Aug 2011 09:17:24 -0700 huffman make Multivariate_Analysis work with separate set type
Thu, 11 Aug 2011 14:24:05 -0700 huffman avoid duplicate rule warnings
Wed, 10 Aug 2011 15:56:48 -0700 huffman remove redundant lemma
Wed, 10 Aug 2011 14:25:56 -0700 huffman simplify proof of lemma bounded_component
Wed, 10 Aug 2011 09:23:42 -0700 huffman split Linear_Algebra.thy from Euclidean_Space.thy
Wed, 10 Aug 2011 01:36:53 -0700 huffman declare tendsto_const [intro] (accidentally removed in 230a8665c919)
Wed, 10 Aug 2011 00:29:31 -0700 huffman simplified definition of class euclidean_space;
Tue, 09 Aug 2011 13:09:35 -0700 huffman bounded_linear interpretation for euclidean_component
Tue, 09 Aug 2011 10:30:00 -0700 huffman mark some redundant theorems as legacy
Mon, 08 Aug 2011 21:17:52 -0700 huffman instance real_basis_with_inner < perfect_space
Mon, 08 Aug 2011 19:26:53 -0700 huffman rename type 'a net to 'a filter, following standard mathematical terminology
Mon, 08 Aug 2011 15:27:24 -0700 huffman generalize sequence lemmas
Mon, 08 Aug 2011 15:11:38 -0700 huffman generalize more lemmas about compactness
Mon, 08 Aug 2011 15:03:34 -0700 huffman generalize compactness equivalence lemmas
Mon, 08 Aug 2011 14:59:01 -0700 huffman lemma bolzano_weierstrass_imp_compact
Mon, 08 Aug 2011 14:44:20 -0700 huffman class perfect_space inherits from topological_space;
Thu, 09 Jun 2011 11:50:16 +0200 hoelzl lemmas about right derivative and limits
Wed, 30 Mar 2011 17:54:01 +0200 hoelzl real multiplication is continuous
Mon, 14 Mar 2011 14:37:35 +0100 hoelzl generalize infinite sums
Mon, 14 Mar 2011 14:37:33 +0100 hoelzl moved t2_spaces to HOL image
Mon, 28 Feb 2011 22:10:57 +0100 boehmes removed dependency on Dense_Linear_Order
Wed, 29 Dec 2010 17:34:41 +0100 wenzelm explicit file specifications -- avoid secondary load path;
Mon, 13 Sep 2010 11:13:15 +0200 nipkow 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 nipkow expand_fun_eq -> ext_iff
Fri, 27 Aug 2010 13:48:10 +0200 hoelzl preimages of open sets over continuous function are open
Mon, 23 Aug 2010 19:35:57 +0200 hoelzl Rewrite the Probability theory.
Mon, 23 Aug 2010 11:17:13 +0200 haftmann dropped type classes mult_mono and mult_mono1; tuned names of technical rule duplicates
Mon, 05 Jul 2010 09:14:51 -0700 huffman generalize type of is_interval to class euclidean_space
Fri, 02 Jul 2010 10:45:25 +0200 haftmann merged
Thu, 01 Jul 2010 16:54:44 +0200 haftmann "prod" and "sum" replace "*" and "+" respectively
Thu, 01 Jul 2010 09:24:04 -0700 huffman generalize more lemmas from ordered_euclidean_space to euclidean_space
Wed, 30 Jun 2010 21:13:46 -0700 huffman add lemma at_within_interior
Tue, 22 Jun 2010 18:15:44 +0200 hoelzl merged
Mon, 21 Jun 2010 19:33:51 +0200 hoelzl Introduce a type class for euclidean spaces, port most lemmas from real^'n to this type class.
Mon, 21 Jun 2010 18:32:16 +0200 blanchet beta-eta was too much, because it transformed SOME x. P x into Eps P, which caused problems later;
Thu, 17 Jun 2010 19:32:05 +0200 haftmann replaced unreliable metis proof
Sun, 09 May 2010 22:51:11 -0700 huffman avoid using real-specific versions of generic lemmas
Tue, 04 May 2010 19:53:57 -0700 huffman generalize some lemmas to class t1_space
Tue, 04 May 2010 19:23:59 -0700 huffman simplify definition of t1_space; generalize lemma closed_sing and related lemmas
Tue, 04 May 2010 18:55:18 -0700 huffman generalize some lemmas
Tue, 04 May 2010 10:06:05 -0700 huffman make (X ----> L) an abbreviation for (X ---> L) sequentially
Tue, 04 May 2010 09:56:34 -0700 huffman adapt to removed premise on tendsto lemma (cf. 88f0125c3bd2)
Mon, 03 May 2010 14:35:10 +0200 hoelzl Moved Convex theory to library.
Thu, 29 Apr 2010 11:41:04 -0700 huffman define linear algebra concepts using scaleR instead of (op *s); generalized many lemmas, though a few theorems that used to work on type int^'n are a bit less general
Thu, 29 Apr 2010 07:22:01 -0700 huffman remove redundant constants pastecart, fstcart, sndcart; users should prefer Pair, fst, snd instead
Wed, 28 Apr 2010 17:48:59 -0700 huffman prove lemma openin_subopen without using choice
Tue, 27 Apr 2010 10:54:24 -0700 huffman generalize more continuity lemmas
Tue, 27 Apr 2010 10:39:52 -0700 huffman generalized many lemmas about continuity
Mon, 26 Apr 2010 22:21:03 -0700 huffman simplify definition of continuous_on; generalize some lemmas
Mon, 26 Apr 2010 20:03:01 -0700 huffman move intervals section heading
less more (0) -60 tip