src/HOL/Multivariate_Analysis/Topology_Euclidean_Space.thy
Wed, 26 Mar 2014 11:05:25 -0700 huffman tuned proofs
Tue, 18 Mar 2014 10:12:58 +0100 immler removed dependencies on theory Ordered_Euclidean_Space
Tue, 18 Mar 2014 10:12:57 +0100 immler use cbox to relax class constraints
Sun, 16 Mar 2014 18:09:04 +0100 haftmann normalising simp rules for compound operators
Sat, 15 Mar 2014 08:31:33 +0100 haftmann more complete set of lemmas wrt. image and composition
Thu, 13 Mar 2014 07:07:07 +0100 nipkow enhanced simplifier solver for preconditions of rewrite rule, can now deal with conjunctions
Wed, 05 Mar 2014 13:59:25 -0800 huffman generalize lemmas
Thu, 27 Feb 2014 16:07:21 +0000 paulson A bit of tidying up
Sun, 16 Feb 2014 21:09:47 +0100 wenzelm tuned proofs;
Wed, 12 Feb 2014 08:35:57 +0100 blanchet renamed 'nat_{case,rec}' to '{case,rec}_nat'
Wed, 25 Dec 2013 17:39:06 +0100 haftmann prefer more canonical names for lemmas on min/max
Wed, 18 Dec 2013 11:53:40 +0100 hoelzl modernized ContNotDenum: use Set_Interval, and finite intersection property to show the nested interval property
Mon, 16 Dec 2013 17:08:22 +0100 immler summarized notions related to ordered_euclidean_space and intervals in separate theory
Mon, 16 Dec 2013 17:08:22 +0100 immler prefer box over greaterThanLessThan on euclidean_space
Tue, 19 Nov 2013 10:05:53 +0100 haftmann eliminiated neg_numeral in favour of - (numeral _)
Tue, 05 Nov 2013 09:45:02 +0100 hoelzl move Lubs from HOL to HOL-Library (replaced by conditionally complete lattices)
Tue, 05 Nov 2013 09:44:59 +0100 hoelzl use INF and SUP on conditionally complete lattices in multivariate analysis
Tue, 05 Nov 2013 09:44:59 +0100 hoelzl add SUP and INF for conditionally complete lattices
Tue, 05 Nov 2013 09:44:58 +0100 hoelzl use bdd_above and bdd_below for conditionally complete lattices
Fri, 01 Nov 2013 18:51:14 +0100 haftmann more simplification rules on unary and binary minus
Mon, 07 Oct 2013 08:39:50 -0700 huffman new topological lemmas; tuned proofs
Tue, 24 Sep 2013 15:03:51 -0700 huffman generalize lemma
Tue, 24 Sep 2013 15:03:50 -0700 huffman removed unused lemma
Tue, 24 Sep 2013 15:03:49 -0700 huffman factor out new lemma
Tue, 24 Sep 2013 15:03:49 -0700 huffman replace lemma with more general simp rule
Mon, 23 Sep 2013 16:56:17 -0700 huffman tuned proofs
Sat, 14 Sep 2013 23:52:36 +0200 wenzelm tuned proofs;
Thu, 12 Sep 2013 09:39:02 -0700 huffman remove duplicate lemmas
Tue, 03 Sep 2013 01:12:40 +0200 wenzelm tuned proofs -- clarified flow of facts wrt. calculation;
Thu, 29 Aug 2013 20:46:55 +0200 wenzelm tuned proofs;
Thu, 29 Aug 2013 19:20:35 +0200 wenzelm tuned proofs;
Thu, 29 Aug 2013 00:18:02 +0200 wenzelm tuned proofs;
Tue, 13 Aug 2013 16:25:47 +0200 wenzelm standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
Fri, 12 Jul 2013 18:16:50 +0200 wenzelm tuned;
Fri, 12 Jul 2013 17:43:18 +0200 wenzelm tuned proofs;
Sat, 25 May 2013 15:44:29 +0200 haftmann weaker precendence of syntax for big intersection and union on sets
Wed, 24 Apr 2013 13:28:30 +0200 hoelzl spell conditional_ly_-complete lattices correct
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)
Tue, 26 Mar 2013 12:21:00 +0100 hoelzl rename eventually_at / _within, to distinguish them from the lemmas in the HOL image
Tue, 26 Mar 2013 12:20:52 +0100 hoelzl separate SupInf into Conditional_Complete_Lattice, move instantiation of real to RealDef
Fri, 22 Mar 2013 10:41:43 +0100 hoelzl move continuous_on_inv to HOL image (simplifies isCont_inverse_function)
Fri, 22 Mar 2013 10:41:43 +0100 hoelzl move connected to HOL image; used to show intermediate value theorem
Fri, 22 Mar 2013 10:41:43 +0100 hoelzl move compact to the HOL image; prove compactness of real closed intervals; show that continuous functions attain supremum and infimum on compact sets
Fri, 22 Mar 2013 10:41:43 +0100 hoelzl move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
Fri, 22 Mar 2013 10:41:43 +0100 hoelzl introduct the conditional_complete_lattice type class; generalize theorems about real Sup and Inf to it
Fri, 22 Mar 2013 10:41:43 +0100 hoelzl move first_countable_topology to the HOL image
Fri, 22 Mar 2013 10:41:43 +0100 hoelzl move metric_space to its own theory
Fri, 22 Mar 2013 10:41:42 +0100 hoelzl move topological_space to its own theory
Wed, 06 Mar 2013 16:56:21 +0100 hoelzl netlimit is abbreviation for Lim
Wed, 06 Mar 2013 16:56:21 +0100 hoelzl tuned proofs
Wed, 06 Mar 2013 16:56:21 +0100 hoelzl changed continuous_on_intros into a named theorems collection
Wed, 06 Mar 2013 16:56:21 +0100 hoelzl changed continuous_intros into a named theorems collection
Tue, 05 Mar 2013 15:43:22 +0100 hoelzl generalized lemmas in Extended_Real_Limits
Tue, 05 Mar 2013 15:43:21 +0100 hoelzl eventually nhds represented using sequentially
Tue, 05 Mar 2013 15:43:20 +0100 hoelzl generalized compact_Times to topological_space
Tue, 05 Mar 2013 15:43:19 +0100 hoelzl move lemma Inf to usage point
Tue, 05 Mar 2013 15:43:18 +0100 hoelzl tuned proof of Edelstein fixed point theorem (use continuity of dist and attains_sup)
Tue, 05 Mar 2013 15:43:17 +0100 hoelzl tuned proofs (used continuity of infdist, dist and continuous_attains_sup)
Tue, 05 Mar 2013 15:43:16 +0100 hoelzl generalized continuous/compact_attains_inf/sup from real to linorder_topology
Tue, 05 Mar 2013 15:43:15 +0100 hoelzl continuity of pair operations
less more (0) -100 -60 tip