src/HOL/Tools/BNF/bnf_gfp_rec_sugar.ML
changeset 61841 4d3527b94f2a
parent 61760 1647bb489522
child 62318 b42858e540bb
equal deleted inserted replaced
61840:a3793600cb93 61841:4d3527b94f2a
  1577   end;
  1577   end;
  1578 
  1578 
  1579 val primcorecursive_cmd = (fn (goalss, after_qed, lthy) =>
  1579 val primcorecursive_cmd = (fn (goalss, after_qed, lthy) =>
  1580   lthy
  1580   lthy
  1581   |> Proof.theorem NONE after_qed goalss
  1581   |> Proof.theorem NONE after_qed goalss
  1582   |> Proof.refine (Method.primitive_text (K I))
  1582   |> Proof.refine_singleton (Method.primitive_text (K I))) ooo primcorec_ursive_cmd false;
  1583   |> Seq.hd) ooo primcorec_ursive_cmd false;
       
  1584 
  1583 
  1585 val primcorec_cmd = (fn (goalss, after_qed, lthy) =>
  1584 val primcorec_cmd = (fn (goalss, after_qed, lthy) =>
  1586     lthy |> after_qed (map (fn [] => [] | _ => use_primcorecursive ()) goalss)) ooo
  1585     lthy |> after_qed (map (fn [] => [] | _ => use_primcorecursive ()) goalss)) ooo
  1587   primcorec_ursive_cmd true;
  1586   primcorec_ursive_cmd true;
  1588 
  1587