src/HOL/Real.thy
Wed, 09 Oct 2019 14:51:54 +0000 haftmann dedicated fact collections for algebraic simplification rules potentially splitting goals
Sat, 22 Jun 2019 07:18:55 +0000 haftmann streamlined setup for linear algebra, particularly removed redundant rule declarations
Wed, 15 May 2019 12:47:15 +0100 paulson Generalisations involving numerals; comparisons should now work for ennreal
Sun, 06 Jan 2019 15:04:34 +0100 wenzelm isabelle update -u path_cartouches;
Fri, 04 Jan 2019 23:22:53 +0100 wenzelm isabelle update -u control_cartouches;
Sun, 23 Dec 2018 20:51:23 +0000 haftmann more rules
Mon, 24 Sep 2018 14:30:09 +0200 nipkow Prefix form of infix with * on either side no longer needs special treatment
Sat, 21 Jul 2018 13:30:43 +0200 paulson de-applying and removing junk
Thu, 19 Jul 2018 17:27:44 +0200 paulson de-applying
Thu, 28 Jun 2018 17:14:52 +0200 nipkow added lemmas
Thu, 28 Jun 2018 14:13:57 +0100 paulson Generalising and renaming some basic results
Fri, 22 Jun 2018 20:31:49 +0200 wenzelm clarified document antiquotation @{theory};
Wed, 10 Jan 2018 15:25:09 +0100 nipkow ran isabelle update_op on all sources
Tue, 19 Dec 2017 13:58:12 +0100 wenzelm isabelle update_cartouches -c -t;
Sat, 11 Nov 2017 18:41:08 +0000 haftmann dedicated definition for coprimality
Tue, 24 Oct 2017 18:48:21 +0200 immler generalized lemmas cancelling real_of_int/real in (in)equalities with power; completed set of related simp rules; lemmas about floorlog/bitlen
Mon, 09 Oct 2017 15:34:23 +0100 paulson new material about connectedness, etc.
Sat, 26 Aug 2017 16:47:25 +0200 nipkow reorganized and added log-related lemmas
Tue, 20 Jun 2017 21:41:59 +0200 haftmann stripped code pre/postprocessor setup for real from superfluous rules
Sun, 21 May 2017 21:37:31 +0200 blanchet added one more simplification to help replay
Mon, 17 Oct 2016 11:46:22 +0200 nipkow setsum -> sum
Thu, 29 Sep 2016 20:54:45 +0200 boehmes invoke argo as part of the tried automatic proof methods
Thu, 29 Sep 2016 20:54:44 +0200 boehmes new proof method "argo" for a combination of quantifier-free propositional logic with equality and linear real arithmetic
Fri, 12 Aug 2016 17:53:55 +0200 wenzelm more symbols;
Fri, 05 Aug 2016 16:22:13 +0200 nipkow added missing lemmas
Fri, 05 Aug 2016 09:30:20 +0200 nipkow tuned floor lemmas
Fri, 15 Jul 2016 11:07:51 +0200 wenzelm misc tuning and modernization;
Thu, 23 Jun 2016 23:08:37 +0200 wenzelm misc tuning and modernization;
Fri, 17 Jun 2016 09:44:16 +0200 hoelzl move Conditional_Complete_Lattices to Main
Mon, 25 Apr 2016 16:09:26 +0200 wenzelm eliminated old 'def';
Wed, 16 Mar 2016 13:57:06 +0000 paulson Contractible sets. Also removal of obsolete theorems and refactoring
Tue, 15 Mar 2016 14:08:25 +0000 paulson rationalisation of theorem names esp about "real Archimedian" etc.
Wed, 24 Feb 2016 16:00:57 +0000 paulson Merge
Wed, 24 Feb 2016 15:51:01 +0000 paulson Substantial new material for multivariate analysis. Also removal of some duplicates.
Tue, 23 Feb 2016 16:25:08 +0100 nipkow more canonical names
Wed, 17 Feb 2016 21:51:57 +0100 haftmann dropped various legacy fact bindings
Wed, 17 Feb 2016 21:51:57 +0100 haftmann generalized some lemmas;
Wed, 06 Jan 2016 12:18:53 +0100 hoelzl add the proof of the central limit theorem
Wed, 06 Jan 2016 13:04:30 +0100 blanchet more complete setup for 'Rat' in Nitpick
Mon, 28 Dec 2015 01:26:34 +0100 wenzelm prefer symbols for "abs";
Sun, 27 Dec 2015 21:46:36 +0100 wenzelm prefer symbols for "floor", "ceiling";
Mon, 07 Dec 2015 10:38:04 +0100 wenzelm isabelle update_cartouches -c -t;
Tue, 17 Nov 2015 12:32:08 +0000 paulson Removed some legacy theorems; minor adjustments to simplification rules; new material on homotopic paths
Fri, 13 Nov 2015 12:27:13 +0000 paulson Tweaks for "real": Removal of [iff] status for some lemmas, adding [simp] for others. Plus fixes.
Tue, 10 Nov 2015 14:18:41 +0000 paulson Coercion "real" now has type nat => real only and is no longer overloaded. Type class "real_of" is gone. Many duplicate theorems removed.
Wed, 30 Sep 2015 16:36:42 +0100 paulson real_of_nat_Suc is now a simprule
Mon, 21 Sep 2015 19:52:13 +0100 paulson new lemmas and movement of lemmas into place
Tue, 01 Sep 2015 22:32:58 +0200 wenzelm eliminated \<Colon>;
Mon, 31 Aug 2015 21:28:08 +0200 wenzelm prefer symbols;
Sat, 18 Jul 2015 22:58:50 +0200 wenzelm isabelle update_cartouches;
Fri, 12 Jun 2015 08:53:23 +0200 haftmann uniform _ div _ as infix syntax for ring division
Mon, 01 Jun 2015 18:59:21 +0200 haftmann separate class for division operator, with particular syntax added in more specific classes
Thu, 30 Apr 2015 15:28:01 +0100 paulson tidying some messy proofs
Thu, 09 Apr 2015 09:12:47 +0200 haftmann conversion between division on nat/int and division in archmedean fields
Tue, 31 Mar 2015 21:54:32 +0200 haftmann given up separate type classes demanding `inverse 0 = 0`
Wed, 04 Mar 2015 23:31:04 +0100 nipkow Removed the obsolete functions "natfloor" and "natceiling"
Thu, 13 Nov 2014 17:19:52 +0100 hoelzl import general theorems from AFP/Markov_Models
Wed, 12 Nov 2014 17:36:32 +0100 immler cancel real of power of numeral also for equality and strict inequality;
Sun, 02 Nov 2014 18:21:45 +0100 wenzelm modernized header uniformly as section;
Thu, 30 Oct 2014 21:02:01 +0100 haftmann more simp rules concerning dvd and even/odd
less more (0) -100 -60 tip