src/Provers/blast.ML
changeset 7272 d20f51e43909
parent 7155 70ba7d640bfe
child 7559 1d2c099e98f7
equal deleted inserted replaced
7271:442456b2a8bb 7272:d20f51e43909
    65 		 xtraIs: thm list, xtraEs: thm list,
    65 		 xtraIs: thm list, xtraEs: thm list,
    66 		 swrappers: (string * wrapper) list, 
    66 		 swrappers: (string * wrapper) list, 
    67 		 uwrappers: (string * wrapper) list,
    67 		 uwrappers: (string * wrapper) list,
    68 		 safe0_netpair: netpair, safep_netpair: netpair,
    68 		 safe0_netpair: netpair, safep_netpair: netpair,
    69 		 haz_netpair: netpair, dup_netpair: netpair, xtra_netpair: netpair}
    69 		 haz_netpair: netpair, dup_netpair: netpair, xtra_netpair: netpair}
    70   val cla_modifiers: (Args.T list -> (Proof.context attribute * Args.T list)) list
    70   val cla_modifiers: (Args.T list -> (Method.modifier * Args.T list)) list
    71   val cla_meth': (claset -> int -> tactic) -> Proof.context -> Proof.method
    71   val cla_meth': (claset -> int -> tactic) -> Proof.context -> Proof.method
    72   end;
    72   end;
    73 
    73 
    74 
    74 
    75 signature BLAST =
    75 signature BLAST =