History log of /seL4-l4v-10.1.1/l4v/isabelle/src/HOL/Complex.thy
Revision Date Author Comments
# 102fb118 26-Jun-2018 paulson <lp15@cam.ac.uk>

Rationalisation of complex transcendentals, esp the Arg function


# a1b2af0a 21-Dec-2017 eberlm <eberlm@in.tum.de>

Some lemmas on complex numbers and coprimality

--HG--
extra : rebase_source : 37434802fd420fdcbc9750dcf9b734797e86eb61


# bf84a1ab 21-Nov-2017 eberlm <eberlm@in.tum.de>

Facts about complex n-th roots


# 5c09067f 09-Oct-2017 paulson <lp15@cam.ac.uk>

new material about connectedness, etc.


# 44a98e21 26-Apr-2017 paulson <lp15@cam.ac.uk>

Further new material. The simprule status of some exp and ln identities was reverted.


# 7af5d61d 25-Apr-2017 paulson <lp15@cam.ac.uk>

Fixed LaTeX issue


# d244f158 25-Apr-2017 paulson <lp15@cam.ac.uk>

New material from PNT proof, as well as more default [simp] declarations. Also removed duplicate theorems about geometric series


# 47187d1b 16-Mar-2017 paulson <lp15@cam.ac.uk>

Removed [simp] status for Complex_eq. Also tidied some proofs


# 246d8de3 28-Feb-2017 paulson <lp15@cam.ac.uk>

Renamed ii to imaginary_unit in order to free up ii as a variable name. Also replaced some legacy def commands


# c8cee3c6 04-Jan-2017 paulson <lp15@cam.ac.uk>

Many new theorems, and more tidying


# 049952fc 18-Oct-2016 haftmann <none@none>

suitable logical type class for abs, sgn

--HG--
extra : rebase_source : 27e95dd7f038f114d0cad11ec69599a166229041


# 593ff4b4 17-Oct-2016 nipkow <none@none>

setprod -> prod


# 351cc2e6 17-Oct-2016 nipkow <none@none>

setsum -> sum


# fbcfe7d0 31-Jul-2016 wenzelm <none@none>

misc tuning and modernization;


# b5509112 23-May-2016 paulson <lp15@cam.ac.uk>

Lots of new material for multivariate analysis


# a2bc0021 25-Apr-2016 wenzelm <none@none>

eliminated old 'def';
tuned comments;


# 6377ced5 14-Mar-2016 paulson <lp15@cam.ac.uk>

New results about paths, segments, etc. The notion of simply_connected.


# 259fcfd2 22-Feb-2016 paulson <lp15@cam.ac.uk>

An assortment of useful lemmas about sums, norm, etc. Also: norm_conv_dist [symmetric] is now a simprule!


# ec265e34 08-Jan-2016 hoelzl <none@none>

fix code generation for uniformity: uniformity is a non-computable pure data.


# da01cc11 08-Jan-2016 hoelzl <none@none>

add uniform spaces


# 82353fd1 30-Dec-2015 wenzelm <none@none>

more symbols;


# 6d3e0a15 29-Dec-2015 wenzelm <none@none>

more symbols;


# 08cabf03 27-Dec-2015 wenzelm <none@none>

prefer symbols for "abs";


# 33a3d60e 15-Dec-2015 paulson <lp15@cam.ac.uk>

New complex analysis material


# 0df376fc 07-Dec-2015 wenzelm <none@none>

isabelle update_cartouches -c -t;


# 4b76bc27 01-Dec-2015 paulson <lp15@cam.ac.uk>

Removal of redundant lemmas (diff_less_iff, diff_le_iff) and of the abbreviation Exp. Addition of some new material.


# 420aaf4c 12-Nov-2015 paulson <lp15@cam.ac.uk>

Tweaks for "real": Removal of [iff] status for some lemmas, adding [simp] for others. Plus fixes.


