src/HOL/Tools/Nitpick/nitpick_mono.ML
author haftmann
Thu, 26 Aug 2010 20:51:17 +0200
changeset 39019 e46e7a9cb622
parent 38426 8a9cace789d6
child 39028 848be46708dc
permissions -rw-r--r--
formerly unnamed infix impliciation now named HOL.implies
blanchet@33982
     1
(*  Title:      HOL/Tools/Nitpick/nitpick_mono.ML
blanchet@33192
     2
    Author:     Jasmin Blanchette, TU Muenchen
blanchet@34969
     3
    Copyright   2009, 2010
blanchet@33192
     4
blanchet@35384
     5
Monotonicity inference for higher-order logic.
blanchet@33192
     6
*)
blanchet@33192
     7
blanchet@33192
     8
signature NITPICK_MONO =
blanchet@33192
     9
sig
blanchet@35067
    10
  type hol_context = Nitpick_HOL.hol_context
blanchet@33192
    11
blanchet@38406
    12
  val trace : bool Unsynchronized.ref
blanchet@33192
    13
  val formulas_monotonic :
blanchet@35386
    14
    hol_context -> bool -> typ -> term list * term list -> bool
blanchet@35665
    15
  val finitize_funs :
blanchet@35665
    16
    hol_context -> bool -> (typ option * bool option) list -> typ
blanchet@35665
    17
    -> term list * term list -> term list * term list
blanchet@33192
    18
end;
blanchet@33192
    19
blanchet@33224
    20
structure Nitpick_Mono : NITPICK_MONO =
blanchet@33192
    21
struct
blanchet@33192
    22
blanchet@33224
    23
open Nitpick_Util
blanchet@33224
    24
open Nitpick_HOL
blanchet@33192
    25
blanchet@33192
    26
type var = int
blanchet@33192
    27
blanchet@34969
    28
datatype sign = Plus | Minus
blanchet@33192
    29
datatype sign_atom = S of sign | V of var
blanchet@33192
    30
blanchet@33192
    31
type literal = var * sign
blanchet@33192
    32
blanchet@35385
    33
datatype mtyp =
blanchet@35385
    34
  MAlpha |
blanchet@35385
    35
  MFun of mtyp * sign_atom * mtyp |
blanchet@35385
    36
  MPair of mtyp * mtyp |
blanchet@35385
    37
  MType of string * mtyp list |
blanchet@35385
    38
  MRec of string * typ list
blanchet@33192
    39
blanchet@35385
    40
datatype mterm =
blanchet@35386
    41
  MRaw of term * mtyp |
blanchet@35385
    42
  MAbs of string * typ * mtyp * sign_atom * mterm |
blanchet@35385
    43
  MApp of mterm * mterm
blanchet@35385
    44
blanchet@35385
    45
type mdata =
blanchet@35067
    46
  {hol_ctxt: hol_context,
blanchet@35190
    47
   binarize: bool,
blanchet@33192
    48
   alpha_T: typ,
blanchet@35665
    49
   no_harmless: bool,
blanchet@33192
    50
   max_fresh: int Unsynchronized.ref,
blanchet@35665
    51
   datatype_mcache: ((string * typ list) * mtyp) list Unsynchronized.ref,
blanchet@35665
    52
   constr_mcache: (styp * mtyp) list Unsynchronized.ref}
blanchet@33192
    53
blanchet@35812
    54
exception UNSOLVABLE of unit
blanchet@35665
    55
exception MTYPE of string * mtyp list * typ list
blanchet@35665
    56
exception MTERM of string * mterm list
blanchet@33192
    57
blanchet@38406
    58
val trace = Unsynchronized.ref false
blanchet@38406
    59
fun trace_msg msg = if !trace then tracing (msg ()) else ()
blanchet@33192
    60
blanchet@33192
    61
val string_for_var = signed_string_of_int
blanchet@33192
    62
fun string_for_vars sep [] = "0\<^bsub>" ^ sep ^ "\<^esub>"
blanchet@33192
    63
  | string_for_vars sep xs = space_implode sep (map string_for_var xs)
blanchet@33192
    64
fun subscript_string_for_vars sep xs =
blanchet@33192
    65
  if null xs then "" else "\<^bsub>" ^ string_for_vars sep xs ^ "\<^esub>"
blanchet@33192
    66
blanchet@34969
    67
fun string_for_sign Plus = "+"
blanchet@34969
    68
  | string_for_sign Minus = "-"
blanchet@33192
    69
blanchet@34969
    70
fun xor sn1 sn2 = if sn1 = sn2 then Plus else Minus
blanchet@34969
    71
val negate = xor Minus
blanchet@33192
    72
blanchet@33192
    73
fun string_for_sign_atom (S sn) = string_for_sign sn
blanchet@35665
    74
  | string_for_sign_atom (V x) = string_for_var x
blanchet@33192
    75
blanchet@33192
    76
fun string_for_literal (x, sn) = string_for_var x ^ " = " ^ string_for_sign sn
blanchet@33192
    77
blanchet@35385
    78
val bool_M = MType (@{type_name bool}, [])
blanchet@35386
    79
val dummy_M = MType (nitpick_prefix ^ "dummy", [])
blanchet@33192
    80
blanchet@35385
    81
fun is_MRec (MRec _) = true
blanchet@35385
    82
  | is_MRec _ = false
blanchet@35385
    83
fun dest_MFun (MFun z) = z
blanchet@35665
    84
  | dest_MFun M = raise MTYPE ("Nitpick_Mono.dest_MFun", [M], [])
blanchet@33192
    85
blanchet@33192
    86
val no_prec = 100
blanchet@33192
    87
blanchet@35385
    88
fun precedence_of_mtype (MFun _) = 1
blanchet@35385
    89
  | precedence_of_mtype (MPair _) = 2
blanchet@35385
    90
  | precedence_of_mtype _ = no_prec
blanchet@33192
    91
blanchet@35385
    92
val string_for_mtype =
blanchet@33192
    93
  let
blanchet@35385
    94
    fun aux outer_prec M =
blanchet@33192
    95
      let
blanchet@35385
    96
        val prec = precedence_of_mtype M
blanchet@33192
    97
        val need_parens = (prec < outer_prec)
blanchet@33192
    98
      in
blanchet@33192
    99
        (if need_parens then "(" else "") ^
blanchet@35386
   100
        (if M = dummy_M then
blanchet@35386
   101
           "_"
blanchet@35386
   102
         else case M of
blanchet@35386
   103
             MAlpha => "\<alpha>"
blanchet@35386
   104
           | MFun (M1, a, M2) =>
blanchet@35386
   105
             aux (prec + 1) M1 ^ " \<Rightarrow>\<^bsup>" ^
blanchet@35386
   106
             string_for_sign_atom a ^ "\<^esup> " ^ aux prec M2
blanchet@35386
   107
           | MPair (M1, M2) => aux (prec + 1) M1 ^ " \<times> " ^ aux prec M2
blanchet@35386
   108
           | MType (s, []) =>
blanchet@35386
   109
             if s = @{type_name prop} orelse s = @{type_name bool} then "o"
blanchet@35386
   110
             else s
blanchet@35386
   111
           | MType (s, Ms) => "(" ^ commas (map (aux 0) Ms) ^ ") " ^ s
blanchet@35386
   112
           | MRec (s, _) => "[" ^ s ^ "]") ^
blanchet@33192
   113
        (if need_parens then ")" else "")
blanchet@33192
   114
      end
blanchet@33192
   115
  in aux 0 end
blanchet@33192
   116
blanchet@35385
   117
fun flatten_mtype (MPair (M1, M2)) = maps flatten_mtype [M1, M2]
blanchet@35385
   118
  | flatten_mtype (MType (_, Ms)) = maps flatten_mtype Ms
blanchet@35385
   119
  | flatten_mtype M = [M]
blanchet@33192
   120
blanchet@35386
   121
fun precedence_of_mterm (MRaw _) = no_prec
blanchet@35385
   122
  | precedence_of_mterm (MAbs _) = 1
blanchet@35385
   123
  | precedence_of_mterm (MApp _) = 2
blanchet@35385
   124
blanchet@35385
   125
fun string_for_mterm ctxt =
blanchet@35385
   126
  let
blanchet@35385
   127
    fun mtype_annotation M = "\<^bsup>" ^ string_for_mtype M ^ "\<^esup>"
blanchet@35385
   128
    fun aux outer_prec m =
blanchet@35385
   129
      let
blanchet@35385
   130
        val prec = precedence_of_mterm m
blanchet@35385
   131
        val need_parens = (prec < outer_prec)
blanchet@35385
   132
      in
blanchet@35385
   133
        (if need_parens then "(" else "") ^
blanchet@35385
   134
        (case m of
blanchet@35386
   135
           MRaw (t, M) => Syntax.string_of_term ctxt t ^ mtype_annotation M
blanchet@35385
   136
         | MAbs (s, _, M, a, m) =>
blanchet@35385
   137
           "\<lambda>" ^ s ^ mtype_annotation M ^ ".\<^bsup>" ^
blanchet@35385
   138
           string_for_sign_atom a ^ "\<^esup> " ^ aux prec m
blanchet@35385
   139
         | MApp (m1, m2) => aux prec m1 ^ " " ^ aux (prec + 1) m2) ^
blanchet@35385
   140
        (if need_parens then ")" else "")
blanchet@35385
   141
      end
blanchet@35385
   142
  in aux 0 end
blanchet@35385
   143
blanchet@35386
   144
fun mtype_of_mterm (MRaw (_, M)) = M
blanchet@35385
   145
  | mtype_of_mterm (MAbs (_, _, M, a, m)) = MFun (M, a, mtype_of_mterm m)
blanchet@35385
   146
  | mtype_of_mterm (MApp (m1, _)) =
blanchet@35385
   147
    case mtype_of_mterm m1 of
blanchet@35385
   148
      MFun (_, _, M12) => M12
blanchet@35665
   149
    | M1 => raise MTYPE ("Nitpick_Mono.mtype_of_mterm", [M1], [])
blanchet@35385
   150
blanchet@35665
   151
fun strip_mcomb (MApp (m1, m2)) = strip_mcomb m1 ||> (fn ms => append ms [m2])
blanchet@35665
   152
  | strip_mcomb m = (m, [])
blanchet@35665
   153
blanchet@35665
   154
fun initial_mdata hol_ctxt binarize no_harmless alpha_T =
blanchet@35190
   155
  ({hol_ctxt = hol_ctxt, binarize = binarize, alpha_T = alpha_T,
blanchet@35665
   156
    no_harmless = no_harmless, max_fresh = Unsynchronized.ref 0,
blanchet@35665
   157
    datatype_mcache = Unsynchronized.ref [],
blanchet@35665
   158
    constr_mcache = Unsynchronized.ref []} : mdata)
