src/HOL/BNF/Tools/bnf_fp_rec_sugar_util.ML
changeset 53329 c31c0c311cf0
parent 53303 ae49b835ca01
child 53411 ab4edf89992f
--- a/src/HOL/BNF/Tools/bnf_fp_rec_sugar_util.ML	Fri Aug 30 14:07:49 2013 +0200
+++ b/src/HOL/BNF/Tools/bnf_fp_rec_sugar_util.ML	Fri Aug 30 14:17:19 2013 +0200
@@ -35,7 +35,7 @@
 
   type rec_spec =
     {recx: term,
-     nested_map_id's: thm list,
+     nested_map_idents: thm list,
      nested_map_comps: thm list,
      ctr_specs: rec_ctr_spec list}
 
@@ -94,7 +94,7 @@
 
 type rec_spec =
   {recx: term,
-   nested_map_id's: thm list,
+   nested_map_idents: thm list,
    nested_map_comps: thm list,
    ctr_specs: rec_ctr_spec list};
 
@@ -336,7 +336,7 @@
 
     fun mk_spec {T, index, ctr_sugars, co_iterss = iterss, co_iter_thmsss = iter_thmsss, ...} =
       {recx = mk_co_iter thy Least_FP (substAT T) perm_Cs' (co_rec_of (nth iterss index)),
-       nested_map_id's = map (unfold_thms lthy [id_def] o map_id0_of_bnf) nested_bnfs,
+       nested_map_idents = map (unfold_thms lthy [id_def] o map_id0_of_bnf) nested_bnfs,
        nested_map_comps = map map_comp_of_bnf nested_bnfs,
        ctr_specs = mk_ctr_specs index ctr_sugars iter_thmsss};
   in