# 3f106d8a 10-Nov-2015 paulson <lp15@cam.ac.uk>

Coercion "real" now has type nat => real only and is no longer overloaded. Type class "real_of" is gone. Many duplicate theorems removed.


# dbea1757 02-Nov-2015 eberlm <none@none>

Added binomial identities to CONTRIBUTORS; small lemmas on of_int/pochhammer


# dd88f1ec 02-Nov-2015 eberlm <none@none>

Rounding function, uniform limits, cotangent, binomial identities


# 0b5cf461 03-Sep-2015 paulson <none@none>

new lemmas about vector_derivative, complex numbers, paths, etc.


# 85ed9565 01-Sep-2015 wenzelm <none@none>

eliminated \<Colon>;


# 1901affb 18-Jul-2015 wenzelm <none@none>

isabelle update_cartouches;


# 603f8dfb 12-Jun-2015 haftmann <none@none>

uniform _ div _ as infix syntax for ring division

--HG--
extra : rebase_source : c4a1892078772c7ce9af33ad66e2abfefe7adea9


# f2ba2c03 01-Jun-2015 haftmann <none@none>

separate class for division operator, with particular syntax added in more specific classes


# d6db773a 11-Apr-2015 paulson <lp15@cam.ac.uk>

Overloading of ln and powr, but "approximation" no longer works for powr. Code generation also fails due to type ambiguity in scala.


# ac517014 31-Mar-2015 haftmann <none@none>

given up separate type classes demanding `inverse 0 = 0`


# 7416c0a5 31-Mar-2015 paulson <lp15@cam.ac.uk>

New material and binomial fix


# ea222974 18-Mar-2015 paulson <lp15@cam.ac.uk>

new HOL Light material about exp, sin, cos


# e7eb131a 18-Mar-2015 paulson <lp15@cam.ac.uk>

Lots of new material on complex-valued functions. Modified simplification of (x/n)^k


# 9c83ffad 09-Mar-2015 paulson <lp15@cam.ac.uk>

sin, cos generalised from type real to any "'a::{real_normed_field,banach}", including complex


# b5ab68e6 05-Mar-2015 paulson <lp15@cam.ac.uk>

The function frac. Various lemmas about limits, series, the exp function, etc.


# ff53cb2b 13-Nov-2014 hoelzl <none@none>

import general theorems from AFP/Markov_Models


# 794edf80 02-Nov-2014 wenzelm <none@none>

modernized header uniformly as section;


# 8153684f 21-Oct-2014 haftmann <none@none>

turn even into an abbreviation


# 3c2ea5d6 19-Oct-2014 haftmann <none@none>

prefer generic elimination rules for even/odd over specialized unfold rules for nat


# e0068d6b 02-Sep-2014 blanchet <none@none>

codatatypes are not datatypes


# e46c07fd 04-Jul-2014 haftmann <none@none>

reduced name variants for assoc and commute on plus and mult


# 0d8a41de 16-Jun-2014 hoelzl <none@none>

add more derivative and continuity rules for complex-values functions


# 61aadd1e 06-May-2014 hoelzl <none@none>

avoid the Complex constructor, use the more natural Re/Im view; moved csqrt to Complex.

--HG--
extra : rebase_source : 899541490c73fe6897445f97dc2a5a3c929cf153


# 838cbeac 11-Apr-2014 nipkow <none@none>

made divide_pos_pos a simp rule


# 77b90a1d 09-Apr-2014 hoelzl <none@none>

revert c1bbd3e22226, a14831ac3023, and 36489d77c484: divide_minus_left/right are again simp rules


# 36a1e2cc 03-Apr-2014 paulson <lp15@cam.ac.uk>

removing simprule status for divide_minus_left and divide_minus_right


# 85993f65 03-Apr-2014 hoelzl <none@none>

merged DERIV_intros, has_derivative_intros into derivative_intros


# 3c2af176 02-Apr-2014 hoelzl <none@none>

