src/HOL/Multivariate_Analysis/Euclidean_Space.thy
Tue, 23 Aug 2011 14:11:02 -0700 huffman declare euclidean_simps [simp] at the point they are proved;
Thu, 18 Aug 2011 17:32:02 -0700 huffman declare euclidean_component_zero[simp] at the point it is proved
Thu, 18 Aug 2011 13:36:58 -0700 huffman remove bounded_(bi)linear locale interpretations, to avoid duplicating so many lemmas
Tue, 16 Aug 2011 09:31:23 -0700 huffman add simp rules for isCont
Mon, 15 Aug 2011 14:50:24 -0700 huffman remove duplicate lemma disjoint_iff
Thu, 11 Aug 2011 13:05:56 -0700 huffman modify euclidean_space class to include basis set
Wed, 10 Aug 2011 09:23:42 -0700 huffman split Linear_Algebra.thy from Euclidean_Space.thy
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
Sun, 24 Jul 2011 22:38:13 +0200 haftmann adjusted to tailored version of bex_simps
Sun, 15 May 2011 17:45:53 +0200 wenzelm simplified/unified method_setup/attribute_setup;
Mon, 14 Mar 2011 14:37:33 +0100 hoelzl moved t2_spaces to HOL image
Sun, 13 Mar 2011 22:55:50 +0100 wenzelm tuned headers;
Thu, 03 Mar 2011 21:43:06 +0100 wenzelm tuned proofs -- eliminated prems;
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;
Sun, 28 Nov 2010 15:20:51 +0100 nipkow gave more standard finite set rules simp and intro attribute
Mon, 22 Nov 2010 10:34:33 +0100 hoelzl Replace surj by abbreviation; remove surj_on.
Fri, 05 Nov 2010 14:17:18 +0100 hoelzl Extend convex analysis by Bogdan Grechuk
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
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
Tue, 03 Aug 2010 16:48:36 +0200 wenzelm tuned headers -- more precise load path;
Mon, 19 Jul 2010 16:09:44 +0200 haftmann diff_minus subsumes diff_def
Wed, 07 Jul 2010 09:26:54 +0200 hoelzl tuned
Mon, 05 Jul 2010 09:12:35 -0700 huffman section -> subsection
Thu, 01 Jul 2010 09:01:09 +0200 hoelzl Instantiate product type as euclidean space.
Wed, 30 Jun 2010 11:51:35 -0700 huffman minimize dependencies on Numeral_Type
Wed, 30 Jun 2010 10:42:38 -0700 huffman change type of 'dimension' to 'a itself => nat
Wed, 30 Jun 2010 10:26:02 -0700 huffman generalize some euclidean_space lemmas
Mon, 28 Jun 2010 15:32:26 +0200 haftmann inner_simps is not enough, need also local facts
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.
Sun, 09 May 2010 22:51:11 -0700 huffman avoid using real-specific versions of generic lemmas
Tue, 04 May 2010 17:37:31 -0700 huffman convert comments to 'text' blocks
Mon, 03 May 2010 14:35:10 +0200 hoelzl Moved Convex theory to library.
Thu, 29 Apr 2010 15:24:22 -0700 huffman generalize lemma adjoint_unique; simplify some proofs
Thu, 29 Apr 2010 14:32:24 -0700 huffman fix latex url
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 09:29:47 -0700 huffman remove unused function vector_power, unused lemma one_plus_of_nat_neq_0
Thu, 29 Apr 2010 09:17:25 -0700 huffman move class instantiations from Euclidean_Space.thy to Finite_Cartesian_Product.thy
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 23:08:31 -0700 huffman generalize LIMSEQ_vector to tendsto_vector
Wed, 28 Apr 2010 22:36:45 -0700 huffman generalize orthogonal_clauses
Wed, 28 Apr 2010 22:20:59 -0700 huffman remove redundant lemma vector_dist_norm
Wed, 28 Apr 2010 22:02:55 -0700 huffman remove redundant lemma norm_0
Wed, 28 Apr 2010 21:39:14 -0700 huffman generalize some euclidean space lemmas
Wed, 28 Apr 2010 15:05:45 -0700 huffman move operator norm stuff to new theory file
Mon, 26 Apr 2010 17:56:39 -0700 huffman remove redundant lemma
Mon, 26 Apr 2010 12:19:57 -0700 huffman move definitions and theorems for type real^1 to separate theory file
Mon, 26 Apr 2010 09:45:22 -0700 huffman merged
Mon, 26 Apr 2010 09:21:25 -0700 huffman fix lots of looping simp calls and other warnings
Mon, 26 Apr 2010 11:34:19 +0200 haftmann dropped group_simps, ring_simps, field_eq_simps
Sat, 24 Apr 2010 14:06:19 -0700 huffman minimize imports
Sat, 24 Apr 2010 13:31:52 -0700 huffman document generation for Multivariate_Analysis
Sat, 24 Apr 2010 11:11:09 -0700 huffman move l2-norm stuff into separate theory file
Fri, 23 Apr 2010 16:17:25 +0200 haftmann epheremal replacement of field_simps by field_eq_simps
Tue, 02 Mar 2010 21:32:37 +0100 himmelma replaced \<bullet> with inner
Tue, 02 Mar 2010 11:07:17 +0100 himmelma tuned
Tue, 02 Mar 2010 09:57:49 +0100 himmelma the ordering on real^1 is linear
less more (0) -60 tip