got rid of hard-coded weights, now that we have TFIDF
(* Title: HOL/HOLCF/Library/HOL_Cpo.thy Author: Brian Huffman*)header {* Cpo class instances for all HOL types *}theory HOL_Cpoimports Bool_Discrete Nat_Discrete Int_Discrete Char_Discrete Sum_Cpo Option_Cpo List_Predomainbeginend