src/HOL/Equiv_Relations.thy
changeset 55024 05cc0dbf3a50
parent 55022 eeba3ba73486
child 58889 5b7a9633cfa8
--- a/src/HOL/Equiv_Relations.thy	Thu Jan 16 20:52:54 2014 +0100
+++ b/src/HOL/Equiv_Relations.thy	Thu Jan 16 21:22:01 2014 +0100
@@ -497,5 +497,6 @@
   "equivp R \<Longrightarrow> R x y \<Longrightarrow> R y z \<Longrightarrow> R x z"
   by (erule equivpE, erule transpE)
 
+hide_const (open) proj
+
 end
-