clarified signature
authorbulwahn
Mon, 31 Oct 2011 08:50:35 +0100
changeset 45314 97b771579000
parent 45313 16bab9f1bb37
child 45315 dfbbc5ac7194
child 45317 bf8b9ac6000c
clarified signature
src/HOL/Tools/Quotient/quotient_typ.ML
--- a/src/HOL/Tools/Quotient/quotient_typ.ML	Mon Oct 31 08:43:21 2011 +0100
+++ b/src/HOL/Tools/Quotient/quotient_typ.ML	Mon Oct 31 08:50:35 2011 +0100
@@ -7,7 +7,7 @@
 signature QUOTIENT_TYPE =
 sig
   val add_quotient_type: ((string list * binding * mixfix) * (typ * term * bool)) * thm
-    -> Proof.context -> Quotient_Info.quotients * local_theory
+    -> local_theory -> Quotient_Info.quotients * local_theory
 
   val quotient_type: ((string list * binding * mixfix) * (typ * term * bool)) list
     -> Proof.context -> Proof.state