moved generic theorems from Complex_Analysis_Basic; fixed some theorem names


# 31965c4d 30-Mar-2014 hoelzl <none@none>

add complex_of_real coercion


# 52d226b9 21-Mar-2014 paulson <lp15@cam.ac.uk>

a few new lemmas and generalisations of old ones


# 956719cb 19-Mar-2014 paulson <lp15@cam.ac.uk>

Some rationalisation of basic lemmas


# 0281a51e 26-Feb-2014 boehmes <none@none>

replaced smt-based proof with metis proof that requires no external tool


# 618e561e 25-Feb-2014 paulson <lp15@cam.ac.uk>

More complex-related lemmas


# 138816de 19-Nov-2013 haftmann <none@none>

eliminiated neg_numeral in favour of - (numeral _)


# d2ef840a 01-Nov-2013 haftmann <none@none>

more simplification rules on unary and binary minus

--HG--
extra : rebase_source : 7c88c9f33c4be8eae76f508a1a73ba79c8b769b1


# 7237bdd9 02-Sep-2013 wenzelm <none@none>

tuned proofs -- clarified flow of facts wrt. calculation;


# 06329277 13-Aug-2013 wenzelm <none@none>

standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;


# 8ea7ea05 31-Jan-2013 hoelzl <none@none>

remove unnecessary assumption from real_normed_vector

--HG--
extra : rebase_source : 4a68de89541842f1b91794ddd73c625b6a822085


# d9333ba5 19-Oct-2012 webertj <none@none>

Renamed {left,right}_distrib to distrib_{right,left}.


# 8bb6233a 25-Mar-2012 huffman <none@none>

merged fork with new numeral representation (see NEWS)


# 93cee60f 12-Sep-2011 huffman <none@none>

move lemmas about complex number 'i' to Complex.thy and Library/Inner_Product.thy


# 20eb8aa2 08-Sep-2011 huffman <none@none>

remove unnecessary intermediate lemmas


# adf75a0a 08-Sep-2011 huffman <none@none>

prove existence, uniqueness, and other properties of complex arg function


# b7e8f839 08-Sep-2011 huffman <none@none>

tuned


# 8b9946f7 08-Sep-2011 huffman <none@none>

remove obsolete intermediate lemma complex_inverse_complex_split


# d23aa661 08-Sep-2011 huffman <none@none>

tuned


# fed3a1d4 07-Sep-2011 huffman <none@none>

add some new lemmas about cis and rcis;
simplify some proofs;


# a1abe539 07-Sep-2011 huffman <none@none>

Complex.thy: move theorems into appropriate subsections


# b5a5716b 07-Sep-2011 huffman <none@none>

remove redundant lemma complex_of_real_minus_one

--HG--
extra : transplant_source : %93%21%A4%91%08%9C%3B%F6h%13%0A%84%F3%2B%ACGz%2B%3AU


# 8e88eb56 07-Sep-2011 huffman <none@none>

simplify proof of lemma DeMoivre, removing unnecessary intermediate lemma


# d9478aab 07-Sep-2011 huffman <none@none>

removed unused lemma sin_cos_squared_add2_mult


# 7e3ead55 06-Sep-2011 huffman <none@none>

remove redundant lemmas i_mult_eq and i_mult_eq2 in favor of i_squared


# 6f7569c4 06-Sep-2011 huffman <none@none>

remove some unnecessary simp rules from simpset


# 80da0e6b 06-Sep-2011 huffman <none@none>

remove redundant lemma real_sum_squared_expand in favor of power2_sum


# d1ff3e8d 06-Sep-2011 huffman <none@none>

remove redundant lemma LIMSEQ_Complex in favor of tendsto_Complex


# ae95dea2 05-Sep-2011 huffman <none@none>

tuned indentation


# f9ec1df2 04-Sep-2011 huffman <none@none>

tuned comments


# 5cd5ec6c 04-Sep-2011 huffman <none@none>

