Quot/QuotMain.thy
changeset 1124 4a4c714ff795
parent 1122 d1eaed018e5d
child 1127 243a5ceaa088
--- a/Quot/QuotMain.thy	Wed Feb 10 17:10:52 2010 +0100
+++ b/Quot/QuotMain.thy	Wed Feb 10 17:22:18 2010 +0100
@@ -12,7 +12,7 @@
   ("quotient_tacs.ML")
 begin
 
-locale Quot_Type =
+locale quot_type =
   fixes R :: "'a \<Rightarrow> 'a \<Rightarrow> bool"
   and   Abs :: "('a \<Rightarrow> bool) \<Rightarrow> 'b"
   and   Rep :: "'b \<Rightarrow> ('a \<Rightarrow> bool)"