src/HOL/Quotient.thy
changeset 47544 e455cdaac479
parent 47488 be6dd389639d
child 47579 28f6f4ad69bf
--- a/src/HOL/Quotient.thy	Wed Apr 18 15:09:07 2012 +0200
+++ b/src/HOL/Quotient.thy	Wed Apr 18 15:48:32 2012 +0200
@@ -34,17 +34,6 @@
   shows "((op =) OOO R) = R"
   by (auto simp add: fun_eq_iff)
 
-subsection {* Respects predicate *}
-
-definition
-  Respects :: "('a \<Rightarrow> 'a \<Rightarrow> bool) \<Rightarrow> 'a set"
-where
-  "Respects R = {x. R x x}"
-
-lemma in_respects:
-  shows "x \<in> Respects R \<longleftrightarrow> R x x"
-  unfolding Respects_def by simp
-
 subsection {* set map (vimage) and set relation *}
 
 definition "set_rel R xs ys \<equiv> \<forall>x y. R x y \<longrightarrow> x \<in> xs \<longleftrightarrow> y \<in> ys"