src/HOL/Tools/TFL/usyntax.ML
author krauss
Sat, 26 Apr 2008 08:49:31 +0200
changeset 26750 b53db47a43b4
parent 23150 073a65f0bc40
child 29265 5b4247055bd7
permissions -rw-r--r--
fixed recdef, broken by my previous commit
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
23150
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
     1
(*  Title:      HOL/Tools/TFL/usyntax.ML
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
     2
    ID:         $Id$
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
     3
    Author:     Konrad Slind, Cambridge University Computer Laboratory
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
     4
    Copyright   1997  University of Cambridge
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
     5
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
     6
Emulation of HOL's abstract syntax functions.
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
     7
*)
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
     8
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
     9
signature USYNTAX =
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
    10
sig
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
    11
  datatype lambda = VAR   of {Name : string, Ty : typ}
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
    12
                  | CONST of {Name : string, Ty : typ}
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
    13
                  | COMB  of {Rator: term, Rand : term}
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
    14
                  | LAMB  of {Bvar : term, Body : term}
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
    15
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
    16
  val alpha : typ
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
    17
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
    18
  (* Types *)
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
    19
  val type_vars  : typ -> typ list
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
    20
  val type_varsl : typ list -> typ list
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
    21
  val mk_vartype : string -> typ
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
    22
  val is_vartype : typ -> bool
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
    23
  val strip_prod_type : typ -> typ list
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
    24
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
    25
  (* Terms *)
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
    26
  val free_vars_lr : term -> term list
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
    27
  val type_vars_in_term : term -> typ list
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
    28
  val dest_term  : term -> lambda
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
    29
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
    30
  (* Prelogic *)
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
    31
  val inst      : (typ*typ) list -> term -> term
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
    32
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
    33
  (* Construction routines *)
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
    34
  val mk_abs    :{Bvar  : term, Body : term} -> term
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
    35
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
    36
  val mk_imp    :{ant : term, conseq :  term} -> term
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
    37
  val mk_select :{Bvar : term, Body : term} -> term
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
    38
  val mk_forall :{Bvar : term, Body : term} -> term
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
    39
  val mk_exists :{Bvar : term, Body : term} -> term
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
    40
  val mk_conj   :{conj1 : term, conj2 : term} -> term
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
    41
  val mk_disj   :{disj1 : term, disj2 : term} -> term
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
    42
  val mk_pabs   :{varstruct : term, body : term} -> term
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
    43
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
    44
  (* Destruction routines *)
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
    45
  val dest_const: term -> {Name : string, Ty : typ}
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
    46
  val dest_comb : term -> {Rator : term, Rand : term}
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
    47
  val dest_abs  : string list -> term -> {Bvar : term, Body : term} * string list
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
    48
  val dest_eq     : term -> {lhs : term, rhs : term}
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
    49
  val dest_imp    : term -> {ant : term, conseq : term}
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
    50
  val dest_forall : term -> {Bvar : term, Body : term}
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
    51
  val dest_exists : term -> {Bvar : term, Body : term}
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
    52
  val dest_neg    : term -> term
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
    53
  val dest_conj   : term -> {conj1 : term, conj2 : term}
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
    54
  val dest_disj   : term -> {disj1 : term, disj2 : term}
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
    55
  val dest_pair   : term -> {fst : term, snd : term}
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
    56
  val dest_pabs   : string list -> term -> {varstruct : term, body : term, used : string list}
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
    57
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
    58
  val lhs   : term -> term
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
    59
  val rhs   : term -> term
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
    60
  val rand  : term -> term
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
    61
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
    62
  (* Query routines *)
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
    63
  val is_imp    : term -> bool
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
    64
  val is_forall : term -> bool
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
    65
  val is_exists : term -> bool
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
    66
  val is_neg    : term -> bool
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
    67
  val is_conj   : term -> bool
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
    68
  val is_disj   : term -> bool
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
    69
  val is_pair   : term -> bool
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
    70
  val is_pabs   : term -> bool
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
    71
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
    72
  (* Construction of a term from a list of Preterms *)
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
    73
  val list_mk_abs    : (term list * term) -> term
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
    74
  val list_mk_imp    : (term list * term) -> term
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
    75
  val list_mk_forall : (term list * term) -> term
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
    76
  val list_mk_conj   : term list -> term
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
    77
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
    78
  (* Destructing a term to a list of Preterms *)
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
    79
  val strip_comb     : term -> (term * term list)
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
    80
  val strip_abs      : term -> (term list * term)
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
    81
  val strip_imp      : term -> (term list * term)
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
    82
  val strip_forall   : term -> (term list * term)
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
    83
  val strip_exists   : term -> (term list * term)
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
    84
  val strip_disj     : term -> term list
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
    85
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
    86
  (* Miscellaneous *)
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
    87
  val mk_vstruct : typ -> term list -> term
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
    88
  val gen_all    : term -> term
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
    89
  val find_term  : (term -> bool) -> term -> term option
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
    90
  val dest_relation : term -> term * term * term
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
    91
  val is_WFR : term -> bool
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
    92
  val ARB : typ -> term
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
    93
