src/HOL/Nominal/nominal_primrec.ML
changeset 32194 966e166d039d
parent 31938 f193d95b4632
child 32196 bda40fb76a65
equal deleted inserted replaced
32193:c314b4836031 32194:966e166d039d
   378            |> snd
   378            |> snd
   379          end)
   379          end)
   380       [goals] |>
   380       [goals] |>
   381     Proof.apply (Method.Basic (fn _ => RAW_METHOD (fn _ =>
   381     Proof.apply (Method.Basic (fn _ => RAW_METHOD (fn _ =>
   382       rewrite_goals_tac defs_thms THEN
   382       rewrite_goals_tac defs_thms THEN
   383       compose_tac (false, rule, length rule_prems) 1), Position.none)) |>
   383       compose_tac (false, rule, length rule_prems) 1)) |>
   384     Seq.hd
   384     Seq.hd
   385   end;
   385   end;
   386 
   386 
   387 in
   387 in
   388 
   388