src/HOLCF/Tools/fixrec_package.ML
author huffman
Fri, 27 Feb 2009 18:34:20 -0800
changeset 30157 40919ebde2c9
parent 30132 243a05a67c41
child 30158 83c50c62cf23
permissions -rw-r--r--
add function taken_names
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
23152
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
     1
(*  Title:      HOLCF/Tools/fixrec_package.ML
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
     2
    Author:     Amber Telfer and Brian Huffman
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
     3
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
     4
Recursive function definition package for HOLCF.
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
     5
*)
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
     6
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
     7
signature FIXREC_PACKAGE =
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
     8
sig
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
     9
  val legacy_infer_term: theory -> term -> term
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
    10
  val legacy_infer_prop: theory -> term -> term
30132
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
    11
28084
a05ca48ef263 type Attrib.binding abbreviates Name.binding without attributes;
wenzelm
parents: 28083
diff changeset
    12
  val add_fixrec: bool -> (Attrib.binding * string) list list -> theory -> theory
29581
b3b33e0298eb binding is alias for Binding.T
haftmann
parents: 29006
diff changeset
    13
  val add_fixrec_i: bool -> ((binding * attribute list) * term) list list -> theory -> theory
28084
a05ca48ef263 type Attrib.binding abbreviates Name.binding without attributes;
wenzelm
parents: 28083
diff changeset
    14
  val add_fixpat: Attrib.binding * string list -> theory -> theory
29581
b3b33e0298eb binding is alias for Binding.T
haftmann
parents: 29006
diff changeset
    15
  val add_fixpat_i: (binding * attribute list) * term list -> theory -> theory
30131
6be1be402ef0 use TheoryData to keep track of pattern match combinators
huffman
parents: 29585
diff changeset
    16
  val add_matchers: (string * string) list -> theory -> theory
6be1be402ef0 use TheoryData to keep track of pattern match combinators
huffman
parents: 29585
diff changeset
    17
  val setup: theory -> theory
23152
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
    18
end;
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
    19
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
    20
structure FixrecPackage: FIXREC_PACKAGE =
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
    21
struct
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
    22
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
    23
(* legacy type inference *)
30132
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
    24
(* used by the domain package *)
23152
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
    25
fun legacy_infer_term thy t =
24493
d4380e9b287b replaced ProofContext.infer_types by general Syntax.check_terms;
wenzelm
parents: 23779
diff changeset
    26
  singleton (Syntax.check_terms (ProofContext.init thy)) (Sign.intern_term thy t);
23152
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
    27
24680
0d355aa59e67 TypeInfer.constrain: canonical argument order;
wenzelm
parents: 24493
diff changeset
    28
fun legacy_infer_prop thy t = legacy_infer_term thy (TypeInfer.constrain propT t);
23152
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
    29
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
    30
26045
02aa3f166c7f use ML antiquotations
huffman
parents: 25557
diff changeset
    31
val fix_eq2 = @{thm fix_eq2};
02aa3f166c7f use ML antiquotations
huffman
parents: 25557
diff changeset
    32
val def_fix_ind = @{thm def_fix_ind};
23152
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
    33
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
    34
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
    35
fun fixrec_err s = error ("fixrec definition error:\n" ^ s);
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
    36
fun fixrec_eq_err thy s eq =
26939
1035c89b4c02 moved global pretty/string_of functions from Sign to Syntax;
wenzelm
parents: 26343
diff changeset
    37
  fixrec_err (s ^ "\nin\n" ^ quote (Syntax.string_of_term_global thy eq));
23152
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
    38
30132
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
    39
(*************************************************************************)
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
    40
(***************************** building types ****************************)
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
    41
(*************************************************************************)
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
    42
23152
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
    43
(* ->> is taken from holcf_logic.ML *)
30132
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
    44
fun cfunT (T, U) = Type(@{type_name "->"}, [T, U]);
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
    45
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
    46
infixr 6 ->>; val (op ->>) = cfunT;
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
    47
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
    48
fun dest_cfunT (Type(@{type_name "->"}, [T, U])) = (T, U)
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
    49
  | dest_cfunT T = raise TYPE ("dest_cfunT", [T], []);
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
    50
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
    51
