src/HOL/Complex.thy
Wed, 26 Apr 2017 15:53:35 +0100 paulson Further new material. The simprule status of some exp and ln identities was reverted.
Tue, 25 Apr 2017 17:10:17 +0100 paulson Fixed LaTeX issue
Tue, 25 Apr 2017 16:39:54 +0100 paulson New material from PNT proof, as well as more default [simp] declarations. Also removed duplicate theorems about geometric series
Thu, 16 Mar 2017 16:02:18 +0000 paulson Removed [simp] status for Complex_eq. Also tidied some proofs
Tue, 28 Feb 2017 13:51:47 +0000 paulson Renamed ii to imaginary_unit in order to free up ii as a variable name. Also replaced some legacy def commands
Wed, 04 Jan 2017 16:18:50 +0000 paulson Many new theorems, and more tidying
Tue, 18 Oct 2016 18:48:53 +0200 haftmann suitable logical type class for abs, sgn
Mon, 17 Oct 2016 17:33:07 +0200 nipkow setprod -> prod
Mon, 17 Oct 2016 11:46:22 +0200 nipkow setsum -> sum
Sun, 31 Jul 2016 17:25:38 +0200 wenzelm misc tuning and modernization;
Mon, 23 May 2016 15:33:24 +0100 paulson Lots of new material for multivariate analysis
Mon, 25 Apr 2016 16:09:26 +0200 wenzelm eliminated old 'def';
Mon, 14 Mar 2016 15:58:02 +0000 paulson New results about paths, segments, etc. The notion of simply_connected.
Mon, 22 Feb 2016 14:37:56 +0000 paulson An assortment of useful lemmas about sums, norm, etc. Also: norm_conv_dist [symmetric] is now a simprule!
Fri, 08 Jan 2016 17:41:04 +0100 hoelzl fix code generation for uniformity: uniformity is a non-computable pure data.
Fri, 08 Jan 2016 17:40:59 +0100 hoelzl add uniform spaces
Wed, 30 Dec 2015 11:21:54 +0100 wenzelm more symbols;
Tue, 29 Dec 2015 23:04:53 +0100 wenzelm more symbols;
Mon, 28 Dec 2015 01:26:34 +0100 wenzelm prefer symbols for "abs";
Tue, 15 Dec 2015 14:40:36 +0000 paulson New complex analysis material
Mon, 07 Dec 2015 10:38:04 +0100 wenzelm isabelle update_cartouches -c -t;
Tue, 01 Dec 2015 14:09:10 +0000 paulson Removal of redundant lemmas (diff_less_iff, diff_le_iff) and of the abbreviation Exp. Addition of some new material.
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.
Mon, 02 Nov 2015 16:17:09 +0100 eberlm Added binomial identities to CONTRIBUTORS; small lemmas on of_int/pochhammer
Mon, 02 Nov 2015 11:56:28 +0100 eberlm Rounding function, uniform limits, cotangent, binomial identities
Thu, 03 Sep 2015 20:27:53 +0100 paulson new lemmas about vector_derivative, complex numbers, paths, etc.
Tue, 01 Sep 2015 22:32:58 +0200 wenzelm eliminated \<Colon>;
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
Sat, 11 Apr 2015 11:56:40 +0100 paulson Overloading of ln and powr, but "approximation" no longer works for powr. Code generation also fails due to type ambiguity in scala.
Tue, 31 Mar 2015 21:54:32 +0200 haftmann given up separate type classes demanding `inverse 0 = 0`
Tue, 31 Mar 2015 15:00:03 +0100 paulson New material and binomial fix
Wed, 18 Mar 2015 17:23:22 +0000 paulson new HOL Light material about exp, sin, cos
Wed, 18 Mar 2015 14:13:27 +0000 paulson Lots of new material on complex-valued functions. Modified simplification of (x/n)^k
Mon, 09 Mar 2015 16:28:19 +0000 paulson sin, cos generalised from type real to any "'a::{real_normed_field,banach}", including complex
Thu, 05 Mar 2015 17:30:29 +0000 paulson The function frac. Various lemmas about limits, series, the exp function, etc.
Thu, 13 Nov 2014 17:19:52 +0100 hoelzl import general theorems from AFP/Markov_Models
Sun, 02 Nov 2014 18:21:45 +0100 wenzelm modernized header uniformly as section;
Tue, 21 Oct 2014 21:10:44 +0200 haftmann turn even into an abbreviation
Sun, 19 Oct 2014 18:05:26 +0200 haftmann prefer generic elimination rules for even/odd over specialized unfold rules for nat
Wed, 03 Sep 2014 00:06:18 +0200 blanchet codatatypes are not datatypes
Fri, 04 Jul 2014 20:18:47 +0200 haftmann reduced name variants for assoc and commute on plus and mult
Mon, 16 Jun 2014 17:52:33 +0200 hoelzl add more derivative and continuity rules for complex-values functions
Wed, 07 May 2014 12:25:35 +0200 hoelzl avoid the Complex constructor, use the more natural Re/Im view; moved csqrt to Complex.
Fri, 11 Apr 2014 22:53:33 +0200 nipkow made divide_pos_pos a simp rule
Wed, 09 Apr 2014 09:37:47 +0200 hoelzl revert c1bbd3e22226, a14831ac3023, and 36489d77c484: divide_minus_left/right are again simp rules
Thu, 03 Apr 2014 23:51:52 +0100 paulson removing simprule status for divide_minus_left and divide_minus_right
Thu, 03 Apr 2014 17:56:08 +0200 hoelzl merged DERIV_intros, has_derivative_intros into derivative_intros
Wed, 02 Apr 2014 18:35:01 +0200 hoelzl moved generic theorems from Complex_Analysis_Basic; fixed some theorem names
Mon, 31 Mar 2014 12:32:15 +0200 hoelzl add complex_of_real coercion
Fri, 21 Mar 2014 15:36:00 +0000 paulson a few new lemmas and generalisations of old ones
Wed, 19 Mar 2014 17:06:02 +0000 paulson Some rationalisation of basic lemmas
Wed, 26 Feb 2014 15:33:52 +0100 boehmes replaced smt-based proof with metis proof that requires no external tool
Tue, 25 Feb 2014 16:17:20 +0000 paulson More complex-related lemmas
Tue, 19 Nov 2013 10:05:53 +0100 haftmann eliminiated neg_numeral in favour of - (numeral _)
Fri, 01 Nov 2013 18:51:14 +0100 haftmann more simplification rules on unary and binary minus
Tue, 03 Sep 2013 01:12:40 +0200 wenzelm tuned proofs -- clarified flow of facts wrt. calculation;
Tue, 13 Aug 2013 16:25:47 +0200 wenzelm standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
Thu, 31 Jan 2013 17:42:12 +0100 hoelzl remove unnecessary assumption from real_normed_vector
Fri, 19 Oct 2012 15:12:52 +0200 webertj Renamed {left,right}_distrib to distrib_{right,left}.
Sun, 25 Mar 2012 20:15:39 +0200 huffman merged fork with new numeral representation (see NEWS)
Mon, 12 Sep 2011 09:21:01 -0700 huffman move lemmas about complex number 'i' to Complex.thy and Library/Inner_Product.thy
Thu, 08 Sep 2011 10:07:53 -0700 huffman remove unnecessary intermediate lemmas
Thu, 08 Sep 2011 08:41:28 -0700 huffman prove existence, uniqueness, and other properties of complex arg function
Thu, 08 Sep 2011 07:27:57 -0700 huffman tuned
Thu, 08 Sep 2011 07:16:47 -0700 huffman remove obsolete intermediate lemma complex_inverse_complex_split
Thu, 08 Sep 2011 07:06:59 -0700 huffman tuned
Wed, 07 Sep 2011 22:44:26 -0700 huffman add some new lemmas about cis and rcis;
Wed, 07 Sep 2011 20:44:39 -0700 huffman Complex.thy: move theorems into appropriate subsections
Wed, 07 Sep 2011 17:41:29 -0700 huffman remove redundant lemma complex_of_real_minus_one
Wed, 07 Sep 2011 18:47:55 -0700 huffman simplify proof of lemma DeMoivre, removing unnecessary intermediate lemma
Wed, 07 Sep 2011 10:04:07 -0700 huffman removed unused lemma sin_cos_squared_add2_mult
Tue, 06 Sep 2011 14:53:51 -0700 huffman remove redundant lemmas i_mult_eq and i_mult_eq2 in favor of i_squared
Tue, 06 Sep 2011 13:16:46 -0700 huffman remove some unnecessary simp rules from simpset
Tue, 06 Sep 2011 07:48:59 -0700 huffman remove redundant lemma real_sum_squared_expand in favor of power2_sum
Tue, 06 Sep 2011 07:45:18 -0700 huffman remove redundant lemma LIMSEQ_Complex in favor of tendsto_Complex
Mon, 05 Sep 2011 08:38:50 -0700 huffman tuned indentation
Sun, 04 Sep 2011 21:03:54 -0700 huffman tuned comments
Sun, 04 Sep 2011 10:29:38 -0700 huffman replace lemma expi_imaginary with reoriented lemma cis_conv_exp
Sun, 04 Sep 2011 10:05:52 -0700 huffman remove redundant lemmas expi_add and expi_zero
Fri, 19 Aug 2011 18:42:41 -0700 huffman move sin_coeff and cos_coeff lemmas to Transcendental.thy; simplify some proofs
Thu, 18 Aug 2011 22:31:52 -0700 huffman define complex exponential 'expi' as abbreviation for 'exp'
Thu, 18 Aug 2011 21:23:31 -0700 huffman remove more bounded_linear locale interpretations (cf. f0de18b62d63)
Tue, 09 Aug 2011 12:50:22 -0700 huffman lemma bounded_linear_intro
Mon, 08 Aug 2011 10:26:26 -0700 huffman standard theorem naming scheme: complex_eqI, complex_eq_iff
Sun, 13 Mar 2011 22:55:50 +0100 wenzelm tuned headers;
Mon, 19 Jul 2010 16:09:44 +0200 haftmann diff_minus subsumes diff_def
Mon, 12 Jul 2010 10:48:37 +0200 haftmann dropped superfluous [code del]s
Tue, 11 May 2010 07:58:48 -0700 huffman add lemma tendsto_Complex
Sun, 09 May 2010 17:47:43 -0700 huffman avoid using real-specific versions of generic lemmas
Mon, 26 Apr 2010 15:37:50 +0200 haftmann use new classes (linordered_)field_inverse_zero
Mon, 26 Apr 2010 11:34:17 +0200 haftmann class division_ring_inverse_zero
Sun, 07 Jun 2009 17:59:54 -0700 huffman replace 'topo' with 'open'; add extra type constraint for 'open'
Wed, 03 Jun 2009 10:29:11 -0700 huffman more [code del] declarations
Wed, 03 Jun 2009 09:58:11 -0700 huffman replace class open with class topo
Wed, 03 Jun 2009 07:44:56 -0700 huffman introduce class topological_space as a superclass of metric_space
Thu, 28 May 2009 22:53:23 -0700 huffman definition of dist for complex
Wed, 29 Apr 2009 14:20:26 +0200 haftmann farewell to class recpower
Wed, 22 Apr 2009 19:09:21 +0200 haftmann power operation defined generic
Thu, 26 Mar 2009 20:08:55 +0100 wenzelm interpretation/interpret: prefixes are mandatory by default;
Wed, 04 Mar 2009 17:12:23 -0800 huffman declare power_Suc [simp]; remove redundant type-specific versions of power_Suc
Wed, 28 Jan 2009 16:29:16 +0100 nipkow Replaced group_ and ring_simps by algebra_simps;
Sun, 14 Dec 2008 18:45:51 +0100 ballarin Ported HOL and HOL-Library to new locales.
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