# HG changeset patch # User traytel # Date 1378998816 -7200 # Node ID f9456284048f48b0ce2d2bd6f2c73194718662d0 # Parent 7f84e5e7a49b71e76bf2c45d2fc78ed858351d1d conceal low-level noted facts (+ FIXME to get rid of the notes altogether eventually) diff -r 7f84e5e7a49b -r f9456284048f src/HOL/BNF/Tools/bnf_gfp.ML --- a/src/HOL/BNF/Tools/bnf_gfp.ML Thu Sep 12 16:58:22 2013 +0200 +++ b/src/HOL/BNF/Tools/bnf_gfp.ML Thu Sep 12 17:13:36 2013 +0200 @@ -2889,7 +2889,11 @@ |> maps (fn (thmN, thmss) => map2 (fn b => fn thms => ((Binding.qualify true (Binding.name_of b) (Binding.name thmN), []), [(thms, [])])) - bs thmss) + bs thmss); + + (*FIXME: once the package exports all the necessary high-level characteristic theorems, + those should not only be concealed but rather not noted at all*) + val maybe_conceal_notes = note_all = false ? map (apfst (apfst Binding.conceal)); in timer; ({Ts = Ts, bnfs = Jbnfs, ctors = ctors, dtors = dtors, @@ -2902,7 +2906,7 @@ xtor_co_iter_thmss = transpose [dtor_unfold_thms, dtor_corec_thms], xtor_co_iter_o_map_thmss = transpose [dtor_unfold_o_map_thms, dtor_corec_o_map_thms], rel_xtor_co_induct_thm = Jrel_coinduct_thm}, - lthy |> Local_Theory.notes (common_notes @ notes @ Jbnf_notes) |> snd) + lthy |> Local_Theory.notes (maybe_conceal_notes (common_notes @ notes @ Jbnf_notes)) |> snd) end; val _ = diff -r 7f84e5e7a49b -r f9456284048f src/HOL/BNF/Tools/bnf_lfp.ML --- a/src/HOL/BNF/Tools/bnf_lfp.ML Thu Sep 12 16:58:22 2013 +0200 +++ b/src/HOL/BNF/Tools/bnf_lfp.ML Thu Sep 12 17:13:36 2013 +0200 @@ -1865,7 +1865,11 @@ |> maps (fn (thmN, thmss) => map2 (fn b => fn thms => ((Binding.qualify true (Binding.name_of b) (Binding.name thmN), []), [(thms, [])])) - bs thmss) + bs thmss); + + (*FIXME: once the package exports all the necessary high-level characteristic theorems, + those should not only be concealed but rather not noted at all*) + val maybe_conceal_notes = note_all = false ? map (apfst (apfst Binding.conceal)); in timer; ({Ts = Ts, bnfs = Ibnfs, ctors = ctors, dtors = dtors, xtor_co_iterss = transpose [folds, recs], @@ -1876,7 +1880,7 @@ xtor_co_iter_thmss = transpose [ctor_fold_thms, ctor_rec_thms], xtor_co_iter_o_map_thmss = transpose [ctor_fold_o_map_thms, ctor_rec_o_map_thms], rel_xtor_co_induct_thm = Irel_induct_thm}, - lthy |> Local_Theory.notes (common_notes @ notes @ Ibnf_notes) |> snd) + lthy |> Local_Theory.notes (maybe_conceal_notes (common_notes @ notes @ Ibnf_notes)) |> snd) end; val _ =