src/HOL/Tools/Function/function.ML
changeset 59582 0fbed69ff081
parent 59159 9312710451f5
child 59859 f9d1442c70f3
equal deleted inserted replaced
59580:cbc38731d42f 59582:0fbed69ff081
   164   let
   164   let
   165     val ((goal_state, afterqed), lthy') =
   165     val ((goal_state, afterqed), lthy') =
   166       prepare_function do_print prep default_constraint fixspec eqns config lthy
   166       prepare_function do_print prep default_constraint fixspec eqns config lthy
   167   in
   167   in
   168     lthy'
   168     lthy'
   169     |> Proof.theorem NONE (snd oo afterqed) [[(Logic.unprotect (concl_of goal_state), [])]]
   169     |> Proof.theorem NONE (snd oo afterqed) [[(Logic.unprotect (Thm.concl_of goal_state), [])]]
   170     |> Proof.refine (Method.primitive_text (K (K goal_state))) |> Seq.hd
   170     |> Proof.refine (Method.primitive_text (K (K goal_state))) |> Seq.hd
   171   end
   171   end
   172 
   172 
   173 val function =
   173 val function =
   174   gen_function false Specification.check_spec (Type_Infer.anyT @{sort type})
   174   gen_function false Specification.check_spec (Type_Infer.anyT @{sort type})