end;
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
    94
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
    95
structure USyntax: USYNTAX =
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
    96
struct
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
    97
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
    98
infix 4 ##;
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
    99
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   100
fun USYN_ERR func mesg = Utils.ERR {module = "USyntax", func = func, mesg = mesg};
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   101
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   102
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   103
(*---------------------------------------------------------------------------
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   104
 *
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   105
 *                            Types
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   106
 *
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   107
 *---------------------------------------------------------------------------*)
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   108
val mk_prim_vartype = TVar;
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   109
fun mk_vartype s = mk_prim_vartype ((s, 0), HOLogic.typeS);
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   110
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   111
(* But internally, it's useful *)
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   112
fun dest_vtype (TVar x) = x
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   113
  | dest_vtype _ = raise USYN_ERR "dest_vtype" "not a flexible type variable";
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   114
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   115
val is_vartype = can dest_vtype;
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   116
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   117
val type_vars  = map mk_prim_vartype o typ_tvars
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   118
fun type_varsl L = distinct (op =) (fold (curry op @ o type_vars) L []);
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   119
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   120
val alpha  = mk_vartype "'a"
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   121
val beta   = mk_vartype "'b"
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   122
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   123
val strip_prod_type = HOLogic.prodT_factors;
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   124
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   125
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   126
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   127
(*---------------------------------------------------------------------------
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   128
 *
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   129
 *                              Terms
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   130
 *
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   131
 *---------------------------------------------------------------------------*)
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   132
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   133
(* Free variables, in order of occurrence, from left to right in the
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   134
 * syntax tree. *)
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   135
fun free_vars_lr tm =
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   136
  let fun memb x = let fun m[] = false | m(y::rst) = (x=y)orelse m rst in m end
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   137
      fun add (t, frees) = case t of
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   138
            Free   _ => if (memb t frees) then frees else t::frees
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   139
          | Abs (_,_,body) => add(body,frees)
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   140
          | f$t =>  add(t, add(f, frees))
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   141
          | _ => frees
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   142
  in rev(add(tm,[]))
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   143
  end;
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   144
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   145
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   146
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   147
val type_vars_in_term = map mk_prim_vartype o term_tvars;
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   148
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   149
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   150
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   151
(* Prelogic *)
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   152
fun dest_tybinding (v,ty) = (#1(dest_vtype v),ty)
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   153
fun inst theta = subst_vars (map dest_tybinding theta,[])
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   154
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   155
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   156
(* Construction routines *)
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   157
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   158
fun mk_abs{Bvar as Var((s,_),ty),Body}  = Abs(s,ty,abstract_over(Bvar,Body))
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   159
  | mk_abs{Bvar as Free(s,ty),Body}  = Abs(s,ty,abstract_over(Bvar,Body))
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   160
  | mk_abs _ = raise USYN_ERR "mk_abs" "Bvar is not a variable";
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   161
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   162
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   163
fun mk_imp{ant,conseq} =
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   164
   let val c = Const("op -->",HOLogic.boolT --> HOLogic.boolT --> HOLogic.boolT)
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   165
   in list_comb(c,[ant,conseq])
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   166
   end;
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   167
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   168
fun mk_select (r as {Bvar,Body}) =
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   169
  let val ty = type_of Bvar
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   170
      val c = Const("Hilbert_Choice.Eps",(ty --> HOLogic.boolT) --> ty)
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   171
  in list_comb(c,[mk_abs r])
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   172
  end;
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   173
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   174
fun mk_forall (r as {Bvar,Body}) =
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   175
  let val ty = type_of Bvar
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   176
      val c = Const("All",(ty --> HOLogic.boolT) --> HOLogic.boolT)
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   177
  in list_comb(c,[mk_abs r])
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   178
  end;
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   179
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   180
fun mk_exists (r as {Bvar,Body}) =
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   181
  let val ty = type_of Bvar
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   182
      val c = Const("Ex",(ty --> HOLogic.boolT) --> HOLogic.boolT)
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   183
  in list_comb(c,[mk_abs r])
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   184
  end;
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   185
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   186
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   187
fun mk_conj{conj1,conj2} =
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   188
   let val c = Const("op &",HOLogic.boolT --> HOLogic.boolT --> HOLogic.boolT)
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   189
   in list_comb(c,[conj1,conj2])
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   190
   end;
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   191
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   192
fun mk_disj{disj1,disj2} =
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   193
   let val c = Const("op |",HOLogic.boolT --> HOLogic.boolT --> HOLogic.boolT)
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   194
   in list_comb(c,[disj1,disj2])
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   195
   end;
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   196
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   197
fun prod_ty ty1 ty2 = HOLogic.mk_prodT (ty1,ty2);
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   198
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   199
local
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   200
fun mk_uncurry(xt,yt,zt) =
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   201
    Const("split",(xt --> yt --> zt) --> prod_ty xt yt --> zt)
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   202
fun dest_pair(Const("Pair",_) $ M $ N) = {fst=M, snd=N}
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   203
  | dest_pair _ = raise USYN_ERR "dest_pair" "not a pair"
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   204
fun is_var (Var _) = true | is_var (Free _) = true | is_var _ = false
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   205
in
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   206
fun mk_pabs{varstruct,body} =
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   207
 let fun mpa (varstruct, body) =
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   208
       if is_var varstruct
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   209
       then mk_abs {Bvar = varstruct, Body = body}
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   210
       else let val {fst, snd} = dest_pair varstruct
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   211
            in mk_uncurry (type_of fst, type_of snd, type_of body) $
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   212
               mpa (fst, mpa (snd, body))
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   213
            end
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   214
 in mpa (varstruct, body) end
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   215
 handle TYPE _ => raise USYN_ERR "mk_pabs" "";
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   216
end;
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   217
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   218
(* Destruction routines *)
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   219
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   220
datatype lambda = VAR   of {Name : string, Ty : typ}
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   221
                | CONST of {Name : string, Ty : typ}
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   222
                | COMB  of {Rator: term, Rand : term}
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   223
                | LAMB  of {Bvar : term, Body : term};
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   224
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   225
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   226
fun dest_term(Var((s,i),ty)) = VAR{Name = s, Ty = ty}
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   227
  | dest_term(Free(s,ty))    = VAR{Name = s, Ty = ty}
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   228
  | dest_term(Const(s,ty))   = CONST{Name = s, Ty = ty}
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   229
  | dest_term(M$N)           = COMB{Rator=M,Rand=N}
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   230
  | dest_term(Abs(s,ty,M))   = let  val v = Free(s,ty)
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   231
                               in LAMB{Bvar = v, Body = Term.betapply (M,v)}
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   232
                               end
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   233
  | dest_term(Bound _)       = raise USYN_ERR "dest_term" "Bound";
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   234
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   235
fun dest_const(Const(s,ty)) = {Name = s, Ty = ty}
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   236
  | dest_const _ = raise USYN_ERR "dest_const" "not a constant";
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   237
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   238
fun dest_comb(t1 $ t2) = {Rator = t1, Rand = t2}
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   239
  | dest_comb _ =  raise USYN_ERR "dest_comb" "not a comb";
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   240
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   241
fun dest_abs used (a as Abs(s, ty, M)) =
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   242
     let
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   243
       val s' = Name.variant used s;
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   244
       val v = Free(s', ty);
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   245
     in ({Bvar = v, Body = Term.betapply (a,v)}, s'::used)
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   246
     end
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   247
  | dest_abs _ _ =  raise USYN_ERR "dest_abs" "not an abstraction";
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   248
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   249
fun dest_eq(Const("op =",_) $ M $ N) = {lhs=M, rhs=N}
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   250
  | dest_eq _ = raise USYN_ERR "dest_eq" "not an equality";
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   251
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   252
fun dest_imp(Const("op -->",_) $ M $ N) = {ant=M, conseq=N}
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   253
  | dest_imp _ = raise USYN_ERR "dest_imp" "not an implication";
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   254
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   255
fun dest_forall(Const("All",_) $ (a as Abs _)) = fst (dest_abs [] a)
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   256
  | dest_forall _ = raise USYN_ERR "dest_forall" "not a forall";
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   257
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   258
fun dest_exists(Const("Ex",_) $ (a as Abs _)) = fst (dest_abs [] a)
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   259
  | dest_exists _ = raise USYN_ERR "dest_exists" "not an existential";
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   260
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   261
fun dest_neg(Const("not",_) $ M) = M
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   262
  | dest_neg _ = raise USYN_ERR "dest_neg" "not a negation";
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   263
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   264
fun dest_conj(Const("op &",_) $ M $ N) = {conj1=M, conj2=N}
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   265
  | dest_conj _ = raise USYN_ERR "dest_conj" "not a conjunction";
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   266
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   267
fun dest_disj(Const("op |",_) $ M $ N) = {disj1=M, disj2=N}
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   268
  | dest_disj _ = raise USYN_ERR "dest_disj" "not a disjunction";
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   269
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   270
fun mk_pair{fst,snd} =
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   271
   let val ty1 = type_of fst
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   272
       val ty2 = type_of snd
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   273
       val c = Const("Pair",ty1 --> ty2 --> prod_ty ty1 ty2)
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   274
   in list_comb(c,[fst,snd])
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   275
   end;
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   276
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   277
fun dest_pair(Const("Pair",_) $ M $ N) = {fst=M, snd=N}
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   278
  | dest_pair _ = raise USYN_ERR "dest_pair" "not a pair";
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   279
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   280
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   281
local  fun ucheck t = (if #Name(dest_const t) = "split" then t
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   282
                       else raise Match)
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   283
in
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   284
fun dest_pabs used tm =
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   285
   let val ({Bvar,Body}, used') = dest_abs used tm
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   286
   in {varstruct = Bvar, body = Body, used = used'}
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   287
   end handle Utils.ERR _ =>
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   288
          let val {Rator,Rand} = dest_comb tm
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   289
              val _ = ucheck Rator
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   290
              val {varstruct = lv, body, used = used'} = dest_pabs used Rand
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   291
              val {varstruct = rv, body, used = used''} = dest_pabs used' body
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   292
          in {varstruct = mk_pair {fst = lv, snd = rv}, body = body, used = used''}
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   293
          end
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   294
end;
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   295
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   296
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   297
val lhs   = #lhs o dest_eq
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   298
val rhs   = #rhs o dest_eq
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   299
val rand  = #Rand o dest_comb
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   300
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   301
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   302
(* Query routines *)
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   303
val is_imp    = can dest_imp
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   304
val is_forall = can dest_forall
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   305
val is_exists = can dest_exists
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   306
val is_neg    = can dest_neg
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   307
val is_conj   = can dest_conj
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   308
val is_disj   = can dest_disj
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   309
val is_pair   = can dest_pair
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   310
val is_pabs   = can (dest_pabs [])
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   311
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   312
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   313
(* Construction of a cterm from a list of Terms *)
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   314
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   315
fun list_mk_abs(L,tm) = fold_rev (fn v => fn M => mk_abs{Bvar=v, Body=M}) L tm;
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   316
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   317
(* These others are almost never used *)
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   318
fun list_mk_imp(A,c) = fold_rev (fn a => fn tm => mk_imp{ant=a,conseq=tm}) A c;
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   319
fun list_mk_forall(V,t) = fold_rev (fn v => fn b => mk_forall{Bvar=v, Body=b})V t;
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   320
val list_mk_conj = Utils.end_itlist(fn c1 => fn tm => mk_conj{conj1=c1, conj2=tm})
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   321
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   322
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   323
(* Need to reverse? *)
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   324
fun gen_all tm = list_mk_forall(term_frees tm, tm);
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   325
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   326
(* Destructing a cterm to a list of Terms *)
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   327
fun strip_comb tm =
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   328
   let fun dest(M$N, A) = dest(M, N::A)
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   329
         | dest x = x
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   330
   in dest(tm,[])
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   331
   end;
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   332
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   333
fun strip_abs(tm as Abs _) =
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   334
       let val ({Bvar,Body}, _) = dest_abs [] tm
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   335
           val (bvs, core) = strip_abs Body
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   336
       in (Bvar::bvs, core)
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   337
       end
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   338
  | strip_abs M = ([],M);
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   339
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   340
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   341
fun strip_imp fm =
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   342
   if (is_imp fm)
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   343
   then let val {ant,conseq} = dest_imp fm
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   344
            val (was,wb) = strip_imp conseq
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   345
        in ((ant::was), wb)
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   346
        end
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   347
   else ([],fm);
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   348
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   349
fun strip_forall fm =
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   350
   if (is_forall fm)
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   351
   then let val {Bvar,Body} = dest_forall fm
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   352
            val (bvs,core) = strip_forall Body
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   353
        in ((Bvar::bvs), core)
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   354
        end
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   355
   else ([],fm);
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   356
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   357
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   358
fun strip_exists fm =
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   359
   if (is_exists fm)
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   360
   then let val {Bvar, Body} = dest_exists fm
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   361
            val (bvs,core) = strip_exists Body
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   362
        in (Bvar::bvs, core)
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   363
        end
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   364
   else ([],fm);
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   365
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   366
fun strip_disj w =
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   367
   if (is_disj w)
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   368
   then let val {disj1,disj2} = dest_disj w
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   369
        in (strip_disj disj1@strip_disj disj2)
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   370
        end
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   371
   else [w];
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   372
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   373
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   374
(* Miscellaneous *)
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   375
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   376
fun mk_vstruct ty V =
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   377
  let fun follow_prod_type (Type("*",[ty1,ty2])) vs =
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   378
              let val (ltm,vs1) = follow_prod_type ty1 vs
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   379
                  val (rtm,vs2) = follow_prod_type ty2 vs1
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   380
              in (mk_pair{fst=ltm, snd=rtm}, vs2) end
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   381
        | follow_prod_type _ (v::vs) = (v,vs)
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   382
  in #1 (follow_prod_type ty V)  end;
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   383
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   384
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   385
(* Search a term for a sub-term satisfying the predicate p. *)
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   386
fun find_term p =
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   387
   let fun find tm =
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   388
      if (p tm) then SOME tm
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   389
      else case tm of
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   390
          Abs(_,_,body) => find body
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   391
        | (t$u)         => (case find t of NONE => find u | some => some)
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   392
        | _             => NONE
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   393
   in find
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   394
   end;
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   395
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   396
fun dest_relation tm =
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   397
   if (type_of tm = HOLogic.boolT)
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   398
   then let val (Const("op :",_) $ (Const("Pair",_)$y$x) $ R) = tm
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   399
        in (R,y,x)
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   400
        end handle Bind => raise USYN_ERR "dest_relation" "unexpected term structure"
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   401
   else raise USYN_ERR "dest_relation" "not a boolean term";
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   402
26750
b53db47a43b4 fixed recdef, broken by my previous commit
krauss
parents: 23150
diff changeset
   403
fun is_WFR (Const(@{const_name "Wellfounded.wf"},_)$_) = true
23150
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   404
  | is_WFR _                 = false;
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   405
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   406
fun ARB ty = mk_select{Bvar=Free("v",ty),
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   407
                       Body=Const("True",HOLogic.boolT)};
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   408
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
   409
end;