src/HOL/Library/Countable.thy
changeset 58155 14dda84afbb3
parent 58112 8081087096ad
child 58158 d2cb7cbb3aaa
--- a/src/HOL/Library/Countable.thy	Wed Sep 03 00:06:26 2014 +0200
+++ b/src/HOL/Library/Countable.thy	Wed Sep 03 00:06:27 2014 +0200
@@ -308,9 +308,11 @@
 hide_const (open) finite_item nth_item
 
 
+(* FIXME
 subsection {* Countable datatypes *}
 
 instance typerep :: countable
   by countable_datatype
+*)
 
 end