blanchet@33192
   159
blanchet@33192
   160
fun could_exist_alpha_subtype alpha_T (T as Type (_, Ts)) =
blanchet@34923
   161
    T = alpha_T orelse (not (is_fp_iterator_type T) andalso
blanchet@34923
   162
                        exists (could_exist_alpha_subtype alpha_T) Ts)
blanchet@33192
   163
  | could_exist_alpha_subtype alpha_T T = (T = alpha_T)
blanchet@35385
   164
fun could_exist_alpha_sub_mtype _ (alpha_T as TFree _) T =
blanchet@34118
   165
    could_exist_alpha_subtype alpha_T T
blanchet@37255
   166
  | could_exist_alpha_sub_mtype ctxt alpha_T T =
blanchet@37255
   167
    (T = alpha_T orelse is_datatype ctxt [(NONE, true)] T)
blanchet@33192
   168
blanchet@35385
   169
fun exists_alpha_sub_mtype MAlpha = true
blanchet@35385
   170
  | exists_alpha_sub_mtype (MFun (M1, _, M2)) =
blanchet@35385
   171
    exists exists_alpha_sub_mtype [M1, M2]
blanchet@35385
   172
  | exists_alpha_sub_mtype (MPair (M1, M2)) =
blanchet@35385
   173
    exists exists_alpha_sub_mtype [M1, M2]
blanchet@35385
   174
  | exists_alpha_sub_mtype (MType (_, Ms)) = exists exists_alpha_sub_mtype Ms
blanchet@35385
   175
  | exists_alpha_sub_mtype (MRec _) = true
blanchet@33192
   176
blanchet@35385
   177
fun exists_alpha_sub_mtype_fresh MAlpha = true
blanchet@35385
   178
  | exists_alpha_sub_mtype_fresh (MFun (_, V _, _)) = true
blanchet@35385
   179
  | exists_alpha_sub_mtype_fresh (MFun (_, _, M2)) =
blanchet@35385
   180
    exists_alpha_sub_mtype_fresh M2
blanchet@35385
   181
  | exists_alpha_sub_mtype_fresh (MPair (M1, M2)) =
blanchet@35385
   182
    exists exists_alpha_sub_mtype_fresh [M1, M2]
blanchet@35385
   183
  | exists_alpha_sub_mtype_fresh (MType (_, Ms)) =
blanchet@35385
   184
    exists exists_alpha_sub_mtype_fresh Ms
blanchet@35385
   185
  | exists_alpha_sub_mtype_fresh (MRec _) = true
blanchet@33192
   186
blanchet@35385
   187
fun constr_mtype_for_binders z Ms =
blanchet@35385
   188
  fold_rev (fn M => curry3 MFun M (S Minus)) Ms (MRec z)
blanchet@33192
   189
blanchet@35385
   190
fun repair_mtype _ _ MAlpha = MAlpha
blanchet@35385
   191
  | repair_mtype cache seen (MFun (M1, a, M2)) =
blanchet@35385
   192
    MFun (repair_mtype cache seen M1, a, repair_mtype cache seen M2)
blanchet@35385
   193
  | repair_mtype cache seen (MPair Mp) =
blanchet@35385
   194
    MPair (pairself (repair_mtype cache seen) Mp)
blanchet@35385
   195
  | repair_mtype cache seen (MType (s, Ms)) =
blanchet@35385
   196
    MType (s, maps (flatten_mtype o repair_mtype cache seen) Ms)
blanchet@35385
   197
  | repair_mtype cache seen (MRec (z as (s, _))) =
blanchet@33192
   198
    case AList.lookup (op =) cache z |> the of
blanchet@35385
   199
      MRec _ => MType (s, [])
blanchet@35385
   200
    | M => if member (op =) seen M then MType (s, [])
blanchet@35385
   201
           else repair_mtype cache (M :: seen) M
blanchet@33192
   202
blanchet@35665
   203
fun repair_datatype_mcache cache =
blanchet@33192
   204
  let
blanchet@35385
   205
    fun repair_one (z, M) =
blanchet@33192
   206
      Unsynchronized.change cache
blanchet@35385
   207
          (AList.update (op =) (z, repair_mtype (!cache) [] M))
blanchet@33192
   208
  in List.app repair_one (rev (!cache)) end
blanchet@33192
   209
blanchet@35665
   210
fun repair_constr_mcache dtype_cache constr_mcache =
blanchet@33192
   211
  let
blanchet@35385
   212
    fun repair_one (x, M) =
blanchet@35665
   213
      Unsynchronized.change constr_mcache
blanchet@35385
   214
          (AList.update (op =) (x, repair_mtype dtype_cache [] M))
blanchet@35665
   215
  in List.app repair_one (!constr_mcache) end
blanchet@35665
   216
blanchet@35665
   217
fun is_fin_fun_supported_type @{typ prop} = true
blanchet@35665
   218
  | is_fin_fun_supported_type @{typ bool} = true
blanchet@35665
   219
  | is_fin_fun_supported_type (Type (@{type_name option}, _)) = true
blanchet@35665
   220
  | is_fin_fun_supported_type _ = false
blanchet@35665
   221
fun fin_fun_body _ _ (t as @{term False}) = SOME t
blanchet@35665
   222
  | fin_fun_body _ _ (t as Const (@{const_name None}, _)) = SOME t
blanchet@35665
   223
  | fin_fun_body dom_T ran_T
