src/HOL/typedef.ML
author oheimb
Tue, 04 Nov 1997 20:48:38 +0100
changeset 4133 0a08c2b9b1ed
parent 4028 01745d56307d
child 4409 2af86fcb97d7
permissions -rw-r--r--
added the, option_map, and case analysis theorems
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
1475
7f5a4cd08209 expanded tabs; renamed subtype to typedef;
clasohm
parents: 1264
diff changeset
     1
(*  Title:      HOL/typedef.ML
923
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
     2
    ID:         $Id$
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
     3
    Author:     Markus Wenzel, TU Muenchen
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
     4
2851
b6a5780e36b9 improved messages;
wenzelm
parents: 2238
diff changeset
     5
Internal interface for typedefs.
923
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
     6
*)
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
     7
1475
7f5a4cd08209 expanded tabs; renamed subtype to typedef;
clasohm
parents: 1264
diff changeset
     8
signature TYPEDEF =
923
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
     9
sig
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    10
  val prove_nonempty: cterm -> thm list -> tactic option -> thm
3955
9666a1ecf3a1 tuned sig;
wenzelm
parents: 3946
diff changeset
    11
  val add_typedef: string -> bstring * string list * mixfix ->
923
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    12
    string -> string list -> thm list -> tactic option -> theory -> theory
3955
9666a1ecf3a1 tuned sig;
wenzelm
parents: 3946
diff changeset
    13
  val add_typedef_i: string -> bstring * string list * mixfix ->
923
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    14
    term -> string list -> thm list -> tactic option -> theory -> theory
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    15
end;
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    16
1475
7f5a4cd08209 expanded tabs; renamed subtype to typedef;
clasohm
parents: 1264
diff changeset
    17
structure Typedef: TYPEDEF =
923
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    18
struct
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    19
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    20
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    21
(* prove non-emptyness of a set *)   (*exception ERROR*)
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    22
3946
wenzelm
parents: 3793
diff changeset
    23
val is_def = Logic.is_equals o #prop o rep_thm;
923
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    24
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    25
fun prove_nonempty cset thms usr_tac =
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    26
  let
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    27
    val {T = setT, t = set, maxidx, sign} = rep_cterm cset;
3946
wenzelm
parents: 3793
diff changeset
    28
    val T = HOLogic.dest_setT setT;
wenzelm
parents: 3793
diff changeset
    29
    val goal = cterm_of sign
wenzelm
parents: 3793
diff changeset
    30
      (HOLogic.mk_Trueprop (HOLogic.mk_mem (Var (("x", maxidx + 1), T), set)));
923
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    31
    val tac =
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    32
      TRY (rewrite_goals_tac (filter is_def thms)) THEN
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    33
      TRY (REPEAT_FIRST (resolve_tac (filter_out is_def thms))) THEN
2928
c0e3f1ceabf2 Added trace output and replaced fast_tac set_cs by Fast_tac.
nipkow
parents: 2851
diff changeset
    34
      if_none usr_tac (TRY (ALLGOALS Fast_tac));
923
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    35
  in
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    36
    prove_goalw_cterm [] goal (K [tac])
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    37
  end
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    38
  handle ERROR =>
2934
bd922fc9001b tuned error msg;
wenzelm
parents: 2928
diff changeset
    39
    error ("Failed to prove nonemptiness of " ^ quote (string_of_cterm cset));
923
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    40
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    41
1475
7f5a4cd08209 expanded tabs; renamed subtype to typedef;
clasohm
parents: 1264
diff changeset
    42
(* ext_typedef *)
923
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    43
1475
7f5a4cd08209 expanded tabs; renamed subtype to typedef;
clasohm
parents: 1264
diff changeset
    44
fun ext_typedef prep_term name (t, vs, mx) raw_set axms thms usr_tac thy =
923
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    45
  let
3946
wenzelm
parents: 3793
diff changeset
    46
    val _ = require_thy thy "Set" "typedefs";
923
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    47
    val sign = sign_of thy;
3946
wenzelm
parents: 3793
diff changeset
    48
    val full_name = Sign.full_name sign;
923
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    49
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    50
    (*rhs*)
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    51
    val cset = prep_term sign raw_set;
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    52
    val {T = setT, t = set, ...} = rep_cterm cset;
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    53
    val rhs_tfrees = term_tfrees set;
3946
wenzelm
parents: 3793
diff changeset
    54
    val oldT = HOLogic.dest_setT setT handle TYPE _ =>
923
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    55
      error ("Not a set type: " ^ quote (Sign.string_of_typ sign setT));
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    56
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    57
    (*lhs*)
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    58
    val lhs_tfrees =
3946
wenzelm
parents: 3793
diff changeset
    59
      map (fn v => (v, if_none (assoc (rhs_tfrees, v)) HOLogic.termS)) vs;
923
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    60
3946
wenzelm
parents: 3793
diff changeset
    61
    val tname = Syntax.type_name t mx;
923
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    62
    val tlen = length vs;
3946
wenzelm
parents: 3793
diff changeset
    63
    val newT = Type (full_name tname, map TFree lhs_tfrees);
923
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    64
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    65
    val Rep_name = "Rep_" ^ name;
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    66
    val Abs_name = "Abs_" ^ name;
3946
wenzelm
parents: 3793
diff changeset
    67
    val setC = Const (full_name name, setT);
wenzelm
parents: 3793
diff changeset
    68
    val RepC = Const (full_name Rep_name, newT --> oldT);
wenzelm
parents: 3793
diff changeset
    69
    val AbsC = Const (full_name Abs_name, oldT --> newT);