fun binder_cfun (Type(@{type_name "->"},[T, U])) = T :: binder_cfun U
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
    52
  | binder_cfun _   =  [];
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
    53
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
    54
fun body_cfun (Type(@{type_name "->"},[T, U])) = body_cfun U
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
    55
  | body_cfun T   =  T;
23152
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
    56
30132
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
    57
fun strip_cfun T : typ list * typ =
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
    58
  (binder_cfun T, body_cfun T);
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
    59
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
    60
fun maybeT T = Type(@{type_name "maybe"}, [T]);
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
    61
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
    62
fun dest_maybeT (Type(@{type_name "maybe"}, [T])) = T
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
    63
  | dest_maybeT T = raise TYPE ("dest_maybeT", [T], []);
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
    64
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
    65
fun tupleT [] = @{typ "unit"}
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
    66
  | tupleT [T] = T
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
    67
  | tupleT (T :: Ts) = HOLogic.mk_prodT (T, tupleT Ts);
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
    68
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
    69
fun matchT T = body_cfun T ->> maybeT (tupleT (binder_cfun T));
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
    70
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
    71
(*************************************************************************)
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
    72
(***************************** building terms ****************************)
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
    73
(*************************************************************************)
23152
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
    74
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
    75
val mk_trp = HOLogic.mk_Trueprop;
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
    76
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
    77
(* splits a cterm into the right and lefthand sides of equality *)
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
    78
fun dest_eqs t = HOLogic.dest_eq (HOLogic.dest_Trueprop t);
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
    79
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
    80
(* similar to Thm.head_of, but for continuous application *)
26045
02aa3f166c7f use ML antiquotations
huffman
parents: 25557
diff changeset
    81
fun chead_of (Const(@{const_name Rep_CFun},_)$f$t) = chead_of f
23152
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
    82
  | chead_of u = u;
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
    83
30132
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
    84
fun capply_const (S, T) =
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
    85
  Const(@{const_name Rep_CFun}, (S ->> T) --> (S --> T));
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
    86
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
    87
fun cabs_const (S, T) =
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
    88
  Const(@{const_name Abs_CFun}, (S --> T) --> (S ->> T));
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
    89
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
    90
fun mk_capply (t, u) =
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
    91
  let val (S, T) =
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
    92
    case Term.fastype_of t of
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
    93
        Type(@{type_name "->"}, [S, T]) => (S, T)
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
    94
      | _ => raise TERM ("mk_capply " ^ ML_Syntax.print_list ML_Syntax.print_term [t, u], [t, u]);
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
    95
  in capply_const (S, T) $ t $ u end;
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
    96
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
    97
infix 0 ==;  val (op ==) = Logic.mk_equals;
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
    98
infix 1 ===; val (op ===) = HOLogic.mk_eq;
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
    99
infix 9 `  ; val (op `) = mk_capply;
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
   100
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
   101
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
   102
fun mk_cpair (t, u) =
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
   103
  let val T = Term.fastype_of t
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
   104
      val U = Term.fastype_of u
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
   105
      val cpairT = T ->> U ->> HOLogic.mk_prodT (T, U)
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
   106
  in Const(@{const_name cpair}, cpairT) ` t ` u end;
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
   107
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
   108
fun mk_cfst t =
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
   109
  let val T = Term.fastype_of t;
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
   110
      val (U, _) = HOLogic.dest_prodT T;
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
   111
  in Const(@{const_name cfst}, T ->> U) ` t end;
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
   112
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
   113
fun mk_csnd t =
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
   114
  let val T = Term.fastype_of t;
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
   115
      val (_, U) = HOLogic.dest_prodT T;
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
   116
  in Const(@{const_name csnd}, T ->> U) ` t end;
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
   117
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
   118