replace lemma expi_imaginary with reoriented lemma cis_conv_exp


# 914fece6 04-Sep-2011 huffman <none@none>

remove redundant lemmas expi_add and expi_zero


# 19dfe100 19-Aug-2011 huffman <none@none>

move sin_coeff and cos_coeff lemmas to Transcendental.thy; simplify some proofs


# 0f89aef6 18-Aug-2011 huffman <none@none>

define complex exponential 'expi' as abbreviation for 'exp'


# 9a2b28b7 18-Aug-2011 huffman <none@none>

remove more bounded_linear locale interpretations (cf. f0de18b62d63)


# ae3b13a5 09-Aug-2011 huffman <none@none>

lemma bounded_linear_intro


# 08b8bb33 08-Aug-2011 huffman <none@none>

standard theorem naming scheme: complex_eqI, complex_eq_iff


# 6b0b29ec 13-Mar-2011 wenzelm <none@none>

tuned headers;


# 8ace0d5f 19-Jul-2010 haftmann <none@none>

diff_minus subsumes diff_def


# 140c6b08 12-Jul-2010 haftmann <none@none>

dropped superfluous [code del]s


# 54f2c5e9 11-May-2010 huffman <none@none>

add lemma tendsto_Complex


# 811241d7 09-May-2010 huffman <none@none>

avoid using real-specific versions of generic lemmas


# 756c3e6e 26-Apr-2010 haftmann <none@none>

use new classes (linordered_)field_inverse_zero


# f2a891d4 26-Apr-2010 haftmann <none@none>

class division_ring_inverse_zero


# 57bfb831 07-Jun-2009 huffman <none@none>

replace 'topo' with 'open'; add extra type constraint for 'open'


# c98b1969 03-Jun-2009 huffman <none@none>

more [code del] declarations


# f1a6d49f 03-Jun-2009 huffman <none@none>

replace class open with class topo


# 187de063 03-Jun-2009 huffman <none@none>

introduce class topological_space as a superclass of metric_space


# 98f3e0ce 28-May-2009 huffman <none@none>

definition of dist for complex


# dcdcebd1 29-Apr-2009 haftmann <none@none>

farewell to class recpower


# 7e4b4782 22-Apr-2009 haftmann <none@none>

power operation defined generic


# 0761d736 26-Mar-2009 wenzelm <none@none>

interpretation/interpret: prefixes are mandatory by default;


# 8ee53001 04-Mar-2009 huffman <none@none>

declare power_Suc [simp]; remove redundant type-specific versions of power_Suc


# abf397f0 28-Jan-2009 nipkow <none@none>

Replaced group_ and ring_simps by algebra_simps;
removed compare_rls - use algebra_simps now


# 590502d1 14-Dec-2008 ballarin <none@none>

Ported HOL and HOL-Library to new locales.


# f21befe1 03-Dec-2008 haftmann <none@none>

made repository layout more coherent with logical distribution structure; stripped some $Id$s

