src/HOL/Real.thy
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
Mon, 27 Oct 2014 12:21:24 +0100 hoelzl further generalization of natfloor_div_nat
Mon, 27 Oct 2014 12:03:13 +0100 hoelzl generalize natfloor_div_nat, add floor variant: floor_divide_real_eq_div
Tue, 02 Sep 2014 08:24:42 +0200 haftmann more convenient printing of real numbers after evaluation
Fri, 29 Aug 2014 11:24:31 +0200 hoelzl add simp rules for divisions of numerals in floor and ceiling.
Thu, 28 Aug 2014 00:40:38 +0200 blanchet renamed new SMT module from 'SMT2' to 'SMT'
Thu, 28 Aug 2014 00:40:37 +0200 blanchet moved old 'smt' method out of 'Main'
Mon, 25 Aug 2014 14:24:05 +0200 hoelzl introduce real_of typeclass for real :: 'a => real
Tue, 19 Aug 2014 18:37:32 +0200 hoelzl better linarith support for floor, ceiling, natfloor, and natceiling
Sat, 05 Jul 2014 11:01:53 +0200 haftmann prefer ac_simps collections over separate name bindings for add and mult
Fri, 04 Jul 2014 20:18:47 +0200 haftmann reduced name variants for assoc and commute on plus and mult
Mon, 30 Jun 2014 15:45:21 +0200 hoelzl import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
Wed, 18 Jun 2014 07:31:12 +0200 hoelzl moved lemmas from the proof of the Central Limit Theorem by Jeremy Avigad and Luke Serafin
Wed, 07 May 2014 12:25:35 +0200 hoelzl avoid the Complex constructor, use the more natural Re/Im view; moved csqrt to Complex.
Mon, 14 Apr 2014 13:08:17 +0200 hoelzl added divide_nonneg_nonneg and co; made it a simp rule
Sat, 12 Apr 2014 17:26:27 +0200 nipkow made mult_pos_pos a simp rule
Fri, 11 Apr 2014 22:53:33 +0200 nipkow made divide_pos_pos a simp rule
Fri, 11 Apr 2014 13:36:57 +0200 nipkow made mult_nonneg_nonneg a simp rule
Wed, 19 Mar 2014 17:06:02 +0000 paulson Some rationalisation of basic lemmas
Thu, 13 Mar 2014 13:18:13 +0100 blanchet moved 'SMT2' (SMT-LIB-2-based SMT module) into Isabelle
Thu, 06 Mar 2014 15:40:33 +0100 blanchet renamed 'fun_rel' to 'rel_fun'
Wed, 25 Dec 2013 17:39:06 +0100 haftmann prefer more canonical names for lemmas on min/max
Tue, 19 Nov 2013 10:05:53 +0100 haftmann eliminiated neg_numeral in favour of - (numeral _)
Tue, 05 Nov 2013 21:23:42 +0100 hoelzl int and nat are conditionally_complete_lattices
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:45:00 +0100 hoelzl generalize bdd_above/below_uminus to ordered_ab_group_add
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, 16 Sep 2013 15:30:20 +0200 kuncar use lifting_forget for deregistering numeric types as a quotient type
Tue, 03 Sep 2013 01:12:40 +0200 wenzelm tuned proofs -- clarified flow of facts wrt. calculation;
Sun, 18 Aug 2013 18:49:45 +0200 wenzelm more symbols;
Mon, 13 May 2013 13:59:04 +0200 kuncar better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
Thu, 25 Apr 2013 11:59:21 +0200 hoelzl revert #916271d52466; add non-topological linear_continuum type class; show linear_continuum_topology is a perfect_space
Wed, 24 Apr 2013 13:28:30 +0200 hoelzl spell conditional_ly_-complete lattices correct
Tue, 26 Mar 2013 15:10:28 +0100 wenzelm merged
Tue, 26 Mar 2013 12:20:56 +0100 hoelzl rename RealDef to Real
Tue, 26 Mar 2013 12:20:55 +0100 hoelzl merge RComplete into RealDef
Wed, 22 Aug 2012 22:55:41 +0200 wenzelm prefer ML_file over old uses;
Wed, 12 May 2010 23:54:04 +0200 boehmes layered SMT setup, adapted SMT clients, added further tests, made Z3 proof abstraction configurable
Wed, 10 Feb 2010 14:12:02 +0100 haftmann moved lemma field_le_epsilon from Real.thy to Fields.thy
Tue, 09 Feb 2010 16:07:09 +0100 haftmann simple proofs make life faster and easier
Fri, 05 Feb 2010 14:33:50 +0100 haftmann more consistent naming of type classes involving orderings (and lattices) -- c.f. NEWS
Mon, 05 Oct 2009 17:27:46 +0100 paulson New lemmas connected with the reals and infinite series
Mon, 29 Dec 2008 14:08:08 +0100 haftmann adapted HOL source structure to distribution layout
Thu, 11 Dec 2008 08:56:02 +0100 nipkow codegen
Wed, 10 Dec 2008 10:23:47 +0100 nipkow moved ContNotDenum into Library
Wed, 03 Dec 2008 15:58:44 +0100 haftmann made repository layout more coherent with logical distribution structure; stripped some $Id$s
less more (0) tip