src/HOL/Quotient.thy
changeset 57960 ee1ba4848896
parent 56073 29e308b56d23
child 58889 5b7a9633cfa8
--- a/src/HOL/Quotient.thy	Sat Aug 16 19:20:11 2014 +0200
+++ b/src/HOL/Quotient.thy	Sat Aug 16 20:14:45 2014 +0200
@@ -748,8 +748,12 @@
 
 text {* Auxiliary data for the quotient package *}
 
+named_theorems quot_equiv "equivalence relation theorems"
+named_theorems quot_respect "respectfulness theorems"
+named_theorems quot_preserve "preservation theorems"
+named_theorems id_simps "identity simp rules for maps"
+named_theorems quot_thm "quotient theorems"
 ML_file "Tools/Quotient/quotient_info.ML"
-setup Quotient_Info.setup
 
 declare [[mapQ3 "fun" = (rel_fun, fun_quotient3)]]