author | nipkow |
Mon, 18 May 2009 23:15:56 +0200 | |
changeset 31198 | ed955d2fbfa9 |
parent 31186 | b458b4ac570f |
child 31204 | 46c0c741c8c2 |
permissions | -rw-r--r-- |
29304 | 1 |
header {* Comprehensive Complex Theory *} |
13984
e055ba9020eb
new theory Complex_Main as basis for analysis developments
paulson
parents:
diff
changeset
|
2 |
|
15131 | 3 |
theory Complex_Main |
27472 | 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 |
29879 | 7 |
Complex |
28952
15a4b2cf8c34
made repository layout more coherent with logical distribution structure; stripped some $Id$s
haftmann
parents:
28944
diff
changeset
|
8 |
Log |
15a4b2cf8c34
made repository layout more coherent with logical distribution structure; stripped some $Id$s
haftmann
parents:
28944
diff
changeset
|
9 |
Ln |
15a4b2cf8c34
made repository layout more coherent with logical distribution structure; stripped some $Id$s
haftmann
parents:
28944
diff
changeset
|
10 |
Taylor |
15a4b2cf8c34
made repository layout more coherent with logical distribution structure; stripped some $Id$s
haftmann
parents:
28944
diff
changeset
|
11 |
Integration |
31186
b458b4ac570f
experimental move of Quickcheck and related theories to HOL image
haftmann
parents:
31179
diff
changeset
|
12 |
Quickcheck |
15131 | 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 |