fun mk_csplit t =
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
   119
  let val (S, TU) = dest_cfunT (Term.fastype_of t);
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
   120
      val (T, U) = dest_cfunT TU;
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
   121
      val csplitT = (S ->> T ->> U) ->> HOLogic.mk_prodT (S, T) ->> U;
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
   122
  in Const(@{const_name csplit}, csplitT) ` t end;
23152
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   123
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   124
(* builds the expression (LAM v. rhs) *)
30132
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
   125
fun big_lambda v rhs =
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
   126
  cabs_const (Term.fastype_of v, Term.fastype_of rhs) $ Term.lambda v rhs;
23152
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   127
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   128
(* builds the expression (LAM v1 v2 .. vn. rhs) *)
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   129
fun big_lambdas [] rhs = rhs
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   130
  | big_lambdas (v::vs) rhs = big_lambda v (big_lambdas vs rhs);
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   131
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   132
(* builds the expression (LAM <v1,v2,..,vn>. rhs) *)
30132
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
   133
fun lambda_ctuple [] rhs = big_lambda (Free("unit", HOLogic.unitT)) rhs
23152
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   134
  | lambda_ctuple (v::[]) rhs = big_lambda v rhs
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   135
  | lambda_ctuple (v::vs) rhs =
30132
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
   136
      mk_csplit (big_lambda v (lambda_ctuple vs rhs));
23152
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   137
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   138
(* builds the expression <v1,v2,..,vn> *)
30132
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
   139
fun mk_ctuple [] = @{term "UU::unit"}
23152
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   140
|   mk_ctuple (t::[]) = t
30132
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
   141
|   mk_ctuple (t::ts) = mk_cpair (t, mk_ctuple ts);
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
   142
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
   143
fun mk_return t =
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
   144
  let val T = Term.fastype_of t
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
   145
  in Const(@{const_name Fixrec.return}, T ->> maybeT T) ` t end;
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
   146
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
   147
fun mk_bind (t, u) =
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
   148
  let val (T, mU) = dest_cfunT (Term.fastype_of u);
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
   149
      val bindT = maybeT T ->> (T ->> mU) ->> mU;
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
   150
  in Const(@{const_name Fixrec.bind}, bindT) ` t ` u end;
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
   151
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
   152
fun mk_mplus (t, u) =
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
   153
  let val mT = Term.fastype_of t
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
   154
  in Const(@{const_name Fixrec.mplus}, mT ->> mT ->> mT) ` t ` u end;
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
   155
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
   156
fun mk_run t =
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
   157
  let val mT = Term.fastype_of t
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
   158
      val T = dest_maybeT mT
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
   159
  in Const(@{const_name Fixrec.run}, mT ->> T) ` t end;
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
   160
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
   161
fun mk_fix t =
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
   162
  let val (T, _) = dest_cfunT (Term.fastype_of t)
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
   163
  in Const(@{const_name fix}, (T ->> T) ->> T) ` t end;
23152
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   164
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   165
(*************************************************************************)
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   166
(************* fixed-point definitions and unfolding theorems ************)
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   167
(*************************************************************************)
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   168
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   169
fun add_fixdefs eqs thy =
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   170
  let
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   171
    val (lhss,rhss) = ListPair.unzip (map dest_eqs eqs);
30132
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
   172
    val fixpoint = mk_fix (lambda_ctuple lhss (mk_ctuple rhss));
23152
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   173
    
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   174
    fun one_def (l as Const(n,T)) r =
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   175
          let val b = Sign.base_name n in (b, (b^"_def", l == r)) end
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   176
      | one_def _ _ = fixrec_err "fixdefs: lhs not of correct form";
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   177
    fun defs [] _ = []
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   178
      | defs (l::[]) r = [one_def l r]
30132
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
   179
      | defs (l::ls) r = one_def l (mk_cfst r) :: defs ls (mk_csnd r);
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
   180
    val (names, fixdefs) = ListPair.unzip (defs lhss fixpoint);
