src/HOL/Tools/Lifting/lifting_info.ML
changeset 53650 71a0a8687d6c
parent 53284 d0153a0a9b2b
child 53651 ee90c67502c9
equal deleted inserted replaced
53649:96814d676c49 53650:71a0a8687d6c
    13   type pcr = {pcrel_def: thm, pcr_cr_eq: thm}
    13   type pcr = {pcrel_def: thm, pcr_cr_eq: thm}
    14   type quotient = {quot_thm: thm, pcr_info: pcr option}
    14   type quotient = {quot_thm: thm, pcr_info: pcr option}
    15   val transform_quotient: morphism -> quotient -> quotient
    15   val transform_quotient: morphism -> quotient -> quotient
    16   val lookup_quotients: Proof.context -> string -> quotient option
    16   val lookup_quotients: Proof.context -> string -> quotient option
    17   val update_quotients: string -> quotient -> Context.generic -> Context.generic
    17   val update_quotients: string -> quotient -> Context.generic -> Context.generic
       
    18   val delete_quotients: thm -> Context.generic -> Context.generic
    18   val print_quotients: Proof.context -> unit
    19   val print_quotients: Proof.context -> unit
    19 
    20 
    20   val get_invariant_commute_rules: Proof.context -> thm list
    21   val get_invariant_commute_rules: Proof.context -> thm list
    21   
    22   
    22   val get_reflexivity_rules: Proof.context -> thm list
    23   val get_reflexivity_rules: Proof.context -> thm list