tuned signature (again, amending f32ac01aef5e), e.g. relevant for Isabelle/DOF;
(* Title: HOL/HOLCF/Library/HOL_Cpo.thy
Author: Brian Huffman
*)
section \<open>Cpo class instances for all HOL types\<close>
theory HOL_Cpo
imports
Bool_Discrete
Nat_Discrete
Int_Discrete
Char_Discrete
Sum_Cpo
Option_Cpo
List_Predomain
begin
end