src/HOLCF/Pcpodef.thy
changeset 40089 8adc57fb8454
parent 40035 a12d35795cb9
child 40321 d065b195ec89
--- a/src/HOLCF/Pcpodef.thy	Fri Oct 22 06:08:51 2010 -0700
+++ b/src/HOLCF/Pcpodef.thy	Fri Oct 22 06:58:45 2010 -0700
@@ -46,15 +46,6 @@
     by (simp only: type_definition.Abs_image [OF type])
 qed
 
-theorem typedef_finite_po:
-  fixes Abs :: "'a::finite_po \<Rightarrow> 'b::po"
-  assumes type: "type_definition Rep Abs A"
-  shows "OFCLASS('b, finite_po_class)"
- apply (intro_classes)
- apply (rule typedef_finite_UNIV [OF type])
- apply (rule finite)
-done
-
 subsection {* Proving a subtype is chain-finite *}
 
 lemma ch2ch_Rep: