src/HOL/Complex.thy
Thu, 08 Nov 2018 09:11:52 +0100 haftmann removed relics of ASCII syntax for indexed big operators
Sat, 04 Aug 2018 01:03:39 +0200 eberlm Small lemmas about analysis
Tue, 26 Jun 2018 14:51:18 +0100 paulson Rationalisation of complex transcendentals, esp the Arg function
Thu, 21 Dec 2017 08:23:19 +0100 eberlm Some lemmas on complex numbers and coprimality
Tue, 21 Nov 2017 17:18:10 +0100 eberlm Facts about complex n-th roots
Mon, 09 Oct 2017 15:34:23 +0100 paulson new material about connectedness, etc.
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
less more (0) -100 -60 tip