--- a/Quot/quotient_info.ML Thu Jan 14 10:47:19 2010 +0100
+++ b/Quot/quotient_info.ML Thu Jan 14 10:51:03 2010 +0100
@@ -21,7 +21,7 @@
val qconsts_lookup: theory -> term -> qconsts_info (* raises NotFound *)
val qconsts_update_thy: string -> qconsts_info -> theory -> theory
val qconsts_update_gen: string -> qconsts_info -> Context.generic -> Context.generic
- val qconsts_dest: theory -> qconsts_info list
+ val qconsts_dest: Proof.context -> qconsts_info list
val print_qconstinfo: Proof.context -> unit
val equiv_rules_get: Proof.context -> thm list
@@ -198,8 +198,8 @@
fun qconsts_update_thy name qcinfo = QConstsData.map (Symtab.cons_list (name, qcinfo))
fun qconsts_update_gen name qcinfo = Context.mapping (qconsts_update_thy name qcinfo) I
-fun qconsts_dest thy =
- flat (map snd (Symtab.dest (QConstsData.get thy)))
+fun qconsts_dest lthy =
+ flat (map snd (Symtab.dest (QConstsData.get (ProofContext.theory_of lthy))))
fun qconsts_lookup thy t =
let