two target language numeral types: integer and natural, as replacement for code_numeral;
former theory HOL/Library/Code_Numeral_Types replaces HOL/Code_Numeral;
refined stack of theories implementing int and/or nat by target language numerals;
reduced number of target language numeral types to exactly one
header {* Comprehensive Complex Theory *}
theory Complex_Main
imports
Main
Real
SupInf
Complex
Log
Ln
Taylor
Deriv
begin
end