src/Provers/blast.ML
changeset 5926 58f9ca06b76b
parent 5734 bebd10cb7a8d
child 5961 6cf4e46ce95a
equal deleted inserted replaced
5925:669d0bc621e1 5926:58f9ca06b76b
    64 		 hazIs: thm list, hazEs: thm list,
    64 		 hazIs: thm list, hazEs: thm list,
    65 		 swrappers: (string * wrapper) list, 
    65 		 swrappers: (string * wrapper) list, 
    66 		 uwrappers: (string * wrapper) list,
    66 		 uwrappers: (string * wrapper) list,
    67 		 safe0_netpair: netpair, safep_netpair: netpair,
    67 		 safe0_netpair: netpair, safep_netpair: netpair,
    68 		 haz_netpair: netpair, dup_netpair: netpair}
    68 		 haz_netpair: netpair, dup_netpair: netpair}
       
    69   val cla_method': (claset -> int -> tactic) -> Args.src -> Proof.context -> Proof.method
    69   end;
    70   end;
    70 
    71 
    71 
    72 
    72 signature BLAST =
    73 signature BLAST =
    73   sig
    74   sig
    85   type branch
    86   type branch
    86   val depth_tac 	: claset -> int -> int -> tactic
    87   val depth_tac 	: claset -> int -> int -> tactic
    87   val blast_tac 	: claset -> int -> tactic
    88   val blast_tac 	: claset -> int -> tactic
    88   val Blast_tac 	: int -> tactic
    89   val Blast_tac 	: int -> tactic
    89   val overloaded 	: string * (Term.typ -> Term.typ) -> unit
    90   val overloaded 	: string * (Term.typ -> Term.typ) -> unit
       
    91   val setup		: (theory -> theory) list
    90   (*debugging tools*)
    92   (*debugging tools*)
    91   val stats	        : bool ref
    93   val stats	        : bool ref
    92   val trace	        : bool ref
    94   val trace	        : bool ref
    93   val fullTrace	        : branch list list ref
    95   val fullTrace	        : branch list list ref
    94   val fromType	        : (indexname * term) list ref -> Term.typ -> term
    96   val fromType	        : (indexname * term) list ref -> Term.typ -> term
  1320 		   Data.claset(), 
  1322 		   Data.claset(), 
  1321 		   [initBranch ([readGoal (sign_of thy) s], lim)], 
  1323 		   [initBranch ([readGoal (sign_of thy) s], lim)], 
  1322 		   I));
  1324 		   I));
  1323 
  1325 
  1324 
  1326 
       
  1327 (** method setup **)
       
  1328 
       
  1329 val setup = [Method.add_methods [("blast", Data.cla_method' blast_tac, "blast")]];
       
  1330 
       
  1331 
  1325 end;
  1332 end;