clarified type ML_Context.antiq: context parser maintains compilation context, declaration is applied to final context;
subtle change of semantics of ML_Context.add_antiq: need to avoid accidental update of context due to concrete syntax parser (cf. Scan.pass);
header {* Comprehensive Complex Theory *}
theory Complex_Main
imports
Main
Real
Complex
Transcendental
Taylor
Deriv
begin
end