src/ZF/UNITY/SubstAx.thy
changeset 74563 042041c0ebeb
parent 69593 3dda49e08b9d
child 76213 e44d86131648
equal deleted inserted replaced
74562:8403bd51f8b1 74563:042041c0ebeb
   371                       ALLGOALS (clarify_tac ctxt),
   371                       ALLGOALS (clarify_tac ctxt),
   372           ALLGOALS (asm_lr_simp_tac ctxt)]);
   372           ALLGOALS (asm_lr_simp_tac ctxt)]);
   373 \<close>
   373 \<close>
   374 
   374 
   375 method_setup ensures = \<open>
   375 method_setup ensures = \<open>
   376     Args.goal_spec -- Scan.lift Args.embedded_inner_syntax >>
   376     Args.goal_spec -- Scan.lift Parse.embedded_inner_syntax >>
   377     (fn (quant, s) => fn ctxt => SIMPLE_METHOD'' quant (ensures_tac ctxt s))
   377     (fn (quant, s) => fn ctxt => SIMPLE_METHOD'' quant (ensures_tac ctxt s))
   378 \<close> "for proving progress properties"
   378 \<close> "for proving progress properties"
   379 
   379 
   380 end
   380 end