923
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    70
    val x_new = Free ("x", newT);
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    71
    val y_old = Free ("y", oldT);
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    72
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    73
    (*axioms*)
3946
wenzelm
parents: 3793
diff changeset
    74
    val rep_type = HOLogic.mk_Trueprop (HOLogic.mk_mem (RepC $ x_new, setC));
wenzelm
parents: 3793
diff changeset
    75
    val rep_type_inv = HOLogic.mk_Trueprop (HOLogic.mk_eq (AbsC $ (RepC $ x_new), x_new));
wenzelm
parents: 3793
diff changeset
    76
    val abs_type_inv = Logic.mk_implies (HOLogic.mk_Trueprop (HOLogic.mk_mem (y_old, setC)),
wenzelm
parents: 3793
diff changeset
    77
      HOLogic.mk_Trueprop (HOLogic.mk_eq (RepC $ (AbsC $ y_old), y_old)));
923
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    78
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    79
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    80
    (* errors *)
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    81
2238
c72a23bbe762 Eta-expanded some declarations that are illegal under value polymorphism
paulson
parents: 1475
diff changeset
    82
    fun show_names pairs = commas_quote (map fst pairs);
923
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    83
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    84
    val illegal_vars =
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    85
      if null (term_vars set) andalso null (term_tvars set) then []
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    86
      else ["Illegal schematic variable(s) on rhs"];
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    87
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    88
    val dup_lhs_tfrees =
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    89
      (case duplicates lhs_tfrees of [] => []
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    90
      | dups => ["Duplicate type variables on lhs: " ^ show_names dups]);
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    91
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    92
    val extra_rhs_tfrees =
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    93
      (case gen_rems (op =) (rhs_tfrees, lhs_tfrees) of [] => []
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    94
      | extras => ["Extra type variables on rhs: " ^ show_names extras]);
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    95
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    96
    val illegal_frees =
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    97
      (case term_frees set of [] => []
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    98
      | xs => ["Illegal variables on rhs: " ^ show_names (map dest_Free xs)]);
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    99
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
   100
    val errs = illegal_vars @ dup_lhs_tfrees @ extra_rhs_tfrees @ illegal_frees;
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
   101
  in
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
   102
    if null errs then ()
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
   103
    else error (cat_lines errs);
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
   104
2928
c0e3f1ceabf2 Added trace output and replaced fast_tac set_cs by Fast_tac.
nipkow
parents: 2851
diff changeset
   105
    writeln("Proving nonemptiness of " ^ quote name ^ " ...");
923
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
   106
    prove_nonempty cset (map (get_axiom thy) axms @ thms) usr_tac;
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
   107
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
   108
    thy
3768
67f4ac759100 fully qualified names: Theory.add_XXX;
wenzelm
parents: 2934
diff changeset
   109
    |> Theory.add_types [(t, tlen, mx)]
3793
6e807b50b6c1 add_arities_i;
wenzelm
parents: 3768
diff changeset
   110
    |> Theory.add_arities_i
3946
wenzelm
parents: 3793
diff changeset
   111
     [(full_name tname, replicate tlen logicS, logicS),
wenzelm
parents: 3793
diff changeset
   112
      (full_name tname, replicate tlen HOLogic.termS, HOLogic.termS)]
3768
67f4ac759100 fully qualified names: Theory.add_XXX;
wenzelm
parents: 2934
diff changeset
   113
    |> Theory.add_consts_i
923
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
   114
     [(name, setT, NoSyn),
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
   115
      (Rep_name, newT --> oldT, NoSyn),
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
   116
      (Abs_name, oldT --> newT, NoSyn)]
4028
01745d56307d PureThy.add_store_defs_i, PureThy.add_store_axioms_i;
wenzelm
parents: 3955
diff changeset
   117
    |> PureThy.add_store_defs_i
3946
wenzelm
parents: 3793
diff changeset
   118
     [(name ^ "_def", Logic.mk_equals (setC, set))]
4028
01745d56307d PureThy.add_store_defs_i, PureThy.add_store_axioms_i;
wenzelm
parents: 3955
diff changeset
   119
    |> PureThy.add_store_axioms_i
923
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
   120
     [(Rep_name, rep_type),
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
   121
      (Rep_name ^ "_inverse", rep_type_inv),
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
   122
      (Abs_name ^ "_inverse", abs_type_inv)]
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
   123
  end
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
   124
  handle ERROR =>
2851
b6a5780e36b9 improved messages;
wenzelm
parents: 2238
diff changeset
   125
    error ("The error(s) above occurred in typedef " ^ quote name);
923
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
   126
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
   127
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
   128
(* external interfaces *)
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
   129
3955
9666a1ecf3a1 tuned sig;
wenzelm
parents: 3946
diff changeset
   130
fun read_term sg str =
9666a1ecf3a1 tuned sig;
wenzelm
parents: 3946
diff changeset
   131
  read_cterm sg (str, HOLogic.termTVar);
9666a1ecf3a1 tuned sig;
wenzelm
parents: 3946
diff changeset
   132
923
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
   133
fun cert_term sg tm =
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
   134
  cterm_of sg tm handle TERM (msg, _) => error msg;
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
   135
1475
7f5a4cd08209 expanded tabs; renamed subtype to typedef;
clasohm
parents: 1264
diff changeset
   136
val add_typedef = ext_typedef read_term;
7f5a4cd08209 expanded tabs; renamed subtype to typedef;
clasohm
parents: 1264
diff changeset
   137
val add_typedef_i = ext_typedef cert_term;
923
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
   138
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
   139
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
   140
end;