src/HOL/Complex.thy
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
less more (0) -60 tip