src/HOL/Tools/BNF/bnf_comp.ML
author wenzelm
Mon, 02 Mar 2020 13:57:03 +0100
changeset 71506 4197e30040f3
parent 71261 4765fec43414
child 74575 ccf599864beb
permissions -rw-r--r--
VSCode extension for official Isabelle release;
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
55061
a0adf838e2d1 adjusted comments
blanchet
parents: 55060
diff changeset
     1
(*  Title:      HOL/Tools/BNF/bnf_comp.ML
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
     2
    Author:     Dmitriy Traytel, TU Muenchen
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
     3
    Author:     Jasmin Blanchette, TU Muenchen
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
     4
    Copyright   2012
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
     5
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
     6
Composition of bounded natural functors.
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
     7
*)
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
     8
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
     9
signature BNF_COMP =
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
    10
sig
59994
19e5f5ac7b59 renamed misleading option
blanchet
parents: 59957
diff changeset
    11
  val typedef_threshold: int Config.T
63800
6489d85ecc98 extended ML signature
blanchet
parents: 62684
diff changeset
    12
  val with_typedef_threshold: int -> (Proof.context -> Proof.context) -> Proof.context ->
6489d85ecc98 extended ML signature
blanchet
parents: 62684
diff changeset
    13
    Proof.context
6489d85ecc98 extended ML signature
blanchet
parents: 62684
diff changeset
    14
  val with_typedef_threshold_yield: int -> (Proof.context -> 'a * Proof.context) -> Proof.context ->
6489d85ecc98 extended ML signature
blanchet
parents: 62684
diff changeset
    15
    'a * Proof.context
59710
4aa63424ba89 inlining threshold
blanchet
parents: 59131
diff changeset
    16
51837
087498724486 lowercase type constructor, for consistency (cf. fp_result not FP_result nor FP_Result)
blanchet
parents: 51782
diff changeset
    17
  val ID_bnf: BNF_Def.bnf
087498724486 lowercase type constructor, for consistency (cf. fp_result not FP_result nor FP_Result)
blanchet
parents: 51782
diff changeset
    18
  val DEADID_bnf: BNF_Def.bnf
49585
5c4a12550491 generate high-level "maps", "sets", and "rels" properties
blanchet
parents: 49538
diff changeset
    19
55706
064c7c249f55 added BNF cache (within one definition)
blanchet
parents: 55705
diff changeset
    20
  type comp_cache
65436
1fd2dca8eb60 tuned signature
traytel
parents: 63837
diff changeset
    21
  type unfold_set =
1fd2dca8eb60 tuned signature
traytel
parents: 63837
diff changeset
    22
    {map_unfolds: thm list,
1fd2dca8eb60 tuned signature
traytel
parents: 63837
diff changeset
    23
     set_unfoldss: thm list list,
71261
4765fec43414 unfold intermediate (internal) pred definitions
traytel
parents: 70494
diff changeset
    24
     rel_unfolds: thm list,
4765fec43414 unfold intermediate (internal) pred definitions
traytel
parents: 70494
diff changeset
    25
     pred_unfolds: thm list}
55706
064c7c249f55 added BNF cache (within one definition)
blanchet
parents: 55705
diff changeset
    26
064c7c249f55 added BNF cache (within one definition)
blanchet
parents: 55705
diff changeset
    27
  val empty_comp_cache: comp_cache
49502
92a7c1842c78 tuned a few ML names
blanchet
parents: 49463
diff changeset
    28
  val empty_unfolds: unfold_set
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
    29
53222
8b159677efb5 better error message
blanchet
parents: 53040
diff changeset
    30
  exception BAD_DEAD of typ * typ
8b159677efb5 better error message
blanchet
parents: 53040
diff changeset
    31
62621
a1e73be79c0b generalized ML function
blanchet
parents: 62324
diff changeset
    32
  val bnf_of_typ: bool -> BNF_Def.inline_policy -> (binding -> binding) ->
55703
a21069381ba5 optimization of 'bnf_of_typ' if all variables are dead
blanchet
parents: 55480
diff changeset
    33
    ((string * sort) list list -> (string * sort) list) -> (string * sort) list ->
55904
0ef30d52c5e4 more caching in composition pipeline
blanchet
parents: 55900
diff changeset
    34
    (string * sort) list -> typ -> (comp_cache * unfold_set) * local_theory ->
0ef30d52c5e4 more caching in composition pipeline
blanchet
parents: 55900
diff changeset
    35
    (BNF_Def.bnf * (typ list * typ list)) * ((comp_cache * unfold_set) * local_theory)
49014
332e5e661675 have "bnf_of_typ" command seal the BNF
blanchet
parents: 48975
diff changeset
    36
  val default_comp_sort: (string * sort) list list -> (string * sort) list
59725
e5dc7e7744f0 export more ML functions
blanchet
parents: 59710
diff changeset
    37
  val clean_compose_bnf: BNF_Def.inline_policy -> (binding -> binding) -> binding -> BNF_Def.bnf ->
e5dc7e7744f0 export more ML functions
blanchet
parents: 59710
diff changeset
    38
    BNF_Def.bnf list -> unfold_set * local_theory -> BNF_Def.bnf * (unfold_set * local_theory)
e5dc7e7744f0 export more ML functions
blanchet
parents: 59710
diff changeset
    39
  val kill_bnf: (binding -> binding) -> int -> BNF_Def.bnf ->
e5dc7e7744f0 export more ML functions
blanchet
parents: 59710
diff changeset
    40
    (comp_cache * unfold_set) * local_theory ->
e5dc7e7744f0 export more ML functions
blanchet
parents: 59710
diff changeset
    41
    BNF_Def.bnf * ((comp_cache * unfold_set) * local_theory)
e5dc7e7744f0 export more ML functions
blanchet
parents: 59710
diff changeset
    42
  val lift_bnf: (binding -> binding) -> int -> BNF_Def.bnf ->
e5dc7e7744f0 export more ML functions
blanchet
parents: 59710
diff changeset
    43
    (comp_cache * unfold_set) * local_theory ->
e5dc7e7744f0 export more ML functions
blanchet
parents: 59710
diff changeset
    44
    BNF_Def.bnf * ((comp_cache * unfold_set) * local_theory)
e5dc7e7744f0 export more ML functions
blanchet
parents: 59710
diff changeset
    45
  val permute_bnf: (binding -> binding) -> int list -> int list -> BNF_Def.bnf ->
e5dc7e7744f0 export more ML functions
blanchet
parents: 59710
diff changeset
    46
    (comp_cache * unfold_set) * local_theory ->
e5dc7e7744f0 export more ML functions
blanchet
parents: 59710
diff changeset
    47
    BNF_Def.bnf * ((comp_cache * unfold_set) * local_theory)
e5dc7e7744f0 export more ML functions
blanchet
parents: 59710
diff changeset
    48
  val permute_and_kill_bnf: (binding -> binding) -> int -> int list -> int list -> BNF_Def.bnf ->
e5dc7e7744f0 export more ML functions
blanchet
parents: 59710
diff changeset
    49
    (comp_cache * unfold_set) * local_theory ->
e5dc7e7744f0 export more ML functions
blanchet
parents: 59710
diff changeset
    50
    BNF_Def.bnf * ((comp_cache * unfold_set) * local_theory)
e5dc7e7744f0 export more ML functions
blanchet
parents: 59710
diff changeset
    51
  val lift_and_permute_bnf: (binding -> binding) -> int -> int list -> int list -> BNF_Def.bnf ->
e5dc7e7744f0 export more ML functions
blanchet
parents: 59710
diff changeset
    52
    (comp_cache * unfold_set) * local_theory ->
e5dc7e7744f0 export more ML functions
blanchet
parents: 59710
diff changeset
    53
    BNF_Def.bnf * ((comp_cache * unfold_set) * local_theory)
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
    54
  val normalize_bnfs: (int -> binding -> binding) -> ''a list list -> ''a list ->
55904
0ef30d52c5e4 more caching in composition pipeline
blanchet
parents: 55900
diff changeset
    55
    (''a list list -> ''a list) -> BNF_Def.bnf list -> (comp_cache * unfold_set) * local_theory ->
0ef30d52c5e4 more caching in composition pipeline
blanchet
parents: 55900
diff changeset
    56
    (int list list * ''a list) * (BNF_Def.bnf list * ((comp_cache * unfold_set) * local_theory))
59725
e5dc7e7744f0 export more ML functions
blanchet
parents: 59710
diff changeset
    57
  val compose_bnf: BNF_Def.inline_policy -> (int -> binding -> binding) ->
e5dc7e7744f0 export more ML functions
blanchet
parents: 59710
diff changeset
    58
    ((string * sort) list list -> (string * sort) list) -> BNF_Def.bnf -> BNF_Def.bnf list ->
e5dc7e7744f0 export more ML functions
blanchet
parents: 59710
diff changeset
    59
    typ list -> typ list list -> typ list list -> (comp_cache * unfold_set) * local_theory ->
e5dc7e7744f0 export more ML functions
blanchet
parents: 59710
diff changeset
    60
    (BNF_Def.bnf * (typ list * typ list)) * ((comp_cache * unfold_set) * local_theory)
55803
74d3fe9031d8 joint work with blanchet: intermediate typedef for the input to fp-operations
traytel
parents: 55707
diff changeset
    61
  type absT_info =
74d3fe9031d8 joint work with blanchet: intermediate typedef for the input to fp-operations
traytel
parents: 55707
diff changeset
    62
    {absT: typ,
74d3fe9031d8 joint work with blanchet: intermediate typedef for the input to fp-operations
traytel
parents: 55707
diff changeset
    63
     repT: typ,
74d3fe9031d8 joint work with blanchet: intermediate typedef for the input to fp-operations
traytel
parents: 55707
diff changeset
    64
     abs: term,
74d3fe9031d8 joint work with blanchet: intermediate typedef for the input to fp-operations
traytel
parents: 55707
diff changeset
    65
     rep: term,
74d3fe9031d8 joint work with blanchet: intermediate typedef for the input to fp-operations
traytel
parents: 55707
diff changeset
    66
     abs_inject: thm,
74d3fe9031d8 joint work with blanchet: intermediate typedef for the input to fp-operations
traytel
parents: 55707
diff changeset
    67
     abs_inverse: thm,
74d3fe9031d8 joint work with blanchet: intermediate typedef for the input to fp-operations
traytel
parents: 55707
diff changeset
    68
     type_definition: thm}
74d3fe9031d8 joint work with blanchet: intermediate typedef for the input to fp-operations
traytel
parents: 55707
diff changeset
    69
74d3fe9031d8 joint work with blanchet: intermediate typedef for the input to fp-operations
traytel
parents: 55707
diff changeset
    70
  val morph_absT_info: morphism -> absT_info -> absT_info
74d3fe9031d8 joint work with blanchet: intermediate typedef for the input to fp-operations
traytel
parents: 55707
diff changeset
    71
  val mk_absT: theory -> typ -> typ -> typ -> typ
74d3fe9031d8 joint work with blanchet: intermediate typedef for the input to fp-operations
traytel
parents: 55707
diff changeset
    72
  val mk_repT: typ -> typ -> typ -> typ
74d3fe9031d8 joint work with blanchet: intermediate typedef for the input to fp-operations
traytel
parents: 55707
diff changeset
    73
  val mk_abs: typ -> term -> term
74d3fe9031d8 joint work with blanchet: intermediate typedef for the input to fp-operations
traytel
parents: 55707
diff changeset
    74
  val mk_rep: typ -> term -> term
63837
fdf90aa59868 provide a mechanism for ensuring dead type variables occur in typedef if desired
blanchet
parents: 63836
diff changeset
    75
  val seal_bnf: (binding -> binding) -> unfold_set -> binding -> bool -> typ list -> typ list ->
fdf90aa59868 provide a mechanism for ensuring dead type variables occur in typedef if desired
blanchet
parents: 63836
diff changeset
    76
    BNF_Def.bnf -> local_theory -> (BNF_Def.bnf * (typ list * absT_info)) * local_theory
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
    77
end;
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
    78
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
    79
structure BNF_Comp : BNF_COMP =
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
    80
struct
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
    81
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
    82
open BNF_Def
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
    83
open BNF_Util
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
    84
open BNF_Tactics
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
    85
open BNF_Comp_Tactics
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
    86
69593
3dda49e08b9d isabelle update -u control_cartouches;
wenzelm
parents: 68960
diff changeset
    87
val typedef_threshold = Attrib.setup_config_int \<^binding>\<open>bnf_typedef_threshold\<close> (K 6);
59710
4aa63424ba89 inlining threshold
blanchet
parents: 59131
diff changeset
    88
63800
6489d85ecc98 extended ML signature
blanchet
parents: 62684
diff changeset
    89
fun with_typedef_threshold threshold f lthy =
6489d85ecc98 extended ML signature
blanchet
parents: 62684
diff changeset
    90
  lthy
6489d85ecc98 extended ML signature
blanchet
parents: 62684
diff changeset
    91
  |> Config.put typedef_threshold threshold
6489d85ecc98 extended ML signature
blanchet
parents: 62684
diff changeset
    92
  |> f
6489d85ecc98 extended ML signature
blanchet
parents: 62684
diff changeset
    93
  |> Config.put typedef_threshold (Config.get lthy typedef_threshold);
6489d85ecc98 extended ML signature
blanchet
parents: 62684
diff changeset
    94
6489d85ecc98 extended ML signature
blanchet
parents: 62684
diff changeset
    95
fun with_typedef_threshold_yield threshold f lthy =
6489d85ecc98 extended ML signature
blanchet
parents: 62684
diff changeset
    96
  lthy
6489d85ecc98 extended ML signature
blanchet
parents: 62684
diff changeset
    97
  |> Config.put typedef_threshold threshold
6489d85ecc98 extended ML signature
blanchet
parents: 62684
diff changeset
    98
  |> f
6489d85ecc98 extended ML signature
blanchet
parents: 62684
diff changeset
    99
  ||> Config.put typedef_threshold (Config.get lthy typedef_threshold);
6489d85ecc98 extended ML signature
blanchet
parents: 62684
diff changeset
   100
69593
3dda49e08b9d isabelle update -u control_cartouches;
wenzelm
parents: 68960
diff changeset
   101
val ID_bnf = the (bnf_of \<^context> "BNF_Composition.ID");
3dda49e08b9d isabelle update -u control_cartouches;
wenzelm
parents: 68960
diff changeset
   102
val DEADID_bnf = the (bnf_of \<^context> "BNF_Composition.DEADID");
49585
5c4a12550491 generate high-level "maps", "sets", and "rels" properties
blanchet
parents: 49538
diff changeset
   103
55706
064c7c249f55 added BNF cache (within one definition)
blanchet
parents: 55705
diff changeset
   104
type comp_cache = (bnf * (typ list * typ list)) Typtab.table;
064c7c249f55 added BNF cache (within one definition)
blanchet
parents: 55705
diff changeset
   105
55904
0ef30d52c5e4 more caching in composition pipeline
blanchet
parents: 55900
diff changeset
   106
fun key_of_types s Ts = Type (s, Ts);
0ef30d52c5e4 more caching in composition pipeline
blanchet
parents: 55900
diff changeset
   107
fun key_of_typess s = key_of_types s o map (key_of_types "");
0ef30d52c5e4 more caching in composition pipeline
blanchet
parents: 55900
diff changeset
   108
fun typ_of_int n = Type (string_of_int n, []);
0ef30d52c5e4 more caching in composition pipeline
blanchet
parents: 55900
diff changeset
   109
fun typ_of_bnf bnf =
0ef30d52c5e4 more caching in composition pipeline
blanchet
parents: 55900
diff changeset
   110
  key_of_typess "" [[T_of_bnf bnf], lives_of_bnf bnf, sort Term_Ord.typ_ord (deads_of_bnf bnf)];
0ef30d52c5e4 more caching in composition pipeline
blanchet
parents: 55900
diff changeset
   111
0ef30d52c5e4 more caching in composition pipeline
blanchet
parents: 55900
diff changeset
   112
fun key_of_kill n bnf = key_of_types "k" [typ_of_int n, typ_of_bnf bnf];
0ef30d52c5e4 more caching in composition pipeline
blanchet
parents: 55900
diff changeset
   113
fun key_of_lift n bnf = key_of_types "l" [typ_of_int n, typ_of_bnf bnf];
0ef30d52c5e4 more caching in composition pipeline
blanchet
parents: 55900
diff changeset
   114
fun key_of_permute src dest bnf =
0ef30d52c5e4 more caching in composition pipeline
blanchet
parents: 55900
diff changeset
   115
  key_of_types "p" (map typ_of_int src @ map typ_of_int dest @ [typ_of_bnf bnf]);
0ef30d52c5e4 more caching in composition pipeline
blanchet
parents: 55900
diff changeset
   116
fun key_of_compose oDs Dss Ass outer inners =
0ef30d52c5e4 more caching in composition pipeline
blanchet
parents: 55900
diff changeset
   117
  key_of_types "c" (map (key_of_typess "") [[oDs], Dss, Ass, [map typ_of_bnf (outer :: inners)]]);
0ef30d52c5e4 more caching in composition pipeline
blanchet
parents: 55900
diff changeset
   118
0ef30d52c5e4 more caching in composition pipeline
blanchet
parents: 55900
diff changeset
   119
fun cache_comp_simple key cache (bnf, (unfold_set, lthy)) =
0ef30d52c5e4 more caching in composition pipeline
blanchet
parents: 55900
diff changeset
   120
  (bnf, ((Typtab.update (key, (bnf, ([], []))) cache, unfold_set), lthy));
0ef30d52c5e4 more caching in composition pipeline
blanchet
parents: 55900
diff changeset
   121
0ef30d52c5e4 more caching in composition pipeline
blanchet
parents: 55900
diff changeset
   122
fun cache_comp key (bnf_Ds_As, ((cache, unfold_set), lthy)) =
0ef30d52c5e4 more caching in composition pipeline
blanchet
parents: 55900
diff changeset
   123
  (bnf_Ds_As, ((Typtab.update (key, bnf_Ds_As) cache, unfold_set), lthy));
0ef30d52c5e4 more caching in composition pipeline
blanchet
parents: 55900
diff changeset
   124
49502
92a7c1842c78 tuned a few ML names
blanchet
parents: 49463
diff changeset
   125
type unfold_set = {
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   126
  map_unfolds: thm list,
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   127
  set_unfoldss: thm list list,
71261
4765fec43414 unfold intermediate (internal) pred definitions
traytel
parents: 70494
diff changeset
   128
  rel_unfolds: thm list,
4765fec43414 unfold intermediate (internal) pred definitions
traytel
parents: 70494
diff changeset
   129
  pred_unfolds: thm list
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   130
};
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   131
55706
064c7c249f55 added BNF cache (within one definition)
blanchet
parents: 55705
diff changeset
   132
val empty_comp_cache = Typtab.empty;
71261
4765fec43414 unfold intermediate (internal) pred definitions
traytel
parents: 70494
diff changeset
   133
val empty_unfolds = {map_unfolds = [], set_unfoldss = [], rel_unfolds = [], pred_unfolds = []};
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   134
49503
dbbde075a42e simplified code
blanchet
parents: 49502
diff changeset
   135
fun add_to_thms thms new = thms |> not (Thm.is_reflexive new) ? insert Thm.eq_thm new;
dbbde075a42e simplified code
blanchet
parents: 49502
diff changeset
   136
fun adds_to_thms thms news = insert (eq_set Thm.eq_thm) (no_reflexive news) thms;
dbbde075a42e simplified code
blanchet
parents: 49502
diff changeset
   137
71261
4765fec43414 unfold intermediate (internal) pred definitions
traytel
parents: 70494
diff changeset
   138
fun add_to_unfolds map sets rel pred
4765fec43414 unfold intermediate (internal) pred definitions
traytel
parents: 70494
diff changeset
   139
  {map_unfolds, set_unfoldss, rel_unfolds, pred_unfolds} =
49503
dbbde075a42e simplified code
blanchet
parents: 49502
diff changeset
   140
  {map_unfolds = add_to_thms map_unfolds map,
dbbde075a42e simplified code
blanchet
parents: 49502
diff changeset
   141
    set_unfoldss = adds_to_thms set_unfoldss sets,
71261
4765fec43414 unfold intermediate (internal) pred definitions
traytel
parents: 70494
diff changeset
   142
    rel_unfolds = add_to_thms rel_unfolds rel,
4765fec43414 unfold intermediate (internal) pred definitions
traytel
parents: 70494
diff changeset
   143
    pred_unfolds = add_to_thms pred_unfolds pred};
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   144
49503
dbbde075a42e simplified code
blanchet
parents: 49502
diff changeset
   145
fun add_bnf_to_unfolds bnf =
71261
4765fec43414 unfold intermediate (internal) pred definitions
traytel
parents: 70494
diff changeset
   146
  add_to_unfolds (map_def_of_bnf bnf) (set_defs_of_bnf bnf) (rel_def_of_bnf bnf) (pred_def_of_bnf bnf);
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   147
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   148
val bdTN = "bdT";
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   149
49425
f27f83f71e94 cleaned up internal naming scheme for bnfs
traytel
parents: 49304
diff changeset
   150
fun mk_killN n = "_kill" ^ string_of_int n;
f27f83f71e94 cleaned up internal naming scheme for bnfs
traytel
parents: 49304
diff changeset
   151
fun mk_liftN n = "_lift" ^ string_of_int n;
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   152
fun mk_permuteN src dest =
49425
f27f83f71e94 cleaned up internal naming scheme for bnfs
traytel
parents: 49304
diff changeset
   153
  "_permute_" ^ implode (map string_of_int src) ^ "_" ^ implode (map string_of_int dest);
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   154
55935
8f20d09d294e move special BNFs used for composition only to BNF_Comp;
traytel
parents: 55930
diff changeset
   155
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   156
(*copied from Envir.expand_term_free*)
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   157
fun expand_term_const defs =
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   158
  let
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   159
    val eqs = map ((fn ((x, U), u) => (x, (U, u))) o apfst dest_Const) defs;
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   160
    val get = fn Const (x, _) => AList.lookup (op =) eqs x | _ => NONE;
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   161
  in Envir.expand_term get end;
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   162
58181
6d527272f7b2 renamed internal constant
blanchet
parents: 58128
diff changeset
   163
val id_bnf_def = @{thm id_bnf_def};
6d527272f7b2 renamed internal constant
blanchet
parents: 58128
diff changeset
   164
val expand_id_bnf_def = expand_term_const [Thm.prop_of id_bnf_def |> Logic.dest_equals];
55937
traytel
parents: 55935
diff changeset
   165
69593
3dda49e08b9d isabelle update -u control_cartouches;
wenzelm
parents: 68960
diff changeset
   166
fun is_sum_prod_natLeq (Const (\<^const_name>\<open>csum\<close>, _) $ t $ u) = forall is_sum_prod_natLeq [t, u]
3dda49e08b9d isabelle update -u control_cartouches;
wenzelm
parents: 68960
diff changeset
   167
  | is_sum_prod_natLeq (Const (\<^const_name>\<open>cprod\<close>, _) $ t $ u) = forall is_sum_prod_natLeq [t, u]
3dda49e08b9d isabelle update -u control_cartouches;
wenzelm
parents: 68960
diff changeset
   168
  | is_sum_prod_natLeq t = t aconv \<^term>\<open>natLeq\<close>;
55851
3d40cf74726c optimize cardinal bounds involving natLeq (omega)
blanchet
parents: 55803
diff changeset
   169
49502
92a7c1842c78 tuned a few ML names
blanchet
parents: 49463
diff changeset
   170
fun clean_compose_bnf const_policy qualify b outer inners (unfold_set, lthy) =
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   171
  let
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   172
    val olive = live_of_bnf outer;
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   173
    val onwits = nwits_of_bnf outer;
60207
81a0900f0ddc allow sorts on dead variables in BNFs
blanchet
parents: 59994
diff changeset
   174
    val odeads = deads_of_bnf outer;
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   175
    val inner = hd inners;
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   176
    val ilive = live_of_bnf inner;
60207
81a0900f0ddc allow sorts on dead variables in BNFs
blanchet
parents: 59994
diff changeset
   177
    val ideadss = map deads_of_bnf inners;
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   178
    val inwitss = map nwits_of_bnf inners;
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   179
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   180
    (* TODO: check olive = length inners > 0,
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   181
                   forall inner from inners. ilive = live,
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   182
                   forall inner from inners. idead = dead  *)
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   183
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   184
    val (oDs, lthy1) = apfst (map TFree)
60207
81a0900f0ddc allow sorts on dead variables in BNFs
blanchet
parents: 59994
diff changeset
   185
      (Variable.invent_types (map Type.sort_of_atyp odeads) lthy);
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   186
    val (Dss, lthy2) = apfst (map (map TFree))
60207
81a0900f0ddc allow sorts on dead variables in BNFs
blanchet
parents: 59994
diff changeset
   187
      (fold_map Variable.invent_types (map (map Type.sort_of_atyp) ideadss) lthy1);
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   188
    val (Ass, lthy3) = apfst (replicate ilive o map TFree)
69593
3dda49e08b9d isabelle update -u control_cartouches;
wenzelm
parents: 68960
diff changeset
   189
      (Variable.invent_types (replicate ilive \<^sort>\<open>type\<close>) lthy2);
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   190
    val As = if ilive > 0 then hd Ass else [];
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   191
    val Ass_repl = replicate olive As;
55906
abf91ebd0820 simplify sets in BNF composition
blanchet
parents: 55904
diff changeset
   192
    val (Bs, names_lthy) = apfst (map TFree)
69593
3dda49e08b9d isabelle update -u control_cartouches;
wenzelm
parents: 68960
diff changeset
   193
      (Variable.invent_types (replicate ilive \<^sort>\<open>type\<close>) lthy3);
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   194
    val Bss_repl = replicate olive Bs;
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   195
62324
ae44f16dcea5 make predicator a first-class bnf citizen
traytel
parents: 62316
diff changeset
   196
    val (((((fs', Qs'), Ps'), Asets), xs), _) = names_lthy
52923
traytel
parents: 52660
diff changeset
   197
      |> apfst snd o mk_Frees' "f" (map2 (curry op -->) As Bs)
49463
83ac281bcdc2 provide predicator, define relator
blanchet
parents: 49461
diff changeset
   198
      ||>> apfst snd o mk_Frees' "Q" (map2 mk_pred2T As Bs)
62324
ae44f16dcea5 make predicator a first-class bnf citizen
traytel
parents: 62316
diff changeset
   199
      ||>> apfst snd o mk_Frees' "P" (map mk_pred1T As)
49456
fa8302c8dea1 adapted BNF composition to new relator approach
blanchet
parents: 49455
diff changeset
   200
      ||>> mk_Frees "A" (map HOLogic.mk_setT As)
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   201
      ||>> mk_Frees "x" As;
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   202
58634
9f10d82e8188 added parameterized ML antiquotations @{map N}, @{fold N}, @{fold_map N}, @{split_list N};
wenzelm
parents: 58359
diff changeset
   203
    val CAs = @{map 3} mk_T_of_bnf Dss Ass_repl inners;
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   204
    val CCA = mk_T_of_bnf oDs CAs outer;
58634
9f10d82e8188 added parameterized ML antiquotations @{map N}, @{fold N}, @{fold_map N}, @{split_list N};
wenzelm
parents: 58359
diff changeset
   205
    val CBs = @{map 3} mk_T_of_bnf Dss Bss_repl inners;
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   206
    val outer_sets = mk_sets_of_bnf (replicate olive oDs) (replicate olive CAs) outer;
61760
1647bb489522 tuned whitespace
blanchet
parents: 61242
diff changeset
   207
    val inner_setss =
1647bb489522 tuned whitespace
blanchet
parents: 61242
diff changeset
   208
      @{map 3} mk_sets_of_bnf (map (replicate ilive) Dss) (replicate olive Ass) inners;
58634
9f10d82e8188 added parameterized ML antiquotations @{map N}, @{fold N}, @{fold_map N}, @{split_list N};
wenzelm
parents: 58359
diff changeset
   209
    val inner_bds = @{map 3} mk_bd_of_bnf Dss Ass_repl inners;
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   210
    val outer_bd = mk_bd_of_bnf oDs CAs outer;
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   211
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   212
    (*%f1 ... fn. outer.map (inner_1.map f1 ... fn) ... (inner_m.map f1 ... fn)*)
49303
blanchet
parents: 49236
diff changeset
   213
    val mapx = fold_rev Term.abs fs'
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   214
      (Term.list_comb (mk_map_of_bnf oDs CAs CBs outer,
49463
83ac281bcdc2 provide predicator, define relator
blanchet
parents: 49461
diff changeset
   215
        map2 (fn Ds => (fn f => Term.list_comb (f, map Bound (ilive - 1 downto 0))) o
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   216
          mk_map_of_bnf Ds As Bs) Dss inners));
49507
8826d5a4332b renamed "pred" to "rel" (relator)
blanchet
parents: 49506
diff changeset
   217
    (*%Q1 ... Qn. outer.rel (inner_1.rel Q1 ... Qn) ... (inner_m.rel Q1 ... Qn)*)
8826d5a4332b renamed "pred" to "rel" (relator)
blanchet
parents: 49506
diff changeset
   218
    val rel = fold_rev Term.abs Qs'
8826d5a4332b renamed "pred" to "rel" (relator)
blanchet
parents: 49506
diff changeset
   219
      (Term.list_comb (mk_rel_of_bnf oDs CAs CBs outer,
49463
83ac281bcdc2 provide predicator, define relator
blanchet
parents: 49461
diff changeset
   220
        map2 (fn Ds => (fn f => Term.list_comb (f, map Bound (ilive - 1 downto 0))) o
49507
8826d5a4332b renamed "pred" to "rel" (relator)
blanchet
parents: 49506
diff changeset
   221
          mk_rel_of_bnf Ds As Bs) Dss inners));
62324
ae44f16dcea5 make predicator a first-class bnf citizen
traytel
parents: 62316
diff changeset
   222
    (*%P1 ... Pn. outer.pred (inner_1.pred P1 ... Pn) ... (inner_m.pred P1 ... Pn)*)
ae44f16dcea5 make predicator a first-class bnf citizen
traytel
parents: 62316
diff changeset
   223
    val pred = fold_rev Term.abs Ps'
ae44f16dcea5 make predicator a first-class bnf citizen
traytel
parents: 62316
diff changeset
   224
      (Term.list_comb (mk_pred_of_bnf oDs CAs outer,
ae44f16dcea5 make predicator a first-class bnf citizen
traytel
parents: 62316
diff changeset
   225
        map2 (fn Ds => (fn f => Term.list_comb (f, map Bound (ilive - 1 downto 0))) o
ae44f16dcea5 make predicator a first-class bnf citizen
traytel
parents: 62316
diff changeset
   226
          mk_pred_of_bnf Ds As) Dss inners));
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   227
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   228
    (*Union o collect {outer.set_1 ... outer.set_m} o outer.map inner_1.set_i ... inner_m.set_i*)
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   229
    (*Union o collect {image inner_1.set_i o outer.set_1 ... image inner_m.set_i o outer.set_m}*)
49303
blanchet
parents: 49236
diff changeset
   230
    fun mk_set i =
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   231
      let
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   232
        val (setTs, T) = `(replicate olive o HOLogic.mk_setT) (nth As i);
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   233
        val outer_set = mk_collect
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   234
          (mk_sets_of_bnf (replicate olive oDs) (replicate olive setTs) outer)
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   235
          (mk_T_of_bnf oDs setTs outer --> HOLogic.mk_setT T);
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   236
        val inner_sets = map (fn sets => nth sets i) inner_setss;
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   237
        val outer_map = mk_map_of_bnf oDs CAs setTs outer;
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   238
        val map_inner_sets = Term.list_comb (outer_map, inner_sets);
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   239
        val collect_image = mk_collect
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   240
          (map2 (fn f => fn set => HOLogic.mk_comp (mk_image f, set)) inner_sets outer_sets)
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   241
          (CCA --> HOLogic.mk_setT T);
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   242
      in
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   243
        (Library.foldl1 HOLogic.mk_comp [mk_Union T, outer_set, map_inner_sets],
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   244
        HOLogic.mk_comp (mk_Union T, collect_image))
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   245
      end;
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   246
49303
blanchet
parents: 49236
diff changeset
   247
    val (sets, sets_alt) = map_split mk_set (0 upto ilive - 1);
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   248
55906
abf91ebd0820 simplify sets in BNF composition
blanchet
parents: 55904
diff changeset
   249
    fun mk_simplified_set set =
abf91ebd0820 simplify sets in BNF composition
blanchet
parents: 55904
diff changeset
   250
      let
abf91ebd0820 simplify sets in BNF composition
blanchet
parents: 55904
diff changeset
   251
        val setT = fastype_of set;
69593
3dda49e08b9d isabelle update -u control_cartouches;
wenzelm
parents: 68960
diff changeset
   252
        val var_set' = Const (\<^const_name>\<open>id_bnf\<close>, setT --> setT) $ Var ((Name.uu, 0), setT);
55908
e6d570cb0f5e no 'sorry' so that the schematic variable gets instantiated
blanchet
parents: 55906
diff changeset
   253
        val goal = mk_Trueprop_eq (var_set', set);
55930
25a90cebbbe5 more careful simplification of sets (cf. abf91ebd0820)---yields smaller terms
traytel
parents: 55908
diff changeset
   254
        fun tac {context = ctxt, prems = _} =
25a90cebbbe5 more careful simplification of sets (cf. abf91ebd0820)---yields smaller terms
traytel
parents: 55908
diff changeset
   255
          mk_simplified_set_tac ctxt (collect_set_map_of_bnf outer);
55906
abf91ebd0820 simplify sets in BNF composition
blanchet
parents: 55904
diff changeset
   256
        val set'_eq_set =
57890
1e13f63fb452 use Goal.prove_sorry instead of Goal.prove where possible (= no schematics in goal and tactic is expected to succeed)
traytel
parents: 57632
diff changeset
   257
          Goal.prove (*no sorry*) names_lthy [] [] goal tac
70494
41108e3e9ca5 formal position for PThm nodes;
wenzelm
parents: 69593
diff changeset
   258
          |> Thm.close_derivation \<^here>;
55906
abf91ebd0820 simplify sets in BNF composition
blanchet
parents: 55904
diff changeset
   259
        val set' = fst (HOLogic.dest_eq (HOLogic.dest_Trueprop (Thm.prop_of set'_eq_set)));
abf91ebd0820 simplify sets in BNF composition
blanchet
parents: 55904
diff changeset
   260
      in
abf91ebd0820 simplify sets in BNF composition
blanchet
parents: 55904
diff changeset
   261
        (set', set'_eq_set)
abf91ebd0820 simplify sets in BNF composition
blanchet
parents: 55904
diff changeset
   262
      end;
abf91ebd0820 simplify sets in BNF composition
blanchet
parents: 55904
diff changeset
   263
abf91ebd0820 simplify sets in BNF composition
blanchet
parents: 55904
diff changeset
   264
    val (sets', set'_eq_sets) =
abf91ebd0820 simplify sets in BNF composition
blanchet
parents: 55904
diff changeset
   265
      map_split mk_simplified_set sets
abf91ebd0820 simplify sets in BNF composition
blanchet
parents: 55904
diff changeset
   266
      ||> Proof_Context.export names_lthy lthy;
abf91ebd0820 simplify sets in BNF composition
blanchet
parents: 55904
diff changeset
   267
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   268
    (*(inner_1.bd +c ... +c inner_m.bd) *c outer.bd*)
54421
632be352a5a3 more explicit syntax for defining a bnf
traytel
parents: 53289
diff changeset
   269
    val bd = mk_cprod (Library.foldr1 (uncurry mk_csum) inner_bds) outer_bd;
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   270
55851
3d40cf74726c optimize cardinal bounds involving natLeq (omega)
blanchet
parents: 55803
diff changeset
   271
    val (bd', bd_ordIso_natLeq_thm_opt) =
3d40cf74726c optimize cardinal bounds involving natLeq (omega)
blanchet
parents: 55803
diff changeset
   272
      if is_sum_prod_natLeq bd then
3d40cf74726c optimize cardinal bounds involving natLeq (omega)
blanchet
parents: 55803
diff changeset
   273
        let
69593
3dda49e08b9d isabelle update -u control_cartouches;
wenzelm
parents: 68960
diff changeset
   274
          val bd' = \<^term>\<open>natLeq\<close>;
55851
3d40cf74726c optimize cardinal bounds involving natLeq (omega)
blanchet
parents: 55803
diff changeset
   275
          val bd_bd' = HOLogic.mk_prod (bd, bd');
69593
3dda49e08b9d isabelle update -u control_cartouches;
wenzelm
parents: 68960
diff changeset
   276
          val ordIso = Const (\<^const_name>\<open>ordIso\<close>, HOLogic.mk_setT (fastype_of bd_bd'));
57567
d554b0097ad4 add mk_Trueprop_mem utility function
desharna
parents: 56634
diff changeset
   277
          val goal = mk_Trueprop_mem (bd_bd', ordIso);
55851
3d40cf74726c optimize cardinal bounds involving natLeq (omega)
blanchet
parents: 55803
diff changeset
   278
        in
60757
c09598a97436 prefer tactics with explicit context;
wenzelm
parents: 60752
diff changeset
   279
          (bd', SOME (Goal.prove_sorry lthy [] [] goal (bd_ordIso_natLeq_tac o #context)
70494
41108e3e9ca5 formal position for PThm nodes;
wenzelm
parents: 69593
diff changeset
   280
            |> Thm.close_derivation \<^here>))
55851
3d40cf74726c optimize cardinal bounds involving natLeq (omega)
blanchet
parents: 55803
diff changeset
   281
        end
3d40cf74726c optimize cardinal bounds involving natLeq (omega)
blanchet
parents: 55803
diff changeset
   282
      else
3d40cf74726c optimize cardinal bounds involving natLeq (omega)
blanchet
parents: 55803
diff changeset
   283
        (bd, NONE);
3d40cf74726c optimize cardinal bounds involving natLeq (omega)
blanchet
parents: 55803
diff changeset
   284
60728
26ffdb966759 {r,e,d,f}tac with proper context in BNF
traytel
parents: 60207
diff changeset
   285
    fun map_id0_tac ctxt =
26ffdb966759 {r,e,d,f}tac with proper context in BNF
traytel
parents: 60207
diff changeset
   286
      mk_comp_map_id0_tac ctxt (map_id0_of_bnf outer) (map_cong0_of_bnf outer)
53270
c8628119d18e renamed BNF axiom
blanchet
parents: 53264
diff changeset
   287
        (map map_id0_of_bnf inners);
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   288
60728
26ffdb966759 {r,e,d,f}tac with proper context in BNF
traytel
parents: 60207
diff changeset
   289
    fun map_comp0_tac ctxt =
26ffdb966759 {r,e,d,f}tac with proper context in BNF
traytel
parents: 60207
diff changeset
   290
      mk_comp_map_comp0_tac ctxt (map_comp0_of_bnf outer) (map_cong0_of_bnf outer)
53287
271b34513bfb renamed BNF axiom
blanchet
parents: 53270
diff changeset
   291
        (map map_comp0_of_bnf inners);
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   292
55906
abf91ebd0820 simplify sets in BNF composition
blanchet
parents: 55904
diff changeset
   293
    fun mk_single_set_map0_tac i ctxt =
abf91ebd0820 simplify sets in BNF composition
blanchet
parents: 55904
diff changeset
   294
      mk_comp_set_map0_tac ctxt (nth set'_eq_sets i) (map_comp0_of_bnf outer)
abf91ebd0820 simplify sets in BNF composition
blanchet
parents: 55904
diff changeset
   295
        (map_cong0_of_bnf outer) (collect_set_map_of_bnf outer)
53289
5e0623448bdb renamed BNF axiom
blanchet
parents: 53288
diff changeset
   296
        (map ((fn thms => nth thms i) o set_map0_of_bnf) inners);
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   297
53289
5e0623448bdb renamed BNF axiom
blanchet
parents: 53288
diff changeset
   298
    val set_map0_tacs = map mk_single_set_map0_tac (0 upto ilive - 1);
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   299
60728
26ffdb966759 {r,e,d,f}tac with proper context in BNF
traytel
parents: 60207
diff changeset
   300
    fun bd_card_order_tac ctxt =
26ffdb966759 {r,e,d,f}tac with proper context in BNF
traytel
parents: 60207
diff changeset
   301
      mk_comp_bd_card_order_tac ctxt (map bd_card_order_of_bnf inners) (bd_card_order_of_bnf outer);
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   302
60728
26ffdb966759 {r,e,d,f}tac with proper context in BNF
traytel
parents: 60207
diff changeset
   303
    fun bd_cinfinite_tac ctxt =
26ffdb966759 {r,e,d,f}tac with proper context in BNF
traytel
parents: 60207
diff changeset
   304
      mk_comp_bd_cinfinite_tac ctxt (bd_cinfinite_of_bnf inner) (bd_cinfinite_of_bnf outer);
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   305
49303
blanchet
parents: 49236
diff changeset
   306
    val set_alt_thms =
52059
2f970c7f722b proper option quick_and_dirty;
wenzelm
parents: 51895
diff changeset
   307
      if Config.get lthy quick_and_dirty then
49456
fa8302c8dea1 adapted BNF composition to new relator approach
blanchet
parents: 49455
diff changeset
   308
        []
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   309
      else
49109
0e5b859e1c91 no more aliases for Local_Theory.note; use Thm.close_derivation in internal theorems;
traytel
parents: 49019
diff changeset
   310
        map (fn goal =>
51551
88d1d19fb74f tuned signature and module arrangement;
wenzelm
parents: 50059
diff changeset
   311
          Goal.prove_sorry lthy [] [] goal
49714
2c7c32f34220 made SML/NJ happier
traytel
parents: 49713
diff changeset
   312
            (fn {context = ctxt, prems = _} =>
51766
f19a4d0ab1bf renamed "set_natural" to "set_map", reflecting {Bl,Po,Tr} concensus
blanchet
parents: 51761
diff changeset
   313
              mk_comp_set_alt_tac ctxt (collect_set_map_of_bnf outer))
70494
41108e3e9ca5 formal position for PThm nodes;
wenzelm
parents: 69593
diff changeset
   314
          |> Thm.close_derivation \<^here>)
63824
blanchet
parents: 63802
diff changeset
   315
        (map2 (curry mk_Trueprop_eq) sets sets_alt);
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   316
55906
abf91ebd0820 simplify sets in BNF composition
blanchet
parents: 55904
diff changeset
   317
    fun map_cong0_tac ctxt =
abf91ebd0820 simplify sets in BNF composition
blanchet
parents: 55904
diff changeset
   318
      mk_comp_map_cong0_tac ctxt set'_eq_sets set_alt_thms (map_cong0_of_bnf outer)
abf91ebd0820 simplify sets in BNF composition
blanchet
parents: 55904
diff changeset
   319
        (map map_cong0_of_bnf inners);
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   320
49303
blanchet
parents: 49236
diff changeset
   321
    val set_bd_tacs =
52059
2f970c7f722b proper option quick_and_dirty;
wenzelm
parents: 51895
diff changeset
   322
      if Config.get lthy quick_and_dirty then
49669
620fa6272c48 fixed quick-and-dirty mode
blanchet
parents: 49630
diff changeset
   323
        replicate ilive (K all_tac)
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   324
      else
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   325
        let
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   326
          val outer_set_bds = set_bd_of_bnf outer;
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   327
          val inner_set_bdss = map set_bd_of_bnf inners;
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   328
          val inner_bd_Card_orders = map bd_Card_order_of_bnf inners;
49303
blanchet
parents: 49236
diff changeset
   329
          fun single_set_bd_thm i j =
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   330
            @{thm comp_single_set_bd} OF [nth inner_bd_Card_orders j, nth (nth inner_set_bdss j) i,
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   331
              nth outer_set_bds j]
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   332
          val single_set_bd_thmss =
49303
blanchet
parents: 49236
diff changeset
   333
            map ((fn f => map f (0 upto olive - 1)) o single_set_bd_thm) (0 upto ilive - 1);
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   334
        in
58634
9f10d82e8188 added parameterized ML antiquotations @{map N}, @{fold N}, @{fold_map N}, @{split_list N};
wenzelm
parents: 58359
diff changeset
   335
          @{map 3} (fn set'_eq_set => fn set_alt => fn single_set_bds => fn ctxt =>
55906
abf91ebd0820 simplify sets in BNF composition
blanchet
parents: 55904
diff changeset
   336
            mk_comp_set_bd_tac ctxt set'_eq_set bd_ordIso_natLeq_thm_opt set_alt single_set_bds)
abf91ebd0820 simplify sets in BNF composition
blanchet
parents: 55904
diff changeset
   337
          set'_eq_sets set_alt_thms single_set_bd_thmss
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   338
        end;
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   339
49303
blanchet
parents: 49236
diff changeset
   340
    val in_alt_thm =
49155
f51ab68f882f do not trivialize important internal theorem in quick_and_dirty mode
traytel
parents: 49123
diff changeset
   341
      let
49303
blanchet
parents: 49236
diff changeset
   342
        val inx = mk_in Asets sets CCA;
blanchet
parents: 49236
diff changeset
   343
        val in_alt = mk_in (map2 (mk_in Asets) inner_setss CAs) outer_sets CCA;
blanchet
parents: 49236
diff changeset
   344
        val goal = fold_rev Logic.all Asets (mk_Trueprop_eq (inx, in_alt));
49155
f51ab68f882f do not trivialize important internal theorem in quick_and_dirty mode
traytel
parents: 49123
diff changeset
   345
      in
51551
88d1d19fb74f tuned signature and module arrangement;
wenzelm
parents: 50059
diff changeset
   346
        Goal.prove_sorry lthy [] [] goal
49714
2c7c32f34220 made SML/NJ happier
traytel
parents: 49713
diff changeset
   347
          (fn {context = ctxt, prems = _} => mk_comp_in_alt_tac ctxt set_alt_thms)
70494
41108e3e9ca5 formal position for PThm nodes;
wenzelm
parents: 69593
diff changeset
   348
        |> Thm.close_derivation \<^here>
49155
f51ab68f882f do not trivialize important internal theorem in quick_and_dirty mode
traytel
parents: 49123
diff changeset
   349
      end;
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   350
60728
26ffdb966759 {r,e,d,f}tac with proper context in BNF
traytel
parents: 60207
diff changeset
   351
    fun le_rel_OO_tac ctxt = mk_le_rel_OO_tac ctxt (le_rel_OO_of_bnf outer) (rel_mono_of_bnf outer)
54841
af71b753c459 express weak pullback property of bnfs only in terms of the relator
traytel
parents: 54742
diff changeset
   352
      (map le_rel_OO_of_bnf inners);
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   353
55906
abf91ebd0820 simplify sets in BNF composition
blanchet
parents: 55904
diff changeset
   354
    fun rel_OO_Grp_tac ctxt =
49456
fa8302c8dea1 adapted BNF composition to new relator approach
blanchet
parents: 49455
diff changeset
   355
      let
51893
596baae88a88 got rid of the set based relator---use (binary) predicate based relator instead
traytel
parents: 51837
diff changeset
   356
        val outer_rel_Grp = rel_Grp_of_bnf outer RS sym;
49463
83ac281bcdc2 provide predicator, define relator
blanchet
parents: 49461
diff changeset
   357
        val thm =
62324
ae44f16dcea5 make predicator a first-class bnf citizen
traytel
parents: 62316
diff changeset
   358
          trans OF [in_alt_thm RS @{thm OO_Grp_cong},
51893
596baae88a88 got rid of the set based relator---use (binary) predicate based relator instead
traytel
parents: 51837
diff changeset
   359
             trans OF [@{thm arg_cong2[of _ _ _ _ relcompp]} OF
596baae88a88 got rid of the set based relator---use (binary) predicate based relator instead
traytel
parents: 51837
diff changeset
   360
               [trans OF [outer_rel_Grp RS @{thm arg_cong[of _ _ conversep]},
596baae88a88 got rid of the set based relator---use (binary) predicate based relator instead
traytel
parents: 51837
diff changeset
   361
                 rel_conversep_of_bnf outer RS sym], outer_rel_Grp],
61242
1f92b0ac9c96 congruence rules for the relator
traytel
parents: 60757
diff changeset
   362
               trans OF [rel_OO_of_bnf outer RS sym, rel_cong0_of_bnf outer OF
62324
ae44f16dcea5 make predicator a first-class bnf citizen
traytel
parents: 62316
diff changeset
   363
                 (map (fn bnf => rel_OO_Grp_of_bnf bnf RS sym) inners)]]] RS sym;
49456
fa8302c8dea1 adapted BNF composition to new relator approach
blanchet
parents: 49455
diff changeset
   364
      in
60728
26ffdb966759 {r,e,d,f}tac with proper context in BNF
traytel
parents: 60207
diff changeset
   365
        unfold_thms_tac ctxt set'_eq_sets THEN rtac ctxt thm 1
49463
83ac281bcdc2 provide predicator, define relator
blanchet
parents: 49461
diff changeset
   366
      end;
49456
fa8302c8dea1 adapted BNF composition to new relator approach
blanchet
parents: 49455
diff changeset
   367
62324
ae44f16dcea5 make predicator a first-class bnf citizen
traytel
parents: 62316
diff changeset
   368
    fun pred_set_tac ctxt =
ae44f16dcea5 make predicator a first-class bnf citizen
traytel
parents: 62316
diff changeset
   369
      let
ae44f16dcea5 make predicator a first-class bnf citizen
traytel
parents: 62316
diff changeset
   370
        val pred_alt = unfold_thms ctxt @{thms Ball_Collect}
ae44f16dcea5 make predicator a first-class bnf citizen
traytel
parents: 62316
diff changeset
   371
          (trans OF [pred_cong0_of_bnf outer OF map pred_set_of_bnf inners, pred_set_of_bnf outer]);
ae44f16dcea5 make predicator a first-class bnf citizen
traytel
parents: 62316
diff changeset
   372
        val in_alt = in_alt_thm RS @{thm Collect_inj} RS sym;
ae44f16dcea5 make predicator a first-class bnf citizen
traytel
parents: 62316
diff changeset
   373
      in
ae44f16dcea5 make predicator a first-class bnf citizen
traytel
parents: 62316
diff changeset
   374
        unfold_thms_tac ctxt (@{thm Ball_Collect} :: set'_eq_sets) THEN
ae44f16dcea5 make predicator a first-class bnf citizen
traytel
parents: 62316
diff changeset
   375
        HEADGOAL (rtac ctxt (trans OF [pred_alt, in_alt]))
ae44f16dcea5 make predicator a first-class bnf citizen
traytel
parents: 62316
diff changeset
   376
      end
ae44f16dcea5 make predicator a first-class bnf citizen
traytel
parents: 62316
diff changeset
   377
53289
5e0623448bdb renamed BNF axiom
blanchet
parents: 53288
diff changeset
   378
    val tacs = zip_axioms map_id0_tac map_comp0_tac map_cong0_tac set_map0_tacs bd_card_order_tac
62324
ae44f16dcea5 make predicator a first-class bnf citizen
traytel
parents: 62316
diff changeset
   379
      bd_cinfinite_tac set_bd_tacs le_rel_OO_tac rel_OO_Grp_tac pred_set_tac;
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   380
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   381
    val outer_wits = mk_wits_of_bnf (replicate onwits oDs) (replicate onwits CAs) outer;
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   382
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   383
    val inner_witss = map (map (fn (I, wit) => Term.list_comb (wit, map (nth xs) I)))
58634
9f10d82e8188 added parameterized ML antiquotations @{map N}, @{fold N}, @{fold_map N}, @{split_list N};
wenzelm
parents: 58359
diff changeset
   384
      (@{map 3} (fn Ds => fn n => mk_wits_of_bnf (replicate n Ds) (replicate n As))
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   385
        Dss inwitss inners);
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   386
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   387
    val inner_witsss = map (map (nth inner_witss) o fst) outer_wits;
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   388
49303
blanchet
parents: 49236
diff changeset
   389
    val wits = (inner_witsss, (map (single o snd) outer_wits))
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   390
      |-> map2 (fold (map_product (fn iwit => fn owit => owit $ iwit)))
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   391
      |> flat
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   392
      |> map (`(fn t => Term.add_frees t []))
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   393
      |> minimize_wits
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   394
      |> map (fn (frees, t) => fold absfree frees t);
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   395
55197
5a54ed681ba2 less hermetic tactics
traytel
parents: 55067
diff changeset
   396
    fun wit_tac ctxt =
55906
abf91ebd0820 simplify sets in BNF composition
blanchet
parents: 55904
diff changeset
   397
      mk_comp_wit_tac ctxt set'_eq_sets (wit_thms_of_bnf outer) (collect_set_map_of_bnf outer)
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   398
        (maps wit_thms_of_bnf inners);
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   399
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   400
    val (bnf', lthy') =
56016
8875cdcfc85b unfold intermediate definitions after sealing the bnf
traytel
parents: 56013
diff changeset
   401
      bnf_def const_policy (K Dont_Note) true qualify tacs wit_tac (SOME (oDs @ flat Dss))
62324
ae44f16dcea5 make predicator a first-class bnf citizen
traytel
parents: 62316
diff changeset
   402
        Binding.empty Binding.empty Binding.empty []
ae44f16dcea5 make predicator a first-class bnf citizen
traytel
parents: 62316
diff changeset
   403
        (((((((b, CCA), mapx), sets'), bd'), wits), SOME rel), SOME pred) lthy;
55906
abf91ebd0820 simplify sets in BNF composition
blanchet
parents: 55904
diff changeset
   404
abf91ebd0820 simplify sets in BNF composition
blanchet
parents: 55904
diff changeset
   405
    val phi =
58181
6d527272f7b2 renamed internal constant
blanchet
parents: 58128
diff changeset
   406
      Morphism.thm_morphism "BNF" (unfold_thms lthy' [id_bnf_def])
6d527272f7b2 renamed internal constant
blanchet
parents: 58128
diff changeset
   407
      $> Morphism.term_morphism "BNF" expand_id_bnf_def;
55906
abf91ebd0820 simplify sets in BNF composition
blanchet
parents: 55904
diff changeset
   408
abf91ebd0820 simplify sets in BNF composition
blanchet
parents: 55904
diff changeset
   409
    val bnf'' = morph_bnf phi bnf';
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   410
  in
55906
abf91ebd0820 simplify sets in BNF composition
blanchet
parents: 55904
diff changeset
   411
    (bnf'', (add_bnf_to_unfolds bnf'' unfold_set, lthy'))
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   412
  end;
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   413
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   414
(* Killing live variables *)
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   415
55904
0ef30d52c5e4 more caching in composition pipeline
blanchet
parents: 55900
diff changeset
   416
fun raw_kill_bnf qualify n bnf (accum as (unfold_set, lthy)) =
0ef30d52c5e4 more caching in composition pipeline
blanchet
parents: 55900
diff changeset
   417
  if n = 0 then (bnf, accum) else
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   418
  let
49425
f27f83f71e94 cleaned up internal naming scheme for bnfs
traytel
parents: 49304
diff changeset
   419
    val b = Binding.suffix_name (mk_killN n) (name_of_bnf bnf);
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   420
    val live = live_of_bnf bnf;
60207
81a0900f0ddc allow sorts on dead variables in BNFs
blanchet
parents: 59994
diff changeset
   421
    val deads = deads_of_bnf bnf;
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   422
    val nwits = nwits_of_bnf bnf;
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   423
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   424
    (* TODO: check 0 < n <= live *)
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   425
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   426
    val (Ds, lthy1) = apfst (map TFree)
60207
81a0900f0ddc allow sorts on dead variables in BNFs
blanchet
parents: 59994
diff changeset
   427
      (Variable.invent_types (map Type.sort_of_atyp deads) lthy);
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   428
    val ((killedAs, As), lthy2) = apfst (`(take n) o map TFree)
69593
3dda49e08b9d isabelle update -u control_cartouches;
wenzelm
parents: 68960
diff changeset
   429
      (Variable.invent_types (replicate live \<^sort>\<open>type\<close>) lthy1);
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   430
    val (Bs, _(*lthy3*)) = apfst (append killedAs o map TFree)
69593
3dda49e08b9d isabelle update -u control_cartouches;
wenzelm
parents: 68960
diff changeset
   431
      (Variable.invent_types (replicate (live - n) \<^sort>\<open>type\<close>) lthy2);
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   432
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   433
    val ((Asets, lives), _(*names_lthy*)) = lthy
49456
fa8302c8dea1 adapted BNF composition to new relator approach
blanchet
parents: 49455
diff changeset
   434
      |> mk_Frees "A" (map HOLogic.mk_setT (drop n As))
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   435
      ||>> mk_Frees "x" (drop n As);
69593
3dda49e08b9d isabelle update -u control_cartouches;
wenzelm
parents: 68960
diff changeset
   436
    val xs = map (fn T => Const (\<^const_name>\<open>undefined\<close>, T)) killedAs @ lives;
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   437
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   438
    val T = mk_T_of_bnf Ds As bnf;
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   439
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   440
    (*bnf.map id ... id*)
49303
blanchet
parents: 49236
diff changeset
   441
    val mapx = Term.list_comb (mk_map_of_bnf Ds As Bs bnf, map HOLogic.id_const killedAs);
49507
8826d5a4332b renamed "pred" to "rel" (relator)
blanchet
parents: 49506
diff changeset
   442
    (*bnf.rel (op =) ... (op =)*)
8826d5a4332b renamed "pred" to "rel" (relator)
blanchet
parents: 49506
diff changeset
   443
    val rel = Term.list_comb (mk_rel_of_bnf Ds As Bs bnf, map HOLogic.eq_const killedAs);
62324
ae44f16dcea5 make predicator a first-class bnf citizen
traytel
parents: 62316
diff changeset
   444
    (*bnf.pred (%_. True) ... (%_ True)*)
ae44f16dcea5 make predicator a first-class bnf citizen
traytel
parents: 62316
diff changeset
   445
    val pred = Term.list_comb (mk_pred_of_bnf Ds As bnf,
69593
3dda49e08b9d isabelle update -u control_cartouches;
wenzelm
parents: 68960
diff changeset
   446
      map (fn T => Term.absdummy T \<^term>\<open>True\<close>) killedAs);
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   447
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   448
    val bnf_sets = mk_sets_of_bnf (replicate live Ds) (replicate live As) bnf;
49303
blanchet
parents: 49236
diff changeset
   449
    val sets = drop n bnf_sets;
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   450
55707
50cf04dd2584 clarified interaction with dead variables in the composition of BNFs
traytel
parents: 55706
diff changeset
   451
    val bd = mk_bd_of_bnf Ds As bnf;
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   452
60728
26ffdb966759 {r,e,d,f}tac with proper context in BNF
traytel
parents: 60207
diff changeset
   453
    fun map_id0_tac ctxt = rtac ctxt (map_id0_of_bnf bnf) 1;
55197
5a54ed681ba2 less hermetic tactics
traytel
parents: 55067
diff changeset
   454
    fun map_comp0_tac ctxt =
55067
a452de24a877 tuned names
blanchet
parents: 55061
diff changeset
   455
      unfold_thms_tac ctxt ((map_comp0_of_bnf bnf RS sym) ::
60728
26ffdb966759 {r,e,d,f}tac with proper context in BNF
traytel
parents: 60207
diff changeset
   456
        @{thms comp_assoc id_comp comp_id}) THEN rtac ctxt refl 1;
55197
5a54ed681ba2 less hermetic tactics
traytel
parents: 55067
diff changeset
   457
    fun map_cong0_tac ctxt =
51761
4c9f08836d87 renamed "map_cong" axiom to "map_cong0" in preparation for real "map_cong"
blanchet
parents: 51758
diff changeset
   458
      mk_kill_map_cong0_tac ctxt n (live - n) (map_cong0_of_bnf bnf);
60728
26ffdb966759 {r,e,d,f}tac with proper context in BNF
traytel
parents: 60207
diff changeset
   459
    val set_map0_tacs = map (fn thm => fn ctxt => rtac ctxt thm 1) (drop n (set_map0_of_bnf bnf));
26ffdb966759 {r,e,d,f}tac with proper context in BNF
traytel
parents: 60207
diff changeset
   460
    fun bd_card_order_tac ctxt = rtac ctxt (bd_card_order_of_bnf bnf) 1;
26ffdb966759 {r,e,d,f}tac with proper context in BNF
traytel
parents: 60207
diff changeset
   461
    fun bd_cinfinite_tac ctxt = rtac ctxt (bd_cinfinite_of_bnf bnf) 1;
26ffdb966759 {r,e,d,f}tac with proper context in BNF
traytel
parents: 60207
diff changeset
   462
    val set_bd_tacs = map (fn thm => fn ctxt => rtac ctxt thm 1) (drop n (set_bd_of_bnf bnf));
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   463
49303
blanchet
parents: 49236
diff changeset
   464
    val in_alt_thm =
49155
f51ab68f882f do not trivialize important internal theorem in quick_and_dirty mode
traytel
parents: 49123
diff changeset
   465
      let
49303
blanchet
parents: 49236
diff changeset
   466
        val inx = mk_in Asets sets T;
blanchet
parents: 49236
diff changeset
   467
        val in_alt = mk_in (map HOLogic.mk_UNIV killedAs @ Asets) bnf_sets T;
blanchet
parents: 49236
diff changeset
   468
        val goal = fold_rev Logic.all Asets (mk_Trueprop_eq (inx, in_alt));
49155
f51ab68f882f do not trivialize important internal theorem in quick_and_dirty mode
traytel
parents: 49123
diff changeset
   469
      in
60728
26ffdb966759 {r,e,d,f}tac with proper context in BNF
traytel
parents: 60207
diff changeset
   470
        Goal.prove_sorry lthy [] [] goal (fn {context = ctxt, prems = _} =>
70494
41108e3e9ca5 formal position for PThm nodes;
wenzelm
parents: 69593
diff changeset
   471
          kill_in_alt_tac ctxt) |> Thm.close_derivation \<^here>
49155
f51ab68f882f do not trivialize important internal theorem in quick_and_dirty mode
traytel
parents: 49123
diff changeset
   472
      end;
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   473
55197
5a54ed681ba2 less hermetic tactics
traytel
parents: 55067
diff changeset
   474
    fun le_rel_OO_tac ctxt =
60728
26ffdb966759 {r,e,d,f}tac with proper context in BNF
traytel
parents: 60207
diff changeset
   475
      EVERY' [rtac ctxt @{thm ord_le_eq_trans}, rtac ctxt (le_rel_OO_of_bnf bnf)] 1 THEN
26ffdb966759 {r,e,d,f}tac with proper context in BNF
traytel
parents: 60207
diff changeset
   476
      unfold_thms_tac ctxt @{thms eq_OO} THEN rtac ctxt refl 1;
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   477
60728
26ffdb966759 {r,e,d,f}tac with proper context in BNF
traytel
parents: 60207
diff changeset
   478
    fun rel_OO_Grp_tac ctxt =
49456
fa8302c8dea1 adapted BNF composition to new relator approach
blanchet
parents: 49455
diff changeset
   479
      let
51893
596baae88a88 got rid of the set based relator---use (binary) predicate based relator instead
traytel
parents: 51837
diff changeset
   480
        val rel_Grp = rel_Grp_of_bnf bnf RS sym
49463
83ac281bcdc2 provide predicator, define relator
blanchet
parents: 49461
diff changeset
   481
        val thm =
51893
596baae88a88 got rid of the set based relator---use (binary) predicate based relator instead
traytel
parents: 51837
diff changeset
   482
          (trans OF [in_alt_thm RS @{thm OO_Grp_cong},
596baae88a88 got rid of the set based relator---use (binary) predicate based relator instead
traytel
parents: 51837
diff changeset
   483
            trans OF [@{thm arg_cong2[of _ _ _ _ relcompp]} OF
596baae88a88 got rid of the set based relator---use (binary) predicate based relator instead
traytel
parents: 51837
diff changeset
   484
              [trans OF [rel_Grp RS @{thm arg_cong[of _ _ conversep]},
596baae88a88 got rid of the set based relator---use (binary) predicate based relator instead
traytel
parents: 51837
diff changeset
   485
                rel_conversep_of_bnf bnf RS sym], rel_Grp],
61242
1f92b0ac9c96 congruence rules for the relator
traytel
parents: 60757
diff changeset
   486
              trans OF [rel_OO_of_bnf bnf RS sym, rel_cong0_of_bnf bnf OF
51893
596baae88a88 got rid of the set based relator---use (binary) predicate based relator instead
traytel
parents: 51837
diff changeset
   487
                (replicate n @{thm trans[OF Grp_UNIV_id[OF refl] eq_alt[symmetric]]} @
52660
7f7311d04727 killed unused theorems
traytel
parents: 52635
diff changeset
   488
                 replicate (live - n) @{thm Grp_fst_snd})]]] RS sym);
49456
fa8302c8dea1 adapted BNF composition to new relator approach
blanchet
parents: 49455
diff changeset
   489
      in
60728
26ffdb966759 {r,e,d,f}tac with proper context in BNF
traytel
parents: 60207
diff changeset
   490
        rtac ctxt thm 1
49456
fa8302c8dea1 adapted BNF composition to new relator approach
blanchet
parents: 49455
diff changeset
   491
      end;
fa8302c8dea1 adapted BNF composition to new relator approach
blanchet
parents: 49455
diff changeset
   492
62324
ae44f16dcea5 make predicator a first-class bnf citizen
traytel
parents: 62316
diff changeset
   493
    fun pred_set_tac ctxt = mk_simple_pred_set_tac ctxt (pred_set_of_bnf bnf) in_alt_thm;
ae44f16dcea5 make predicator a first-class bnf citizen
traytel
parents: 62316
diff changeset
   494
53289
5e0623448bdb renamed BNF axiom
blanchet
parents: 53288
diff changeset
   495
    val tacs = zip_axioms map_id0_tac map_comp0_tac map_cong0_tac set_map0_tacs bd_card_order_tac
62324
ae44f16dcea5 make predicator a first-class bnf citizen
traytel
parents: 62316
diff changeset
   496
      bd_cinfinite_tac set_bd_tacs le_rel_OO_tac rel_OO_Grp_tac pred_set_tac;
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   497
49303
blanchet
parents: 49236
diff changeset
   498
    val bnf_wits = mk_wits_of_bnf (replicate nwits Ds) (replicate nwits As) bnf;
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   499
49303
blanchet
parents: 49236
diff changeset
   500
    val wits = map (fn t => fold absfree (Term.add_frees t []) t)
blanchet
parents: 49236
diff changeset
   501
      (map (fn (I, wit) => Term.list_comb (wit, map (nth xs) I)) bnf_wits);
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   502
60752
b48830b670a1 prefer tactics with explicit context;
wenzelm
parents: 60728
diff changeset
   503
    fun wit_tac ctxt = mk_simple_wit_tac ctxt (wit_thms_of_bnf bnf);
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   504
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   505
    val (bnf', lthy') =
58297
e3a01b73579f new deads go to the end
traytel
parents: 58181
diff changeset
   506
      bnf_def Smart_Inline (K Dont_Note) true qualify tacs wit_tac (SOME (Ds @ killedAs))
62324
ae44f16dcea5 make predicator a first-class bnf citizen
traytel
parents: 62316
diff changeset
   507
        Binding.empty Binding.empty Binding.empty []
ae44f16dcea5 make predicator a first-class bnf citizen
traytel
parents: 62316
diff changeset
   508
        (((((((b, T), mapx), sets), bd), wits), SOME rel), SOME pred) lthy;
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   509
  in
49503
dbbde075a42e simplified code
blanchet
parents: 49502
diff changeset
   510
    (bnf', (add_bnf_to_unfolds bnf' unfold_set, lthy'))
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   511
  end;
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   512
55904
0ef30d52c5e4 more caching in composition pipeline
blanchet
parents: 55900
diff changeset
   513
fun kill_bnf qualify n bnf (accum as ((cache, unfold_set), lthy)) =
0ef30d52c5e4 more caching in composition pipeline
blanchet
parents: 55900
diff changeset
   514
  let val key = key_of_kill n bnf in
0ef30d52c5e4 more caching in composition pipeline
blanchet
parents: 55900
diff changeset
   515
    (case Typtab.lookup cache key of
0ef30d52c5e4 more caching in composition pipeline
blanchet
parents: 55900
diff changeset
   516
      SOME (bnf, _) => (bnf, accum)
0ef30d52c5e4 more caching in composition pipeline
blanchet
parents: 55900
diff changeset
   517
    | NONE => cache_comp_simple key cache (raw_kill_bnf qualify n bnf (unfold_set, lthy)))
0ef30d52c5e4 more caching in composition pipeline
blanchet
parents: 55900
diff changeset
   518
  end;
0ef30d52c5e4 more caching in composition pipeline
blanchet
parents: 55900
diff changeset
   519
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   520
(* Adding dummy live variables *)
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   521
55904
0ef30d52c5e4 more caching in composition pipeline
blanchet
parents: 55900
diff changeset
   522
fun raw_lift_bnf qualify n bnf (accum as (unfold_set, lthy)) =
0ef30d52c5e4 more caching in composition pipeline
blanchet
parents: 55900
diff changeset
   523
  if n = 0 then (bnf, accum) else
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   524
  let
49425
f27f83f71e94 cleaned up internal naming scheme for bnfs
traytel
parents: 49304
diff changeset
   525
    val b = Binding.suffix_name (mk_liftN n) (name_of_bnf bnf);
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   526
    val live = live_of_bnf bnf;
60207
81a0900f0ddc allow sorts on dead variables in BNFs
blanchet
parents: 59994
diff changeset
   527
    val deads = deads_of_bnf bnf;
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   528
    val nwits = nwits_of_bnf bnf;
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   529
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   530
    (* TODO: check 0 < n *)
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   531
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   532
    val (Ds, lthy1) = apfst (map TFree)
60207
81a0900f0ddc allow sorts on dead variables in BNFs
blanchet
parents: 59994
diff changeset
   533
      (Variable.invent_types (map Type.sort_of_atyp deads) lthy);
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   534
    val ((newAs, As), lthy2) = apfst (chop n o map TFree)
69593
3dda49e08b9d isabelle update -u control_cartouches;
wenzelm
parents: 68960
diff changeset
   535
      (Variable.invent_types (replicate (n + live) \<^sort>\<open>type\<close>) lthy1);
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   536
    val ((newBs, Bs), _(*lthy3*)) = apfst (chop n o map TFree)
69593
3dda49e08b9d isabelle update -u control_cartouches;
wenzelm
parents: 68960
diff changeset
   537
      (Variable.invent_types (replicate (n + live) \<^sort>\<open>type\<close>) lthy2);
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   538
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   539
    val (Asets, _(*names_lthy*)) = lthy
49456
fa8302c8dea1 adapted BNF composition to new relator approach
blanchet
parents: 49455
diff changeset
   540
      |> mk_Frees "A" (map HOLogic.mk_setT (newAs @ As));
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   541
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   542
    val T = mk_T_of_bnf Ds As bnf;
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   543
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   544
    (*%f1 ... fn. bnf.map*)
49303
blanchet
parents: 49236
diff changeset
   545
    val mapx =
52923
traytel
parents: 52660
diff changeset
   546
      fold_rev Term.absdummy (map2 (curry op -->) newAs newBs) (mk_map_of_bnf Ds As Bs bnf);
49507
8826d5a4332b renamed "pred" to "rel" (relator)
blanchet
parents: 49506
diff changeset
   547
    (*%Q1 ... Qn. bnf.rel*)
8826d5a4332b renamed "pred" to "rel" (relator)
blanchet
parents: 49506
diff changeset
   548
    val rel = fold_rev Term.absdummy (map2 mk_pred2T newAs newBs) (mk_rel_of_bnf Ds As Bs bnf);
62324
ae44f16dcea5 make predicator a first-class bnf citizen
traytel
parents: 62316
diff changeset
   549
    (*%P1 ... Pn. bnf.pred*)
ae44f16dcea5 make predicator a first-class bnf citizen
traytel
parents: 62316
diff changeset
   550
    val pred = fold_rev Term.absdummy (map mk_pred1T newAs) (mk_pred_of_bnf Ds As bnf);
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   551
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   552
    val bnf_sets = mk_sets_of_bnf (replicate live Ds) (replicate live As) bnf;
49303
blanchet
parents: 49236
diff changeset
   553
    val sets = map (fn A => absdummy T (HOLogic.mk_set A [])) newAs @ bnf_sets;
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   554
49303
blanchet
parents: 49236
diff changeset
   555
    val bd = mk_bd_of_bnf Ds As bnf;
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   556
60728
26ffdb966759 {r,e,d,f}tac with proper context in BNF
traytel
parents: 60207
diff changeset
   557
    fun map_id0_tac ctxt = rtac ctxt (map_id0_of_bnf bnf) 1;
55197
5a54ed681ba2 less hermetic tactics
traytel
parents: 55067
diff changeset
   558
    fun map_comp0_tac ctxt =
55067
a452de24a877 tuned names
blanchet
parents: 55061
diff changeset
   559
      unfold_thms_tac ctxt ((map_comp0_of_bnf bnf RS sym) ::
60728
26ffdb966759 {r,e,d,f}tac with proper context in BNF
traytel
parents: 60207
diff changeset
   560
        @{thms comp_assoc id_comp comp_id}) THEN rtac ctxt refl 1;
55197
5a54ed681ba2 less hermetic tactics
traytel
parents: 55067
diff changeset
   561
    fun map_cong0_tac ctxt =
60728
26ffdb966759 {r,e,d,f}tac with proper context in BNF
traytel
parents: 60207
diff changeset
   562
      rtac ctxt (map_cong0_of_bnf bnf) 1 THEN REPEAT_DETERM_N live (Goal.assume_rule_tac ctxt 1);
53289
5e0623448bdb renamed BNF axiom
blanchet
parents: 53288
diff changeset
   563
    val set_map0_tacs =
52059
2f970c7f722b proper option quick_and_dirty;
wenzelm
parents: 51895
diff changeset
   564
      if Config.get lthy quick_and_dirty then
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   565
        replicate (n + live) (K all_tac)
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   566
      else
60728
26ffdb966759 {r,e,d,f}tac with proper context in BNF
traytel
parents: 60207
diff changeset
   567
        replicate n empty_natural_tac @
26ffdb966759 {r,e,d,f}tac with proper context in BNF
traytel
parents: 60207
diff changeset
   568
        map (fn thm => fn ctxt => rtac ctxt thm 1) (set_map0_of_bnf bnf);
26ffdb966759 {r,e,d,f}tac with proper context in BNF
traytel
parents: 60207
diff changeset
   569
    fun bd_card_order_tac ctxt = rtac ctxt (bd_card_order_of_bnf bnf) 1;
26ffdb966759 {r,e,d,f}tac with proper context in BNF
traytel
parents: 60207
diff changeset
   570
    fun bd_cinfinite_tac ctxt = rtac ctxt (bd_cinfinite_of_bnf bnf) 1;
49303
blanchet
parents: 49236
diff changeset
   571
    val set_bd_tacs =
52059
2f970c7f722b proper option quick_and_dirty;
wenzelm
parents: 51895
diff changeset
   572
      if Config.get lthy quick_and_dirty then
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   573
        replicate (n + live) (K all_tac)
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   574
      else
60728
26ffdb966759 {r,e,d,f}tac with proper context in BNF
traytel
parents: 60207
diff changeset
   575
        replicate n (fn ctxt => mk_lift_set_bd_tac ctxt (bd_Card_order_of_bnf bnf)) @
26ffdb966759 {r,e,d,f}tac with proper context in BNF
traytel
parents: 60207
diff changeset
   576
        (map (fn thm => fn ctxt => rtac ctxt thm 1) (set_bd_of_bnf bnf));
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   577
49303
blanchet
parents: 49236
diff changeset
   578
    val in_alt_thm =
49155
f51ab68f882f do not trivialize important internal theorem in quick_and_dirty mode
traytel
parents: 49123
diff changeset
   579
      let
49303
blanchet
parents: 49236
diff changeset
   580
        val inx = mk_in Asets sets T;
blanchet
parents: 49236
diff changeset
   581
        val in_alt = mk_in (drop n Asets) bnf_sets T;
blanchet
parents: 49236
diff changeset
   582
        val goal = fold_rev Logic.all Asets (mk_Trueprop_eq (inx, in_alt));
49155
f51ab68f882f do not trivialize important internal theorem in quick_and_dirty mode
traytel
parents: 49123
diff changeset
   583
      in
60728
26ffdb966759 {r,e,d,f}tac with proper context in BNF
traytel
parents: 60207
diff changeset
   584
        Goal.prove_sorry lthy [] [] goal (fn {context = ctxt, prems = _} => lift_in_alt_tac ctxt)
70494
41108e3e9ca5 formal position for PThm nodes;
wenzelm
parents: 69593
diff changeset
   585
        |> Thm.close_derivation \<^here>
49155
f51ab68f882f do not trivialize important internal theorem in quick_and_dirty mode
traytel
parents: 49123
diff changeset
   586
      end;
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   587
60728
26ffdb966759 {r,e,d,f}tac with proper context in BNF
traytel
parents: 60207
diff changeset
   588
    fun le_rel_OO_tac ctxt = rtac ctxt (le_rel_OO_of_bnf bnf) 1;
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   589
60728
26ffdb966759 {r,e,d,f}tac with proper context in BNF
traytel
parents: 60207
diff changeset
   590
    fun rel_OO_Grp_tac ctxt = mk_simple_rel_OO_Grp_tac ctxt (rel_OO_Grp_of_bnf bnf) in_alt_thm;
49456
fa8302c8dea1 adapted BNF composition to new relator approach
blanchet
parents: 49455
diff changeset
   591
62324
ae44f16dcea5 make predicator a first-class bnf citizen
traytel
parents: 62316
diff changeset
   592
    fun pred_set_tac ctxt = mk_simple_pred_set_tac ctxt (pred_set_of_bnf bnf) in_alt_thm;
ae44f16dcea5 make predicator a first-class bnf citizen
traytel
parents: 62316
diff changeset
   593
53289
5e0623448bdb renamed BNF axiom
blanchet
parents: 53288
diff changeset
   594
    val tacs = zip_axioms map_id0_tac map_comp0_tac map_cong0_tac set_map0_tacs bd_card_order_tac
62324
ae44f16dcea5 make predicator a first-class bnf citizen
traytel
parents: 62316
diff changeset
   595
      bd_cinfinite_tac set_bd_tacs le_rel_OO_tac rel_OO_Grp_tac pred_set_tac;
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   596
49303
blanchet
parents: 49236
diff changeset
   597
    val wits = map snd (mk_wits_of_bnf (replicate nwits Ds) (replicate nwits As) bnf);
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   598
60752
b48830b670a1 prefer tactics with explicit context;
wenzelm
parents: 60728
diff changeset
   599
    fun wit_tac ctxt = mk_simple_wit_tac ctxt (wit_thms_of_bnf bnf);
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   600
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   601
    val (bnf', lthy') =
56016
8875cdcfc85b unfold intermediate definitions after sealing the bnf
traytel
parents: 56013
diff changeset
   602
      bnf_def Smart_Inline (K Dont_Note) true qualify tacs wit_tac (SOME Ds) Binding.empty
62324
ae44f16dcea5 make predicator a first-class bnf citizen
traytel
parents: 62316
diff changeset
   603
        Binding.empty Binding.empty []
ae44f16dcea5 make predicator a first-class bnf citizen
traytel
parents: 62316
diff changeset
   604
        (((((((b, T), mapx), sets), bd), wits), SOME rel), SOME pred) lthy;
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   605
  in
49503
dbbde075a42e simplified code
blanchet
parents: 49502
diff changeset
   606
    (bnf', (add_bnf_to_unfolds bnf' unfold_set, lthy'))
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   607
  end;
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   608
55904
0ef30d52c5e4 more caching in composition pipeline
blanchet
parents: 55900
diff changeset
   609
fun lift_bnf qualify n bnf (accum as ((cache, unfold_set), lthy)) =
0ef30d52c5e4 more caching in composition pipeline
blanchet
parents: 55900
diff changeset
   610
  let val key = key_of_lift n bnf in
0ef30d52c5e4 more caching in composition pipeline
blanchet
parents: 55900
diff changeset
   611
    (case Typtab.lookup cache key of
0ef30d52c5e4 more caching in composition pipeline
blanchet
parents: 55900
diff changeset
   612
      SOME (bnf, _) => (bnf, accum)
0ef30d52c5e4 more caching in composition pipeline
blanchet
parents: 55900
diff changeset
   613
    | NONE => cache_comp_simple key cache (raw_lift_bnf qualify n bnf (unfold_set, lthy)))
0ef30d52c5e4 more caching in composition pipeline
blanchet
parents: 55900
diff changeset
   614
  end;
0ef30d52c5e4 more caching in composition pipeline
blanchet
parents: 55900
diff changeset
   615
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   616
(* Changing the order of live variables *)
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   617
55904
0ef30d52c5e4 more caching in composition pipeline
blanchet
parents: 55900
diff changeset
   618
fun raw_permute_bnf qualify src dest bnf (accum as (unfold_set, lthy)) =
0ef30d52c5e4 more caching in composition pipeline
blanchet
parents: 55900
diff changeset
   619
  if src = dest then (bnf, accum) else
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   620
  let
68960
b85d509e7cbf smash position to avoid position of other file "~~/src/HOL/BNF_Composition.thy" (due to "bnf ID"), e.g. relevant for "HOL-Nominal-Examples.Class1";
wenzelm
parents: 67091
diff changeset
   621
    val b = Binding.suffix_name (mk_permuteN src dest) (name_of_bnf bnf) |> Binding.reset_pos;
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   622
    val live = live_of_bnf bnf;
60207
81a0900f0ddc allow sorts on dead variables in BNFs
blanchet
parents: 59994
diff changeset
   623
    val deads = deads_of_bnf bnf;
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   624
    val nwits = nwits_of_bnf bnf;
55480
59cc4a8bc28a allow different functions to recurse on the same type, like in the old package
blanchet
parents: 55197
diff changeset
   625
59cc4a8bc28a allow different functions to recurse on the same type, like in the old package
blanchet
parents: 55197
diff changeset
   626
    fun permute xs = permute_like_unique (op =) src dest xs;
59cc4a8bc28a allow different functions to recurse on the same type, like in the old package
blanchet
parents: 55197
diff changeset
   627
    fun unpermute xs = permute_like_unique (op =) dest src xs;
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   628
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   629
    val (Ds, lthy1) = apfst (map TFree)
60207
81a0900f0ddc allow sorts on dead variables in BNFs
blanchet
parents: 59994
diff changeset
   630
      (Variable.invent_types (map Type.sort_of_atyp deads) lthy);
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   631
    val (As, lthy2) = apfst (map TFree)
69593
3dda49e08b9d isabelle update -u control_cartouches;
wenzelm
parents: 68960
diff changeset
   632
      (Variable.invent_types (replicate live \<^sort>\<open>type\<close>) lthy1);
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   633
    val (Bs, _(*lthy3*)) = apfst (map TFree)
69593
3dda49e08b9d isabelle update -u control_cartouches;
wenzelm
parents: 68960
diff changeset
   634
      (Variable.invent_types (replicate live \<^sort>\<open>type\<close>) lthy2);
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   635
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   636
    val (Asets, _(*names_lthy*)) = lthy
49456
fa8302c8dea1 adapted BNF composition to new relator approach
blanchet
parents: 49455
diff changeset
   637
      |> mk_Frees "A" (map HOLogic.mk_setT (permute As));
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   638
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   639
    val T = mk_T_of_bnf Ds As bnf;
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   640
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   641
    (*%f(1) ... f(n). bnf.map f\<sigma>(1) ... f\<sigma>(n)*)
49303
blanchet
parents: 49236
diff changeset
   642
    val mapx = fold_rev Term.absdummy (permute (map2 (curry op -->) As Bs))
53038
dd5ea8a51af0 generalized "mk_permute"
blanchet
parents: 52985
diff changeset
   643
      (Term.list_comb (mk_map_of_bnf Ds As Bs bnf, unpermute (map Bound (live - 1 downto 0))));
49507
8826d5a4332b renamed "pred" to "rel" (relator)
blanchet
parents: 49506
diff changeset
   644
    (*%Q(1) ... Q(n). bnf.rel Q\<sigma>(1) ... Q\<sigma>(n)*)
8826d5a4332b renamed "pred" to "rel" (relator)
blanchet
parents: 49506
diff changeset
   645
    val rel = fold_rev Term.absdummy (permute (map2 mk_pred2T As Bs))
53038
dd5ea8a51af0 generalized "mk_permute"
blanchet
parents: 52985
diff changeset
   646
      (Term.list_comb (mk_rel_of_bnf Ds As Bs bnf, unpermute (map Bound (live - 1 downto 0))));
62324
ae44f16dcea5 make predicator a first-class bnf citizen
traytel
parents: 62316
diff changeset
   647
    (*%P(1) ... P(n). bnf.pred P\<sigma>(1) ... P\<sigma>(n)*)
ae44f16dcea5 make predicator a first-class bnf citizen
traytel
parents: 62316
diff changeset
   648
    val pred = fold_rev Term.absdummy (permute (map mk_pred1T As))
ae44f16dcea5 make predicator a first-class bnf citizen
traytel
parents: 62316
diff changeset
   649
      (Term.list_comb (mk_pred_of_bnf Ds As bnf, unpermute (map Bound (live - 1 downto 0))));
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   650
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   651
    val bnf_sets = mk_sets_of_bnf (replicate live Ds) (replicate live As) bnf;
49303
blanchet
parents: 49236
diff changeset
   652
    val sets = permute bnf_sets;
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   653
49303
blanchet
parents: 49236
diff changeset
   654
    val bd = mk_bd_of_bnf Ds As bnf;
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   655
60728
26ffdb966759 {r,e,d,f}tac with proper context in BNF
traytel
parents: 60207
diff changeset
   656
    fun map_id0_tac ctxt = rtac ctxt (map_id0_of_bnf bnf) 1;
26ffdb966759 {r,e,d,f}tac with proper context in BNF
traytel
parents: 60207
diff changeset
   657
    fun map_comp0_tac ctxt = rtac ctxt (map_comp0_of_bnf bnf) 1;
55197
5a54ed681ba2 less hermetic tactics
traytel
parents: 55067
diff changeset
   658
    fun map_cong0_tac ctxt =
60728
26ffdb966759 {r,e,d,f}tac with proper context in BNF
traytel
parents: 60207
diff changeset
   659
      rtac ctxt (map_cong0_of_bnf bnf) 1 THEN REPEAT_DETERM_N live (Goal.assume_rule_tac ctxt 1);
26ffdb966759 {r,e,d,f}tac with proper context in BNF
traytel
parents: 60207
diff changeset
   660
    val set_map0_tacs = permute (map (fn thm => fn ctxt => rtac ctxt thm 1) (set_map0_of_bnf bnf));
26ffdb966759 {r,e,d,f}tac with proper context in BNF
traytel
parents: 60207
diff changeset
   661
    fun bd_card_order_tac ctxt = rtac ctxt (bd_card_order_of_bnf bnf) 1;
26ffdb966759 {r,e,d,f}tac with proper context in BNF
traytel
parents: 60207
diff changeset
   662
    fun bd_cinfinite_tac ctxt = rtac ctxt (bd_cinfinite_of_bnf bnf) 1;
26ffdb966759 {r,e,d,f}tac with proper context in BNF
traytel
parents: 60207
diff changeset
   663
    val set_bd_tacs = permute (map (fn thm => fn ctxt => rtac ctxt thm 1) (set_bd_of_bnf bnf));
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   664
49303
blanchet
parents: 49236
diff changeset
   665
    val in_alt_thm =
49155
f51ab68f882f do not trivialize important internal theorem in quick_and_dirty mode
traytel
parents: 49123
diff changeset
   666
      let
49303
blanchet
parents: 49236
diff changeset
   667
        val inx = mk_in Asets sets T;
53038
dd5ea8a51af0 generalized "mk_permute"
blanchet
parents: 52985
diff changeset
   668
        val in_alt = mk_in (unpermute Asets) bnf_sets T;
49303
blanchet
parents: 49236
diff changeset
   669
        val goal = fold_rev Logic.all Asets (mk_Trueprop_eq (inx, in_alt));
49155
f51ab68f882f do not trivialize important internal theorem in quick_and_dirty mode
traytel
parents: 49123
diff changeset
   670
      in
60728
26ffdb966759 {r,e,d,f}tac with proper context in BNF
traytel
parents: 60207
diff changeset
   671
        Goal.prove_sorry lthy [] [] goal (fn {context = ctxt, prems = _} =>
26ffdb966759 {r,e,d,f}tac with proper context in BNF
traytel
parents: 60207
diff changeset
   672
          mk_permute_in_alt_tac ctxt src dest)
70494
41108e3e9ca5 formal position for PThm nodes;
wenzelm
parents: 69593
diff changeset
   673
        |> Thm.close_derivation \<^here>
49155
f51ab68f882f do not trivialize important internal theorem in quick_and_dirty mode
traytel
parents: 49123
diff changeset
   674
      end;
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   675
60728
26ffdb966759 {r,e,d,f}tac with proper context in BNF
traytel
parents: 60207
diff changeset
   676
    fun le_rel_OO_tac ctxt = rtac ctxt (le_rel_OO_of_bnf bnf) 1;
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   677
60728
26ffdb966759 {r,e,d,f}tac with proper context in BNF
traytel
parents: 60207
diff changeset
   678
    fun rel_OO_Grp_tac ctxt = mk_simple_rel_OO_Grp_tac ctxt (rel_OO_Grp_of_bnf bnf) in_alt_thm;
49456
fa8302c8dea1 adapted BNF composition to new relator approach
blanchet
parents: 49455
diff changeset
   679
62324
ae44f16dcea5 make predicator a first-class bnf citizen
traytel
parents: 62316
diff changeset
   680
    fun pred_set_tac ctxt = mk_simple_pred_set_tac ctxt (pred_set_of_bnf bnf) in_alt_thm;
ae44f16dcea5 make predicator a first-class bnf citizen
traytel
parents: 62316
diff changeset
   681
53289
5e0623448bdb renamed BNF axiom
blanchet
parents: 53288
diff changeset
   682
    val tacs = zip_axioms map_id0_tac map_comp0_tac map_cong0_tac set_map0_tacs bd_card_order_tac
62324
ae44f16dcea5 make predicator a first-class bnf citizen
traytel
parents: 62316
diff changeset
   683
      bd_cinfinite_tac set_bd_tacs le_rel_OO_tac rel_OO_Grp_tac pred_set_tac;
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   684
49303
blanchet
parents: 49236
diff changeset
   685
    val wits = map snd (mk_wits_of_bnf (replicate nwits Ds) (replicate nwits As) bnf);
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   686
60752
b48830b670a1 prefer tactics with explicit context;
wenzelm
parents: 60728
diff changeset
   687
    fun wit_tac ctxt = mk_simple_wit_tac ctxt (wit_thms_of_bnf bnf);
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   688
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   689
    val (bnf', lthy') =
56016
8875cdcfc85b unfold intermediate definitions after sealing the bnf
traytel
parents: 56013
diff changeset
   690
      bnf_def Smart_Inline (K Dont_Note) true qualify tacs wit_tac (SOME Ds) Binding.empty
62324
ae44f16dcea5 make predicator a first-class bnf citizen
traytel
parents: 62316
diff changeset
   691
        Binding.empty Binding.empty []
ae44f16dcea5 make predicator a first-class bnf citizen
traytel
parents: 62316
diff changeset
   692
        (((((((b, T), mapx), sets), bd), wits), SOME rel), SOME pred) lthy;
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   693
  in
49503
dbbde075a42e simplified code
blanchet
parents: 49502
diff changeset
   694
    (bnf', (add_bnf_to_unfolds bnf' unfold_set, lthy'))
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   695
  end;
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   696
55904
0ef30d52c5e4 more caching in composition pipeline
blanchet
parents: 55900
diff changeset
   697
fun permute_bnf qualify src dest bnf (accum as ((cache, unfold_set), lthy)) =
0ef30d52c5e4 more caching in composition pipeline
blanchet
parents: 55900
diff changeset
   698
  let val key = key_of_permute src dest bnf in
0ef30d52c5e4 more caching in composition pipeline
blanchet
parents: 55900
diff changeset
   699
    (case Typtab.lookup cache key of
0ef30d52c5e4 more caching in composition pipeline
blanchet
parents: 55900
diff changeset
   700
      SOME (bnf, _) => (bnf, accum)
0ef30d52c5e4 more caching in composition pipeline
blanchet
parents: 55900
diff changeset
   701
    | NONE => cache_comp_simple key cache (raw_permute_bnf qualify src dest bnf (unfold_set, lthy)))
0ef30d52c5e4 more caching in composition pipeline
blanchet
parents: 55900
diff changeset
   702
  end;
0ef30d52c5e4 more caching in composition pipeline
blanchet
parents: 55900
diff changeset
   703
49014
332e5e661675 have "bnf_of_typ" command seal the BNF
blanchet
parents: 48975
diff changeset
   704
(* Composition pipeline *)
332e5e661675 have "bnf_of_typ" command seal the BNF
blanchet
parents: 48975
diff changeset
   705
59725
e5dc7e7744f0 export more ML functions
blanchet
parents: 59710
diff changeset
   706
fun permute_and_kill_bnf qualify n src dest bnf =
55703
a21069381ba5 optimization of 'bnf_of_typ' if all variables are dead
blanchet
parents: 55480
diff changeset
   707
  permute_bnf qualify src dest bnf
49304
blanchet
parents: 49303
diff changeset
   708
  #> uncurry (kill_bnf qualify n);
49014
332e5e661675 have "bnf_of_typ" command seal the BNF
blanchet
parents: 48975
diff changeset
   709
59725
e5dc7e7744f0 export more ML functions
blanchet
parents: 59710
diff changeset
   710
fun lift_and_permute_bnf qualify n src dest bnf =
55703
a21069381ba5 optimization of 'bnf_of_typ' if all variables are dead
blanchet
parents: 55480
diff changeset
   711
  lift_bnf qualify n bnf
49014
332e5e661675 have "bnf_of_typ" command seal the BNF
blanchet
parents: 48975
diff changeset
   712
  #> uncurry (permute_bnf qualify src dest);
332e5e661675 have "bnf_of_typ" command seal the BNF
blanchet
parents: 48975
diff changeset
   713
58332
be0f5d8d511b imported patch phantoms
blanchet
parents: 58297
diff changeset
   714
fun normalize_bnfs qualify Ass Ds flatten_tyargs bnfs accum =
49014
332e5e661675 have "bnf_of_typ" command seal the BNF
blanchet
parents: 48975
diff changeset
   715
  let
332e5e661675 have "bnf_of_typ" command seal the BNF
blanchet
parents: 48975
diff changeset
   716
    val before_kill_src = map (fn As => 0 upto (length As - 1)) Ass;
52985
9e22d6264277 generalized library function
traytel
parents: 52923
diff changeset
   717
    val kill_poss = map (find_indices op = Ds) Ass;
9e22d6264277 generalized library function
traytel
parents: 52923
diff changeset
   718
    val live_poss = map2 (subtract op =) kill_poss before_kill_src;
49014
332e5e661675 have "bnf_of_typ" command seal the BNF
blanchet
parents: 48975
diff changeset
   719
    val before_kill_dest = map2 append kill_poss live_poss;
332e5e661675 have "bnf_of_typ" command seal the BNF
blanchet
parents: 48975
diff changeset
   720
    val kill_ns = map length kill_poss;
55904
0ef30d52c5e4 more caching in composition pipeline
blanchet
parents: 55900
diff changeset
   721
    val (inners', accum') =
59725
e5dc7e7744f0 export more ML functions
blanchet
parents: 59710
diff changeset
   722
      @{fold_map 5} (permute_and_kill_bnf o qualify)
e5dc7e7744f0 export more ML functions
blanchet
parents: 59710
diff changeset
   723
        (if length bnfs = 1 then [0] else 1 upto length bnfs)
55904
0ef30d52c5e4 more caching in composition pipeline
blanchet
parents: 55900
diff changeset
   724
        kill_ns before_kill_src before_kill_dest bnfs accum;
49014
332e5e661675 have "bnf_of_typ" command seal the BNF
blanchet
parents: 48975
diff changeset
   725
332e5e661675 have "bnf_of_typ" command seal the BNF
blanchet
parents: 48975
diff changeset
   726
    val Ass' = map2 (map o nth) Ass live_poss;
58332
be0f5d8d511b imported patch phantoms
blanchet
parents: 58297
diff changeset
   727
    val As = flatten_tyargs Ass';
49014
332e5e661675 have "bnf_of_typ" command seal the BNF
blanchet
parents: 48975
diff changeset
   728
    val after_lift_dest = replicate (length Ass') (0 upto (length As - 1));
332e5e661675 have "bnf_of_typ" command seal the BNF
blanchet
parents: 48975
diff changeset
   729
    val old_poss = map (map (fn x => find_index (fn y => x = y) As)) Ass';
52985
9e22d6264277 generalized library function
traytel
parents: 52923
diff changeset
   730
    val new_poss = map2 (subtract op =) old_poss after_lift_dest;
49014
332e5e661675 have "bnf_of_typ" command seal the BNF
blanchet
parents: 48975
diff changeset
   731
    val after_lift_src = map2 append new_poss old_poss;
332e5e661675 have "bnf_of_typ" command seal the BNF
blanchet
parents: 48975
diff changeset
   732
    val lift_ns = map (fn xs => length As - length xs) Ass';
332e5e661675 have "bnf_of_typ" command seal the BNF
blanchet
parents: 48975
diff changeset
   733
  in
59725
e5dc7e7744f0 export more ML functions
blanchet
parents: 59710
diff changeset
   734
    ((kill_poss, As), @{fold_map 5} (lift_and_permute_bnf o qualify)
55703
a21069381ba5 optimization of 'bnf_of_typ' if all variables are dead
blanchet
parents: 55480
diff changeset
   735
      (if length bnfs = 1 then [0] else 1 upto length bnfs)
55904
0ef30d52c5e4 more caching in composition pipeline
blanchet
parents: 55900
diff changeset
   736
      lift_ns after_lift_src after_lift_dest inners' accum')
49014
332e5e661675 have "bnf_of_typ" command seal the BNF
blanchet
parents: 48975
diff changeset
   737
  end;
332e5e661675 have "bnf_of_typ" command seal the BNF
blanchet
parents: 48975
diff changeset
   738
332e5e661675 have "bnf_of_typ" command seal the BNF
blanchet
parents: 48975
diff changeset
   739
fun default_comp_sort Ass =
59058
a78612c67ec0 renamed "pairself" to "apply2", in accordance to @{apply 2};
wenzelm
parents: 58959
diff changeset
   740
  Library.sort (Term_Ord.typ_ord o apply2 TFree) (fold (fold (insert (op =))) Ass []);
49014
332e5e661675 have "bnf_of_typ" command seal the BNF
blanchet
parents: 48975
diff changeset
   741
58332
be0f5d8d511b imported patch phantoms
blanchet
parents: 58297
diff changeset
   742
fun raw_compose_bnf const_policy qualify flatten_tyargs outer inners oDs Dss tfreess accum =
49014
332e5e661675 have "bnf_of_typ" command seal the BNF
blanchet
parents: 48975
diff changeset
   743
  let
49425
f27f83f71e94 cleaned up internal naming scheme for bnfs
traytel
parents: 49304
diff changeset
   744
    val b = name_of_bnf outer;
49014
332e5e661675 have "bnf_of_typ" command seal the BNF
blanchet
parents: 48975
diff changeset
   745
49121
9e0acaa470ab more work on FP sugar
blanchet
parents: 49109
diff changeset
   746
    val Ass = map (map Term.dest_TFree) tfreess;
49014
332e5e661675 have "bnf_of_typ" command seal the BNF
blanchet
parents: 48975
diff changeset
   747
    val Ds = fold (fold Term.add_tfreesT) (oDs :: Dss) [];
332e5e661675 have "bnf_of_typ" command seal the BNF
blanchet
parents: 48975
diff changeset
   748
55904
0ef30d52c5e4 more caching in composition pipeline
blanchet
parents: 55900
diff changeset
   749
    val ((kill_poss, As), (inners', ((cache', unfold_set'), lthy'))) =
58332
be0f5d8d511b imported patch phantoms
blanchet
parents: 58297
diff changeset
   750
      normalize_bnfs qualify Ass Ds flatten_tyargs inners accum;
49014
332e5e661675 have "bnf_of_typ" command seal the BNF
blanchet
parents: 48975
diff changeset
   751
61760
1647bb489522 tuned whitespace
blanchet
parents: 61242
diff changeset
   752
    val Ds =
1647bb489522 tuned whitespace
blanchet
parents: 61242
diff changeset
   753
      oDs @ flat (@{map 3} (uncurry append oo curry swap oo map o nth) tfreess kill_poss Dss);
49014
332e5e661675 have "bnf_of_typ" command seal the BNF
blanchet
parents: 48975
diff changeset
   754
    val As = map TFree As;
332e5e661675 have "bnf_of_typ" command seal the BNF
blanchet
parents: 48975
diff changeset
   755
  in
49425
f27f83f71e94 cleaned up internal naming scheme for bnfs
traytel
parents: 49304
diff changeset
   756
    apfst (rpair (Ds, As))
55904
0ef30d52c5e4 more caching in composition pipeline
blanchet
parents: 55900
diff changeset
   757
      (apsnd (apfst (pair cache'))
0ef30d52c5e4 more caching in composition pipeline
blanchet
parents: 55900
diff changeset
   758
        (clean_compose_bnf const_policy (qualify 0) b outer inners' (unfold_set', lthy')))
0ef30d52c5e4 more caching in composition pipeline
blanchet
parents: 55900
diff changeset
   759
  end;
0ef30d52c5e4 more caching in composition pipeline
blanchet
parents: 55900
diff changeset
   760
58332
be0f5d8d511b imported patch phantoms
blanchet
parents: 58297
diff changeset
   761
fun compose_bnf const_policy qualify flatten_tyargs outer inners oDs Dss tfreess
be0f5d8d511b imported patch phantoms
blanchet
parents: 58297
diff changeset
   762
    (accum as ((cache, _), _)) =
55904
0ef30d52c5e4 more caching in composition pipeline
blanchet
parents: 55900
diff changeset
   763
  let val key = key_of_compose oDs Dss tfreess outer inners in
0ef30d52c5e4 more caching in composition pipeline
blanchet
parents: 55900
diff changeset
   764
    (case Typtab.lookup cache key of
0ef30d52c5e4 more caching in composition pipeline
blanchet
parents: 55900
diff changeset
   765
      SOME bnf_Ds_As => (bnf_Ds_As, accum)
0ef30d52c5e4 more caching in composition pipeline
blanchet
parents: 55900
diff changeset
   766
    | NONE =>
58332
be0f5d8d511b imported patch phantoms
blanchet
parents: 58297
diff changeset
   767
      cache_comp key
be0f5d8d511b imported patch phantoms
blanchet
parents: 58297
diff changeset
   768
        (raw_compose_bnf const_policy qualify flatten_tyargs outer inners oDs Dss tfreess accum))
49014
332e5e661675 have "bnf_of_typ" command seal the BNF
blanchet
parents: 48975
diff changeset
   769
  end;
332e5e661675 have "bnf_of_typ" command seal the BNF
blanchet
parents: 48975
diff changeset
   770
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   771
(* Hide the type of the bound (optimization) and unfold the definitions (nicer to the user) *)
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   772
55803
74d3fe9031d8 joint work with blanchet: intermediate typedef for the input to fp-operations
traytel
parents: 55707
diff changeset
   773
type absT_info =
74d3fe9031d8 joint work with blanchet: intermediate typedef for the input to fp-operations
traytel
parents: 55707
diff changeset
   774
  {absT: typ,
74d3fe9031d8 joint work with blanchet: intermediate typedef for the input to fp-operations
traytel
parents: 55707
diff changeset
   775
   repT: typ,
74d3fe9031d8 joint work with blanchet: intermediate typedef for the input to fp-operations
traytel
parents: 55707
diff changeset
   776
   abs: term,
74d3fe9031d8 joint work with blanchet: intermediate typedef for the input to fp-operations
traytel
parents: 55707
diff changeset
   777
   rep: term,
74d3fe9031d8 joint work with blanchet: intermediate typedef for the input to fp-operations
traytel
parents: 55707
diff changeset
   778
   abs_inject: thm,
74d3fe9031d8 joint work with blanchet: intermediate typedef for the input to fp-operations
traytel
parents: 55707
diff changeset
   779
   abs_inverse: thm,
74d3fe9031d8 joint work with blanchet: intermediate typedef for the input to fp-operations
traytel
parents: 55707
diff changeset
   780
   type_definition: thm};
74d3fe9031d8 joint work with blanchet: intermediate typedef for the input to fp-operations
traytel
parents: 55707
diff changeset
   781
74d3fe9031d8 joint work with blanchet: intermediate typedef for the input to fp-operations
traytel
parents: 55707
diff changeset
   782
fun morph_absT_info phi
74d3fe9031d8 joint work with blanchet: intermediate typedef for the input to fp-operations
traytel
parents: 55707
diff changeset
   783
  {absT, repT, abs, rep, abs_inject, abs_inverse, type_definition} =
74d3fe9031d8 joint work with blanchet: intermediate typedef for the input to fp-operations
traytel
parents: 55707
diff changeset
   784
  {absT = Morphism.typ phi absT,
74d3fe9031d8 joint work with blanchet: intermediate typedef for the input to fp-operations
traytel
parents: 55707
diff changeset
   785
   repT = Morphism.typ phi repT,
74d3fe9031d8 joint work with blanchet: intermediate typedef for the input to fp-operations
traytel
parents: 55707
diff changeset
   786
   abs = Morphism.term phi abs,
74d3fe9031d8 joint work with blanchet: intermediate typedef for the input to fp-operations
traytel
parents: 55707
diff changeset
   787
   rep = Morphism.term phi rep,
74d3fe9031d8 joint work with blanchet: intermediate typedef for the input to fp-operations
traytel
parents: 55707
diff changeset
   788
   abs_inject = Morphism.thm phi abs_inject,
74d3fe9031d8 joint work with blanchet: intermediate typedef for the input to fp-operations
traytel
parents: 55707
diff changeset
   789
   abs_inverse = Morphism.thm phi abs_inverse,
74d3fe9031d8 joint work with blanchet: intermediate typedef for the input to fp-operations
traytel
parents: 55707
diff changeset
   790
   type_definition = Morphism.thm phi type_definition};
74d3fe9031d8 joint work with blanchet: intermediate typedef for the input to fp-operations
traytel
parents: 55707
diff changeset
   791
74d3fe9031d8 joint work with blanchet: intermediate typedef for the input to fp-operations
traytel
parents: 55707
diff changeset
   792
fun mk_absT thy repT absT repU =
55900
21aa30ea6806 propagate the exception that is expected later on
traytel
parents: 55856
diff changeset
   793
  let
56634
a001337c8d24 tuned whitespace
blanchet
parents: 56254
diff changeset
   794
    val rho = Vartab.fold (cons o apsnd snd) (Sign.typ_match thy (repT, repU) Vartab.empty) [];
55900
21aa30ea6806 propagate the exception that is expected later on
traytel
parents: 55856
diff changeset
   795
  in Term.typ_subst_TVars rho absT end
21aa30ea6806 propagate the exception that is expected later on
traytel
parents: 55856
diff changeset
   796
  handle Type.TYPE_MATCH => raise Term.TYPE ("mk_absT", [repT, absT, repU], []);
55803
74d3fe9031d8 joint work with blanchet: intermediate typedef for the input to fp-operations
traytel
parents: 55707
diff changeset
   797
55854
ee270328a781 make 'typedef' optional, depending on size of original type
blanchet
parents: 55853
diff changeset
   798
fun mk_repT absT repT absU =
ee270328a781 make 'typedef' optional, depending on size of original type
blanchet
parents: 55853
diff changeset
   799
  if absT = repT then absU
ee270328a781 make 'typedef' optional, depending on size of original type
blanchet
parents: 55853
diff changeset
   800
  else
ee270328a781 make 'typedef' optional, depending on size of original type
blanchet
parents: 55853
diff changeset
   801
    (case (absT, absU) of
ee270328a781 make 'typedef' optional, depending on size of original type
blanchet
parents: 55853
diff changeset
   802
      (Type (C, Ts), Type (C', Us)) =>
ee270328a781 make 'typedef' optional, depending on size of original type
blanchet
parents: 55853
diff changeset
   803
        if C = C' then Term.typ_subst_atomic (Ts ~~ Us) repT
62684
cb20e8828196 document that n2m does not depend on most things in fp_sugar in its type
traytel
parents: 62621
diff changeset
   804
        else raise Term.TYPE ("mk_repT", [absT, repT, absU], [])
cb20e8828196 document that n2m does not depend on most things in fp_sugar in its type
traytel
parents: 62621
diff changeset
   805
    | _ => raise Term.TYPE ("mk_repT", [absT, repT, absU], []));
55803
74d3fe9031d8 joint work with blanchet: intermediate typedef for the input to fp-operations
traytel
parents: 55707
diff changeset
   806
69593
3dda49e08b9d isabelle update -u control_cartouches;
wenzelm
parents: 68960
diff changeset
   807
fun mk_abs_or_rep _ absU (Const (\<^const_name>\<open>id_bnf\<close>, _)) =
3dda49e08b9d isabelle update -u control_cartouches;
wenzelm
parents: 68960
diff changeset
   808
    Const (\<^const_name>\<open>id_bnf\<close>, absU --> absU)
55854
ee270328a781 make 'typedef' optional, depending on size of original type
blanchet
parents: 55853
diff changeset
   809
  | mk_abs_or_rep getT (Type (_, Us)) abs =
ee270328a781 make 'typedef' optional, depending on size of original type
blanchet
parents: 55853
diff changeset
   810
    let val Ts = snd (dest_Type (getT (fastype_of abs)))
ee270328a781 make 'typedef' optional, depending on size of original type
blanchet
parents: 55853
diff changeset
   811
    in Term.subst_atomic_types (Ts ~~ Us) abs end;
55803
74d3fe9031d8 joint work with blanchet: intermediate typedef for the input to fp-operations
traytel
parents: 55707
diff changeset
   812
74d3fe9031d8 joint work with blanchet: intermediate typedef for the input to fp-operations
traytel
parents: 55707
diff changeset
   813
val mk_abs = mk_abs_or_rep range_type;
74d3fe9031d8 joint work with blanchet: intermediate typedef for the input to fp-operations
traytel
parents: 55707
diff changeset
   814
val mk_rep = mk_abs_or_rep domain_type;
74d3fe9031d8 joint work with blanchet: intermediate typedef for the input to fp-operations
traytel
parents: 55707
diff changeset
   815
63802
94336cf98486 generalized ML signature
blanchet
parents: 63800
diff changeset
   816
fun maybe_typedef force_out_of_line (b, As, mx) set opt_morphs tac lthy =
55854
ee270328a781 make 'typedef' optional, depending on size of original type
blanchet
parents: 55853
diff changeset
   817
  let
63802
94336cf98486 generalized ML signature
blanchet
parents: 63800
diff changeset
   818
    val threshold = Config.get lthy typedef_threshold;
55854
ee270328a781 make 'typedef' optional, depending on size of original type
blanchet
parents: 55853
diff changeset
   819
    val repT = HOLogic.dest_setT (fastype_of set);
59710
4aa63424ba89 inlining threshold
blanchet
parents: 59131
diff changeset
   820
    val out_of_line = force_out_of_line orelse
59994
19e5f5ac7b59 renamed misleading option
blanchet
parents: 59957
diff changeset
   821
      (threshold >= 0 andalso Term.size_of_typ repT >= threshold);
55854
ee270328a781 make 'typedef' optional, depending on size of original type
blanchet
parents: 55853
diff changeset
   822
  in
58332
be0f5d8d511b imported patch phantoms
blanchet
parents: 58297
diff changeset
   823
    if out_of_line then
63802
94336cf98486 generalized ML signature
blanchet
parents: 63800
diff changeset
   824
      typedef (b, As, mx) set opt_morphs tac lthy
94336cf98486 generalized ML signature
blanchet
parents: 63800
diff changeset
   825
      |>> (fn (T_name, ({Rep_name, Abs_name, ...},
58332
be0f5d8d511b imported patch phantoms
blanchet
parents: 58297
diff changeset
   826
          {type_definition, Abs_inverse, Abs_inject, Abs_cases, ...}) : Typedef.info) =>
be0f5d8d511b imported patch phantoms
blanchet
parents: 58297
diff changeset
   827
        (Type (T_name, map TFree As),
be0f5d8d511b imported patch phantoms
blanchet
parents: 58297
diff changeset
   828
          (Rep_name, Abs_name, type_definition, Abs_inverse, Abs_inject, Abs_cases)))
be0f5d8d511b imported patch phantoms
blanchet
parents: 58297
diff changeset
   829
    else
63802
94336cf98486 generalized ML signature
blanchet
parents: 63800
diff changeset
   830
      ((repT,
69593
3dda49e08b9d isabelle update -u control_cartouches;
wenzelm
parents: 68960
diff changeset
   831
        (\<^const_name>\<open>id_bnf\<close>, \<^const_name>\<open>id_bnf\<close>,
58181
6d527272f7b2 renamed internal constant
blanchet
parents: 58128
diff changeset
   832
         @{thm type_definition_id_bnf_UNIV},
6d527272f7b2 renamed internal constant
blanchet
parents: 58128
diff changeset
   833
         @{thm type_definition.Abs_inverse[OF type_definition_id_bnf_UNIV]},
6d527272f7b2 renamed internal constant
blanchet
parents: 58128
diff changeset
   834
         @{thm type_definition.Abs_inject[OF type_definition_id_bnf_UNIV]},
63802
94336cf98486 generalized ML signature
blanchet
parents: 63800
diff changeset
   835
         @{thm type_definition.Abs_cases[OF type_definition_id_bnf_UNIV]})), lthy)
55854
ee270328a781 make 'typedef' optional, depending on size of original type
blanchet
parents: 55853
diff changeset
   836
  end;
ee270328a781 make 'typedef' optional, depending on size of original type
blanchet
parents: 55853
diff changeset
   837
63837
fdf90aa59868 provide a mechanism for ensuring dead type variables occur in typedef if desired
blanchet
parents: 63836
diff changeset
   838
fun seal_bnf qualify (unfold_set : unfold_set) b force_out_of_line Ds all_Ds bnf lthy =
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   839
  let
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   840
    val live = live_of_bnf bnf;
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   841
    val nwits = nwits_of_bnf bnf;
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   842
58332
be0f5d8d511b imported patch phantoms
blanchet
parents: 58297
diff changeset
   843
    val ((As, As'), lthy1) = apfst (`(map TFree))
69593
3dda49e08b9d isabelle update -u control_cartouches;
wenzelm
parents: 68960
diff changeset
   844
      (Variable.invent_types (replicate live \<^sort>\<open>type\<close>) (fold Variable.declare_typ all_Ds lthy));
3dda49e08b9d isabelle update -u control_cartouches;
wenzelm
parents: 68960
diff changeset
   845
    val (Bs, _) = apfst (map TFree) (Variable.invent_types (replicate live \<^sort>\<open>type\<close>) lthy1);
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   846
62324
ae44f16dcea5 make predicator a first-class bnf citizen
traytel
parents: 62316
diff changeset
   847
    val ((((fs, fs'), (Rs, Rs')), (Ps, Ps')), _(*names_lthy*)) = lthy
55803
74d3fe9031d8 joint work with blanchet: intermediate typedef for the input to fp-operations
traytel
parents: 55707
diff changeset
   848
      |> mk_Frees' "f" (map2 (curry op -->) As Bs)
62324
ae44f16dcea5 make predicator a first-class bnf citizen
traytel
parents: 62316
diff changeset
   849
      ||>> mk_Frees' "R" (map2 mk_pred2T As Bs)
ae44f16dcea5 make predicator a first-class bnf citizen
traytel
parents: 62316
diff changeset
   850
      ||>> mk_Frees' "P" (map mk_pred1T As);
55803
74d3fe9031d8 joint work with blanchet: intermediate typedef for the input to fp-operations
traytel
parents: 55707
diff changeset
   851
74d3fe9031d8 joint work with blanchet: intermediate typedef for the input to fp-operations
traytel
parents: 55707
diff changeset
   852
    val repTA = mk_T_of_bnf Ds As bnf;
74d3fe9031d8 joint work with blanchet: intermediate typedef for the input to fp-operations
traytel
parents: 55707
diff changeset
   853
    val T_bind = qualify b;
63836
2f9ee7d85d85 preserve order of dead variables
blanchet
parents: 63824
diff changeset
   854
    val repTA_tfrees = Term.add_tfreesT repTA [];
63837
fdf90aa59868 provide a mechanism for ensuring dead type variables occur in typedef if desired
blanchet
parents: 63836
diff changeset
   855
    val all_TA_params_in_order = fold_rev Term.add_tfreesT all_Ds As';
59821
fd3a7692e083 preserve order of type arguments in pre-FP BNF typedef
blanchet
parents: 59820
diff changeset
   856
    val TA_params =
63802
94336cf98486 generalized ML signature
blanchet
parents: 63800
diff changeset
   857
      (if force_out_of_line then all_TA_params_in_order
63836
2f9ee7d85d85 preserve order of dead variables
blanchet
parents: 63824
diff changeset
   858
       else inter (op =) repTA_tfrees all_TA_params_in_order);
56012
158dc03db8be made typedef for the type of the bound optional (size-based)
traytel
parents: 56010
diff changeset
   859
    val ((TA, (Rep_name, Abs_name, type_definition, Abs_inverse, Abs_inject, _)), lthy) =
63802
94336cf98486 generalized ML signature
blanchet
parents: 63800
diff changeset
   860
      maybe_typedef force_out_of_line (T_bind, TA_params, NoSyn) (HOLogic.mk_UNIV repTA) NONE
60728
26ffdb966759 {r,e,d,f}tac with proper context in BNF
traytel
parents: 60207
diff changeset
   861
        (fn ctxt => EVERY' [rtac ctxt exI, rtac ctxt UNIV_I] 1) lthy;
55854
ee270328a781 make 'typedef' optional, depending on size of original type
blanchet
parents: 55853
diff changeset
   862
ee270328a781 make 'typedef' optional, depending on size of original type
blanchet
parents: 55853
diff changeset
   863
    val repTB = mk_T_of_bnf Ds Bs bnf;
ee270328a781 make 'typedef' optional, depending on size of original type
blanchet
parents: 55853
diff changeset
   864
    val TB = Term.typ_subst_atomic (As ~~ Bs) TA;
ee270328a781 make 'typedef' optional, depending on size of original type
blanchet
parents: 55853
diff changeset
   865
    val RepA = Const (Rep_name, TA --> repTA);
ee270328a781 make 'typedef' optional, depending on size of original type
blanchet
parents: 55853
diff changeset
   866
    val RepB = Const (Rep_name, TB --> repTB);
ee270328a781 make 'typedef' optional, depending on size of original type
blanchet
parents: 55853
diff changeset
   867
    val AbsA = Const (Abs_name, repTA --> TA);
ee270328a781 make 'typedef' optional, depending on size of original type
blanchet
parents: 55853
diff changeset
   868
    val AbsB = Const (Abs_name, repTB --> TB);
ee270328a781 make 'typedef' optional, depending on size of original type
blanchet
parents: 55853
diff changeset
   869
    val Abs_inject' = Abs_inject OF @{thms UNIV_I UNIV_I};
ee270328a781 make 'typedef' optional, depending on size of original type
blanchet
parents: 55853
diff changeset
   870
    val Abs_inverse' = Abs_inverse OF @{thms UNIV_I};
55803
74d3fe9031d8 joint work with blanchet: intermediate typedef for the input to fp-operations
traytel
parents: 55707
diff changeset
   871
74d3fe9031d8 joint work with blanchet: intermediate typedef for the input to fp-operations
traytel
parents: 55707
diff changeset
   872
    val absT_info = {absT = TA, repT = repTA, abs = AbsA, rep = RepA, abs_inject = Abs_inject',
55854
ee270328a781 make 'typedef' optional, depending on size of original type
blanchet
parents: 55853
diff changeset
   873
      abs_inverse = Abs_inverse', type_definition = type_definition};
55803
74d3fe9031d8 joint work with blanchet: intermediate typedef for the input to fp-operations
traytel
parents: 55707
diff changeset
   874
74d3fe9031d8 joint work with blanchet: intermediate typedef for the input to fp-operations
traytel
parents: 55707
diff changeset
   875
    val bnf_map = fold_rev Term.absfree fs' (HOLogic.mk_comp (HOLogic.mk_comp (AbsB,
56016
8875cdcfc85b unfold intermediate definitions after sealing the bnf
traytel
parents: 56013
diff changeset
   876
      Term.list_comb (mk_map_of_bnf Ds As Bs bnf, fs)), RepA));
8875cdcfc85b unfold intermediate definitions after sealing the bnf
traytel
parents: 56013
diff changeset
   877
    val bnf_sets = map ((fn t => HOLogic.mk_comp (t, RepA)))
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   878
      (mk_sets_of_bnf (replicate live Ds) (replicate live As) bnf);
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   879
    val bnf_bd = mk_bd_of_bnf Ds As bnf;
55803
74d3fe9031d8 joint work with blanchet: intermediate typedef for the input to fp-operations
traytel
parents: 55707
diff changeset
   880
    val bnf_rel = fold_rev Term.absfree Rs' (mk_vimage2p RepA RepB $
56016
8875cdcfc85b unfold intermediate definitions after sealing the bnf
traytel
parents: 56013
diff changeset
   881
      (Term.list_comb (mk_rel_of_bnf Ds As Bs bnf, Rs)));
62324
ae44f16dcea5 make predicator a first-class bnf citizen
traytel
parents: 62316
diff changeset
   882
    val bnf_pred = fold_rev Term.absfree Ps' (HOLogic.mk_comp
ae44f16dcea5 make predicator a first-class bnf citizen
traytel
parents: 62316
diff changeset
   883
      (Term.list_comb (mk_pred_of_bnf Ds As bnf, Ps), RepA));
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   884
55704
a97b9b81e195 optimized 'bnf_of_typ' further w.r.t. dead variables
blanchet
parents: 55703
diff changeset
   885
    (*bd may depend only on dead type variables*)
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   886
    val bd_repT = fst (dest_relT (fastype_of bnf_bd));
53264
1973b821168c qualify generated constants uniformly
blanchet
parents: 53222
diff changeset
   887
    val bdT_bind = qualify (Binding.suffix_name ("_" ^ bdTN) b);
55707
50cf04dd2584 clarified interaction with dead variables in the composition of BNFs
traytel
parents: 55706
diff changeset
   888
    val params = Term.add_tfreesT bd_repT [];
63837
fdf90aa59868 provide a mechanism for ensuring dead type variables occur in typedef if desired
blanchet
parents: 63836
diff changeset
   889
    val all_deads = map TFree (fold_rev Term.add_tfreesT all_Ds []);
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   890
56012
158dc03db8be made typedef for the type of the bound optional (size-based)
traytel
parents: 56010
diff changeset
   891
    val ((bdT, (_, Abs_bd_name, _, _, Abs_bdT_inject, Abs_bdT_cases)), lthy) =
63802
94336cf98486 generalized ML signature
blanchet
parents: 63800
diff changeset
   892
      maybe_typedef false (bdT_bind, params, NoSyn) (HOLogic.mk_UNIV bd_repT) NONE
94336cf98486 generalized ML signature
blanchet
parents: 63800
diff changeset
   893
        (fn ctxt => EVERY' [rtac ctxt exI, rtac ctxt UNIV_I] 1) lthy;
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   894
56012
158dc03db8be made typedef for the type of the bound optional (size-based)
traytel
parents: 56010
diff changeset
   895
    val (bnf_bd', bd_ordIso, bd_card_order, bd_cinfinite) =
158dc03db8be made typedef for the type of the bound optional (size-based)
traytel
parents: 56010
diff changeset
   896
      if bdT = bd_repT then (bnf_bd, bd_Card_order_of_bnf bnf RS @{thm ordIso_refl},
158dc03db8be made typedef for the type of the bound optional (size-based)
traytel
parents: 56010
diff changeset
   897
        bd_card_order_of_bnf bnf, bd_cinfinite_of_bnf bnf)
158dc03db8be made typedef for the type of the bound optional (size-based)
traytel
parents: 56010
diff changeset
   898
      else
158dc03db8be made typedef for the type of the bound optional (size-based)
traytel
parents: 56010
diff changeset
   899
        let
158dc03db8be made typedef for the type of the bound optional (size-based)
traytel
parents: 56010
diff changeset
   900
          val bnf_bd' = mk_dir_image bnf_bd (Const (Abs_bd_name, bd_repT --> bdT));
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   901
56012
158dc03db8be made typedef for the type of the bound optional (size-based)
traytel
parents: 56010
diff changeset
   902
          val Abs_bdT_inj = mk_Abs_inj_thm Abs_bdT_inject;
158dc03db8be made typedef for the type of the bound optional (size-based)
traytel
parents: 56010
diff changeset
   903
          val Abs_bdT_bij = mk_Abs_bij_thm lthy Abs_bdT_inj Abs_bdT_cases;
57567
d554b0097ad4 add mk_Trueprop_mem utility function
desharna
parents: 56634
diff changeset
   904
56012
158dc03db8be made typedef for the type of the bound optional (size-based)
traytel
parents: 56010
diff changeset
   905
          val bd_ordIso = @{thm dir_image} OF [Abs_bdT_inj, bd_Card_order_of_bnf bnf];
158dc03db8be made typedef for the type of the bound optional (size-based)
traytel
parents: 56010
diff changeset
   906
          val bd_card_order =
158dc03db8be made typedef for the type of the bound optional (size-based)
traytel
parents: 56010
diff changeset
   907
            @{thm card_order_dir_image} OF [Abs_bdT_bij, bd_card_order_of_bnf bnf];
158dc03db8be made typedef for the type of the bound optional (size-based)
traytel
parents: 56010
diff changeset
   908
          val bd_cinfinite =
158dc03db8be made typedef for the type of the bound optional (size-based)
traytel
parents: 56010
diff changeset
   909
            (@{thm Cinfinite_cong} OF [bd_ordIso, bd_Cinfinite_of_bnf bnf]) RS conjunct1;
158dc03db8be made typedef for the type of the bound optional (size-based)
traytel
parents: 56010
diff changeset
   910
        in
158dc03db8be made typedef for the type of the bound optional (size-based)
traytel
parents: 56010
diff changeset
   911
          (bnf_bd', bd_ordIso, bd_card_order, bd_cinfinite)
158dc03db8be made typedef for the type of the bound optional (size-based)
traytel
parents: 56010
diff changeset
   912
        end;
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   913
60728
26ffdb966759 {r,e,d,f}tac with proper context in BNF
traytel
parents: 60207
diff changeset
   914
    fun map_id0_tac ctxt =
26ffdb966759 {r,e,d,f}tac with proper context in BNF
traytel
parents: 60207
diff changeset
   915
      rtac ctxt (@{thm type_copy_map_id0} OF [type_definition, map_id0_of_bnf bnf]) 1;
26ffdb966759 {r,e,d,f}tac with proper context in BNF
traytel
parents: 60207
diff changeset
   916
    fun map_comp0_tac ctxt =
26ffdb966759 {r,e,d,f}tac with proper context in BNF
traytel
parents: 60207
diff changeset
   917
      rtac ctxt (@{thm type_copy_map_comp0} OF [type_definition, map_comp0_of_bnf bnf]) 1;
26ffdb966759 {r,e,d,f}tac with proper context in BNF
traytel
parents: 60207
diff changeset
   918
    fun map_cong0_tac ctxt =
26ffdb966759 {r,e,d,f}tac with proper context in BNF
traytel
parents: 60207
diff changeset
   919
      EVERY' (rtac ctxt @{thm type_copy_map_cong0} :: rtac ctxt (map_cong0_of_bnf bnf) ::
26ffdb966759 {r,e,d,f}tac with proper context in BNF
traytel
parents: 60207
diff changeset
   920
        map (fn i => EVERY' [select_prem_tac ctxt live (dtac ctxt meta_spec) i, etac ctxt meta_mp,
26ffdb966759 {r,e,d,f}tac with proper context in BNF
traytel
parents: 60207
diff changeset
   921
          etac ctxt (o_apply RS equalityD2 RS set_mp)]) (1 upto live)) 1;
26ffdb966759 {r,e,d,f}tac with proper context in BNF
traytel
parents: 60207
diff changeset
   922
    fun set_map0_tac thm ctxt =
26ffdb966759 {r,e,d,f}tac with proper context in BNF
traytel
parents: 60207
diff changeset
   923
      rtac ctxt (@{thm type_copy_set_map0} OF [type_definition, thm]) 1;
26ffdb966759 {r,e,d,f}tac with proper context in BNF
traytel
parents: 60207
diff changeset
   924
    val set_bd_tacs = map (fn thm => fn ctxt => rtac ctxt (@{thm ordLeq_ordIso_trans} OF
56016
8875cdcfc85b unfold intermediate definitions after sealing the bnf
traytel
parents: 56013
diff changeset
   925
        [thm, bd_ordIso] RS @{thm type_copy_set_bd}) 1) (set_bd_of_bnf bnf);
60728
26ffdb966759 {r,e,d,f}tac with proper context in BNF
traytel
parents: 60207
diff changeset
   926
    fun le_rel_OO_tac ctxt =
26ffdb966759 {r,e,d,f}tac with proper context in BNF
traytel
parents: 60207
diff changeset
   927
      rtac ctxt (le_rel_OO_of_bnf bnf RS @{thm vimage2p_relcompp_mono}) 1;
55803
74d3fe9031d8 joint work with blanchet: intermediate typedef for the input to fp-operations
traytel
parents: 55707
diff changeset
   928
    fun rel_OO_Grp_tac ctxt =
60728
26ffdb966759 {r,e,d,f}tac with proper context in BNF
traytel
parents: 60207
diff changeset
   929
      (rtac ctxt (rel_OO_Grp_of_bnf bnf RS @{thm vimage2p_cong} RS trans) THEN'
63802
94336cf98486 generalized ML signature
blanchet
parents: 63800
diff changeset
   930
       (if force_out_of_line then subst_tac ctxt NONE else SELECT_GOAL o unfold_thms_tac ctxt)
58359
3782c7b0d1cc avoid 'subst_tac' when possible (it is suspected of not helping 'HOL-Proofs')
blanchet
parents: 58332
diff changeset
   931
         [type_definition RS @{thm vimage2p_relcompp_converse}] THEN'
58332
be0f5d8d511b imported patch phantoms
blanchet
parents: 58297
diff changeset
   932
       SELECT_GOAL (unfold_thms_tac ctxt [o_apply,
be0f5d8d511b imported patch phantoms
blanchet
parents: 58297
diff changeset
   933
         type_definition RS @{thm type_copy_vimage2p_Grp_Rep},
be0f5d8d511b imported patch phantoms
blanchet
parents: 58297
diff changeset
   934
         type_definition RS @{thm vimage2p_relcompp_converse}]) THEN'
60728
26ffdb966759 {r,e,d,f}tac with proper context in BNF
traytel
parents: 60207
diff changeset
   935
       rtac ctxt refl) 1;
62324
ae44f16dcea5 make predicator a first-class bnf citizen
traytel
parents: 62316
diff changeset
   936
    fun pred_set_tac ctxt =
ae44f16dcea5 make predicator a first-class bnf citizen
traytel
parents: 62316
diff changeset
   937
      HEADGOAL (EVERY'
67091
1393c2340eec more symbols;
wenzelm
parents: 65436
diff changeset
   938
        [rtac ctxt (pred_set_of_bnf bnf RS @{thm arg_cong[of _ _ "\<lambda>f. f \<circ> _"]} RS trans),
62324
ae44f16dcea5 make predicator a first-class bnf citizen
traytel
parents: 62316
diff changeset
   939
        SELECT_GOAL (unfold_thms_tac ctxt (@{thms Ball_comp_iff conj_comp_iff})), rtac ctxt refl]);
49456
fa8302c8dea1 adapted BNF composition to new relator approach
blanchet
parents: 49455
diff changeset
   940
55803
74d3fe9031d8 joint work with blanchet: intermediate typedef for the input to fp-operations
traytel
parents: 55707
diff changeset
   941
    val tacs = zip_axioms map_id0_tac map_comp0_tac map_cong0_tac
60728
26ffdb966759 {r,e,d,f}tac with proper context in BNF
traytel
parents: 60207
diff changeset
   942
      (map set_map0_tac (set_map0_of_bnf bnf))
26ffdb966759 {r,e,d,f}tac with proper context in BNF
traytel
parents: 60207
diff changeset
   943
      (fn ctxt => rtac ctxt bd_card_order 1) (fn ctxt => rtac ctxt bd_cinfinite 1)
62324
ae44f16dcea5 make predicator a first-class bnf citizen
traytel
parents: 62316
diff changeset
   944
      set_bd_tacs le_rel_OO_tac rel_OO_Grp_tac pred_set_tac;
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   945
55803
74d3fe9031d8 joint work with blanchet: intermediate typedef for the input to fp-operations
traytel
parents: 55707
diff changeset
   946
    val bnf_wits = map (fn (I, t) =>
74d3fe9031d8 joint work with blanchet: intermediate typedef for the input to fp-operations
traytel
parents: 55707
diff changeset
   947
        fold Term.absdummy (map (nth As) I)
56016
8875cdcfc85b unfold intermediate definitions after sealing the bnf
traytel
parents: 56013
diff changeset
   948
          (AbsA $ Term.list_comb (t, map Bound (0 upto length I - 1))))
55803
74d3fe9031d8 joint work with blanchet: intermediate typedef for the input to fp-operations
traytel
parents: 55707
diff changeset
   949
      (mk_wits_of_bnf (replicate nwits Ds) (replicate nwits As) bnf);
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   950
60752
b48830b670a1 prefer tactics with explicit context;
wenzelm
parents: 60728
diff changeset
   951
    fun wit_tac ctxt =
b48830b670a1 prefer tactics with explicit context;
wenzelm
parents: 60728
diff changeset
   952
      ALLGOALS (dtac ctxt (type_definition RS @{thm type_copy_wit})) THEN
b48830b670a1 prefer tactics with explicit context;
wenzelm
parents: 60728
diff changeset
   953
      mk_simple_wit_tac ctxt (wit_thms_of_bnf bnf);
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   954
53264
1973b821168c qualify generated constants uniformly
blanchet
parents: 53222
diff changeset
   955
    val (bnf', lthy') =
56016
8875cdcfc85b unfold intermediate definitions after sealing the bnf
traytel
parents: 56013
diff changeset
   956
      bnf_def Hardly_Inline (user_policy Dont_Note) true qualify tacs wit_tac (SOME all_deads)
62324
ae44f16dcea5 make predicator a first-class bnf citizen
traytel
parents: 62316
diff changeset
   957
        Binding.empty Binding.empty Binding.empty []
ae44f16dcea5 make predicator a first-class bnf citizen
traytel
parents: 62316
diff changeset
   958
        (((((((b, TA), bnf_map), bnf_sets), bnf_bd'), bnf_wits), SOME bnf_rel), SOME bnf_pred) lthy;
56016
8875cdcfc85b unfold intermediate definitions after sealing the bnf
traytel
parents: 56013
diff changeset
   959
58181
6d527272f7b2 renamed internal constant
blanchet
parents: 58128
diff changeset
   960
    val unfolds = @{thm id_bnf_apply} ::
71261
4765fec43414 unfold intermediate (internal) pred definitions
traytel
parents: 70494
diff changeset
   961
      (#map_unfolds unfold_set @ flat (#set_unfoldss unfold_set) @
4765fec43414 unfold intermediate (internal) pred definitions
traytel
parents: 70494
diff changeset
   962
       #rel_unfolds unfold_set @ #pred_unfolds unfold_set);
56016
8875cdcfc85b unfold intermediate definitions after sealing the bnf
traytel
parents: 56013
diff changeset
   963
8875cdcfc85b unfold intermediate definitions after sealing the bnf
traytel
parents: 56013
diff changeset
   964
    val bnf'' = bnf' |> morph_bnf_defs (Morphism.thm_morphism "BNF" (unfold_thms lthy' unfolds));
57567
d554b0097ad4 add mk_Trueprop_mem utility function
desharna
parents: 56634
diff changeset
   965
56016
8875cdcfc85b unfold intermediate definitions after sealing the bnf
traytel
parents: 56013
diff changeset
   966
    val map_def = map_def_of_bnf bnf'';
8875cdcfc85b unfold intermediate definitions after sealing the bnf
traytel
parents: 56013
diff changeset
   967
    val set_defs = set_defs_of_bnf bnf'';
56018
c3fc8692dbc1 copy-paste typo
traytel
parents: 56016
diff changeset
   968
    val rel_def = rel_def_of_bnf bnf'';
56016
8875cdcfc85b unfold intermediate definitions after sealing the bnf
traytel
parents: 56013
diff changeset
   969
8875cdcfc85b unfold intermediate definitions after sealing the bnf
traytel
parents: 56013
diff changeset
   970
    val bnf_b = qualify b;
8875cdcfc85b unfold intermediate definitions after sealing the bnf
traytel
parents: 56013
diff changeset
   971
    val def_qualify =
59859
f9d1442c70f3 tuned signature;
wenzelm
parents: 59821
diff changeset
   972
      Thm.def_binding o Binding.concealed o Binding.qualify false (Binding.name_of bnf_b);
56016
8875cdcfc85b unfold intermediate definitions after sealing the bnf
traytel
parents: 56013
diff changeset
   973
    fun mk_prefix_binding pre = Binding.prefix_name (pre ^ "_") bnf_b;
8875cdcfc85b unfold intermediate definitions after sealing the bnf
traytel
parents: 56013
diff changeset
   974
    val map_b = def_qualify (mk_prefix_binding mapN);
8875cdcfc85b unfold intermediate definitions after sealing the bnf
traytel
parents: 56013
diff changeset
   975
    val rel_b = def_qualify (mk_prefix_binding relN);
8875cdcfc85b unfold intermediate definitions after sealing the bnf
traytel
parents: 56013
diff changeset
   976
    val set_bs = if live = 1 then [def_qualify (mk_prefix_binding setN)]
59725
e5dc7e7744f0 export more ML functions
blanchet
parents: 59710
diff changeset
   977
      else map (def_qualify o mk_prefix_binding o mk_setN) (1 upto live);
56016
8875cdcfc85b unfold intermediate definitions after sealing the bnf
traytel
parents: 56013
diff changeset
   978
8875cdcfc85b unfold intermediate definitions after sealing the bnf
traytel
parents: 56013
diff changeset
   979
    val notes = (map_b, map_def) :: (rel_b, rel_def) :: (set_bs ~~ set_defs)
8875cdcfc85b unfold intermediate definitions after sealing the bnf
traytel
parents: 56013
diff changeset
   980
      |> map (fn (b, def) => ((b, []), [([def], [])]))
57632
231e90cf2892 use the noted theorems in 'BNF_Comp'
blanchet
parents: 57567
diff changeset
   981
59820
0e9a0a5f4424 register pre-fixpoint BNFs in database to enable lookup later (e.g. in 'corec')
blanchet
parents: 59794
diff changeset
   982
    val (noted, lthy'') = lthy'
0e9a0a5f4424 register pre-fixpoint BNFs in database to enable lookup later (e.g. in 'corec')
blanchet
parents: 59794
diff changeset
   983
      |> Local_Theory.notes notes
0e9a0a5f4424 register pre-fixpoint BNFs in database to enable lookup later (e.g. in 'corec')
blanchet
parents: 59794
diff changeset
   984
      ||> (if repTA = TA then I else register_bnf_raw (fst (dest_Type TA)) bnf'')
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   985
  in
57632
231e90cf2892 use the noted theorems in 'BNF_Comp'
blanchet
parents: 57567
diff changeset
   986
    ((morph_bnf (substitute_noted_thm noted) bnf'', (all_deads, absT_info)), lthy'')
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   987
  end;
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
   988
53222
8b159677efb5 better error message
blanchet
parents: 53040
diff changeset
   989
exception BAD_DEAD of typ * typ;
8b159677efb5 better error message
blanchet
parents: 53040
diff changeset
   990
62621
a1e73be79c0b generalized ML function
blanchet
parents: 62324
diff changeset
   991
fun bnf_of_typ _ _ _ _ _ Ds0 (T as TFree T') accum =
55704
a97b9b81e195 optimized 'bnf_of_typ' further w.r.t. dead variables
blanchet
parents: 55703
diff changeset
   992
    (if member (op =) Ds0 T' then (DEADID_bnf, ([T], [])) else (ID_bnf, ([], [T])), accum)
62621
a1e73be79c0b generalized ML function
blanchet
parents: 62324
diff changeset
   993
  | bnf_of_typ _ _ _ _ _ _ (TVar _) _ = error "Unexpected schematic variable"
a1e73be79c0b generalized ML function
blanchet
parents: 62324
diff changeset
   994
  | bnf_of_typ optim const_policy qualify' flatten_tyargs Xs Ds0 (T as Type (C, Ts))
58332
be0f5d8d511b imported patch phantoms
blanchet
parents: 58297
diff changeset
   995
      (accum as (_, lthy)) =
49186
4b5fa9d5e330 handle type constructors not known to be a BNF using the DEADID BNF
traytel
parents: 49185
diff changeset
   996
    let
53222
8b159677efb5 better error message
blanchet
parents: 53040
diff changeset
   997
      fun check_bad_dead ((_, (deads, _)), _) =
8b159677efb5 better error message
blanchet
parents: 53040
diff changeset
   998
        let val Ds = fold Term.add_tfreesT deads [] in
8b159677efb5 better error message
blanchet
parents: 53040
diff changeset
   999
          (case Library.inter (op =) Ds Xs of [] => ()
55705
a98a045a6169 updated docs
blanchet
parents: 55704
diff changeset
  1000
          | X :: _ => raise BAD_DEAD (TFree X, T))
53222
8b159677efb5 better error message
blanchet
parents: 53040
diff changeset
  1001
        end;
8b159677efb5 better error message
blanchet
parents: 53040
diff changeset
  1002
55704
a97b9b81e195 optimized 'bnf_of_typ' further w.r.t. dead variables
blanchet
parents: 55703
diff changeset
  1003
      val tfrees = subtract (op =) Ds0 (Term.add_tfreesT T []);
a97b9b81e195 optimized 'bnf_of_typ' further w.r.t. dead variables
blanchet
parents: 55703
diff changeset
  1004
      val bnf_opt = if null tfrees then NONE else bnf_of lthy C;
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
  1005
    in
49186
4b5fa9d5e330 handle type constructors not known to be a BNF using the DEADID BNF
traytel
parents: 49185
diff changeset
  1006
      (case bnf_opt of
55704
a97b9b81e195 optimized 'bnf_of_typ' further w.r.t. dead variables
blanchet
parents: 55703
diff changeset
  1007
        NONE => ((DEADID_bnf, ([T], [])), accum)
49186
4b5fa9d5e330 handle type constructors not known to be a BNF using the DEADID BNF
traytel
parents: 49185
diff changeset
  1008
      | SOME bnf =>
62621
a1e73be79c0b generalized ML function
blanchet
parents: 62324
diff changeset
  1009
        if optim andalso forall (can Term.dest_TFree) Ts andalso length Ts = length tfrees then
49186
4b5fa9d5e330 handle type constructors not known to be a BNF using the DEADID BNF
traytel
parents: 49185
diff changeset
  1010
          let
4b5fa9d5e330 handle type constructors not known to be a BNF using the DEADID BNF
traytel
parents: 49185
diff changeset
  1011
            val T' = T_of_bnf bnf;
4b5fa9d5e330 handle type constructors not known to be a BNF using the DEADID BNF
traytel
parents: 49185
diff changeset
  1012
            val deads = deads_of_bnf bnf;
4b5fa9d5e330 handle type constructors not known to be a BNF using the DEADID BNF
traytel
parents: 49185
diff changeset
  1013
            val lives = lives_of_bnf bnf;
4b5fa9d5e330 handle type constructors not known to be a BNF using the DEADID BNF
traytel
parents: 49185
diff changeset
  1014
            val tvars' = Term.add_tvarsT T' [];
55904
0ef30d52c5e4 more caching in composition pipeline
blanchet
parents: 55900
diff changeset
  1015
            val Ds_As =
59058
a78612c67ec0 renamed "pairself" to "apply2", in accordance to @{apply 2};
wenzelm
parents: 58959
diff changeset
  1016
              apply2 (map (Term.typ_subst_TVars (map fst tvars' ~~ map TFree tfrees)))
49186
4b5fa9d5e330 handle type constructors not known to be a BNF using the DEADID BNF
traytel
parents: 49185
diff changeset
  1017
                (deads, lives);
55904
0ef30d52c5e4 more caching in composition pipeline
blanchet
parents: 55900
diff changeset
  1018
          in ((bnf, Ds_As), accum) end
49186
4b5fa9d5e330 handle type constructors not known to be a BNF using the DEADID BNF
traytel
parents: 49185
diff changeset
  1019
        else
4b5fa9d5e330 handle type constructors not known to be a BNF using the DEADID BNF
traytel
parents: 49185
diff changeset
  1020
          let
49425
f27f83f71e94 cleaned up internal naming scheme for bnfs
traytel
parents: 49304
diff changeset
  1021
            val name = Long_Name.base_name C;
f27f83f71e94 cleaned up internal naming scheme for bnfs
traytel
parents: 49304
diff changeset
  1022
            fun qualify i =
f27f83f71e94 cleaned up internal naming scheme for bnfs
traytel
parents: 49304
diff changeset
  1023
              let val namei = name ^ nonzero_string_of_int i;
f27f83f71e94 cleaned up internal naming scheme for bnfs
traytel
parents: 49304
diff changeset
  1024
              in qualify' o Binding.qualify true namei end;
49186
4b5fa9d5e330 handle type constructors not known to be a BNF using the DEADID BNF
traytel
parents: 49185
diff changeset
  1025
            val odead = dead_of_bnf bnf;
4b5fa9d5e330 handle type constructors not known to be a BNF using the DEADID BNF
traytel
parents: 49185
diff changeset
  1026
            val olive = live_of_bnf bnf;
59131
894d613f7f7c respect order of deads when retrieving bnfs from the database
traytel
parents: 59058
diff changeset
  1027
            val Ds = map (fn i => TFree (string_of_int i, [])) (1 upto odead);
894d613f7f7c respect order of deads when retrieving bnfs from the database
traytel
parents: 59058
diff changeset
  1028
            val Us = snd (Term.dest_Type (mk_T_of_bnf Ds (replicate olive dummyT) bnf));
894d613f7f7c respect order of deads when retrieving bnfs from the database
traytel
parents: 59058
diff changeset
  1029
            val oDs_pos = map (fn x => find_index (fn y => x = y) Us) Ds
894d613f7f7c respect order of deads when retrieving bnfs from the database
traytel
parents: 59058
diff changeset
  1030
              |> filter (fn x => x >= 0);
49186
4b5fa9d5e330 handle type constructors not known to be a BNF using the DEADID BNF
traytel
parents: 49185
diff changeset
  1031
            val oDs = map (nth Ts) oDs_pos;
4b5fa9d5e330 handle type constructors not known to be a BNF using the DEADID BNF
traytel
parents: 49185
diff changeset
  1032
            val Ts' = map (nth Ts) (subtract (op =) oDs_pos (0 upto length Ts - 1));
55904
0ef30d52c5e4 more caching in composition pipeline
blanchet
parents: 55900
diff changeset
  1033
            val ((inners, (Dss, Ass)), (accum', lthy')) =
62621
a1e73be79c0b generalized ML function
blanchet
parents: 62324
diff changeset
  1034
              apfst (apsnd split_list o split_list) (@{fold_map 2}
a1e73be79c0b generalized ML function
blanchet
parents: 62324
diff changeset
  1035
                (fn i => bnf_of_typ optim Smart_Inline (qualify i) flatten_tyargs Xs Ds0)
59725
e5dc7e7744f0 export more ML functions
blanchet
parents: 59710
diff changeset
  1036
                (if length Ts' = 1 then [0] else 1 upto length Ts') Ts' accum);
49186
4b5fa9d5e330 handle type constructors not known to be a BNF using the DEADID BNF
traytel
parents: 49185
diff changeset
  1037
          in
58332
be0f5d8d511b imported patch phantoms
blanchet
parents: 58297
diff changeset
  1038
            compose_bnf const_policy qualify flatten_tyargs bnf inners oDs Dss Ass (accum', lthy')
49186
4b5fa9d5e330 handle type constructors not known to be a BNF using the DEADID BNF
traytel
parents: 49185
diff changeset
  1039
          end)
53222
8b159677efb5 better error message
blanchet
parents: 53040
diff changeset
  1040
      |> tap check_bad_dead
48975
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
  1041
    end;
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
  1042
7f79f94a432c added new (co)datatype package + theories of ordinals and cardinals (with Dmitriy and Andrei)
blanchet
parents:
diff changeset
  1043
end;