--HG--
rename : src/HOL/Library/Code_Message.thy => src/HOL/Code_Message.thy
rename : src/HOL/Complex/Complex.thy => src/HOL/Complex.thy
rename : src/HOL/Complex/Complex_Main.thy => src/HOL/Complex_Main.thy
rename : src/HOL/Real/ContNotDenum.thy => src/HOL/ContNotDenum.thy
rename : src/HOL/Hyperreal/Deriv.thy => src/HOL/Deriv.thy
rename : src/HOL/Hyperreal/Fact.thy => src/HOL/Fact.thy
rename : src/HOL/Hyperreal/FrechetDeriv.thy => src/HOL/FrechetDeriv.thy
rename : src/HOL/Library/GCD.thy => src/HOL/GCD.thy
rename : src/HOL/Hyperreal/Integration.thy => src/HOL/Integration.thy
rename : src/HOL/Real/Float.thy => src/HOL/Library/Float.thy
rename : src/HOL/Hyperreal/Lim.thy => src/HOL/Lim.thy
rename : src/HOL/Hyperreal/Ln.thy => src/HOL/Ln.thy
rename : src/HOL/Hyperreal/Log.thy => src/HOL/Log.thy
rename : src/HOL/Real/Lubs.thy => src/HOL/Lubs.thy
rename : src/HOL/Hyperreal/MacLaurin.thy => src/HOL/MacLaurin.thy
rename : src/HOL/Hyperreal/NthRoot.thy => src/HOL/NthRoot.thy
rename : src/HOL/Library/Order_Relation.thy => src/HOL/Order_Relation.thy
rename : src/HOL/Real/PReal.thy => src/HOL/PReal.thy
rename : src/HOL/Library/Parity.thy => src/HOL/Parity.thy
rename : src/HOL/Real/RComplete.thy => src/HOL/RComplete.thy
rename : src/HOL/Real/Rational.thy => src/HOL/Rational.thy
rename : src/HOL/Real/Real.thy => src/HOL/Real.thy
rename : src/HOL/Real/RealDef.thy => src/HOL/RealDef.thy
rename : src/HOL/Real/RealPow.thy => src/HOL/RealPow.thy
rename : src/HOL/Hyperreal/Series.thy => src/HOL/Series.thy
rename : src/HOL/Hyperreal/Taylor.thy => src/HOL/Taylor.thy
rename : src/HOL/arith_data.ML => src/HOL/Tools/arith_data.ML
rename : src/HOL/Real/float_arith.ML => src/HOL/Tools/float_arith.ML
rename : src/HOL/Real/float_syntax.ML => src/HOL/Tools/float_syntax.ML
rename : src/HOL/hologic.ML => src/HOL/Tools/hologic.ML
rename : src/HOL/int_arith1.ML => src/HOL/Tools/int_arith.ML
rename : src/HOL/int_factor_simprocs.ML => src/HOL/Tools/int_factor_simprocs.ML
rename : src/HOL/nat_simprocs.ML => src/HOL/Tools/nat_simprocs.ML
rename : src/HOL/Real/rat_arith.ML => src/HOL/Tools/rat_arith.ML
rename : src/HOL/Real/real_arith.ML => src/HOL/Tools/real_arith.ML
rename : src/HOL/simpdata.ML => src/HOL/Tools/simpdata.ML
rename : src/HOL/Hyperreal/Transcendental.thy => src/HOL/Transcendental.thy
rename : src/HOL/Library/RType.thy => src/HOL/Typerep.thy
rename : src/HOL/Library/Univ_Poly.thy => src/HOL/Univ_Poly.thy
rename : src/HOL/Complex/ex/Arithmetic_Series_Complex.thy => src/HOL/ex/Arithmetic_Series_Complex.thy
rename : src/HOL/Complex/ex/BigO_Complex.thy => src/HOL/ex/BigO_Complex.thy
rename : src/HOL/Complex/ex/HarmonicSeries.thy => src/HOL/ex/HarmonicSeries.thy
rename : src/HOL/Complex/ex/MIR.thy => src/HOL/ex/MIR.thy
rename : src/HOL/Complex/ex/ReflectedFerrack.thy => src/HOL/ex/ReflectedFerrack.thy
rename : src/HOL/Complex/ex/Sqrt.thy => src/HOL/ex/Sqrt.thy
rename : src/HOL/Complex/ex/Sqrt_Script.thy => src/HOL/ex/Sqrt_Script.thy
rename : src/HOL/Complex/ex/linrtac.ML => src/HOL/ex/linrtac.ML
rename : src/HOL/Complex/ex/mirtac.ML => src/HOL/ex/mirtac.ML
rename : src/Pure/Tools/quickcheck.ML => src/Tools/quickcheck.ML
rename : src/Pure/Tools/value.ML => src/Tools/value.ML