reintroduce mutually (co)rec check, since the underlying N2M code doesn't quite handle the general case (esp. in presence of type variables)
theory HOLCF_Library
imports
Bool_Discrete
Char_Discrete
Defl_Bifinite
Int_Discrete
List_Cpo
List_Predomain
Nat_Discrete
Option_Cpo
Stream
Sum_Cpo
begin
end