src/HOL/Tools/Function/function.ML
changeset 61841 4d3527b94f2a
parent 61112 e966c311e9a7
child 62774 cfcb20bbdbd8
equal deleted inserted replaced
61840:a3793600cb93 61841:4d3527b94f2a
   169     val ((goal_state, afterqed), lthy') =
   169     val ((goal_state, afterqed), lthy') =
   170       prepare_function do_print prep default_constraint fixspec eqns config lthy
   170       prepare_function do_print prep default_constraint fixspec eqns config lthy
   171   in
   171   in
   172     lthy'
   172     lthy'
   173     |> Proof.theorem NONE (snd oo afterqed) [[(Logic.unprotect (Thm.concl_of goal_state), [])]]
   173     |> Proof.theorem NONE (snd oo afterqed) [[(Logic.unprotect (Thm.concl_of goal_state), [])]]
   174     |> Proof.refine (Method.primitive_text (K (K goal_state))) |> Seq.hd
   174     |> Proof.refine_singleton (Method.primitive_text (K (K goal_state)))
   175   end
   175   end
   176 
   176 
   177 val function =
   177 val function =
   178   gen_function false Specification.check_spec default_constraint_any
   178   gen_function false Specification.check_spec default_constraint_any
   179 fun function_cmd a b c int =
   179 fun function_cmd a b c int =