src/Pure/Isar/method.ML
changeset 8381 4fc7e63781f6
parent 8372 7b2cec1e789c
child 8519 981f52707e5d
equal deleted inserted replaced
8380:c96953faf0a4 8381:4fc7e63781f6
   456 
   456 
   457 type modifier = (Proof.context -> Proof.context) * Proof.context attribute;
   457 type modifier = (Proof.context -> Proof.context) * Proof.context attribute;
   458 
   458 
   459 local
   459 local
   460 
   460 
   461 fun sect ss = Scan.first (map (fn s => Scan.lift (s --| Args.$$$ ":")) ss);
   461 fun sect ss = Scan.first (map Scan.lift ss);
   462 fun thms ss = Scan.unless (sect ss) Attrib.local_thms;
   462 fun thms ss = Scan.unless (sect ss) Attrib.local_thms;
   463 fun thmss ss = Scan.repeat (thms ss) >> flat;
   463 fun thmss ss = Scan.repeat (thms ss) >> flat;
   464 
   464 
   465 fun apply (f, att) (ctxt, ths) = Thm.applys_attributes ((f ctxt, ths), [att]);
   465 fun apply (f, att) (ctxt, ths) = Thm.applys_attributes ((f ctxt, ths), [att]);
   466 
   466