src/Provers/blast.ML
changeset 7272 d20f51e43909
parent 7155 70ba7d640bfe
child 7559 1d2c099e98f7
--- a/src/Provers/blast.ML	Wed Aug 18 20:45:52 1999 +0200
+++ b/src/Provers/blast.ML	Wed Aug 18 20:47:31 1999 +0200
@@ -67,7 +67,7 @@
 		 uwrappers: (string * wrapper) list,
 		 safe0_netpair: netpair, safep_netpair: netpair,
 		 haz_netpair: netpair, dup_netpair: netpair, xtra_netpair: netpair}
-  val cla_modifiers: (Args.T list -> (Proof.context attribute * Args.T list)) list
+  val cla_modifiers: (Args.T list -> (Method.modifier * Args.T list)) list
   val cla_meth': (claset -> int -> tactic) -> Proof.context -> Proof.method
   end;