23152
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   181
    
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   182
    val (fixdef_thms, thy') =
29585
c23295521af5 binding replaces bstring
haftmann
parents: 29581
diff changeset
   183
      PureThy.add_defs false (map (Thm.no_attributes o apfst Binding.name) fixdefs) thy;
25132
dffe405b090d removed obsolete ML bindings;
wenzelm
parents: 24867
diff changeset
   184
    val ctuple_fixdef_thm = foldr1 (fn (x,y) => @{thm cpair_equalI} OF [x,y]) fixdef_thms;
23152
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   185
    
30132
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
   186
    val ctuple_unfold = mk_trp (mk_ctuple lhss === mk_ctuple rhss);
23152
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   187
    val ctuple_unfold_thm = Goal.prove_global thy' [] [] ctuple_unfold
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   188
          (fn _ => EVERY [rtac (ctuple_fixdef_thm RS fix_eq2 RS trans) 1,
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   189
                    simp_tac (simpset_of thy') 1]);
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   190
    val ctuple_induct_thm =
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   191
          (space_implode "_" names ^ "_induct", ctuple_fixdef_thm RS def_fix_ind);
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   192
    
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   193
    fun unfolds [] thm = []
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   194
      | unfolds (n::[]) thm = [(n^"_unfold", thm)]
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   195
      | unfolds (n::ns) thm = let
25132
dffe405b090d removed obsolete ML bindings;
wenzelm
parents: 24867
diff changeset
   196
          val thmL = thm RS @{thm cpair_eqD1};
dffe405b090d removed obsolete ML bindings;
wenzelm
parents: 24867
diff changeset
   197
          val thmR = thm RS @{thm cpair_eqD2};
23152
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   198
        in (n^"_unfold", thmL) :: unfolds ns thmR end;
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   199
    val unfold_thms = unfolds names ctuple_unfold_thm;
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   200
    val thms = ctuple_induct_thm :: unfold_thms;
29585
c23295521af5 binding replaces bstring
haftmann
parents: 29581
diff changeset
   201
    val (_, thy'') = PureThy.add_thms (map (Thm.no_attributes o apfst Binding.name) thms) thy';
23152
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   202
  in
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   203
    (thy'', names, fixdef_thms, map snd unfold_thms)
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   204
  end;
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   205
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   206
(*************************************************************************)
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   207
(*********** monadic notation and pattern matching compilation ***********)
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   208
(*************************************************************************)
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   209
30131
6be1be402ef0 use TheoryData to keep track of pattern match combinators
huffman
parents: 29585
diff changeset
   210
structure FixrecMatchData = TheoryDataFun (
6be1be402ef0 use TheoryData to keep track of pattern match combinators
huffman
parents: 29585
diff changeset
   211
  type T = string Symtab.table;
6be1be402ef0 use TheoryData to keep track of pattern match combinators
huffman
parents: 29585
diff changeset
   212
  val empty = Symtab.empty;
6be1be402ef0 use TheoryData to keep track of pattern match combinators
huffman
parents: 29585
diff changeset
   213
  val copy = I;
6be1be402ef0 use TheoryData to keep track of pattern match combinators
huffman
parents: 29585
diff changeset
   214
  val extend = I;
6be1be402ef0 use TheoryData to keep track of pattern match combinators
huffman
parents: 29585
diff changeset
   215
  fun merge _ tabs : T = Symtab.merge (K true) tabs;
6be1be402ef0 use TheoryData to keep track of pattern match combinators
huffman
parents: 29585
diff changeset
   216
);
6be1be402ef0 use TheoryData to keep track of pattern match combinators
huffman
parents: 29585
diff changeset
   217
6be1be402ef0 use TheoryData to keep track of pattern match combinators
huffman
parents: 29585
diff changeset
   218
(* associate match functions with pattern constants *)
6be1be402ef0 use TheoryData to keep track of pattern match combinators
huffman
parents: 29585
diff changeset
   219
fun add_matchers ms = FixrecMatchData.map (fold Symtab.update ms);
6be1be402ef0 use TheoryData to keep track of pattern match combinators
huffman
parents: 29585
diff changeset
   220
30157
40919ebde2c9 add function taken_names
huffman
parents: 30132
diff changeset
   221
fun taken_names (t : term) : bstring list =
40919ebde2c9 add function taken_names
huffman
parents: 30132
diff changeset
   222
  let
40919ebde2c9 add function taken_names
huffman
parents: 30132
diff changeset
   223
    fun taken (Const(a,_), bs) = insert (op =) (Sign.base_name a) bs
40919ebde2c9 add function taken_names
huffman
parents: 30132
diff changeset
   224
      | taken (Free(a,_) , bs) = insert (op =) a bs
40919ebde2c9 add function taken_names
huffman
parents: 30132
diff changeset
   225
      | taken (f $ u     , bs) = taken (f, taken (u, bs))
40919ebde2c9 add function taken_names
huffman
parents: 30132
diff changeset
   226
      | taken (Abs(a,_,t), bs) = taken (t, insert (op =) a bs)
40919ebde2c9 add function taken_names
huffman
parents: 30132
diff changeset
   227
      | taken (_         , bs) = bs;
40919ebde2c9 add function taken_names
huffman
parents: 30132
diff changeset
   228
  in
40919ebde2c9 add function taken_names
huffman
parents: 30132
diff changeset
   229
    taken (t, [])
40919ebde2c9 add function taken_names
huffman
parents: 30132
diff changeset
   230
  end;
23152
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   231
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   232
(* builds a monadic term for matching a constructor pattern *)
30131
6be1be402ef0 use TheoryData to keep track of pattern match combinators
huffman
parents: 29585
diff changeset
   233
fun pre_build match_name pat rhs vs taken =
23152
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   234
  case pat of
26045
02aa3f166c7f use ML antiquotations
huffman
parents: 25557
diff changeset
   235
    Const(@{const_name Rep_CFun},_)$f$(v as Free(n,T)) =>
30131
6be1be402ef0 use TheoryData to keep track of pattern match combinators
huffman
parents: 29585
diff changeset
   236
      pre_build match_name f rhs (v::vs) taken
26045
02aa3f166c7f use ML antiquotations
huffman
parents: 25557
diff changeset
   237
  | Const(@{const_name Rep_CFun},_)$f$x =>
30131
6be1be402ef0 use TheoryData to keep track of pattern match combinators
huffman
parents: 29585
diff changeset
   238
      let val (rhs', v, taken') = pre_build match_name x rhs [] taken;
6be1be402ef0 use TheoryData to keep track of pattern match combinators
huffman
parents: 29585
diff changeset
   239
      in pre_build match_name f rhs' (v::vs) taken' end
23152
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   240
  | Const(c,T) =>
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   241
      let
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   242
        val n = Name.variant taken "v";
26045
02aa3f166c7f use ML antiquotations
huffman
parents: 25557
diff changeset
   243
        fun result_type (Type(@{type_name "->"},[_,T])) (x::xs) = result_type T xs
23152
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   244
          | result_type T _ = T;
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   245
        val v = Free(n, result_type T vs);
30132
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
   246
        val m = Const(match_name c, matchT T);
23152
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   247
        val k = lambda_ctuple vs rhs;
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   248
      in
30132
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
   249
        (mk_bind (m`v, k), v, n::taken)
23152
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   250
      end
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   251
  | Free(n,_) => fixrec_err ("expected constructor, found free variable " ^ quote n)
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   252
  | _ => fixrec_err "pre_build: invalid pattern";
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   253
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   254
(* builds a monadic term for matching a function definition pattern *)
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   255
(* returns (name, arity, matcher) *)
30131
6be1be402ef0 use TheoryData to keep track of pattern match combinators
huffman
parents: 29585
diff changeset
   256
fun building match_name pat rhs vs taken =
23152
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   257
  case pat of
26045
02aa3f166c7f use ML antiquotations
huffman
parents: 25557
diff changeset
   258
    Const(@{const_name Rep_CFun}, _)$f$(v as Free(n,T)) =>
30131
6be1be402ef0 use TheoryData to keep track of pattern match combinators
huffman
parents: 29585
diff changeset
   259
      building match_name f rhs (v::vs) taken
26045
02aa3f166c7f use ML antiquotations
huffman
parents: 25557
diff changeset
   260
  | Const(@{const_name Rep_CFun}, _)$f$x =>
30131
6be1be402ef0 use TheoryData to keep track of pattern match combinators
huffman
parents: 29585
diff changeset
   261
      let val (rhs', v, taken') = pre_build match_name x rhs [] taken;
6be1be402ef0 use TheoryData to keep track of pattern match combinators
huffman
parents: 29585
diff changeset
   262
      in building match_name f rhs' (v::vs) taken' end
30132
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
   263
  | Const(name,_) => (pat, length vs, big_lambdas vs rhs)
23152
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   264
  | _ => fixrec_err "function is not declared as constant in theory";
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   265
30131
6be1be402ef0 use TheoryData to keep track of pattern match combinators
huffman
parents: 29585
diff changeset
   266
fun match_eq match_name eq = 
23152
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   267
  let val (lhs,rhs) = dest_eqs eq;
30131
6be1be402ef0 use TheoryData to keep track of pattern match combinators
huffman
parents: 29585
diff changeset
   268
  in
30157
40919ebde2c9 add function taken_names
huffman
parents: 30132
diff changeset
   269
    building match_name lhs (mk_return rhs) [] (taken_names eq)
30131
6be1be402ef0 use TheoryData to keep track of pattern match combinators
huffman
parents: 29585
diff changeset
   270
  end;
23152
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   271
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   272
(* returns the sum (using +++) of the terms in ms *)
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   273
(* also applies "run" to the result! *)
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   274
fun fatbar arity ms =
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   275
  let
30132
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
   276
    fun LAM_Ts 0 t = ([], Term.fastype_of t)
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
   277
      | LAM_Ts n (_ $ Abs(_,T,t)) =
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
   278
          let val (Ts, U) = LAM_Ts (n-1) t in (T::Ts, U) end
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
   279
      | LAM_Ts _ _ = fixrec_err "fatbar: internal error, not enough LAMs";
23152
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   280
    fun unLAM 0 t = t
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   281
      | unLAM n (_$Abs(_,_,t)) = unLAM (n-1) t
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   282
      | unLAM _ _ = fixrec_err "fatbar: internal error, not enough LAMs";
30132
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
   283
    fun reLAM ([], U) t = t
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
   284
      | reLAM (T::Ts, U) t = reLAM (Ts, T ->> U) (cabs_const(T,U)$Abs("",T,t));
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
   285
    val msum = foldr1 mk_mplus (map (unLAM arity) ms);
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
   286
    val (Ts, U) = LAM_Ts arity (hd ms)
23152
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   287
  in
30132
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
   288
    reLAM (rev Ts, dest_maybeT U) (mk_run msum)
23152
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   289
  end;
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   290
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   291
fun unzip3 [] = ([],[],[])
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   292
  | unzip3 ((x,y,z)::ts) =
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   293
      let val (xs,ys,zs) = unzip3 ts
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   294
      in (x::xs, y::ys, z::zs) end;
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   295
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   296
(* this is the pattern-matching compiler function *)
30131
6be1be402ef0 use TheoryData to keep track of pattern match combinators
huffman
parents: 29585
diff changeset
   297
fun compile_pats match_name eqs = 
23152
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   298
  let
30131
6be1be402ef0 use TheoryData to keep track of pattern match combinators
huffman
parents: 29585
diff changeset
   299
    val ((n::names),(a::arities),mats) = unzip3 (map (match_eq match_name) eqs);
23152
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   300
    val cname = if forall (fn x => n=x) names then n
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   301
          else fixrec_err "all equations in block must define the same function";
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   302
    val arity = if forall (fn x => a=x) arities then a
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   303
          else fixrec_err "all equations in block must have the same arity";
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   304
    val rhs = fatbar arity mats;
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   305
  in
30132
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
   306
    mk_trp (cname === rhs)
23152
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   307
  end;
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   308
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   309
(*************************************************************************)
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   310
(********************** Proving associated theorems **********************)
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   311
(*************************************************************************)
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   312
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   313
(* proves a block of pattern matching equations as theorems, using unfold *)
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   314
fun make_simps thy (unfold_thm, eqns) =
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   315
  let
25132
dffe405b090d removed obsolete ML bindings;
wenzelm
parents: 24867
diff changeset
   316
    val tacs = [rtac (unfold_thm RS @{thm ssubst_lhs}) 1, asm_simp_tac (simpset_of thy) 1];
23152
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   317
    fun prove_term t = Goal.prove_global thy [] [] t (K (EVERY tacs));
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   318
    fun prove_eqn ((name, eqn_t), atts) = ((name, prove_term eqn_t), atts);
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   319
  in
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   320
    map prove_eqn eqns
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   321
  end;
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   322
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   323
(*************************************************************************)
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   324
(************************* Main fixrec function **************************)
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   325
(*************************************************************************)
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   326
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   327
fun gen_add_fixrec prep_prop prep_attrib strict blocks thy =
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   328
  let
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   329
    val eqns = List.concat blocks;
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   330
    val lengths = map length blocks;
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   331
    
28083
103d9282a946 explicit type Name.binding for higher-specification elements;
wenzelm
parents: 27691
diff changeset
   332
    val ((bindings, srcss), strings) = apfst split_list (split_list eqns);
29006
abe0f11cfa4e Name.name_of -> Binding.base_name
haftmann
parents: 28965
diff changeset
   333
    val names = map Binding.base_name bindings;
23152
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   334
    val atts = map (map (prep_attrib thy)) srcss;
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   335
    val eqn_ts = map (prep_prop thy) strings;
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   336
    val rec_ts = map (fn eq => chead_of (fst (dest_eqs (Logic.strip_imp_concl eq)))
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   337
      handle TERM _ => fixrec_eq_err thy "not a proper equation" eq) eqn_ts;
25557
ea6b11021e79 added new primrec package
haftmann
parents: 25132
diff changeset
   338
    val (_, eqn_ts') = OldPrimrecPackage.unify_consts thy rec_ts eqn_ts;
23152
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   339
    
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   340
    fun unconcat [] _ = []
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   341
      | unconcat (n::ns) xs = List.take (xs,n) :: unconcat ns (List.drop (xs,n));
30131
6be1be402ef0 use TheoryData to keep track of pattern match combinators
huffman
parents: 29585
diff changeset
   342
    val matcher_tab = FixrecMatchData.get thy;
6be1be402ef0 use TheoryData to keep track of pattern match combinators
huffman
parents: 29585
diff changeset
   343
    fun match_name c =
6be1be402ef0 use TheoryData to keep track of pattern match combinators
huffman
parents: 29585
diff changeset
   344
          case Symtab.lookup matcher_tab c of SOME m => m
6be1be402ef0 use TheoryData to keep track of pattern match combinators
huffman
parents: 29585
diff changeset
   345
            | NONE => fixrec_err ("unknown pattern constructor: " ^ c);
6be1be402ef0 use TheoryData to keep track of pattern match combinators
huffman
parents: 29585
diff changeset
   346
23152
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   347
    val pattern_blocks = unconcat lengths (map Logic.strip_imp_concl eqn_ts');
30131
6be1be402ef0 use TheoryData to keep track of pattern match combinators
huffman
parents: 29585
diff changeset
   348
    val compiled_ts =
30132
243a05a67c41 avoid using legacy type inference
huffman
parents: 30131
diff changeset
   349
          map (compile_pats match_name) pattern_blocks;
23152
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   350
    val (thy', cnames, fixdef_thms, unfold_thms) = add_fixdefs compiled_ts thy;
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   351
  in
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   352
    if strict then let (* only prove simp rules if strict = true *)
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   353
      val eqn_blocks = unconcat lengths ((names ~~ eqn_ts') ~~ atts);
29585
c23295521af5 binding replaces bstring
haftmann
parents: 29581
diff changeset
   354
      val simps = maps (make_simps thy') (unfold_thms ~~ eqn_blocks);
c23295521af5 binding replaces bstring
haftmann
parents: 29581
diff changeset
   355
      val (simp_thms, thy'') = PureThy.add_thms ((map o apfst o apfst) Binding.name simps) thy';
23152
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   356
      
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   357
      val simp_names = map (fn name => name^"_simps") cnames;
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   358
      val simp_attribute = rpair [Simplifier.simp_add];
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   359
      val simps' = map simp_attribute (simp_names ~~ unconcat lengths simp_thms);
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   360
    in
29585
c23295521af5 binding replaces bstring
haftmann
parents: 29581
diff changeset
   361
      (snd o PureThy.add_thmss ((map o apfst o apfst) Binding.name simps')) thy''
23152
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   362
    end
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   363
    else thy'
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   364
  end;
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   365
24707
dfeb98f84e93 Syntax.parse/check/read;
wenzelm
parents: 24680
diff changeset
   366
val add_fixrec = gen_add_fixrec Syntax.read_prop_global Attrib.attribute;
23152
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   367
val add_fixrec_i = gen_add_fixrec Sign.cert_prop (K I);
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   368
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   369
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   370
(*************************************************************************)
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   371
(******************************** Fixpat *********************************)
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   372
(*************************************************************************)
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   373
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   374
fun fix_pat thy t = 
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   375
  let
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   376
    val T = fastype_of t;
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   377
    val eq = mk_trp (HOLogic.eq_const T $ t $ Var (("x",0),T));
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   378
    val cname = case chead_of t of Const(c,_) => c | _ =>
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   379
              fixrec_err "function is not declared as constant in theory";
26343
0dd2eab7b296 simplified get_thm(s): back to plain name argument;
wenzelm
parents: 26336
diff changeset
   380
    val unfold_thm = PureThy.get_thm thy (cname^"_unfold");
23152
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   381
    val simp = Goal.prove_global thy [] [] eq
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   382
          (fn _ => EVERY [stac unfold_thm 1, simp_tac (simpset_of thy) 1]);
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   383
  in simp end;
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   384
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   385
fun gen_add_fixpat prep_term prep_attrib ((name, srcs), strings) thy =
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   386
  let
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   387
    val atts = map (prep_attrib thy) srcs;
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   388
    val ts = map (prep_term thy) strings;
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   389
    val simps = map (fix_pat thy) ts;
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   390
  in
29585
c23295521af5 binding replaces bstring
haftmann
parents: 29581
diff changeset
   391
    (snd o PureThy.add_thmss [((name, simps), atts)]) thy
23152
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   392
  end;
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   393
24707
dfeb98f84e93 Syntax.parse/check/read;
wenzelm
parents: 24680
diff changeset
   394
val add_fixpat = gen_add_fixpat Syntax.read_term_global Attrib.attribute;
23152
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   395
val add_fixpat_i = gen_add_fixpat Sign.cert_term (K I);
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   396
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   397
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   398
(*************************************************************************)
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   399
(******************************** Parsers ********************************)
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   400
(*************************************************************************)
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   401
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   402
local structure P = OuterParse and K = OuterKeyword in
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   403
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   404
val fixrec_eqn = SpecParse.opt_thm_name ":" -- P.prop;
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   405
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   406
val fixrec_strict = P.opt_keyword "permissive" >> not;
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   407
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   408
val fixrec_decl = fixrec_strict -- P.and_list1 (Scan.repeat1 fixrec_eqn);
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   409
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   410
(* this builds a parser for a new keyword, fixrec, whose functionality 
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   411
is defined by add_fixrec *)
24867
e5b55d7be9bb simplified interfaces for outer syntax;
wenzelm
parents: 24707
diff changeset
   412
val _ =
23152
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   413
  OuterSyntax.command "fixrec" "define recursive functions (HOLCF)" K.thy_decl
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   414
    (fixrec_decl >> (Toplevel.theory o uncurry add_fixrec));
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   415
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   416
(* fixpat parser *)
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   417
val fixpat_decl = SpecParse.opt_thm_name ":" -- Scan.repeat1 P.prop;
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   418
24867
e5b55d7be9bb simplified interfaces for outer syntax;
wenzelm
parents: 24707
diff changeset
   419
val _ =
23152
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   420
  OuterSyntax.command "fixpat" "define rewrites for fixrec functions" K.thy_decl
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   421
    (fixpat_decl >> (Toplevel.theory o add_fixpat));
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   422
26045
02aa3f166c7f use ML antiquotations
huffman
parents: 25557
diff changeset
   423
end; (* local structure *)
23152
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents:
diff changeset
   424
30131
6be1be402ef0 use TheoryData to keep track of pattern match combinators
huffman
parents: 29585
diff changeset
   425
val setup = FixrecMatchData.init;
6be1be402ef0 use TheoryData to keep track of pattern match combinators
huffman
parents: 29585
diff changeset
   426
24867
e5b55d7be9bb simplified interfaces for outer syntax;
wenzelm
parents: 24707
diff changeset
   427
end;