src/HOL/HOLCF/Library/HOLCF_Library.thy
changeset 41112 866148b76247
parent 40774 0437dbc127b3
--- a/src/HOL/HOLCF/Library/HOLCF_Library.thy	Sat Dec 11 11:26:37 2010 -0800
+++ b/src/HOL/HOLCF/Library/HOLCF_Library.thy	Sat Dec 11 21:27:53 2010 -0800
@@ -1,7 +1,13 @@
 theory HOLCF_Library
 imports
+  Bool_Discrete
+  Char_Discrete
   Defl_Bifinite
+  Int_Discrete
   List_Cpo
+  List_Predomain
+  Nat_Discrete
+  Option_Cpo
   Stream
   Sum_Cpo
 begin