src/HOL/Tools/function_package/fundef_prep.ML
changeset 21793 74409847e349
parent 21746 9d0652354513
child 22130 0906fd95e0b5
equal deleted inserted replaced
21792:266a1056a2a3 21793:74409847e349
   505       val trees = PROFILE "inst_trees" (map (FundefCtxTree.inst_tree (ProofContext.theory_of lthy) fvar f)) trees
   505       val trees = PROFILE "inst_trees" (map (FundefCtxTree.inst_tree (ProofContext.theory_of lthy) fvar f)) trees
   506 
   506 
   507       val ((R, RIntro_thmss, R_elim), lthy) = 
   507       val ((R, RIntro_thmss, R_elim), lthy) = 
   508           PROFILE "def_rel" (define_recursion_relation (rel_name defname) domT ranT fvar f abstract_qglrs clauses RCss) lthy
   508           PROFILE "def_rel" (define_recursion_relation (rel_name defname) domT ranT fvar f abstract_qglrs clauses RCss) lthy
   509 
   509 
   510       val lthy = PROFILE "abbrev"
   510       val (_, lthy) = PROFILE "abbrev"
   511         (LocalTheory.abbrev Syntax.default_mode ((defname ^ "_dom", NoSyn), mk_acc domT R)) lthy
   511         (LocalTheory.abbrev Syntax.default_mode ((defname ^ "_dom", NoSyn), mk_acc domT R)) lthy
   512 
   512 
   513       val newthy = ProofContext.theory_of lthy
   513       val newthy = ProofContext.theory_of lthy
   514       val clauses = map (transfer_clause_ctx newthy) clauses
   514       val clauses = map (transfer_clause_ctx newthy) clauses
   515 
   515