Quot/quotient_tacs.ML
changeset 814 cd3fa86be45f
parent 804 ba7e81531c6d
child 826 e3732ed89dfc
equal deleted inserted replaced
813:77506496e6fd 814:cd3fa86be45f
     1 signature QUOTIENT_TACS =
     1 signature QUOTIENT_TACS =
     2 sig
     2 sig
     3     val regularize_tac: Proof.context -> int -> tactic
     3     val regularize_tac: Proof.context -> int -> tactic
       
     4     val injection_tac: Proof.context -> int -> tactic
     4     val all_injection_tac: Proof.context -> int -> tactic
     5     val all_injection_tac: Proof.context -> int -> tactic
     5     val clean_tac: Proof.context -> int -> tactic
     6     val clean_tac: Proof.context -> int -> tactic
     6     val procedure_tac: Proof.context -> thm -> int -> tactic
     7     val procedure_tac: Proof.context -> thm -> int -> tactic
     7     val lift_tac: Proof.context -> thm -> int -> tactic
     8     val lift_tac: Proof.context -> thm -> int -> tactic
     8     val quotient_tac: Proof.context -> int -> tactic
     9     val quotient_tac: Proof.context -> int -> tactic
       
    10     val quot_true_tac: Proof.context -> (term -> term) -> int -> tactic
     9 end;
    11 end;
    10 
    12 
    11 structure Quotient_Tacs: QUOTIENT_TACS =
    13 structure Quotient_Tacs: QUOTIENT_TACS =
    12 struct
    14 struct
    13 
    15