| Sun, 25 Mar 2012 20:15:39 +0200 | 
huffman | 
merged fork with new numeral representation (see NEWS)
 | 
file |
diff |
annotate
 | 
| Tue, 20 Sep 2011 10:52:08 -0700 | 
huffman | 
add lemmas within_empty and tendsto_bot;
 | 
file |
diff |
annotate
 | 
| Mon, 12 Sep 2011 11:54:20 -0700 | 
huffman | 
remove redundant lemma Lim_sequentially in favor of lemma LIMSEQ_def
 | 
file |
diff |
annotate
 | 
| Thu, 01 Sep 2011 09:02:14 -0700 | 
huffman | 
modernize lemmas about 'continuous' and 'continuous_on';
 | 
file |
diff |
annotate
 | 
| Sun, 28 Aug 2011 20:56:49 -0700 | 
huffman | 
move class perfect_space into RealVector.thy;
 | 
file |
diff |
annotate
 | 
| Thu, 25 Aug 2011 12:43:55 -0700 | 
huffman | 
rename subset_{interior,closure} to {interior,closure}_mono;
 | 
file |
diff |
annotate
 | 
| Thu, 25 Aug 2011 11:57:42 -0700 | 
huffman | 
simplify many proofs about subspace and span;
 | 
file |
diff |
annotate
 | 
| Tue, 23 Aug 2011 14:11:02 -0700 | 
huffman | 
declare euclidean_simps [simp] at the point they are proved;
 | 
file |
diff |
annotate
 | 
| Mon, 22 Aug 2011 10:43:10 -0700 | 
huffman | 
legacy theorem names
 | 
file |
diff |
annotate
 | 
| Sun, 21 Aug 2011 09:46:20 -0700 | 
huffman | 
section -> subsection
 | 
file |
diff |
annotate
 | 
| Thu, 18 Aug 2011 13:36:58 -0700 | 
huffman | 
remove bounded_(bi)linear locale interpretations, to avoid duplicating so many lemmas
 | 
file |
diff |
annotate
 | 
| Tue, 16 Aug 2011 09:31:23 -0700 | 
huffman | 
add simp rules for isCont
 | 
file |
diff |
annotate
 | 
| Mon, 15 Aug 2011 18:35:36 -0700 | 
huffman | 
generalize lemmas open_Collect_less, closed_Collect_le, closed_Collect_eq to class topological_space
 | 
file |
diff |
annotate
 | 
| Mon, 15 Aug 2011 14:09:39 -0700 | 
huffman | 
add lemmas open_Collect_less, closed_Collect_le, closed_Collect_eq;
 | 
file |
diff |
annotate
 | 
| Mon, 15 Aug 2011 12:13:46 -0700 | 
huffman | 
remove duplicate lemmas eventually_conjI, eventually_and, eventually_false
 | 
file |
diff |
annotate
 | 
| Fri, 12 Aug 2011 09:17:24 -0700 | 
huffman | 
make Multivariate_Analysis work with separate set type
 | 
file |
diff |
annotate
 | 
| Thu, 11 Aug 2011 14:24:05 -0700 | 
huffman | 
avoid duplicate rule warnings
 | 
file |
diff |
annotate
 | 
| Thu, 11 Aug 2011 13:05:56 -0700 | 
huffman | 
modify euclidean_space class to include basis set
 | 
file |
diff |
annotate
 | 
| Thu, 11 Aug 2011 09:11:15 -0700 | 
huffman | 
remove lemma stupid_ext
 | 
file |
diff |
annotate
 | 
| Wed, 10 Aug 2011 16:35:50 -0700 | 
huffman | 
remove several redundant and unused theorems about derivatives
 | 
file |
diff |
annotate
 | 
| Wed, 10 Aug 2011 13:13:37 -0700 | 
huffman | 
more uniform naming scheme for finite cartesian product type and related theorems
 | 
file |
diff |
annotate
 | 
| Wed, 10 Aug 2011 10:13:16 -0700 | 
huffman | 
move euclidean_space instance from Cartesian_Euclidean_Space.thy to Finite_Cartesian_Product.thy
 | 
file |
diff |
annotate
 | 
| Wed, 10 Aug 2011 00:29:31 -0700 | 
huffman | 
simplified definition of class euclidean_space;
 | 
file |
diff |
annotate
 | 
| Mon, 08 Aug 2011 16:04:58 -0700 | 
huffman | 
fix perfect_space instance proof for finite cartesian product (cf. 5b970711fb39)
 | 
file |
diff |
annotate
 | 
| Thu, 28 Jul 2011 10:42:24 +0200 | 
hoelzl | 
simplified definition of vector (also removed Cartesian_Euclidean_Space.from_nat which collides with Countable.from_nat)
 | 
file |
diff |
annotate
 | 
| Sun, 15 May 2011 17:45:53 +0200 | 
wenzelm | 
simplified/unified method_setup/attribute_setup;
 | 
file |
diff |
annotate
 | 
| Sun, 28 Nov 2010 15:20:51 +0100 | 
nipkow | 
gave more standard finite set rules simp and intro attribute
 | 
file |
diff |
annotate
 | 
| 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
 | 
file |
diff |
annotate
 | 
| Tue, 07 Sep 2010 10:05:19 +0200 | 
nipkow | 
expand_fun_eq -> ext_iff
 | 
file |
diff |
annotate
 | 
| Mon, 23 Aug 2010 19:35:57 +0200 | 
hoelzl | 
Rewrite the Probability theory.
 | 
file |
diff |
annotate
 | 
| Fri, 20 Aug 2010 17:46:56 +0200 | 
haftmann | 
more concise characterization of of_nat operation and class semiring_char_0
 | 
file |
diff |
annotate
 | 
| Thu, 01 Jul 2010 16:54:44 +0200 | 
haftmann | 
"prod" and "sum" replace "*" and "+" respectively
 | 
file |
diff |
annotate
 | 
| Thu, 01 Jul 2010 11:48:42 +0200 | 
hoelzl | 
Add theory for indicator function.
 | 
file |
diff |
annotate
 | 
| Thu, 01 Jul 2010 09:01:09 +0200 | 
hoelzl | 
Instantiate product type as euclidean space.
 | 
file |
diff |
annotate
 | 
| Wed, 23 Jun 2010 10:05:13 +0200 | 
hoelzl | 
Make latex happy
 | 
file |
diff |
annotate
 | 
| 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.
 | 
file |
diff |
annotate
 |