src/HOL/Quotient.thy
changeset 47361 87c0eaf04bad
parent 47308 9caab698dbe4
child 47362 b1f099bdfbba
--- a/src/HOL/Quotient.thy	Wed Apr 04 16:29:17 2012 +0100
+++ b/src/HOL/Quotient.thy	Wed Apr 04 17:51:12 2012 +0200
@@ -772,24 +772,6 @@
 using assms
 by (rule OOO_quotient3) auto
 
-subsection {* Invariant *}
-
-lemma copy_type_to_Quotient3:
-  assumes "type_definition Rep Abs UNIV"
-  shows "Quotient3 (op =) Abs Rep"
-proof -
-  interpret type_definition Rep Abs UNIV by fact
-  from Abs_inject Rep_inverse show ?thesis by (auto intro!: Quotient3I)
-qed
-
-lemma invariant_type_to_Quotient3:
-  assumes "type_definition Rep Abs {x. P x}"
-  shows "Quotient3 (Lifting.invariant P) Abs Rep"
-proof -
-  interpret type_definition Rep Abs "{x. P x}" by fact
-  from Rep Abs_inject Rep_inverse show ?thesis by (auto intro!: Quotient3I simp: invariant_def)
-qed
-
 subsection {* ML setup *}
 
 text {* Auxiliary data for the quotient package *}