blanchet@35665
   224
                 ((t0 as Const (@{const_name If}, _))
blanchet@35665
   225
                  $ (t1 as Const (@{const_name "op ="}, _) $ Bound 0 $ t1')
blanchet@35665
   226
                  $ t2 $ t3) =
blanchet@35665
   227
    (if loose_bvar1 (t1', 0) then
blanchet@35665
   228
       NONE
blanchet@35665
   229
     else case fin_fun_body dom_T ran_T t3 of
blanchet@35665
   230
       NONE => NONE
blanchet@35665
   231
     | SOME t3 =>
blanchet@35665
   232
       SOME (t0 $ (Const (@{const_name is_unknown}, dom_T --> bool_T) $ t1')
blanchet@35665
   233
                $ (Const (@{const_name unknown}, ran_T)) $ (t0 $ t1 $ t2 $ t3)))
blanchet@35665
   234
  | fin_fun_body _ _ _ = NONE
blanchet@33192
   235
blanchet@35667
   236
fun fresh_mfun_for_fun_type (mdata as {max_fresh, ...} : mdata) all_minus
blanchet@35667
   237
                            T1 T2 =
blanchet@33192
   238
  let
blanchet@35667
   239
    val M1 = fresh_mtype_for_type mdata all_minus T1
blanchet@35667
   240
    val M2 = fresh_mtype_for_type mdata all_minus T2
blanchet@35667
   241
    val a = if not all_minus andalso exists_alpha_sub_mtype_fresh M1 andalso
blanchet@35667
   242
               is_fin_fun_supported_type (body_type T2) then
blanchet@35385
   243
              V (Unsynchronized.inc max_fresh)
blanchet@35385
   244
            else
blanchet@35385
   245
              S Minus
blanchet@35385
   246
  in (M1, a, M2) end
blanchet@37255
   247
and fresh_mtype_for_type (mdata as {hol_ctxt as {ctxt, ...}, binarize, alpha_T,
blanchet@35667
   248
                                    datatype_mcache, constr_mcache, ...})
blanchet@35667
   249
                         all_minus =
blanchet@35385
   250
  let
blanchet@35385
   251
    fun do_type T =
blanchet@33192
   252
      if T = alpha_T then
blanchet@35385
   253
        MAlpha
blanchet@33192
   254
      else case T of
blanchet@35665
   255
        Type (@{type_name fun}, [T1, T2]) =>
blanchet@35667
   256
        MFun (fresh_mfun_for_fun_type mdata false T1 T2)
blanchet@38417
   257
      | Type (@{type_name prod}, [T1, T2]) => MPair (pairself do_type (T1, T2))
blanchet@33192
   258
      | Type (z as (s, _)) =>
blanchet@37255
   259
        if could_exist_alpha_sub_mtype ctxt alpha_T T then
blanchet@35665
   260
          case AList.lookup (op =) (!datatype_mcache) z of
blanchet@35385
   261
            SOME M => M
blanchet@33192
   262
          | NONE =>
blanchet@33192
   263
            let
blanchet@35665
   264
              val _ = Unsynchronized.change datatype_mcache (cons (z, MRec z))
blanchet@35219
   265
              val xs = binarized_and_boxed_datatype_constrs hol_ctxt binarize T
blanchet@35385
   266
              val (all_Ms, constr_Ms) =
blanchet@35385
   267
                fold_rev (fn (_, T') => fn (all_Ms, constr_Ms) =>
blanchet@33192
   268
                             let
blanchet@35385
   269
                               val binder_Ms = map do_type (binder_types T')
blanchet@35385
   270
                               val new_Ms = filter exists_alpha_sub_mtype_fresh
blanchet@35385
   271
                                                   binder_Ms
blanchet@35385
   272
                               val constr_M = constr_mtype_for_binders z
blanchet@35385
   273
                                                                       binder_Ms
blanchet@33192
   274
                             in
blanchet@35385
   275
                               (union (op =) new_Ms all_Ms,
blanchet@35385
   276
                                constr_M :: constr_Ms)
blanchet@33192
   277
                             end)
blanchet@33192
   278
                         xs ([], [])
blanchet@35385
   279
              val M = MType (s, all_Ms)
blanchet@35665
   280
              val _ = Unsynchronized.change datatype_mcache
blanchet@35385
   281
                          (AList.update (op =) (z, M))
blanchet@35665
   282
              val _ = Unsynchronized.change constr_mcache
blanchet@35385
   283
                          (append (xs ~~ constr_Ms))
blanchet@33192
   284
            in
blanchet@35665
   285
              if forall (not o is_MRec o snd) (!datatype_mcache) then
blanchet@35665
   286
                (repair_datatype_mcache datatype_mcache;
blanchet@35665
   287
                 repair_constr_mcache (!datatype_mcache) constr_mcache;
blanchet@35665
   288
                 AList.lookup (op =) (!datatype_mcache) z |> the)
blanchet@33192
   289
              else
blanchet@35385
   290
                M
blanchet@33192
   291
            end
blanchet@33192
   292
        else
blanchet@35385
   293
          MType (s, [])
blanchet@37259
   294
      | _ => MType (simple_string_of_typ T, [])
blanchet@33192
   295
  in do_type end
blanchet@33192
   296
blanchet@35385
   297
fun prodM_factors (MPair (M1, M2)) = maps prodM_factors [M1, M2]
blanchet@35385
   298
  | prodM_factors M = [M]
blanchet@35665
   299
fun curried_strip_mtype (MFun (M1, _, M2)) =
blanchet@35385
   300
    curried_strip_mtype M2 |>> append (prodM_factors M1)
blanchet@35385
   301
  | curried_strip_mtype M = ([], M)
blanchet@35385
   302
fun sel_mtype_from_constr_mtype s M =
blanchet@35385
   303
  let val (arg_Ms, dataM) = curried_strip_mtype M in
blanchet@35385
   304
    MFun (dataM, S Minus,
blanchet@35385
   305
          case sel_no_from_name s of ~1 => bool_M | n => nth arg_Ms n)
blanchet@33192
   306
  end
blanchet@33192
   307
blanchet@37255
   308
fun mtype_for_constr (mdata as {hol_ctxt = {ctxt, ...}, alpha_T, constr_mcache,
blanchet@33192
   309
                                ...}) (x as (_, T)) =
blanchet@37255
   310
  if could_exist_alpha_sub_mtype ctxt alpha_T T then
blanchet@35665
   311
    case AList.lookup (op =) (!constr_mcache) x of
blanchet@35385
   312
      SOME M => M
blanchet@35384
   313
    | NONE => if T = alpha_T then
blanchet@35667
   314
                let val M = fresh_mtype_for_type mdata false T in
blanchet@35665
   315
                  (Unsynchronized.change constr_mcache (cons (x, M)); M)
blanchet@35384
   316
                end
blanchet@35384
   317
              else
blanchet@35667
   318
                (fresh_mtype_for_type mdata false (body_type T);
blanchet@35665
   319
                 AList.lookup (op =) (!constr_mcache) x |> the)
blanchet@33192
   320
  else
blanchet@35667
   321
    fresh_mtype_for_type mdata false T
blanchet@35385
   322
fun mtype_for_sel (mdata as {hol_ctxt, binarize, ...}) (x as (s, _)) =
blanchet@35190
   323
  x |> binarized_and_boxed_constr_for_sel hol_ctxt binarize
blanchet@35385
   324
    |> mtype_for_constr mdata |> sel_mtype_from_constr_mtype s
blanchet@33192
   325
blanchet@35665
   326
fun resolve_sign_atom lits (V x) =
blanchet@35665
   327
    x |> AList.lookup (op =) lits |> Option.map S |> the_default (V x)
blanchet@35665
   328
  | resolve_sign_atom _ a = a
blanchet@35665
   329
fun resolve_mtype lits =
blanchet@33192
   330
  let
blanchet@35385
   331
    fun aux MAlpha = MAlpha
blanchet@35665
   332
      | aux (MFun (M1, a, M2)) = MFun (aux M1, resolve_sign_atom lits a, aux M2)
blanchet@35385
   333
      | aux (MPair Mp) = MPair (pairself aux Mp)
blanchet@35385
   334
      | aux (MType (s, Ms)) = MType (s, map aux Ms)
blanchet@35385
   335
      | aux (MRec z) = MRec z
blanchet@33192
   336
  in aux end
blanchet@33192
   337
blanchet@33192
   338
datatype comp_op = Eq | Leq
blanchet@33192
   339
blanchet@33192
   340
type comp = sign_atom * sign_atom * comp_op * var list
blanchet@33192
   341
type sign_expr = literal list
blanchet@33192
   342
blanchet@35812
   343
type constraint_set = literal list * comp list * sign_expr list
blanchet@33192
   344
blanchet@33192
   345
fun string_for_comp_op Eq = "="
blanchet@33192
   346
  | string_for_comp_op Leq = "\<le>"
blanchet@33192
   347
blanchet@33192
   348
fun string_for_sign_expr [] = "\<bot>"
blanchet@33192
   349
  | string_for_sign_expr lits =
blanchet@33192
   350
    space_implode " \<or> " (map string_for_literal lits)
blanchet@33192
   351
blanchet@33192
   352
fun do_literal _ NONE = NONE
blanchet@33192
   353
  | do_literal (x, sn) (SOME lits) =
blanchet@33192
   354
    case AList.lookup (op =) lits x of
blanchet@33192
   355
      SOME sn' => if sn = sn' then SOME lits else NONE
blanchet@33192
   356
    | NONE => SOME ((x, sn) :: lits)
blanchet@33192
   357
blanchet@33192
   358
fun do_sign_atom_comp Eq [] a1 a2 (accum as (lits, comps)) =
blanchet@33192
   359
    (case (a1, a2) of
blanchet@33192
   360
       (S sn1, S sn2) => if sn1 = sn2 then SOME accum else NONE
blanchet@33192
   361
     | (V x1, S sn2) =>
blanchet@33192
   362
       Option.map (rpair comps) (do_literal (x1, sn2) (SOME lits))
blanchet@33192
   363
     | (V _, V _) => SOME (lits, insert (op =) (a1, a2, Eq, []) comps)
blanchet@33192
   364
     | _ => do_sign_atom_comp Eq [] a2 a1 accum)
blanchet@33192
   365
  | do_sign_atom_comp Leq [] a1 a2 (accum as (lits, comps)) =
blanchet@33192
   366
    (case (a1, a2) of
blanchet@34969
   367
       (_, S Minus) => SOME accum
blanchet@34969
   368
     | (S Plus, _) => SOME accum
blanchet@34969
   369
     | (S Minus, S Plus) => NONE
blanchet@33192
   370
     | (V _, V _) => SOME (lits, insert (op =) (a1, a2, Leq, []) comps)
blanchet@33192
   371
     | _ => do_sign_atom_comp Eq [] a1 a2 accum)
blanchet@35280
   372
  | do_sign_atom_comp cmp xs a1 a2 (lits, comps) =
blanchet@33192
   373
    SOME (lits, insert (op =) (a1, a2, cmp, xs) comps)
blanchet@33192
   374
blanchet@35385
   375
fun do_mtype_comp _ _ _ _ NONE = NONE
blanchet@35385
   376
  | do_mtype_comp _ _ MAlpha MAlpha accum = accum
blanchet@35385
   377
  | do_mtype_comp Eq xs (MFun (M11, a1, M12)) (MFun (M21, a2, M22))
blanchet@33192
   378
                  (SOME accum) =
blanchet@35385
   379
     accum |> do_sign_atom_comp Eq xs a1 a2 |> do_mtype_comp Eq xs M11 M21
blanchet@35385
   380
           |> do_mtype_comp Eq xs M12 M22
blanchet@35385
   381
  | do_mtype_comp Leq xs (MFun (M11, a1, M12)) (MFun (M21, a2, M22))
blanchet@33192
   382
                  (SOME accum) =
blanchet@35385
   383
    (if exists_alpha_sub_mtype M11 then
blanchet@33192
   384
       accum |> do_sign_atom_comp Leq xs a1 a2
blanchet@35385
   385
             |> do_mtype_comp Leq xs M21 M11
blanchet@33192
   386
             |> (case a2 of
blanchet@34969
   387
                   S Minus => I
blanchet@35385
   388
                 | S Plus => do_mtype_comp Leq xs M11 M21
blanchet@35385
   389
                 | V x => do_mtype_comp Leq (x :: xs) M11 M21)
blanchet@33192
   390
     else
blanchet@33192
   391
       SOME accum)
blanchet@35385
   392
    |> do_mtype_comp Leq xs M12 M22
blanchet@35385
   393
  | do_mtype_comp cmp xs (M1 as MPair (M11, M12)) (M2 as MPair (M21, M22))
blanchet@33192
   394
                  accum =
blanchet@35385
   395
    (accum |> fold (uncurry (do_mtype_comp cmp xs)) [(M11, M21), (M12, M22)]
blanchet@33192
   396
     handle Library.UnequalLengths =>
blanchet@35665
   397
            raise MTYPE ("Nitpick_Mono.do_mtype_comp", [M1, M2], []))
blanchet@35385
   398
  | do_mtype_comp _ _ (MType _) (MType _) accum =
blanchet@33192
   399
    accum (* no need to compare them thanks to the cache *)
blanchet@35665
   400
  | do_mtype_comp cmp _ M1 M2 _ =
blanchet@35665
   401
    raise MTYPE ("Nitpick_Mono.do_mtype_comp (" ^ string_for_comp_op cmp ^ ")",
blanchet@35665
   402
                 [M1, M2], [])
blanchet@33192
   403
blanchet@35832
   404
fun add_mtype_comp cmp M1 M2 ((lits, comps, sexps) : constraint_set) =
blanchet@38406
   405
    (trace_msg (fn () => "*** Add " ^ string_for_mtype M1 ^ " " ^
blanchet@38406
   406
                         string_for_comp_op cmp ^ " " ^ string_for_mtype M2);
blanchet@35385
   407
     case do_mtype_comp cmp [] M1 M2 (SOME (lits, comps)) of
blanchet@38406
   408
       NONE => (trace_msg (K "**** Unsolvable"); raise UNSOLVABLE ())
blanchet@35812
   409
     | SOME (lits, comps) => (lits, comps, sexps))
blanchet@33192
   410
blanchet@35385
   411
val add_mtypes_equal = add_mtype_comp Eq
blanchet@35385
   412
val add_is_sub_mtype = add_mtype_comp Leq
blanchet@33192
   413
blanchet@35385
   414
fun do_notin_mtype_fv _ _ _ NONE = NONE
blanchet@35385
   415
  | do_notin_mtype_fv Minus _ MAlpha accum = accum
blanchet@35385
   416
  | do_notin_mtype_fv Plus [] MAlpha _ = NONE
blanchet@35385
   417
  | do_notin_mtype_fv Plus [(x, sn)] MAlpha (SOME (lits, sexps)) =
blanchet@33192
   418
    SOME lits |> do_literal (x, sn) |> Option.map (rpair sexps)
blanchet@35385
   419
  | do_notin_mtype_fv Plus sexp MAlpha (SOME (lits, sexps)) =
blanchet@33192
   420
    SOME (lits, insert (op =) sexp sexps)
blanchet@35385
   421
  | do_notin_mtype_fv sn sexp (MFun (M1, S sn', M2)) accum =
blanchet@34969
   422
    accum |> (if sn' = Plus andalso sn = Plus then
blanchet@35385
   423
                do_notin_mtype_fv Plus sexp M1
blanchet@34969
   424
              else
blanchet@34969
   425
                I)
blanchet@34969
   426
          |> (if sn' = Minus orelse sn = Plus then
blanchet@35385
   427
                do_notin_mtype_fv Minus sexp M1
blanchet@34969
   428
              else
blanchet@34969
   429
                I)
blanchet@35385
   430
          |> do_notin_mtype_fv sn sexp M2
blanchet@35385
   431
  | do_notin_mtype_fv Plus sexp (MFun (M1, V x, M2)) accum =
blanchet@34969
   432
    accum |> (case do_literal (x, Minus) (SOME sexp) of
blanchet@33192
   433
                NONE => I
blanchet@35385
   434
              | SOME sexp' => do_notin_mtype_fv Plus sexp' M1)
blanchet@35385
   435
          |> do_notin_mtype_fv Minus sexp M1
blanchet@35385
   436
          |> do_notin_mtype_fv Plus sexp M2
blanchet@35385
   437
  | do_notin_mtype_fv Minus sexp (MFun (M1, V x, M2)) accum =
blanchet@34969
   438
    accum |> (case do_literal (x, Plus) (SOME sexp) of
blanchet@33192
   439
                NONE => I
blanchet@35385
   440
              | SOME sexp' => do_notin_mtype_fv Plus sexp' M1)
blanchet@35385
   441
          |> do_notin_mtype_fv Minus sexp M2
blanchet@35385
   442
  | do_notin_mtype_fv sn sexp (MPair (M1, M2)) accum =
blanchet@35385
   443
    accum |> fold (do_notin_mtype_fv sn sexp) [M1, M2]
blanchet@35385
   444
  | do_notin_mtype_fv sn sexp (MType (_, Ms)) accum =
blanchet@35385
   445
    accum |> fold (do_notin_mtype_fv sn sexp) Ms
blanchet@35385
   446
  | do_notin_mtype_fv _ _ M _ =
blanchet@35665
   447
    raise MTYPE ("Nitpick_Mono.do_notin_mtype_fv", [M], [])
blanchet@33192
   448
blanchet@35832
   449
fun add_notin_mtype_fv sn M ((lits, comps, sexps) : constraint_set) =
blanchet@38406
   450
    (trace_msg (fn () => "*** Add " ^ string_for_mtype M ^ " is " ^
blanchet@38406
   451
                         (case sn of Minus => "concrete" | Plus => "complete") ^
blanchet@38406
   452
                         ".");
blanchet@35385
   453
     case do_notin_mtype_fv sn [] M (SOME (lits, sexps)) of
blanchet@38406
   454
       NONE => (trace_msg (K "**** Unsolvable"); raise UNSOLVABLE ())
blanchet@35812
   455
     | SOME (lits, sexps) => (lits, comps, sexps))
blanchet@33192
   456
blanchet@35665
   457
val add_mtype_is_concrete = add_notin_mtype_fv Minus
blanchet@35665
   458
val add_mtype_is_complete = add_notin_mtype_fv Plus
blanchet@33192
   459
blanchet@35384
   460
val bool_from_minus = true
blanchet@35384
   461
blanchet@35384
   462
fun bool_from_sign Plus = not bool_from_minus
blanchet@35384
   463
  | bool_from_sign Minus = bool_from_minus
blanchet@35384
   464
fun sign_from_bool b = if b = bool_from_minus then Minus else Plus
blanchet@33192
   465
blanchet@33192
   466
fun prop_for_literal (x, sn) =
blanchet@33192
   467
  (not (bool_from_sign sn) ? PropLogic.Not) (PropLogic.BoolVar x)
blanchet@33192
   468
fun prop_for_sign_atom_eq (S sn', sn) =
blanchet@33192
   469
    if sn = sn' then PropLogic.True else PropLogic.False
blanchet@33192
   470
  | prop_for_sign_atom_eq (V x, sn) = prop_for_literal (x, sn)
blanchet@33192
   471
fun prop_for_sign_expr xs = PropLogic.exists (map prop_for_literal xs)
blanchet@33192
   472
fun prop_for_exists_eq xs sn =
blanchet@33192
   473
  PropLogic.exists (map (fn x => prop_for_literal (x, sn)) xs)
blanchet@33192
   474
fun prop_for_comp (a1, a2, Eq, []) =
blanchet@33192
   475
    PropLogic.SAnd (prop_for_comp (a1, a2, Leq, []),
blanchet@33192
   476
                    prop_for_comp (a2, a1, Leq, []))
blanchet@33192
   477
  | prop_for_comp (a1, a2, Leq, []) =
blanchet@34969
   478
    PropLogic.SOr (prop_for_sign_atom_eq (a1, Plus),
blanchet@34969
   479
                   prop_for_sign_atom_eq (a2, Minus))
blanchet@33192
   480
  | prop_for_comp (a1, a2, cmp, xs) =
blanchet@34969
   481
    PropLogic.SOr (prop_for_exists_eq xs Minus, prop_for_comp (a1, a2, cmp, []))
blanchet@33192
   482
blanchet@34120
   483
fun literals_from_assignments max_var assigns lits =
blanchet@33192
   484
  fold (fn x => fn accum =>
blanchet@33192
   485
           if AList.defined (op =) lits x then
blanchet@33192
   486
             accum
blanchet@34120
   487
           else case assigns x of
blanchet@33192
   488
             SOME b => (x, sign_from_bool b) :: accum
blanchet@33192
   489
           | NONE => accum) (max_var downto 1) lits
blanchet@33192
   490
blanchet@33192
   491
fun string_for_comp (a1, a2, cmp, xs) =
blanchet@33192
   492
  string_for_sign_atom a1 ^ " " ^ string_for_comp_op cmp ^
blanchet@33192
   493
  subscript_string_for_vars " \<and> " xs ^ " " ^ string_for_sign_atom a2
blanchet@33192
   494
blanchet@33192
   495
fun print_problem lits comps sexps =
blanchet@38406
   496
  trace_msg (fn () => "*** Problem:\n" ^
blanchet@38406
   497
                      cat_lines (map string_for_literal lits @
blanchet@38406
   498
                                 map string_for_comp comps @
blanchet@38406
   499
                                 map string_for_sign_expr sexps))
blanchet@33192
   500
blanchet@33192
   501
fun print_solution lits =
blanchet@34969
   502
  let val (pos, neg) = List.partition (curry (op =) Plus o snd) lits in
blanchet@38406
   503
    trace_msg (fn () => "*** Solution:\n" ^
blanchet@38406
   504
                        "+: " ^ commas (map (string_for_var o fst) pos) ^ "\n" ^
blanchet@38406
   505
                        "-: " ^ commas (map (string_for_var o fst) neg))
blanchet@33192
   506
  end
blanchet@33192
   507
blanchet@35812
   508
fun solve max_var (lits, comps, sexps) =
blanchet@33192
   509
    let
blanchet@35386
   510
      fun do_assigns assigns =
blanchet@35386
   511
        SOME (literals_from_assignments max_var assigns lits
blanchet@35386
   512
              |> tap print_solution)
blanchet@33192
   513
      val _ = print_problem lits comps sexps
blanchet@33192
   514
      val prop = PropLogic.all (map prop_for_literal lits @
blanchet@33192
   515
                                map prop_for_comp comps @
blanchet@33192
   516
                                map prop_for_sign_expr sexps)
blanchet@35386
   517
      val default_val = bool_from_sign Minus
blanchet@33192
   518
    in
blanchet@35386
   519
      if PropLogic.eval (K default_val) prop then
blanchet@35386
   520
        do_assigns (K (SOME default_val))
blanchet@35386
   521
      else
blanchet@35386
   522
        let
blanchet@35386
   523
          (* use the first ML solver (to avoid startup overhead) *)
blanchet@35386
   524
          val solvers = !SatSolver.solvers
blanchet@35386
   525
                        |> filter (member (op =) ["dptsat", "dpll"] o fst)
blanchet@35386
   526
        in
blanchet@35386
   527
          case snd (hd solvers) prop of
blanchet@35386
   528
            SatSolver.SATISFIABLE assigns => do_assigns assigns
blanchet@35386
   529
          | _ => NONE
blanchet@35386
   530
        end
blanchet@33192
   531
    end
blanchet@33192
   532
blanchet@35385
   533
type mtype_schema = mtyp * constraint_set
blanchet@35385
   534
type mtype_context =
blanchet@35665
   535
  {bound_Ts: typ list,
blanchet@35665
   536
   bound_Ms: mtyp list,
blanchet@35385
   537
   frees: (styp * mtyp) list,
blanchet@35385
   538
   consts: (styp * mtyp) list}
blanchet@33192
   539
blanchet@35385
   540
type accumulator = mtype_context * constraint_set
blanchet@33192
   541
blanchet@35665
   542
val initial_gamma = {bound_Ts = [], bound_Ms = [], frees = [], consts = []}
blanchet@33192
   543
blanchet@35665
   544
fun push_bound T M {bound_Ts, bound_Ms, frees, consts} =
blanchet@35665
   545
  {bound_Ts = T :: bound_Ts, bound_Ms = M :: bound_Ms, frees = frees,
blanchet@35665
   546
   consts = consts}
blanchet@35665
   547
fun pop_bound {bound_Ts, bound_Ms, frees, consts} =
blanchet@35665
   548
  {bound_Ts = tl bound_Ts, bound_Ms = tl bound_Ms, frees = frees,
blanchet@35665
   549
   consts = consts}
blanchet@35665
   550
  handle List.Empty => initial_gamma (* FIXME: needed? *)
blanchet@33192
   551
blanchet@35386
   552
fun consider_term (mdata as {hol_ctxt as {thy, ctxt, stds, fast_descrs,
blanchet@35665
   553
                                          def_table, ...},
blanchet@35220
   554
                             alpha_T, max_fresh, ...}) =
blanchet@33192
   555
  let
blanchet@37451
   556
    fun is_enough_eta_expanded t =
blanchet@37451
   557
      case strip_comb t of
blanchet@37451
   558
        (Const x, ts) =>
blanchet@37451
   559
        the_default 0 (arity_of_built_in_const thy stds fast_descrs x)
blanchet@37451
   560
        <= length ts
blanchet@37451
   561
      | _ => true
blanchet@35667
   562
    val mtype_for = fresh_mtype_for_type mdata false
blanchet@35665
   563
    fun plus_set_mtype_for_dom M =
blanchet@35385
   564
      MFun (M, S (if exists_alpha_sub_mtype M then Plus else Minus), bool_M)
blanchet@35385
   565
    fun do_all T (gamma, cset) =
blanchet@33192
   566
      let
blanchet@35385
   567
        val abs_M = mtype_for (domain_type (domain_type T))
blanchet@35386
   568
        val body_M = mtype_for (body_type T)
blanchet@33192
   569
      in
blanchet@35385
   570
        (MFun (MFun (abs_M, S Minus, body_M), S Minus, body_M),
blanchet@35665
   571
         (gamma, cset |> add_mtype_is_complete abs_M))
blanchet@33192
   572
      end
blanchet@33192
   573
    fun do_equals T (gamma, cset) =
blanchet@35385
   574
      let val M = mtype_for (domain_type T) in
blanchet@35385
   575
        (MFun (M, S Minus, MFun (M, V (Unsynchronized.inc max_fresh),
blanchet@35385
   576
                                 mtype_for (nth_range_type 2 T))),
blanchet@35665
   577
         (gamma, cset |> add_mtype_is_concrete M))
blanchet@33192
   578
      end
blanchet@33192
   579
    fun do_robust_set_operation T (gamma, cset) =
blanchet@33192
   580
      let
blanchet@33192
   581
        val set_T = domain_type T
blanchet@35385
   582
        val M1 = mtype_for set_T
blanchet@35385
   583
        val M2 = mtype_for set_T
blanchet@35385
   584
        val M3 = mtype_for set_T
blanchet@33192
   585
      in
blanchet@35385
   586
        (MFun (M1, S Minus, MFun (M2, S Minus, M3)),
blanchet@35385
   587
         (gamma, cset |> add_is_sub_mtype M1 M3 |> add_is_sub_mtype M2 M3))
blanchet@33192
   588
      end
blanchet@33192
   589
    fun do_fragile_set_operation T (gamma, cset) =
blanchet@33192
   590
      let
blanchet@33192
   591
        val set_T = domain_type T
blanchet@35385
   592
        val set_M = mtype_for set_T
blanchet@35665
   593
        fun custom_mtype_for (T as Type (@{type_name fun}, [T1, T2])) =
blanchet@35385
   594
            if T = set_T then set_M
blanchet@35385
   595
            else MFun (custom_mtype_for T1, S Minus, custom_mtype_for T2)
blanchet@35385
   596
          | custom_mtype_for T = mtype_for T
blanchet@33192
   597
      in
blanchet@35665
   598
        (custom_mtype_for T, (gamma, cset |> add_mtype_is_concrete set_M))
blanchet@33192
   599
      end
blanchet@33192
   600
    fun do_pair_constr T accum =
blanchet@35385
   601
      case mtype_for (nth_range_type 2 T) of
blanchet@35385
   602
        M as MPair (a_M, b_M) =>
blanchet@35385
   603
        (MFun (a_M, S Minus, MFun (b_M, S Minus, M)), accum)
blanchet@35665
   604
      | M => raise MTYPE ("Nitpick_Mono.consider_term.do_pair_constr", [M], [])
blanchet@33192
   605
    fun do_nth_pair_sel n T =
blanchet@35385
   606
      case mtype_for (domain_type T) of
blanchet@35385
   607
        M as MPair (a_M, b_M) =>
blanchet@35385
   608
        pair (MFun (M, S Minus, if n = 0 then a_M else b_M))
blanchet@35665
   609
      | M => raise MTYPE ("Nitpick_Mono.consider_term.do_nth_pair_sel", [M], [])
blanchet@35385
   610
    fun do_bounded_quantifier t0 abs_s abs_T connective_t bound_t body_t accum =
blanchet@33192
   611
      let
blanchet@35385
   612
        val abs_M = mtype_for abs_T
blanchet@35665
   613
        val (bound_m, accum) =
blanchet@35665
   614
          accum |>> push_bound abs_T abs_M |> do_term bound_t
blanchet@35665
   615
        val expected_bound_M = plus_set_mtype_for_dom abs_M
blanchet@35385
   616
        val (body_m, accum) =
blanchet@35385
   617
          accum ||> add_mtypes_equal expected_bound_M (mtype_of_mterm bound_m)
blanchet@35385
   618
                |> do_term body_t ||> apfst pop_bound
blanchet@35385
   619
        val bound_M = mtype_of_mterm bound_m
blanchet@35385
   620
        val (M1, a, M2) = dest_MFun bound_M
blanchet@33192
   621
      in
blanchet@35386
   622
        (MApp (MRaw (t0, MFun (bound_M, S Minus, bool_M)),
blanchet@35385
   623
               MAbs (abs_s, abs_T, M1, a,
blanchet@35386
   624
                     MApp (MApp (MRaw (connective_t,
blanchet@35386
   625
                                       mtype_for (fastype_of connective_t)),
blanchet@35386
   626
                                 MApp (bound_m, MRaw (Bound 0, M1))),
blanchet@35385
   627
                           body_m))), accum)
blanchet@33192
   628
      end
blanchet@35812
   629
    and do_term t (accum as (gamma as {bound_Ts, bound_Ms, frees, consts},
blanchet@35665
   630
                             cset)) =
blanchet@38406
   631
        (trace_msg (fn () => "  \<Gamma> \<turnstile> " ^
blanchet@38406
   632
                             Syntax.string_of_term ctxt t ^ " : _?");
blanchet@37695
   633
         case t of
blanchet@33192
   634
           Const (x as (s, T)) =>
blanchet@33192
   635
           (case AList.lookup (op =) consts x of
blanchet@35385
   636
              SOME M => (M, accum)
blanchet@33192
   637
            | NONE =>
blanchet@33192
   638
              if not (could_exist_alpha_subtype alpha_T T) then
blanchet@35385
   639
                (mtype_for T, accum)
blanchet@33192
   640
              else case s of
blanchet@35385
   641
                @{const_name all} => do_all T accum
blanchet@33192
   642
              | @{const_name "=="} => do_equals T accum
blanchet@35385
   643
              | @{const_name All} => do_all T accum
blanchet@35385
   644
              | @{const_name Ex} =>
blanchet@35386
   645
                let val set_T = domain_type T in
blanchet@35386
   646
                  do_term (Abs (Name.uu, set_T,
blanchet@35386
   647
                                @{const Not} $ (HOLogic.mk_eq
blanchet@35386
   648
                                    (Abs (Name.uu, domain_type set_T,
blanchet@35386
   649
                                          @{const False}),
blanchet@35386
   650
                                     Bound 0)))) accum
blanchet@35386
   651
                  |>> mtype_of_mterm
blanchet@35386
   652
                end
blanchet@33192
   653
              | @{const_name "op ="} => do_equals T accum
blanchet@37451
   654
              | @{const_name The} =>
blanchet@38406
   655
                (trace_msg (K "*** The"); raise UNSOLVABLE ())
blanchet@37451
   656
              | @{const_name Eps} =>
blanchet@38406
   657
                (trace_msg (K "*** Eps"); raise UNSOLVABLE ())
blanchet@33192
   658
              | @{const_name If} =>
blanchet@33192
   659
                do_robust_set_operation (range_type T) accum
blanchet@35385
   660
                |>> curry3 MFun bool_M (S Minus)
blanchet@33192
   661
              | @{const_name Pair} => do_pair_constr T accum
blanchet@33192
   662
              | @{const_name fst} => do_nth_pair_sel 0 T accum
blanchet@33192
   663
              | @{const_name snd} => do_nth_pair_sel 1 T accum 
blanchet@33192
   664
              | @{const_name Id} =>
blanchet@35385
   665
                (MFun (mtype_for (domain_type T), S Minus, bool_M), accum)
blanchet@33192
   666
              | @{const_name converse} =>
blanchet@33192
   667
                let
blanchet@33192
   668
                  val x = Unsynchronized.inc max_fresh
blanchet@35385
   669
                  fun mtype_for_set T =
blanchet@35385
   670
                    MFun (mtype_for (domain_type T), V x, bool_M)
blanchet@35385
   671
                  val ab_set_M = domain_type T |> mtype_for_set
blanchet@35385
   672
                  val ba_set_M = range_type T |> mtype_for_set
blanchet@35385
   673
                in (MFun (ab_set_M, S Minus, ba_set_M), accum) end
blanchet@33192
   674
              | @{const_name trancl} => do_fragile_set_operation T accum
blanchet@33192
   675
              | @{const_name rel_comp} =>
blanchet@33192
   676
                let
blanchet@33192
   677
                  val x = Unsynchronized.inc max_fresh
blanchet@35385
   678
                  fun mtype_for_set T =
blanchet@35385
   679
                    MFun (mtype_for (domain_type T), V x, bool_M)
blanchet@35385
   680
                  val bc_set_M = domain_type T |> mtype_for_set
blanchet@35385
   681
                  val ab_set_M = domain_type (range_type T) |> mtype_for_set
blanchet@35385
   682
                  val ac_set_M = nth_range_type 2 T |> mtype_for_set
blanchet@33192
   683
                in
blanchet@35385
   684
                  (MFun (bc_set_M, S Minus, MFun (ab_set_M, S Minus, ac_set_M)),
blanchet@33192
   685
                   accum)
blanchet@33192
   686
                end
blanchet@33192
   687
              | @{const_name image} =>
blanchet@33192
   688
                let
blanchet@35385
   689
                  val a_M = mtype_for (domain_type (domain_type T))
blanchet@35385
   690
                  val b_M = mtype_for (range_type (domain_type T))
blanchet@33192
   691
                in
blanchet@35385
   692
                  (MFun (MFun (a_M, S Minus, b_M), S Minus,
blanchet@35665
   693
                         MFun (plus_set_mtype_for_dom a_M, S Minus,
blanchet@35665
   694
                               plus_set_mtype_for_dom b_M)), accum)
blanchet@33192
   695
                end
blanchet@35667
   696
              | @{const_name finite} =>
blanchet@35667
   697
                let val M1 = mtype_for (domain_type (domain_type T)) in
blanchet@35667
   698
                  (MFun (plus_set_mtype_for_dom M1, S Minus, bool_M), accum)
blanchet@35667
   699
                end
blanchet@33192
   700
              | @{const_name Sigma} =>
blanchet@33192
   701
                let
blanchet@33192
   702
                  val x = Unsynchronized.inc max_fresh
blanchet@35385
   703
                  fun mtype_for_set T =
blanchet@35385
   704
                    MFun (mtype_for (domain_type T), V x, bool_M)
blanchet@33192
   705
                  val a_set_T = domain_type T
blanchet@35385
   706
                  val a_M = mtype_for (domain_type a_set_T)
blanchet@35385
   707
                  val b_set_M = mtype_for_set (range_type (domain_type
blanchet@33192
   708
                                                               (range_type T)))
blanchet@35385
   709
                  val a_set_M = mtype_for_set a_set_T
blanchet@35385
   710
                  val a_to_b_set_M = MFun (a_M, S Minus, b_set_M)
blanchet@35385
   711
                  val ab_set_M = mtype_for_set (nth_range_type 2 T)
blanchet@33192
   712
                in
blanchet@35385
   713
                  (MFun (a_set_M, S Minus,
blanchet@35385
   714
                         MFun (a_to_b_set_M, S Minus, ab_set_M)), accum)
blanchet@33192
   715
                end
blanchet@35220
   716
              | _ =>
blanchet@35666
   717
                if s = @{const_name safe_The} orelse
blanchet@35666
   718
                   s = @{const_name safe_Eps} then
blanchet@35666
   719
                  let
blanchet@35666
   720
                    val a_set_M = mtype_for (domain_type T)
blanchet@35666
   721
                    val a_M = dest_MFun a_set_M |> #1
blanchet@35666
   722
                  in (MFun (a_set_M, S Minus, a_M), accum) end
blanchet@35220
   723
                else if s = @{const_name ord_class.less_eq} andalso
blanchet@35220
   724
                        is_set_type (domain_type T) then
blanchet@35220
   725
                  do_fragile_set_operation T accum
blanchet@35220
   726
                else if is_sel s then
blanchet@35665
   727
                  (mtype_for_sel mdata x, accum)
blanchet@37255
   728
                else if is_constr ctxt stds x then
blanchet@35385
   729
                  (mtype_for_constr mdata x, accum)
blanchet@35667
   730
                else if is_built_in_const thy stds fast_descrs x then
blanchet@35667
   731
                  (fresh_mtype_for_type mdata true T, accum)
blanchet@35220
   732
                else
blanchet@35385
   733
                  let val M = mtype_for T in
blanchet@35665
   734
                    (M, ({bound_Ts = bound_Ts, bound_Ms = bound_Ms,
blanchet@35665
   735
                          frees = frees, consts = (x, M) :: consts}, cset))
blanchet@35386
   736
                  end) |>> curry MRaw t
blanchet@33192
   737
         | Free (x as (_, T)) =>
blanchet@33192
   738
           (case AList.lookup (op =) frees x of
blanchet@35385
   739
              SOME M => (M, accum)
blanchet@33192
   740
            | NONE =>
blanchet@35385
   741
              let val M = mtype_for T in
blanchet@35665
   742
                (M, ({bound_Ts = bound_Ts, bound_Ms = bound_Ms,
blanchet@35665
   743
                      frees = (x, M) :: frees, consts = consts}, cset))
blanchet@35386
   744
              end) |>> curry MRaw t
blanchet@38406
   745
         | Var _ => (trace_msg (K "*** Var"); raise UNSOLVABLE ())
blanchet@35665
   746
         | Bound j => (MRaw (t, nth bound_Ms j), accum)
blanchet@35385
   747
         | Abs (s, T, t') =>
blanchet@35665
   748
           (case fin_fun_body T (fastype_of1 (T :: bound_Ts, t')) t' of
blanchet@35665
   749
              SOME t' =>
blanchet@35665
   750
              let
blanchet@35665
   751
                val M = mtype_for T
blanchet@35665
   752
                val a = V (Unsynchronized.inc max_fresh)
blanchet@35665
   753
                val (m', accum) = do_term t' (accum |>> push_bound T M)
blanchet@35665
   754
              in (MAbs (s, T, M, a, m'), accum |>> pop_bound) end
blanchet@35665
   755
            | NONE =>
blanchet@35665
   756
              ((case t' of
blanchet@35665
   757
                  t1' $ Bound 0 =>
blanchet@37451
   758
                  if not (loose_bvar1 (t1', 0)) andalso
blanchet@37451
   759
                     is_enough_eta_expanded t1' then
blanchet@35665
   760
                    do_term (incr_boundvars ~1 t1') accum
blanchet@35665
   761
                  else
blanchet@35665
   762
                    raise SAME ()
blanchet@37451
   763
                | (t11 as Const (@{const_name "op ="}, _)) $ Bound 0 $ t13 =>
blanchet@37451
   764
                  if not (loose_bvar1 (t13, 0)) then
blanchet@37451
   765
                    do_term (incr_boundvars ~1 (t11 $ t13)) accum
blanchet@37451
   766
                  else
blanchet@37451
   767
                    raise SAME ()
blanchet@35665
   768
                | _ => raise SAME ())
blanchet@35665
   769
               handle SAME () =>
blanchet@35665
   770
                      let
blanchet@35665
   771
                        val M = mtype_for T
blanchet@35665
   772
                        val (m', accum) = do_term t' (accum |>> push_bound T M)
blanchet@35665
   773
                      in
blanchet@35665
   774
                        (MAbs (s, T, M, S Minus, m'), accum |>> pop_bound)
blanchet@35665
   775
                      end))
blanchet@35385
   776
         | (t0 as Const (@{const_name All}, _))
haftmann@39019
   777
           $ Abs (s', T', (t10 as @{const HOL.implies}) $ (t11 $ Bound 0) $ t12) =>
blanchet@35385
   778
           do_bounded_quantifier t0 s' T' t10 t11 t12 accum
blanchet@35385
   779
         | (t0 as Const (@{const_name Ex}, _))
blanchet@35385
   780
           $ Abs (s', T', (t10 as @{const "op &"}) $ (t11 $ Bound 0) $ t12) =>
blanchet@35385
   781
           do_bounded_quantifier t0 s' T' t10 t11 t12 accum
blanchet@33192
   782
         | Const (@{const_name Let}, _) $ t1 $ t2 =>
blanchet@33192
   783
           do_term (betapply (t2, t1)) accum
blanchet@33192
   784
         | t1 $ t2 =>
blanchet@33192
   785
           let
blanchet@35385
   786
             val (m1, accum) = do_term t1 accum
blanchet@35385
   787
             val (m2, accum) = do_term t2 accum
blanchet@33192
   788
           in
blanchet@35812
   789
             let
blanchet@35812
   790
               val T11 = domain_type (fastype_of1 (bound_Ts, t1))
blanchet@35812
   791
               val T2 = fastype_of1 (bound_Ts, t2)
blanchet@35812
   792
               val M11 = mtype_of_mterm m1 |> dest_MFun |> #1
blanchet@35812
   793
               val M2 = mtype_of_mterm m2
blanchet@35812
   794
             in (MApp (m1, m2), accum ||> add_is_sub_mtype M2 M11) end
blanchet@33192
   795
           end)
blanchet@38406
   796
        |> tap (fn (m, _) => trace_msg (fn () => "  \<Gamma> \<turnstile> " ^
blanchet@38406
   797
                                                 string_for_mterm ctxt m))
blanchet@33192
   798
  in do_term end
blanchet@33192
   799
blanchet@35665
   800
fun force_minus_funs 0 _ = I
blanchet@35665
   801
  | force_minus_funs n (M as MFun (M1, _, M2)) =
blanchet@35665
   802
    add_mtypes_equal M (MFun (M1, S Minus, M2))
blanchet@35665
   803
    #> force_minus_funs (n - 1) M2
blanchet@35665
   804
  | force_minus_funs _ M =
blanchet@35665
   805
    raise MTYPE ("Nitpick_Mono.force_minus_funs", [M], [])
blanchet@35665
   806
fun consider_general_equals mdata def (x as (_, T)) t1 t2 accum =
blanchet@35386
   807
  let
blanchet@35386
   808
    val (m1, accum) = consider_term mdata t1 accum
blanchet@35386
   809
    val (m2, accum) = consider_term mdata t2 accum
blanchet@35386
   810
    val M1 = mtype_of_mterm m1
blanchet@35386
   811
    val M2 = mtype_of_mterm m2
blanchet@35665
   812
    val accum = accum ||> add_mtypes_equal M1 M2
blanchet@35667
   813
    val body_M = fresh_mtype_for_type mdata false (nth_range_type 2 T)
blanchet@35665
   814
    val m = MApp (MApp (MRaw (Const x,
blanchet@35665
   815
                MFun (M1, S Minus, MFun (M2, S Minus, body_M))), m1), m2)
blanchet@35386
   816
  in
blanchet@35665
   817
    (m, if def then
blanchet@35665
   818
          let val (head_m, arg_ms) = strip_mcomb m1 in
blanchet@35665
   819
            accum ||> force_minus_funs (length arg_ms) (mtype_of_mterm head_m)
blanchet@35665
   820
          end
blanchet@35665
   821
        else
blanchet@35665
   822
          accum)
blanchet@35386
   823
  end
blanchet@35386
   824
blanchet@35385
   825
fun consider_general_formula (mdata as {hol_ctxt = {ctxt, ...}, ...}) =
blanchet@33192
   826
  let
blanchet@35667
   827
    val mtype_for = fresh_mtype_for_type mdata false
blanchet@35386
   828
    val do_term = consider_term mdata
blanchet@35812
   829
    fun do_formula sn t accum =
blanchet@33192
   830
        let
blanchet@35386
   831
          fun do_quantifier (quant_x as (quant_s, _)) abs_s abs_T body_t =
blanchet@33192
   832
            let
blanchet@35385
   833
              val abs_M = mtype_for abs_T
blanchet@34969
   834
              val side_cond = ((sn = Minus) = (quant_s = @{const_name Ex}))
blanchet@35386
   835
              val (body_m, accum) =
blanchet@35665
   836
                accum ||> side_cond ? add_mtype_is_complete abs_M
blanchet@35665
   837
                      |>> push_bound abs_T abs_M |> do_formula sn body_t
blanchet@35386
   838
              val body_M = mtype_of_mterm body_m
blanchet@33192
   839
            in
blanchet@35665
   840
              (MApp (MRaw (Const quant_x,
blanchet@35665
   841
                           MFun (MFun (abs_M, S Minus, body_M), S Minus,
blanchet@35665
   842
                                 body_M)),
blanchet@35386
   843
                     MAbs (abs_s, abs_T, abs_M, S Minus, body_m)),
blanchet@35386
   844
               accum |>> pop_bound)
blanchet@33192
   845
            end
blanchet@35386
   846
          fun do_equals x t1 t2 =
blanchet@33192
   847
            case sn of
blanchet@35386
   848
              Plus => do_term t accum
blanchet@35665
   849
            | Minus => consider_general_equals mdata false x t1 t2 accum
blanchet@33192
   850
        in
blanchet@38406
   851
          (trace_msg (fn () => "  \<Gamma> \<turnstile> " ^
blanchet@38406
   852
                               Syntax.string_of_term ctxt t ^ " : o\<^sup>" ^
blanchet@38406
   853
                               string_for_sign sn ^ "?");
blanchet@37695
   854
           case t of
blanchet@37695
   855
             Const (x as (@{const_name all}, _)) $ Abs (s1, T1, t1) =>
blanchet@37695
   856
             do_quantifier x s1 T1 t1
blanchet@37695
   857
           | Const (x as (@{const_name "=="}, _)) $ t1 $ t2 => do_equals x t1 t2
blanchet@37695
   858
           | @{const Trueprop} $ t1 =>
blanchet@37695
   859
             let val (m1, accum) = do_formula sn t1 accum in
blanchet@37695
   860
               (MApp (MRaw (@{const Trueprop}, mtype_for (bool_T --> prop_T)),
blanchet@37695
   861
                      m1), accum)
blanchet@37695
   862
             end
blanchet@37695
   863
           | @{const Not} $ t1 =>
blanchet@37695
   864
             let val (m1, accum) = do_formula (negate sn) t1 accum in
blanchet@37695
   865
               (MApp (MRaw (@{const Not}, mtype_for (bool_T --> bool_T)), m1),
blanchet@37695
   866
                accum)
blanchet@37695
   867
             end
blanchet@37695
   868
           | Const (x as (@{const_name All}, _)) $ Abs (s1, T1, t1) =>
blanchet@37695
   869
             do_quantifier x s1 T1 t1
blanchet@37695
   870
           | Const (x0 as (s0 as @{const_name Ex}, T0))
blanchet@37695
   871
             $ (t1 as Abs (s1, T1, t1')) =>
blanchet@37695
   872
             (case sn of
blanchet@37695
   873
                Plus => do_quantifier x0 s1 T1 t1'
blanchet@37695
   874
              | Minus =>
blanchet@37695
   875
                (* FIXME: Move elsewhere *)
blanchet@37695
   876
                do_term (@{const Not}
blanchet@37695
   877
                         $ (HOLogic.eq_const (domain_type T0) $ t1
blanchet@37695
   878
                            $ Abs (Name.uu, T1, @{const False}))) accum)
blanchet@37695
   879
           | Const (x as (@{const_name "op ="}, _)) $ t1 $ t2 =>
blanchet@37695
   880
             do_equals x t1 t2
blanchet@37695
   881
           | Const (@{const_name Let}, _) $ t1 $ t2 =>
blanchet@37695
   882
             do_formula sn (betapply (t2, t1)) accum
blanchet@37695
   883
           | (t0 as Const (s0, _)) $ t1 $ t2 =>
blanchet@38426
   884
             if s0 = @{const_name "==>"} orelse
blanchet@38426
   885
                s0 = @{const_name Pure.conjunction} orelse
blanchet@38426
   886
                s0 = @{const_name "op &"} orelse
blanchet@37695
   887
                s0 = @{const_name "op |"} orelse
haftmann@39019
   888
                s0 = @{const_name HOL.implies} then
blanchet@37695
   889
               let
blanchet@37695
   890
                 val impl = (s0 = @{const_name "==>"} orelse
haftmann@39019
   891
                             s0 = @{const_name HOL.implies})
blanchet@37695
   892
                 val (m1, accum) = do_formula (sn |> impl ? negate) t1 accum
blanchet@37695
   893
                 val (m2, accum) = do_formula sn t2 accum
blanchet@37695
   894
               in
blanchet@37695
   895
                 (MApp (MApp (MRaw (t0, mtype_for (fastype_of t0)), m1), m2),
blanchet@37695
   896
                  accum)
blanchet@37695
   897
               end 
blanchet@37695
   898
             else
blanchet@37695
   899
               do_term t accum
blanchet@37695
   900
           | _ => do_term t accum)
blanchet@33192
   901
        end
blanchet@35386
   902
        |> tap (fn (m, _) =>
blanchet@38406
   903
                   trace_msg (fn () => "\<Gamma> \<turnstile> " ^
blanchet@38406
   904
                                       string_for_mterm ctxt m ^ " : o\<^sup>" ^
blanchet@38406
   905
                                       string_for_sign sn))
blanchet@33192
   906
  in do_formula end
blanchet@33192
   907
blanchet@33192
   908
(* The harmless axiom optimization below is somewhat too aggressive in the face
blanchet@33192
   909
   of (rather peculiar) user-defined axioms. *)
blanchet@33192
   910
val harmless_consts =
blanchet@33192
   911
  [@{const_name ord_class.less}, @{const_name ord_class.less_eq}]
blanchet@33192
   912
val bounteous_consts = [@{const_name bisim}]
blanchet@33192
   913
blanchet@35665
   914
fun is_harmless_axiom ({no_harmless = true, ...} : mdata) _ = false
blanchet@35665
   915
  | is_harmless_axiom {hol_ctxt = {thy, stds, fast_descrs, ...}, ...} t =
blanchet@35665
   916
    Term.add_consts t []
blanchet@35665
   917
    |> filter_out (is_built_in_const thy stds fast_descrs)
blanchet@35665
   918
    |> (forall (member (op =) harmless_consts o original_name o fst) orf
blanchet@35665
   919
        exists (member (op =) bounteous_consts o fst))
blanchet@33192
   920
blanchet@35665
   921
fun consider_nondefinitional_axiom mdata t =
blanchet@35665
   922
  if is_harmless_axiom mdata t then pair (MRaw (t, dummy_M))
blanchet@35386
   923
  else consider_general_formula mdata Plus t
blanchet@33192
   924
blanchet@37255
   925
fun consider_definitional_axiom (mdata as {hol_ctxt = {ctxt, ...}, ...}) t =
blanchet@37255
   926
  if not (is_constr_pattern_formula ctxt t) then
blanchet@35386
   927
    consider_nondefinitional_axiom mdata t
blanchet@35665
   928
  else if is_harmless_axiom mdata t then
blanchet@35386
   929
    pair (MRaw (t, dummy_M))
blanchet@33192
   930
  else
blanchet@33192
   931
    let
blanchet@35667
   932
      val mtype_for = fresh_mtype_for_type mdata false
blanchet@35386
   933
      val do_term = consider_term mdata
blanchet@35386
   934
      fun do_all quant_t abs_s abs_T body_t accum =
blanchet@35386
   935
        let
blanchet@35386
   936
          val abs_M = mtype_for abs_T
blanchet@35386
   937
          val (body_m, accum) =
blanchet@35665
   938
            accum |>> push_bound abs_T abs_M |> do_formula body_t
blanchet@35386
   939
          val body_M = mtype_of_mterm body_m
blanchet@35386
   940
        in
blanchet@35665
   941
          (MApp (MRaw (quant_t,
blanchet@35665
   942
                       MFun (MFun (abs_M, S Minus, body_M), S Minus, body_M)),
blanchet@35386
   943
                 MAbs (abs_s, abs_T, abs_M, S Minus, body_m)),
blanchet@35386
   944
           accum |>> pop_bound)
blanchet@33192
   945
        end
blanchet@35386
   946
      and do_conjunction t0 t1 t2 accum =
blanchet@33192
   947
        let
blanchet@35386
   948
          val (m1, accum) = do_formula t1 accum
blanchet@35386
   949
          val (m2, accum) = do_formula t2 accum
blanchet@35386
   950
        in
blanchet@35386
   951
          (MApp (MApp (MRaw (t0, mtype_for (fastype_of t0)), m1), m2), accum)
blanchet@35386
   952
        end
blanchet@35386
   953
      and do_implies t0 t1 t2 accum =
blanchet@35386
   954
        let
blanchet@35386
   955
          val (m1, accum) = do_term t1 accum
blanchet@35386
   956
          val (m2, accum) = do_formula t2 accum
blanchet@35386
   957
        in
blanchet@35386
   958
          (MApp (MApp (MRaw (t0, mtype_for (fastype_of t0)), m1), m2), accum)
blanchet@35386
   959
        end
blanchet@35812
   960
      and do_formula t accum =
blanchet@33192
   961
          case t of
blanchet@35386
   962
            (t0 as Const (@{const_name all}, _)) $ Abs (s1, T1, t1) =>
blanchet@35386
   963
            do_all t0 s1 T1 t1 accum
blanchet@35665
   964
          | @{const Trueprop} $ t1 =>
blanchet@35665
   965
            let val (m1, accum) = do_formula t1 accum in
blanchet@35665
   966
              (MApp (MRaw (@{const Trueprop}, mtype_for (bool_T --> prop_T)),
blanchet@35665
   967
                     m1), accum)
blanchet@35665
   968
            end
blanchet@35386
   969
          | Const (x as (@{const_name "=="}, _)) $ t1 $ t2 =>
blanchet@35665
   970
            consider_general_equals mdata true x t1 t2 accum
blanchet@35386
   971
          | (t0 as @{const "==>"}) $ t1 $ t2 => do_implies t0 t1 t2 accum
blanchet@35386
   972
          | (t0 as @{const Pure.conjunction}) $ t1 $ t2 =>
blanchet@35386
   973
            do_conjunction t0 t1 t2 accum
blanchet@35386
   974
          | (t0 as Const (@{const_name All}, _)) $ Abs (s0, T1, t1) =>
blanchet@35386
   975
            do_all t0 s0 T1 t1 accum
blanchet@35386
   976
          | Const (x as (@{const_name "op ="}, _)) $ t1 $ t2 =>
blanchet@35665
   977
            consider_general_equals mdata true x t1 t2 accum
blanchet@35386
   978
          | (t0 as @{const "op &"}) $ t1 $ t2 => do_conjunction t0 t1 t2 accum
haftmann@39019
   979
          | (t0 as @{const HOL.implies}) $ t1 $ t2 => do_implies t0 t1 t2 accum
blanchet@33224
   980
          | _ => raise TERM ("Nitpick_Mono.consider_definitional_axiom.\
blanchet@33192
   981
                             \do_formula", [t])
blanchet@33192
   982
    in do_formula t end
blanchet@33192
   983
blanchet@35385
   984
fun string_for_mtype_of_term ctxt lits t M =
blanchet@35665
   985
  Syntax.string_of_term ctxt t ^ " : " ^ string_for_mtype (resolve_mtype lits M)
blanchet@33192
   986
blanchet@35385
   987
fun print_mtype_context ctxt lits ({frees, consts, ...} : mtype_context) =
blanchet@38406
   988
  trace_msg (fn () =>
blanchet@37451
   989
      map (fn (x, M) => string_for_mtype_of_term ctxt lits (Free x) M) frees @
blanchet@37451
   990
      map (fn (x, M) => string_for_mtype_of_term ctxt lits (Const x) M) consts
blanchet@37451
   991
      |> cat_lines)
blanchet@33192
   992
blanchet@35665
   993
fun amass f t (ms, accum) =
blanchet@35386
   994
  let val (m, accum) = f t accum in (m :: ms, accum) end
blanchet@35386
   995
blanchet@35665
   996
fun infer which no_harmless (hol_ctxt as {ctxt, ...}) binarize alpha_T
blanchet@35665
   997
          (nondef_ts, def_ts) =
blanchet@33192
   998
  let
blanchet@38406
   999
    val _ = trace_msg (fn () => "****** " ^ which ^ " analysis: " ^
blanchet@38406
  1000
                                string_for_mtype MAlpha ^ " is " ^
blanchet@38406
  1001
                                Syntax.string_of_typ ctxt alpha_T)
blanchet@35665
  1002
    val mdata as {max_fresh, constr_mcache, ...} =
blanchet@35665
  1003
      initial_mdata hol_ctxt binarize no_harmless alpha_T
blanchet@35812
  1004
    val accum = (initial_gamma, ([], [], []))
blanchet@35386
  1005
    val (nondef_ms, accum) =
blanchet@35665
  1006
      ([], accum) |> amass (consider_general_formula mdata Plus) (hd nondef_ts)
blanchet@35665
  1007
                  |> fold (amass (consider_nondefinitional_axiom mdata))
blanchet@35386
  1008
                          (tl nondef_ts)
blanchet@35386
  1009
    val (def_ms, (gamma, cset)) =
blanchet@35665
  1010
      ([], accum) |> fold (amass (consider_definitional_axiom mdata)) def_ts
blanchet@33192
  1011
  in
blanchet@33192
  1012
    case solve (!max_fresh) cset of
blanchet@35665
  1013
      SOME lits => (print_mtype_context ctxt lits gamma;
blanchet@35665
  1014
                    SOME (lits, (nondef_ms, def_ms), !constr_mcache))
blanchet@35665
  1015
    | _ => NONE
blanchet@33192
  1016
  end
blanchet@35812
  1017
  handle UNSOLVABLE () => NONE
blanchet@35812
  1018
       | MTYPE (loc, Ms, Ts) =>
blanchet@35665
  1019
         raise BAD (loc, commas (map string_for_mtype Ms @
blanchet@35665
  1020
                                 map (Syntax.string_of_typ ctxt) Ts))
blanchet@35665
  1021
       | MTERM (loc, ms) =>
blanchet@35665
  1022
         raise BAD (loc, commas (map (string_for_mterm ctxt) ms))
blanchet@35665
  1023
blanchet@35665
  1024
val formulas_monotonic = is_some oooo infer "Monotonicity" false
blanchet@35665
  1025
blanchet@35665
  1026
fun fin_fun_constr T1 T2 =
blanchet@35665
  1027
  (@{const_name FinFun}, (T1 --> T2) --> Type (@{type_name fin_fun}, [T1, T2]))
blanchet@35665
  1028
blanchet@37255
  1029
fun finitize_funs (hol_ctxt as {thy, ctxt, stds, fast_descrs, constr_cache,
blanchet@37255
  1030
                                ...})
blanchet@35665
  1031
                  binarize finitizes alpha_T tsp =
blanchet@35665
  1032
  case infer "Finiteness" true hol_ctxt binarize alpha_T tsp of
blanchet@35665
  1033
    SOME (lits, msp, constr_mtypes) =>
blanchet@35812
  1034
    if forall (curry (op =) Minus o snd) lits then
blanchet@35812
  1035
      tsp
blanchet@35812
  1036
    else
blanchet@35812
  1037
      let
blanchet@35812
  1038
        fun should_finitize T a =
blanchet@35812
  1039
          case triple_lookup (type_match thy) finitizes T of
blanchet@35812
  1040
            SOME (SOME false) => false
blanchet@35812
  1041
          | _ => resolve_sign_atom lits a = S Plus
blanchet@35812
  1042
        fun type_from_mtype T M =
blanchet@35812
  1043
          case (M, T) of
blanchet@35812
  1044
            (MAlpha, _) => T
blanchet@35812
  1045
          | (MFun (M1, a, M2), Type (@{type_name fun}, Ts)) =>
blanchet@35812
  1046
            Type (if should_finitize T a then @{type_name fin_fun}
blanchet@35812
  1047
                  else @{type_name fun}, map2 type_from_mtype Ts [M1, M2])
blanchet@38417
  1048
          | (MPair (M1, M2), Type (@{type_name prod}, Ts)) =>
blanchet@38417
  1049
            Type (@{type_name prod}, map2 type_from_mtype Ts [M1, M2])
blanchet@35812
  1050
          | (MType _, _) => T
blanchet@35812
  1051
          | _ => raise MTYPE ("Nitpick_Mono.finitize_funs.type_from_mtype",
blanchet@35812
  1052
                              [M], [T])
blanchet@35812
  1053
        fun finitize_constr (x as (s, T)) =
blanchet@35812
  1054
          (s, case AList.lookup (op =) constr_mtypes x of
blanchet@35812
  1055
                SOME M => type_from_mtype T M
blanchet@35812
  1056
              | NONE => T)
blanchet@37266
  1057
        fun term_from_mterm new_Ts old_Ts m =
blanchet@35812
  1058
          case m of
blanchet@35812
  1059
            MRaw (t, M) =>
blanchet@35812
  1060
            let
blanchet@37266
  1061
              val T = fastype_of1 (old_Ts, t)
blanchet@35812
  1062
              val T' = type_from_mtype T M
blanchet@35812
  1063
            in
blanchet@35812
  1064
              case t of
blanchet@35812
  1065
                Const (x as (s, _)) =>
blanchet@37451
  1066
                if s = @{const_name finite} then
blanchet@35812
  1067
                  case domain_type T' of
blanchet@35812
  1068
                    set_T' as Type (@{type_name fin_fun}, _) =>
blanchet@35812
  1069
                    Abs (Name.uu, set_T', @{const True})
blanchet@35812
  1070
                  | _ => Const (s, T')
blanchet@35812
  1071
                else if s = @{const_name "=="} orelse
blanchet@35812
  1072
                        s = @{const_name "op ="} then
blanchet@37451
  1073
                  let
blanchet@37451
  1074
                    val T =
blanchet@37451
  1075
                      case T' of
blanchet@37451
  1076
                        Type (_, [T1, Type (_, [T2, T3])]) =>
blanchet@37451
  1077
                        T1 --> T2 --> T3
blanchet@37451
  1078
                      | _ => raise TYPE ("Nitpick_Mono.finitize_funs.\
blanchet@37451
  1079
                                         \term_from_mterm", [T, T'], [])
blanchet@37451
  1080
                  in coerce_term hol_ctxt new_Ts T' T (Const (s, T)) end
blanchet@35812
  1081
                else if is_built_in_const thy stds fast_descrs x then
blanchet@37266
  1082
                  coerce_term hol_ctxt new_Ts T' T t
blanchet@37255
  1083
                else if is_constr ctxt stds x then
blanchet@35812
  1084
                  Const (finitize_constr x)
blanchet@35812
  1085
                else if is_sel s then
blanchet@35812
  1086
                  let
blanchet@35812
  1087
                    val n = sel_no_from_name s
blanchet@35812
  1088
                    val x' =
blanchet@35812
  1089
                      x |> binarized_and_boxed_constr_for_sel hol_ctxt binarize
blanchet@35812
  1090
                        |> finitize_constr
blanchet@35812
  1091
                    val x'' =
blanchet@35812
  1092
                      binarized_and_boxed_nth_sel_for_constr hol_ctxt binarize
blanchet@35812
  1093
                                                             x' n
blanchet@35812
  1094
                  in Const x'' end
blanchet@35812
  1095
                else
blanchet@35812
  1096
                  Const (s, T')
blanchet@35812
  1097
              | Free (s, T) => Free (s, type_from_mtype T M)
blanchet@35812
  1098
              | Bound _ => t
blanchet@35812
  1099
              | _ => raise MTERM ("Nitpick_Mono.finitize_funs.term_from_mterm",
blanchet@35812
  1100
                                  [m])
blanchet@35812
  1101
            end
blanchet@35812
  1102
          | MApp (m1, m2) =>
blanchet@35812
  1103
            let
blanchet@37266
  1104
              val (t1, t2) = pairself (term_from_mterm new_Ts old_Ts) (m1, m2)
blanchet@37266
  1105
              val (T1, T2) = pairself (curry fastype_of1 new_Ts) (t1, t2)
blanchet@35812
  1106
              val (t1', T2') =
blanchet@35812
  1107
                case T1 of
blanchet@35812
  1108
                  Type (s, [T11, T12]) => 
blanchet@35812
  1109
                  (if s = @{type_name fin_fun} then
blanchet@37255
  1110
                     select_nth_constr_arg ctxt stds (fin_fun_constr T11 T12) t1
blanchet@35812
  1111
                                           0 (T11 --> T12)
blanchet@35812
  1112
                   else
blanchet@35812
  1113
                     t1, T11)
blanchet@35812
  1114
                | _ => raise TYPE ("Nitpick_Mono.finitize_funs.term_from_mterm",
blanchet@35812
  1115
                                   [T1], [])
blanchet@37266
  1116
            in betapply (t1', coerce_term hol_ctxt new_Ts T2' T2 t2) end
blanchet@37266
  1117
          | MAbs (s, old_T, M, a, m') =>
blanchet@35812
  1118
            let
blanchet@37266
  1119
              val new_T = type_from_mtype old_T M
blanchet@37266
  1120
              val t' = term_from_mterm (new_T :: new_Ts) (old_T :: old_Ts) m'
blanchet@37266
  1121
              val T' = fastype_of1 (new_T :: new_Ts, t')
blanchet@35812
  1122
            in
blanchet@37266
  1123
              Abs (s, new_T, t')
blanchet@37266
  1124
              |> should_finitize (new_T --> T') a
blanchet@37266
  1125
                 ? construct_value ctxt stds (fin_fun_constr new_T T') o single
blanchet@35812
  1126
            end
blanchet@35812
  1127
      in
blanchet@35812
  1128
        Unsynchronized.change constr_cache (map (apsnd (map finitize_constr)));
blanchet@37266
  1129
        pairself (map (term_from_mterm [] [])) msp
blanchet@35812
  1130
      end
blanchet@35665
  1131
  | NONE => tsp
blanchet@33192
  1132
blanchet@33192
  1133
end;