Sun, 02 Nov 2014 17:09:04 +0100 |
wenzelm |
modernized header;
|
file |
diff |
annotate
|
Tue, 05 Aug 2014 16:58:19 +0200 |
wenzelm |
tuned proofs -- fewer warnings;
|
file |
diff |
annotate
|
Sat, 05 Jul 2014 11:01:53 +0200 |
haftmann |
prefer ac_simps collections over separate name bindings for add and mult
|
file |
diff |
annotate
|
Fri, 04 Jul 2014 20:18:47 +0200 |
haftmann |
reduced name variants for assoc and commute on plus and mult
|
file |
diff |
annotate
|
Sat, 28 Jun 2014 09:16:42 +0200 |
haftmann |
fact consolidation
|
file |
diff |
annotate
|
Tue, 25 Mar 2014 14:20:58 +0100 |
hoelzl |
cleanup auxiliary proofs for Brouwer fixpoint theorem (removes ~2400 lines)
|
file |
diff |
annotate
|
Tue, 18 Mar 2014 09:39:07 -0700 |
huffman |
remove unnecessary finiteness assumptions from lemmas about setsum
|
file |
diff |
annotate
|
Tue, 18 Mar 2014 15:53:48 +0100 |
hoelzl |
cleanup Series: sorted according to typeclass hierarchy, use {..<_} instead of {0..<_}
|
file |
diff |
annotate
|
Tue, 18 Mar 2014 10:12:58 +0100 |
immler |
removed dependencies on theory Ordered_Euclidean_Space
|
file |
diff |
annotate
|
Tue, 18 Mar 2014 10:12:57 +0100 |
immler |
use cbox to relax class constraints
|
file |
diff |
annotate
|
Sun, 16 Feb 2014 21:09:47 +0100 |
wenzelm |
tuned proofs;
|
file |
diff |
annotate
|
Mon, 16 Dec 2013 17:08:22 +0100 |
immler |
ordered_euclidean_space compatible with more standard pointwise ordering on products; conditionally complete lattice with product order
|
file |
diff |
annotate
|
Mon, 16 Dec 2013 17:08:22 +0100 |
immler |
prefer box over greaterThanLessThan on euclidean_space
|
file |
diff |
annotate
|
Tue, 19 Nov 2013 10:05:53 +0100 |
haftmann |
eliminiated neg_numeral in favour of - (numeral _)
|
file |
diff |
annotate
|
Fri, 01 Nov 2013 18:51:14 +0100 |
haftmann |
more simplification rules on unary and binary minus
|
file |
diff |
annotate
|
Thu, 12 Sep 2013 18:09:17 -0700 |
huffman |
make 'linear' into a sublocale of 'bounded_linear';
|
file |
diff |
annotate
|
Thu, 12 Sep 2013 09:06:46 -0700 |
huffman |
prefer theorem name over 'long_thm_list(n)'
|
file |
diff |
annotate
|
Thu, 12 Sep 2013 09:03:52 -0700 |
huffman |
removed outdated comments
|
file |
diff |
annotate
|
Thu, 18 Apr 2013 17:07:01 +0200 |
wenzelm |
simplifier uses proper Proof.context instead of historic type simpset;
|
file |
diff |
annotate
|
Tue, 09 Apr 2013 14:04:41 +0200 |
hoelzl |
remove the within-filter, replace "at" by "at _ within UNIV" (This allows to remove a couple of redundant lemmas)
|
file |
diff |
annotate
|
Sat, 23 Mar 2013 20:50:39 +0100 |
haftmann |
fundamental revision of big operators on sets
|
file |
diff |
annotate
|
Thu, 31 Jan 2013 11:31:22 +0100 |
hoelzl |
simplify heine_borel type class
|
file |
diff |
annotate
|
Fri, 14 Dec 2012 15:46:01 +0100 |
hoelzl |
Remove the indexed basis from the definition of euclidean spaces and only use the set of Basis vectors
|
file |
diff |
annotate
|
Fri, 19 Oct 2012 15:12:52 +0200 |
webertj |
Renamed {left,right}_distrib to distrib_{right,left}.
|
file |
diff |
annotate
|
Fri, 28 Sep 2012 15:05:16 +0200 |
wenzelm |
tuned proofs;
|
file |
diff |
annotate
|
Fri, 07 Sep 2012 15:15:07 +0200 |
wenzelm |
tuned proofs;
|
file |
diff |
annotate
|
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
|