src/HOL/Complex_Main.thy
author wenzelm
Sun, 15 Nov 2009 00:23:26 +0100
changeset 33689 d0a9ce721e0c
parent 33269 3b7e2dbbd684
child 35292 e4a431b6d9b7
permissions -rw-r--r--
properly inlined @{lemma} antiqutations -- might also reduce proof terms a bit;
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
29304
5c71a6da989d tuned header and description of boot files;
wenzelm
parents: 29197
diff changeset
     1
header {* Comprehensive Complex Theory *}
13984
e055ba9020eb new theory Complex_Main as basis for analysis developments
paulson
parents:
diff changeset
     2
15131
c69542757a4d New theory header syntax.
nipkow
parents: 13984
diff changeset
     3
theory Complex_Main
27472
47bc28e011d5 removed nonstandard analysis theories to HOL-NSA
huffman
parents: 27368
diff changeset
     4
imports
28952
15a4b2cf8c34 made repository layout more coherent with logical distribution structure; stripped some $Id$s
haftmann
parents: 28944
diff changeset
     5
  Main
15a4b2cf8c34 made repository layout more coherent with logical distribution structure; stripped some $Id$s
haftmann
parents: 28944
diff changeset
     6
  Real
33269
3b7e2dbbd684 New theory SupInf of the supremum and infimum operators for sets of reals.
paulson
parents: 31204
diff changeset
     7
  SupInf
29879
4425849f5db7 Moved FTA into Lib and cleaned it up a little.
nipkow
parents: 29304
diff changeset
     8
  Complex
28952
15a4b2cf8c34 made repository layout more coherent with logical distribution structure; stripped some $Id$s
haftmann
parents: 28944
diff changeset
     9
  Log
15a4b2cf8c34 made repository layout more coherent with logical distribution structure; stripped some $Id$s
haftmann
parents: 28944
diff changeset
    10
  Ln
15a4b2cf8c34 made repository layout more coherent with logical distribution structure; stripped some $Id$s
haftmann
parents: 28944
diff changeset
    11
  Taylor
15a4b2cf8c34 made repository layout more coherent with logical distribution structure; stripped some $Id$s
haftmann
parents: 28944
diff changeset
    12
  Integration
15131
c69542757a4d New theory header syntax.
nipkow
parents: 13984
diff changeset
    13
begin
13984
e055ba9020eb new theory Complex_Main as basis for analysis developments
paulson
parents:
diff changeset
    14
e055ba9020eb new theory Complex_Main as basis for analysis developments
paulson
parents:
diff changeset
    15
end