| author | boehmes | 
| Wed, 21 Oct 2009 14:08:04 +0200 | |
| changeset 33048 | af06b784814d | 
| parent 32970 | fbd2bb2489a8 | 
| child 33056 | 791a4655cae3 | 
| permissions | -rw-r--r-- | 
| 31775 | 1 | (* Title: HOL/Tools/Function/size.ML | 
| 29495 | 2 | Author: Stefan Berghofer, Florian Haftmann & Alexander Krauss, TU Muenchen | 
| 24710 | 3 | |
| 4 | Size functions for datatypes. | |
| 5 | *) | |
| 6 | ||
| 7 | signature SIZE = | |
| 8 | sig | |
| 9 | val size_thms: theory -> string -> thm list | |
| 10 | val setup: theory -> theory | |
| 11 | end; | |
| 12 | ||
| 13 | structure Size: SIZE = | |
| 14 | struct | |
| 15 | ||
| 16 | open DatatypeAux; | |
| 17 | ||
| 24714 
1618c2ac1b74
proper Sign operations instead of Theory aliases;
 wenzelm parents: 
24711diff
changeset | 18 | structure SizeData = TheoryDataFun | 
| 
1618c2ac1b74
proper Sign operations instead of Theory aliases;
 wenzelm parents: 
24711diff
changeset | 19 | ( | 
| 25679 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 20 | type T = (string * thm list) Symtab.table; | 
| 24710 | 21 | val empty = Symtab.empty; | 
| 22 | val copy = I | |
| 23 | val extend = I | |
| 24 | fun merge _ = Symtab.merge (K true); | |
| 24714 
1618c2ac1b74
proper Sign operations instead of Theory aliases;
 wenzelm parents: 
24711diff
changeset | 25 | ); | 
| 24710 | 26 | |
| 25679 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 27 | val lookup_size = SizeData.get #> Symtab.lookup; | 
| 24710 | 28 | |
| 29 | fun plus (t1, t2) = Const ("HOL.plus_class.plus",
 | |
| 30 | HOLogic.natT --> HOLogic.natT --> HOLogic.natT) $ t1 $ t2; | |
| 31 | ||
| 25679 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 32 | fun size_of_type f g h (T as Type (s, Ts)) = | 
| 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 33 | (case f s of | 
| 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 34 | SOME t => SOME t | 
| 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 35 | | NONE => (case g s of | 
| 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 36 | SOME size_name => | 
| 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 37 | SOME (list_comb (Const (size_name, | 
| 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 38 | map (fn U => U --> HOLogic.natT) Ts @ [T] ---> HOLogic.natT), | 
| 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 39 | map (size_of_type' f g h) Ts)) | 
| 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 40 | | NONE => NONE)) | 
| 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 41 | | size_of_type f g h (TFree (s, _)) = h s | 
| 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 42 | and size_of_type' f g h T = (case size_of_type f g h T of | 
| 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 43 |       NONE => Abs ("x", T, HOLogic.zero)
 | 
| 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 44 | | SOME t => t); | 
| 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 45 | |
| 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 46 | fun is_poly thy (DtType (name, dts)) = | 
| 31784 | 47 | (case Datatype.get_info thy name of | 
| 25679 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 48 | NONE => false | 
| 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 49 | | SOME _ => exists (is_poly thy) dts) | 
| 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 50 | | is_poly _ _ = true; | 
| 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 51 | |
| 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 52 | fun constrs_of thy name = | 
| 24710 | 53 | let | 
| 31784 | 54 |     val {descr, index, ...} = Datatype.the_info thy name
 | 
| 25679 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 55 | val SOME (_, _, constrs) = AList.lookup op = descr index | 
| 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 56 | in constrs end; | 
| 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 57 | |
| 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 58 | val app = curry (list_comb o swap); | 
| 24710 | 59 | |
| 31737 | 60 | fun prove_size_thms (info : info) new_type_names thy = | 
| 25679 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 61 | let | 
| 32727 | 62 |     val {descr, alt_names, sorts, rec_names, rec_rewrites, induct, ...} = info;
 | 
| 25679 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 63 | val l = length new_type_names; | 
| 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 64 | val alt_names' = (case alt_names of | 
| 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 65 | NONE => replicate l NONE | SOME names => map SOME names); | 
| 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 66 | val descr' = List.take (descr, l); | 
| 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 67 | val (rec_names1, rec_names2) = chop l rec_names; | 
| 25864 | 68 | val recTs = get_rec_types descr sorts; | 
| 25679 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 69 | val (recTs1, recTs2) = chop l recTs; | 
| 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 70 | val (_, (_, paramdts, _)) :: _ = descr; | 
| 25864 | 71 | val paramTs = map (typ_of_dtyp descr sorts) paramdts; | 
| 25679 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 72 | val ((param_size_fs, param_size_fTs), f_names) = paramTs |> | 
| 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 73 | map (fn T as TFree (s, _) => | 
| 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 74 | let | 
| 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 75 | val name = "f" ^ implode (tl (explode s)); | 
| 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 76 | val U = T --> HOLogic.natT | 
| 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 77 | in | 
| 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 78 | (((s, Free (name, U)), U), name) | 
| 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 79 | end) |> split_list |>> split_list; | 
| 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 80 | val param_size = AList.lookup op = param_size_fs; | 
| 24710 | 81 | |
| 25679 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 82 | val extra_rewrites = descr |> map (#1 o snd) |> distinct op = |> | 
| 29495 | 83 | map_filter (Option.map snd o lookup_size thy) |> flat; | 
| 25679 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 84 | val extra_size = Option.map fst o lookup_size thy; | 
| 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 85 | |
| 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 86 | val (((size_names, size_fns), def_names), def_names') = | 
| 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 87 | recTs1 ~~ alt_names' |> | 
| 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 88 | map (fn (T as Type (s, _), optname) => | 
| 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 89 | let | 
| 30364 
577edc39b501
moved basic algebra of long names from structure NameSpace to Long_Name;
 wenzelm parents: 
30345diff
changeset | 90 | val s' = the_default (Long_Name.base_name s) optname ^ "_size"; | 
| 28965 | 91 | val s'' = Sign.full_bname thy s' | 
| 25679 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 92 | in | 
| 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 93 | (s'', | 
| 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 94 | (list_comb (Const (s'', param_size_fTs @ [T] ---> HOLogic.natT), | 
| 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 95 | map snd param_size_fs), | 
| 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 96 | (s' ^ "_def", s' ^ "_overloaded_def"))) | 
| 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 97 | end) |> split_list ||>> split_list ||>> split_list; | 
| 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 98 | val overloaded_size_fns = map HOLogic.size_const recTs1; | 
| 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 99 | |
| 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 100 | (* instantiation for primrec combinator *) | 
| 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 101 | fun size_of_constr b size_ofp ((_, cargs), (_, cargs')) = | 
| 24710 | 102 | let | 
| 25864 | 103 | val Ts = map (typ_of_dtyp descr sorts) cargs; | 
| 24710 | 104 | val k = length (filter is_rec_type cargs); | 
| 25679 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 105 | val (ts, _, _) = fold_rev (fn ((dt, dt'), T) => fn (us, i, j) => | 
| 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 106 | if is_rec_type dt then (Bound i :: us, i + 1, j + 1) | 
| 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 107 | else | 
| 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 108 | (if b andalso is_poly thy dt' then | 
| 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 109 | case size_of_type (K NONE) extra_size size_ofp T of | 
| 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 110 | NONE => us | SOME sz => sz $ Bound j :: us | 
| 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 111 | else us, i, j + 1)) | 
| 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 112 | (cargs ~~ cargs' ~~ Ts) ([], 0, k); | 
| 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 113 | val t = | 
| 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 114 | if null ts andalso (not b orelse not (exists (is_poly thy) cargs')) | 
| 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 115 | then HOLogic.zero | 
| 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 116 | else foldl1 plus (ts @ [HOLogic.Suc_zero]) | 
| 24710 | 117 | in | 
| 30190 | 118 |         List.foldr (fn (T, t') => Abs ("x", T, t')) t (Ts @ replicate k HOLogic.natT)
 | 
| 24710 | 119 | end; | 
| 120 | ||
| 25679 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 121 | val fs = maps (fn (_, (name, _, constrs)) => | 
| 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 122 | map (size_of_constr true param_size) (constrs ~~ constrs_of thy name)) descr; | 
| 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 123 | val fs' = maps (fn (n, (name, _, constrs)) => | 
| 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 124 | map (size_of_constr (l <= n) (K NONE)) (constrs ~~ constrs_of thy name)) descr; | 
| 24710 | 125 | val fTs = map fastype_of fs; | 
| 126 | ||
| 25679 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 127 | val (rec_combs1, rec_combs2) = chop l (map (fn (T, rec_name) => | 
| 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 128 | Const (rec_name, fTs @ [T] ---> HOLogic.natT)) | 
| 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 129 | (recTs ~~ rec_names)); | 
| 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 130 | |
| 25835 | 131 | fun define_overloaded (def_name, eq) lthy = | 
| 132 | let | |
| 133 | val (Free (c, _), rhs) = (Logic.dest_equals o Syntax.check_term lthy) eq; | |
| 28083 
103d9282a946
explicit type Name.binding for higher-specification elements;
 wenzelm parents: 
27691diff
changeset | 134 | val ((_, (_, thm)), lthy') = lthy |> LocalTheory.define Thm.definitionK | 
| 28965 | 135 | ((Binding.name c, NoSyn), ((Binding.name def_name, []), rhs)); | 
| 25835 | 136 | val ctxt_thy = ProofContext.init (ProofContext.theory_of lthy'); | 
| 25864 | 137 | val thm' = singleton (ProofContext.export lthy' ctxt_thy) thm; | 
| 25835 | 138 | in (thm', lthy') end; | 
| 139 | ||
| 25679 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 140 | val ((size_def_thms, size_def_thms'), thy') = | 
| 24710 | 141 | thy | 
| 24714 
1618c2ac1b74
proper Sign operations instead of Theory aliases;
 wenzelm parents: 
24711diff
changeset | 142 | |> Sign.add_consts_i (map (fn (s, T) => | 
| 30364 
577edc39b501
moved basic algebra of long names from structure NameSpace to Long_Name;
 wenzelm parents: 
30345diff
changeset | 143 | (Binding.name (Long_Name.base_name s), param_size_fTs @ [T] ---> HOLogic.natT, NoSyn)) | 
| 25679 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 144 | (size_names ~~ recTs1)) | 
| 27691 
ce171cbd4b93
PureThy: dropped note_thmss_qualified, dropped _i suffix
 haftmann parents: 
25890diff
changeset | 145 | |> PureThy.add_defs false | 
| 25679 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 146 | (map (Thm.no_attributes o apsnd (Logic.mk_equals o apsnd (app fs))) | 
| 29579 | 147 | (map Binding.name def_names ~~ (size_fns ~~ rec_combs1))) | 
| 25835 | 148 | ||> TheoryTarget.instantiation | 
| 25890 
0ba401ddbaed
Now uses more carefully designed simpsets to prevent proofs from
 berghofe parents: 
25864diff
changeset | 149 | (map (#1 o snd) descr', map dest_TFree paramTs, [HOLogic.class_size]) | 
| 25835 | 150 | ||>> fold_map define_overloaded | 
| 151 | (def_names' ~~ map Logic.mk_equals (overloaded_size_fns ~~ map (app fs') rec_combs1)) | |
| 152 | ||> Class.prove_instantiation_instance (K (Class.intro_classes_tac [])) | |
| 28394 | 153 | ||> LocalTheory.exit_global; | 
| 25679 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 154 | |
| 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 155 | val ctxt = ProofContext.init thy'; | 
| 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 156 | |
| 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 157 |     val simpset1 = HOL_basic_ss addsimps @{thm add_0} :: @{thm add_0_right} ::
 | 
| 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 158 | size_def_thms @ size_def_thms' @ rec_rewrites @ extra_rewrites; | 
| 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 159 | val xs = map (fn i => "x" ^ string_of_int i) (1 upto length recTs2); | 
| 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 160 | |
| 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 161 | fun mk_unfolded_size_eq tab size_ofp fs (p as (x, T), r) = | 
| 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 162 | HOLogic.mk_eq (app fs r $ Free p, | 
| 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 163 | the (size_of_type tab extra_size size_ofp T) $ Free p); | 
| 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 164 | |
| 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 165 | fun prove_unfolded_size_eqs size_ofp fs = | 
| 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 166 | if null recTs2 then [] | 
| 32970 
fbd2bb2489a8
operations of structure Skip_Proof (formerly SkipProof) no longer require quick_and_dirty mode;
 wenzelm parents: 
32957diff
changeset | 167 | else split_conj_thm (Skip_Proof.prove ctxt xs [] | 
| 25679 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 168 | (HOLogic.mk_Trueprop (mk_conj (replicate l HOLogic.true_const @ | 
| 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 169 | map (mk_unfolded_size_eq (AList.lookup op = | 
| 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 170 | (new_type_names ~~ map (app fs) rec_combs1)) size_ofp fs) | 
| 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 171 | (xs ~~ recTs2 ~~ rec_combs2)))) | 
| 32712 
ec5976f4d3d8
registering split rules and projected induction rules; ML identifiers more close to Isar theorem names
 haftmann parents: 
31902diff
changeset | 172 | (fn _ => (indtac induct xs THEN_ALL_NEW asm_simp_tac simpset1) 1)); | 
| 25679 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 173 | |
| 25890 
0ba401ddbaed
Now uses more carefully designed simpsets to prevent proofs from
 berghofe parents: 
25864diff
changeset | 174 | val unfolded_size_eqs1 = prove_unfolded_size_eqs param_size fs; | 
| 
0ba401ddbaed
Now uses more carefully designed simpsets to prevent proofs from
 berghofe parents: 
25864diff
changeset | 175 | val unfolded_size_eqs2 = prove_unfolded_size_eqs (K NONE) fs'; | 
| 24710 | 176 | |
| 25679 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 177 | (* characteristic equations for size functions *) | 
| 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 178 | fun gen_mk_size_eq p size_of size_ofp size_const T (cname, cargs) = | 
| 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 179 | let | 
| 25864 | 180 | val Ts = map (typ_of_dtyp descr sorts) cargs; | 
| 25679 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 181 | val tnames = Name.variant_list f_names (DatatypeProp.make_tnames Ts); | 
| 29495 | 182 | val ts = map_filter (fn (sT as (s, T), dt) => | 
| 25679 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 183 | Option.map (fn sz => sz $ Free sT) | 
| 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 184 | (if p dt then size_of_type size_of extra_size size_ofp T | 
| 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 185 | else NONE)) (tnames ~~ Ts ~~ cargs) | 
| 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 186 | in | 
| 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 187 | HOLogic.mk_Trueprop (HOLogic.mk_eq | 
| 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 188 | (size_const $ list_comb (Const (cname, Ts ---> T), | 
| 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 189 | map2 (curry Free) tnames Ts), | 
| 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 190 | if null ts then HOLogic.zero | 
| 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 191 | else foldl1 plus (ts @ [HOLogic.Suc_zero]))) | 
| 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 192 | end; | 
| 24710 | 193 | |
| 25679 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 194 | val simpset2 = HOL_basic_ss addsimps | 
| 25890 
0ba401ddbaed
Now uses more carefully designed simpsets to prevent proofs from
 berghofe parents: 
25864diff
changeset | 195 | rec_rewrites @ size_def_thms @ unfolded_size_eqs1; | 
| 
0ba401ddbaed
Now uses more carefully designed simpsets to prevent proofs from
 berghofe parents: 
25864diff
changeset | 196 | val simpset3 = HOL_basic_ss addsimps | 
| 
0ba401ddbaed
Now uses more carefully designed simpsets to prevent proofs from
 berghofe parents: 
25864diff
changeset | 197 | rec_rewrites @ size_def_thms' @ unfolded_size_eqs2; | 
| 25679 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 198 | |
| 25890 
0ba401ddbaed
Now uses more carefully designed simpsets to prevent proofs from
 berghofe parents: 
25864diff
changeset | 199 | fun prove_size_eqs p size_fns size_ofp simpset = | 
| 25679 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 200 | maps (fn (((_, (_, _, constrs)), size_const), T) => | 
| 32970 
fbd2bb2489a8
operations of structure Skip_Proof (formerly SkipProof) no longer require quick_and_dirty mode;
 wenzelm parents: 
32957diff
changeset | 201 | map (fn constr => Drule.standard (Skip_Proof.prove ctxt [] [] | 
| 25679 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 202 | (gen_mk_size_eq p (AList.lookup op = (new_type_names ~~ size_fns)) | 
| 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 203 | size_ofp size_const T constr) | 
| 25890 
0ba401ddbaed
Now uses more carefully designed simpsets to prevent proofs from
 berghofe parents: 
25864diff
changeset | 204 | (fn _ => simp_tac simpset 1))) constrs) | 
| 25679 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 205 | (descr' ~~ size_fns ~~ recTs1); | 
| 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 206 | |
| 25890 
0ba401ddbaed
Now uses more carefully designed simpsets to prevent proofs from
 berghofe parents: 
25864diff
changeset | 207 | val size_eqns = prove_size_eqs (is_poly thy') size_fns param_size simpset2 @ | 
| 
0ba401ddbaed
Now uses more carefully designed simpsets to prevent proofs from
 berghofe parents: 
25864diff
changeset | 208 | prove_size_eqs is_rec_type overloaded_size_fns (K NONE) simpset3; | 
| 25679 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 209 | |
| 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 210 | val ([size_thms], thy'') = PureThy.add_thmss | 
| 29579 | 211 | [((Binding.name "size", size_eqns), | 
| 31902 | 212 | [Simplifier.simp_add, Nitpick_Const_Simps.add, | 
| 29863 
dadad1831e9d
Added "nitpick_const_simps" and "nitpick_ind_intros" attributes for theorems;
 blanchet parents: 
29579diff
changeset | 213 | Thm.declaration_attribute | 
| 
dadad1831e9d
Added "nitpick_const_simps" and "nitpick_ind_intros" attributes for theorems;
 blanchet parents: 
29579diff
changeset | 214 | (fn thm => Context.mapping (Code.add_default_eqn thm) I)])] thy' | 
| 24710 | 215 | |
| 216 | in | |
| 25679 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 217 | SizeData.map (fold (Symtab.update_new o apsnd (rpair size_thms)) | 
| 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 218 | (new_type_names ~~ size_names)) thy'' | 
| 24710 | 219 | end; | 
| 220 | ||
| 31668 
a616e56a5ec8
datatype packages: record datatype_config for configuration flags; less verbose signatures
 haftmann parents: 
30364diff
changeset | 221 | fun add_size_thms config (new_type_names as name :: _) thy = | 
| 24710 | 222 | let | 
| 31784 | 223 |     val info as {descr, alt_names, ...} = Datatype.the_info thy name;
 | 
| 30364 
577edc39b501
moved basic algebra of long names from structure NameSpace to Long_Name;
 wenzelm parents: 
30345diff
changeset | 224 | val prefix = Long_Name.map_base_name (K (space_implode "_" | 
| 
577edc39b501
moved basic algebra of long names from structure NameSpace to Long_Name;
 wenzelm parents: 
30345diff
changeset | 225 | (the_default (map Long_Name.base_name new_type_names) alt_names))) name; | 
| 24710 | 226 | val no_size = exists (fn (_, (_, _, constrs)) => exists (fn (_, cargs) => exists (fn dt => | 
| 25679 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 227 | is_rec_type dt andalso not (null (fst (strip_dtyp dt)))) cargs) constrs) descr | 
| 24710 | 228 | in if no_size then thy | 
| 229 | else | |
| 230 | thy | |
| 25679 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 231 | |> Sign.root_path | 
| 24714 
1618c2ac1b74
proper Sign operations instead of Theory aliases;
 wenzelm parents: 
24711diff
changeset | 232 | |> Sign.add_path prefix | 
| 28361 
232fcbba2e4e
explicit checkpoint for low-level (global) theory operations, admits concurrent proofs;
 wenzelm parents: 
28083diff
changeset | 233 | |> Theory.checkpoint | 
| 25679 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 234 | |> prove_size_thms info new_type_names | 
| 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 235 | |> Sign.restore_naming thy | 
| 24710 | 236 | end; | 
| 237 | ||
| 25679 
b77f797b528a
size functions for nested datatypes are now expressed using
 berghofe parents: 
25569diff
changeset | 238 | val size_thms = snd oo (the oo lookup_size); | 
| 24710 | 239 | |
| 31723 
f5cafe803b55
discontinued ancient tradition to suffix certain ML module names with "_package"
 haftmann parents: 
31668diff
changeset | 240 | val setup = Datatype.interpretation add_size_thms; | 
| 24710 | 241 | |
| 29866 
6e93ae65c678
Added Nitpick_Const_Psimp attribute, dropped the 's' in Nitpick_Const_Simps, and killed the Nitpick_Ind_Intros attribute.
 blanchet parents: 
29863diff
changeset | 242 | end; |