src/Provers/blast.ML
author paulson
Fri, 04 Apr 1997 11:28:28 +0200
changeset 2894 d2ffee4f811b
parent 2883 fd1c0b8e9b61
child 2924 af506c35b4ed
permissions -rw-r--r--
Re-organization of the order of haz rules
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
2894
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
     1
(*  Title: 	Provers/blast
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
     2
    ID:         $Id$
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
     3
    Author: 	Lawrence C Paulson, Cambridge University Computer Laboratory
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
     4
    Copyright   1992  University of Cambridge
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
     5
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
     6
Generic tableau prover with proof reconstruction
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
     7
2854
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
     8
  SKOLEMIZES ReplaceI WRONGLY: allow new vars in prems, or forbid such rules??
2894
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
     9
  Needs explicit instantiation of assumptions?
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
    10
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
    11
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
    12
Limitations compared with fast_tac:
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
    13
  * ignores addss, addbefore, addafter; this restriction is intrinsic
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
    14
  * seems to loop given transitivity and similar rules
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
    15
  * ignores elimination rules that don't have the correct format
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
    16
	(conclusion must be a formula variable)
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
    17
  * ignores types, which can make HOL proofs fail
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
    18
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
    19
Known problems:
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
    20
  With hyp_subst_tac:
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
    21
    1.  Sometimes hyp_subst_tac will fail due to occurrence of the parameter
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
    22
        as the argument of a function variable
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
    23
    2.  When a literal is affected, it is moved back to the active formulae.
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
    24
        But there's no way of putting it in the right place.
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
    25
    3.  Affected haz formulae should also be moved, but they are not.
2854
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
    26
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
    27
*)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
    28
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
    29
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
    30
(*Should be a type abbreviation?*)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
    31
type netpair = (int*(bool*thm)) Net.net * (int*(bool*thm)) Net.net;
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
    32
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
    33
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
    34
(*Assumptions about constants:
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
    35
  --The negation symbol is "Not"
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
    36
  --The equality symbol is "op ="
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
    37
  --The is-true judgement symbol is "Trueprop"
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
    38
  --There are no constants named "*Goal* or "*False*"
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
    39
*)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
    40
signature BLAST_DATA =
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
    41
  sig
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
    42
  type claset
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
    43
  val notE		: thm		(* [| ~P;  P |] ==> R *)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
    44
  val ccontr		: thm		
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
    45
  val contr_tac 	: int -> tactic
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
    46
  val dup_intr		: thm -> thm
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
    47
  val vars_gen_hyp_subst_tac : bool -> int -> tactic
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
    48
  val claset		: claset ref
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
    49
  val rep_claset	: 
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
    50
      claset -> {safeIs: thm list, safeEs: thm list, 
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
    51
		 hazIs: thm list, hazEs: thm list,
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
    52
		 uwrapper: (int -> tactic) -> (int -> tactic),
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
    53
		 swrapper: (int -> tactic) -> (int -> tactic),
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
    54
		 safe0_netpair: netpair, safep_netpair: netpair,
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
    55
		 haz_netpair: netpair, dup_netpair: netpair}
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
    56
  end;
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
    57
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
    58
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
    59
signature BLAST =
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
    60
  sig
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
    61
  type claset
2883
fd1c0b8e9b61 Now exports declConsts!
paulson
parents: 2854
diff changeset
    62
  val depth_tac 	: claset -> int -> int -> tactic
fd1c0b8e9b61 Now exports declConsts!
paulson
parents: 2854
diff changeset
    63
  val blast_tac 	: claset -> int -> tactic
fd1c0b8e9b61 Now exports declConsts!
paulson
parents: 2854
diff changeset
    64
  val Blast_tac 	: int -> tactic
fd1c0b8e9b61 Now exports declConsts!
paulson
parents: 2854
diff changeset
    65
  val declConsts 	: string list * thm list -> unit
2854
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
    66
  end;
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
    67
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
    68
2883
fd1c0b8e9b61 Now exports declConsts!
paulson
parents: 2854
diff changeset
    69
functor BlastFun(Data: BLAST_DATA) = 
2854
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
    70
struct
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
    71
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
    72
type claset = Data.claset;
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
    73
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
    74
val trace = ref false;
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
    75
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
    76
datatype term = 
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
    77
    Const of string
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
    78
  | OConst of string * int
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
    79
  | Skolem of string * term option ref list
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
    80
  | Free  of string
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
    81
  | Var   of term option ref
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
    82
  | Bound of int
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
    83
  | Abs   of string*term
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
    84
  | op $  of term*term;
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
    85
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
    86
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
    87
exception DEST_EQ;
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
    88
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
    89
  (*Take apart an equality (plain or overloaded).  NO constant Trueprop*)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
    90
  fun dest_eq (Const  "op ="     $ t $ u) = (t,u)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
    91
    | dest_eq (OConst("op =",_)  $ t $ u) = (t,u)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
    92
    | dest_eq _                      = raise DEST_EQ;
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
    93
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
    94
(** Basic syntactic operations **)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
    95
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
    96
fun is_Var (Var _) = true
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
    97
  | is_Var _ = false;
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
    98
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
    99
fun dest_Var (Var x) =  x;
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   100
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   101
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   102
fun rand (f$x) = x;
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   103
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   104
(* maps   (f, [t1,...,tn])  to  f(t1,...,tn) *)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   105
val list_comb : term * term list -> term = foldl (op $);
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   106
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   107
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   108
(* maps   f(t1,...,tn)  to  (f, [t1,...,tn]) ; naturally tail-recursive*)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   109
fun strip_comb u : term * term list = 
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   110
    let fun stripc (f$t, ts) = stripc (f, t::ts)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   111
        |   stripc  x =  x 
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   112
    in  stripc(u,[])  end;
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   113
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   114
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   115
(* maps   f(t1,...,tn)  to  f , which is never a combination *)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   116
fun head_of (f$t) = head_of f
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   117
  | head_of u = u;
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   118
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   119
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   120
(** Particular constants **)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   121
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   122
fun negate P = Const"Not" $ P;
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   123
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   124
fun mkGoal P = Const"*Goal*" $ P;
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   125
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   126
fun isGoal (Const"*Goal*" $ _) = true
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   127
  | isGoal _                   = false;
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   128
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   129
val Trueprop = Term.Const("Trueprop", Type("o",[])-->propT);
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   130
fun mk_tprop P = Term.$ (Trueprop, P);
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   131
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   132
fun isTrueprop (Term.Const("Trueprop",_)) = true
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   133
  | isTrueprop _                          = false;
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   134
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   135
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   136
(** Dealing with overloaded constants **)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   137
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   138
(*Result is a symbol table, indexed by names of overloaded constants.
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   139
  Each constant maps to a list of (pattern,Blast.Const) pairs.
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   140
  Any Term.Const that matches a pattern gets replaced by the Blast.Const.
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   141
*)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   142
fun addConsts (t as Term.Const(a,_), tab) =
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   143
     (case Symtab.lookup (tab,a) of
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   144
	  None    => tab  (*ignore: not a constant that we are looking for*)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   145
	| Some patList => 
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   146
	      (case gen_assoc (op aconv) (patList, t) of
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   147
		  None => Symtab.update
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   148
		           ((a, (t, OConst (a, length patList)) :: patList), 
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   149
			    tab)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   150
		 | _    => tab))
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   151
  | addConsts (Term.Abs(_,_,body), tab) = addConsts (body, tab)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   152
  | addConsts (Term.$ (t,u), tab) = addConsts (t, addConsts (u, tab))
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   153
  | addConsts (_,            tab) = tab (*ignore others*);
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   154
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   155
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   156
fun addRules (rls,tab) = foldr addConsts (map (#prop o rep_thm) rls, tab);
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   157
2883
fd1c0b8e9b61 Now exports declConsts!
paulson
parents: 2854
diff changeset
   158
fun declConst (a,tab) = 
fd1c0b8e9b61 Now exports declConsts!
paulson
parents: 2854
diff changeset
   159
    case Symtab.lookup (tab,a) of
fd1c0b8e9b61 Now exports declConsts!
paulson
parents: 2854
diff changeset
   160
	None   => Symtab.update((a,[]), tab)	(*create a brand new entry*)
fd1c0b8e9b61 Now exports declConsts!
paulson
parents: 2854
diff changeset
   161
      | Some _ => tab				(*preserve old entry*);
2854
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   162
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   163
(*maps the name of each overloaded constant to a list of archetypal constants,
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   164
  which may be polymorphic.*)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   165
local
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   166
val overLoadTab = ref (Symtab.null : (Term.term * term) list Symtab.table)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   167
    (*The alists in this table should only be increased*)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   168
in
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   169
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   170
fun declConsts (names, rls) =
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   171
    overLoadTab := addRules (rls, foldr declConst (names, !overLoadTab));
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   172
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   173
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   174
(*Convert a possibly overloaded Term.Const to a Blast.Const*)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   175
fun fromConst tsig (t as Term.Const (a,_)) =
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   176
  let fun find []                  = Const a
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   177
	| find ((pat,t')::patList) =
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   178
		if Pattern.matches tsig (pat,t) then t' 
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   179
		else find patList
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   180
  in  case Symtab.lookup(!overLoadTab, a) of
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   181
	   None         => Const a
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   182
	 | Some patList => find patList
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   183
  end;
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   184
end;
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   185
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   186
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   187
(*Tests whether 2 terms are alpha-convertible; chases instantiations*)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   188
fun (Const a)      aconv (Const b)      = a=b
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   189
  | (OConst ai)    aconv (OConst bj)    = ai=bj
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   190
  | (Skolem (a,_)) aconv (Skolem (b,_)) = a=b  (*arglists must then be equal*)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   191
  | (Free a)       aconv (Free b)       = a=b
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   192
  | (Var(ref(Some t))) aconv u          = t aconv u
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   193
  | t aconv (Var(ref(Some u)))          = t aconv u
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   194
  | (Var v)        aconv (Var w)        = v=w	(*both Vars are un-assigned*)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   195
  | (Bound i)      aconv (Bound j)      = i=j
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   196
  | (Abs(_,t))     aconv (Abs(_,u))     = t aconv u
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   197
  | (f$t)          aconv (g$u)          = (f aconv g) andalso (t aconv u)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   198
  | _ aconv _  =  false;
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   199
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   200
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   201
fun mem_term (_, [])     = false
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   202
  | mem_term (t, t'::ts) = t aconv t' orelse mem_term(t,ts);
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   203
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   204
fun ins_term(t,ts) = if mem_term(t,ts) then ts else t :: ts;
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   205
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   206
fun mem_var (v: term option ref, []) = false
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   207
  | mem_var (v, v'::vs)              = v=v' orelse mem_var(v,vs);
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   208
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   209
fun ins_var(v,vs) = if mem_var(v,vs) then vs else v :: vs;
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   210
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   211
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   212
(** Vars **)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   213
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   214
(*Accumulates the Vars in the term, suppressing duplicates*)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   215
fun add_term_vars (Skolem(a,args),	vars) = add_vars_vars(args,vars)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   216
  | add_term_vars (Var (v as ref None),	vars) = ins_var (v, vars)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   217
  | add_term_vars (Var (ref (Some u)), vars)  = add_term_vars(u,vars)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   218
  | add_term_vars (Abs (_,body),	vars) = add_term_vars(body,vars)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   219
  | add_term_vars (f$t,	vars) =  add_term_vars (f, add_term_vars(t, vars))
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   220
  | add_term_vars (_,	vars) = vars
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   221
(*Term list version.  [The fold functionals are slow]*)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   222
and add_terms_vars ([],    vars) = vars
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   223
  | add_terms_vars (t::ts, vars) = add_terms_vars (ts, add_term_vars(t,vars))
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   224
(*Var list version.*)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   225
and add_vars_vars ([],    vars) = vars
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   226
  | add_vars_vars (ref (Some u) :: vs, vars) = 
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   227
	add_vars_vars (vs, add_term_vars(u,vars))
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   228
  | add_vars_vars (v::vs, vars) =   (*v must be a ref None*)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   229
	add_vars_vars (vs, ins_var (v, vars));
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   230
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   231
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   232
(*Chase assignments in "vars"; return a list of unassigned variables*)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   233
fun vars_in_vars vars = add_vars_vars(vars,[]);
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   234
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   235
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   236
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   237
(*increment a term's non-local bound variables
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   238
     inc is  increment for bound variables
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   239
     lev is  level at which a bound variable is considered 'loose'*)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   240
fun incr_bv (inc, lev, u as Bound i) = if i>=lev then Bound(i+inc) else u 
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   241
  | incr_bv (inc, lev, Abs(a,body)) = Abs(a, incr_bv(inc,lev+1,body))
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   242
  | incr_bv (inc, lev, f$t) = incr_bv(inc,lev,f) $ incr_bv(inc,lev,t)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   243
  | incr_bv (inc, lev, u) = u;
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   244
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   245
fun incr_boundvars  0  t = t
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   246
  | incr_boundvars inc t = incr_bv(inc,0,t);
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   247
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   248
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   249
(*Accumulate all 'loose' bound vars referring to level 'lev' or beyond.
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   250
   (Bound 0) is loose at level 0 *)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   251
fun add_loose_bnos (Bound i, lev, js)   = if i<lev then js  
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   252
					  else  (i-lev) ins_int js
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   253
  | add_loose_bnos (Abs (_,t), lev, js) = add_loose_bnos (t, lev+1, js)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   254
  | add_loose_bnos (f$t, lev, js)       =
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   255
	        add_loose_bnos (f, lev, add_loose_bnos (t, lev, js)) 
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   256
  | add_loose_bnos (_, _, js)           = js;
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   257
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   258
fun loose_bnos t = add_loose_bnos (t, 0, []);
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   259
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   260
fun subst_bound (arg, t) : term = 
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   261
  let fun subst (t as Bound i, lev) =
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   262
 	    if i<lev then  t    (*var is locally bound*)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   263
	    else  if i=lev then incr_boundvars lev arg
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   264
		           else Bound(i-1)  (*loose: change it*)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   265
	| subst (Abs(a,body), lev) = Abs(a, subst(body,lev+1))
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   266
	| subst (f$t, lev) =  subst(f,lev)  $  subst(t,lev)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   267
	| subst (t,lev)    = t
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   268
  in  subst (t,0)  end;
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   269
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   270
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   271
(*Normalize...but not the bodies of ABSTRACTIONS*)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   272
fun norm t = case t of
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   273
    Skolem(a,args)       => Skolem(a, vars_in_vars args)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   274
  | (Var (ref None))     => t
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   275
  | (Var (ref (Some u))) => norm u
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   276
  | (f $ u) => (case norm f of
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   277
		    Abs(_,body) => norm (subst_bound (u, body))
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   278
		  | nf => nf $ norm u)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   279
  | _ => t;
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   280
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   281
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   282
(*Weak (one-level) normalize for use in unification*)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   283
fun wkNormAux t = case t of
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   284
    (Var v) => (case !v of
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   285
		    Some u => wkNorm u
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   286
		  | None   => t)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   287
  | (f $ u) => (case wkNormAux f of
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   288
		    Abs(_,body) => wkNorm (subst_bound (u, body))
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   289
		  | nf          => nf $ u)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   290
  | _ => t
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   291
and wkNorm t = case head_of t of
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   292
    Const _        => t
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   293
  | OConst _       => t
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   294
  | Skolem(a,args) => t
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   295
  | Free _         => t
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   296
  | _              => wkNormAux t;
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   297
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   298
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   299
(*Does variable v occur in u?  For unification.*)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   300
fun varOccur v = 
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   301
  let fun occL [] = false	(*same as (exists occ), but faster*)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   302
	| occL (u::us) = occ u orelse occL us
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   303
      and occ (Var w) = 
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   304
	      v=w orelse
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   305
              (case !w of None   => false
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   306
	                | Some u => occ u)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   307
        | occ (Skolem(_,args)) = occL (map Var args)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   308
        | occ (Abs(_,u)) = occ u
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   309
        | occ (f$u)      = occ u  orelse  occ f
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   310
        | occ (_)        = false;
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   311
  in  occ  end;
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   312
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   313
exception UNIFY;
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   314
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   315
val trail = ref [] : term option ref list ref;
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   316
val ntrail = ref 0;
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   317
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   318
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   319
(*Restore the trail to some previous state: for backtracking*)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   320
fun clearTo n =
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   321
    while !ntrail>n do
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   322
	(hd(!trail) := None;
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   323
	 trail := tl (!trail);
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   324
	 ntrail := !ntrail - 1);
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   325
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   326
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   327
(*First-order unification with bound variables.  
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   328
  "vars" is a list of variables local to the rule and NOT to be put
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   329
	on the trail (no point in doing so)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   330
*)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   331
fun unify(vars,t,u) =
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   332
    let val n = !ntrail 
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   333
	fun update (t as Var v, u) =
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   334
	    if t aconv u then ()
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   335
	    else if varOccur v u then raise UNIFY 
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   336
	    else if mem_var(v, vars) then v := Some u
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   337
		 else (*avoid updating Vars in the branch if possible!*)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   338
		      if is_Var u andalso mem_var(dest_Var u, vars)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   339
		      then dest_Var u := Some t
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   340
		      else (v := Some u;
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   341
			    trail := v :: !trail;  ntrail := !ntrail + 1)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   342
	fun unifyAux (t,u) = 
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   343
	    case (wkNorm t,  wkNorm u) of
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   344
		(nt as Var v,  nu) => update(nt,nu)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   345
	      | (nu,  nt as Var v) => update(nt,nu)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   346
	      | (Abs(_,t'),  Abs(_,u')) => unifyAux(t',u')
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   347
		    (*NB: can yield unifiers having dangling Bound vars!*)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   348
	      | (f$t',  g$u') => (unifyAux(f,g); unifyAux(t',u'))
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   349
	      | (nt,  nu)    => if nt aconv nu then () else raise UNIFY
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   350
    in  unifyAux(t,u) handle UNIFY => (clearTo n; raise UNIFY)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   351
    end;
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   352
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   353
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   354
(*Convert from "real" terms to prototerms; eta-contract*)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   355
fun fromTerm tsig t =
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   356
  let val alist = ref []
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   357
      fun from (t as Term.Const _) = fromConst tsig t
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   358
	| from (Term.Free  (a,_)) = Free a
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   359
	| from (Term.Bound i)     = Bound i
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   360
	| from (Term.Var (ixn,T)) = 
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   361
	      (case (assoc_string_int(!alist,ixn)) of
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   362
		   None => let val t' = Var(ref None)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   363
		           in  alist := (ixn, (t', T)) :: !alist;  t'
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   364
			   end
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   365
		 | Some (v,_) => v)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   366
	| from (Term.Abs (a,_,u)) = 
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   367
	      (case  from u  of
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   368
		u' as (f $ Bound 0) => 
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   369
		  if (0 mem_int loose_bnos f) then Abs(a,u')
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   370
		  else incr_boundvars ~1 f 
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   371
	      | u' => Abs(a,u'))
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   372
	| from (Term.$ (f,u)) = from f $ from u
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   373
  in  from t  end;
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   374
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   375
(* A1==>...An==>B  goes to  [A1,...,An], where B is not an implication *)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   376
fun strip_imp_prems (Const"==>" $ (Const"Trueprop" $ A) $ B) = 
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   377
           A :: strip_imp_prems B
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   378
  | strip_imp_prems (Const"==>" $ A $ B) = A :: strip_imp_prems B
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   379
  | strip_imp_prems _ = [];
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   380
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   381
(* A1==>...An==>B  goes to B, where B is not an implication *)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   382
fun strip_imp_concl (Const"==>" $ A $ B) = strip_imp_concl B
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   383
  | strip_imp_concl (Const"Trueprop" $ A) = A
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   384
  | strip_imp_concl A = A : term;
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   385
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   386
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   387
(*** Conversion of Elimination Rules to Tableau Operations ***)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   388
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   389
(*The conclusion becomes the goal/negated assumption *False*: delete it!*)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   390
fun squash_nots [] = []
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   391
  | squash_nots (Const "*Goal*" $ (Var (ref (Some (Const"*False*")))) :: Ps) =
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   392
	squash_nots Ps
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   393
  | squash_nots (Const "Not" $ (Var (ref (Some (Const"*False*")))) :: Ps) =
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   394
	squash_nots Ps
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   395
  | squash_nots (P::Ps) = P :: squash_nots Ps;
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   396
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   397
fun skoPrem vars (Const "all" $ Abs (_, P)) =
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   398
        skoPrem vars (subst_bound (Skolem (gensym "S_", vars), P))
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   399
  | skoPrem vars P = P;
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   400
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   401
fun convertPrem t = 
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   402
    squash_nots (mkGoal (strip_imp_concl t) :: strip_imp_prems t);
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   403
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   404
(*Expects elimination rules to have a formula variable as conclusion*)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   405
fun convertRule vars t =
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   406
  let val (P::Ps) = strip_imp_prems t
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   407
      val Var v   = strip_imp_concl t
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   408
  in  v := Some (Const"*False*");
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   409
      (P, map (convertPrem o skoPrem vars) Ps) 
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   410
  end;
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   411
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   412
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   413
(*Like dup_elim, but puts the duplicated major premise FIRST*)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   414
fun rev_dup_elim th = th RSN (2, revcut_rl) |> assumption 2 |> Sequence.hd;
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   415
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   416
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   417
(*Count new hyps so that they can be rotated*)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   418
fun nNewHyps []                         = 0
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   419
  | nNewHyps (Const "*Goal*" $ _ :: Ps) = nNewHyps Ps
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   420
  | nNewHyps (P::Ps)                    = 1 + nNewHyps Ps;
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   421
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   422
fun rot_subgoals_tac [] i st      = Sequence.single st
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   423
  | rot_subgoals_tac (k::ks) i st =
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   424
      rot_subgoals_tac ks (i+1) (Sequence.hd (rotate_tac (~k) i st))
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   425
      handle OPTION _ => Sequence.null;
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   426
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   427
fun TRACE rl tac st = if !trace then (prth rl; tac st) else tac st;
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   428
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   429
(*Tableau rule from elimination rule.  Flag "dup" requests duplication of the
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   430
  affected formula.*)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   431
fun fromRule vars rl = 
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   432
  let val {tsig,...} = Sign.rep_sg (#sign (rep_thm rl))
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   433
      val trl = rl |> rep_thm |> #prop |> fromTerm tsig |> convertRule vars
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   434
      fun tac dup i = 
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   435
	  TRACE rl
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   436
	  (DETERM (etac (if dup then rev_dup_elim rl else rl) i))
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   437
	  THEN rot_subgoals_tac (map nNewHyps (#2 trl)) i
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   438
	  
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   439
  in General.SOME (trl, tac) end
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   440
  handle Bind => General.NONE  (*reject: conclusion is not just a variable*);
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   441
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   442
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   443
(*** Conversion of Introduction Rules (needed for efficiency in 
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   444
               proof reconstruction) ***)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   445
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   446
fun convertIntrPrem t = mkGoal (strip_imp_concl t) :: strip_imp_prems t;
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   447
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   448
fun convertIntrRule vars t =
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   449
  let val Ps = strip_imp_prems t
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   450
      val P  = strip_imp_concl t
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   451
  in  (mkGoal P, map (convertIntrPrem o skoPrem vars) Ps) 
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   452
  end;
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   453
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   454
(*Tableau rule from introduction rule.  Since haz rules are now delayed, 
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   455
  "dup" is always FALSE for introduction rules.*)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   456
fun fromIntrRule vars rl = 
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   457
  let val {tsig,...} = Sign.rep_sg (#sign (rep_thm rl))
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   458
      val trl = rl |> rep_thm |> #prop |> fromTerm tsig |> convertIntrRule vars
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   459
      fun tac dup i = 
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   460
	  TRACE rl (DETERM (rtac (if dup then Data.dup_intr rl else rl) i))
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   461
	  THEN rot_subgoals_tac (map nNewHyps (#2 trl)) i
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   462
  in (trl, tac) end;
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   463
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   464
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   465
val dummyVar = Term.Var (("Doom",666), dummyT);
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   466
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   467
(*Convert from prototerms to ordinary terms with dummy types
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   468
  Ignore abstractions; identify all Vars*)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   469
fun dummyTerm 0 _             = dummyVar
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   470
  | dummyTerm d (Const a)     = Term.Const (a,dummyT)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   471
  | dummyTerm d (OConst(a,_)) = Term.Const (a,dummyT)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   472
  | dummyTerm d (Skolem(a,_)) = Term.Const (a,dummyT)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   473
  | dummyTerm d (Free a)      = Term.Free  (a,dummyT)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   474
  | dummyTerm d (Bound i)     = Term.Bound i
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   475
  | dummyTerm d (Var _)       = dummyVar
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   476
  | dummyTerm d (Abs(a,_))    = dummyVar
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   477
  | dummyTerm d (f $ u)       = Term.$ (dummyTerm d f, dummyTerm (d-1) u);
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   478
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   479
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   480
fun netMkRules P vars (nps: netpair list) =
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   481
  case P of
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   482
      (Const "*Goal*" $ G) =>
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   483
	let val pG = mk_tprop (dummyTerm 2 G)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   484
	    val intrs = List.concat 
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   485
		             (map (fn (inet,_) => Net.unify_term inet pG) 
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   486
			      nps)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   487
	in  map (fromIntrRule vars o #2) (orderlist intrs)  end
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   488
    | _ =>
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   489
	let val pP = mk_tprop (dummyTerm 3 P)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   490
	    val elims = List.concat 
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   491
		             (map (fn (_,enet) => Net.unify_term enet pP) 
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   492
			      nps)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   493
	in  List.mapPartial (fromRule vars o #2) (orderlist elims)  end;
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   494
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   495
(**
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   496
end;
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   497
**)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   498
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   499
(*** Code for handling equality: naive substitution, like hyp_subst_tac ***)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   500
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   501
(*Replace the ATOMIC term "old" by "new" in t*)  
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   502
fun subst_atomic (old,new) t =
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   503
    let fun subst (Var(ref(Some u))) = subst u
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   504
	  | subst (Abs(a,body))      = Abs(a, subst body)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   505
	  | subst (f$t)              = subst f $ subst t
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   506
	  | subst t                  = if t aconv old then new else t
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   507
    in  subst t  end;
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   508
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   509
(*Eta-contract a term from outside: just enough to reduce it to an atom*)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   510
fun eta_contract_atom (t0 as Abs(a, body)) = 
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   511
      (case  eta_contract2 body  of
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   512
        f $ Bound 0 => if (0 mem_int loose_bnos f) then t0
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   513
		       else eta_contract_atom (incr_boundvars ~1 f)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   514
      | _ => t0)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   515
  | eta_contract_atom t = t
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   516
and eta_contract2 (f$t) = f $ eta_contract_atom t
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   517
  | eta_contract2 t     = eta_contract_atom t;
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   518
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   519
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   520
(*When can we safely delete the equality?
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   521
    Not if it equates two constants; consider 0=1.
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   522
    Not if it resembles x=t[x], since substitution does not eliminate x.
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   523
    Not if it resembles ?x=0; another goal could instantiate ?x to Suc(i)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   524
  Prefer to eliminate Bound variables if possible.
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   525
  Result:  true = use as is,  false = reorient first *)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   526
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   527
(*Does t occur in u?  For substitution.  
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   528
  Does NOT check args of Skolem terms: substitution does not affect them.
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   529
  NOT reflexive since hyp_subst_tac fails on x=x.*)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   530
fun substOccur t = 
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   531
  let fun occEq u = (t aconv u) orelse occ u
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   532
      and occ (Var(ref None))    = false
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   533
	| occ (Var(ref(Some u))) = occEq u
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   534
        | occ (Abs(_,u))         = occEq u
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   535
        | occ (f$u)              = occEq u  orelse  occEq f
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   536
        | occ (_)                = false;
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   537
  in  occEq  end;
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   538
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   539
fun check (t,u,v) = if substOccur t u then raise DEST_EQ else v;
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   540
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   541
(*IF the goal is an equality with a substitutable variable 
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   542
  THEN orient that equality ELSE raise exception DEST_EQ*)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   543
fun orientGoal (t,u) =
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   544
  case (eta_contract_atom t, eta_contract_atom u) of
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   545
       (Skolem _, _) => check(t,u,(t,u))	(*eliminates t*)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   546
     | (_, Skolem _) => check(u,t,(u,t))	(*eliminates u*)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   547
     | (Free _, _)   => check(t,u,(t,u))	(*eliminates t*)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   548
     | (_, Free _)   => check(u,t,(u,t))	(*eliminates u*)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   549
     | _             => raise DEST_EQ;
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   550
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   551
2894
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
   552
(*Substitute through the branch if an equality goal (else raise DEST_EQ).
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
   553
  Moves affected literals back into the branch, but it is not clear where
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
   554
  they should go: this could make proofs fail.  ??? *)
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
   555
fun equalSubst (G, pairs, lits, vars, lim) = 
2854
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   556
  let val subst = subst_atomic (orientGoal(dest_eq G))
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   557
      fun subst2(G,md) = (subst G, md)
2894
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
   558
      val pairs' = map (fn(Gs,Hs) => (map subst2 Gs, map subst2 Hs)) pairs
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
   559
      (*substitute throughout literals and note those affected*)
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
   560
      fun subLits ([], [], nlits) =          (pairs', nlits, vars, lim)
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
   561
	| subLits ([], Gs, nlits) = ((Gs,[])::pairs', nlits, vars, lim)
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
   562
	| subLits (lit::lits, Gs, nlits) =
2854
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   563
	    let val nlit = subst lit
2894
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
   564
	    in  if nlit aconv lit then subLits (lits, Gs, nlit::nlits)
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
   565
		                  else subLits (lits, (nlit,true)::Gs, nlits)
2854
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   566
            end
2894
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
   567
  in  subLits (rev lits, [], [])  
2854
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   568
  end;
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   569
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   570
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   571
exception NEWBRANCHES and CLOSEF;
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   572
2894
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
   573
(*Pending formulae carry md (may duplicate) flags*)
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
   574
type branch = ((term*bool) list *	(*safe formulae on this level*)
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
   575
               (term*bool) list) list * (*haz formulae  on this level*)
2854
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   576
	      term list *               (*literals: irreducible formulae*)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   577
	      term option ref list *    (*variables occurring in branch*)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   578
	      int;                      (*resource limit*)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   579
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   580
val fullTrace = ref[] : branch list list ref;
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   581
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   582
exception PROVE;
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   583
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   584
val eq_contr_tac = eresolve_tac [Data.notE]  THEN'  eq_assume_tac;
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   585
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   586
val eContr_tac  = TRACE Data.notE (eq_contr_tac ORELSE' Data.contr_tac);
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   587
val eAssume_tac = TRACE asm_rl   (eq_assume_tac ORELSE' assume_tac);
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   588
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   589
(*Try to unify complementary literals and return the corresponding tactic. *) 
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   590
fun tryClose (Const"*Goal*" $ G,  L) = (unify([],G,L); eAssume_tac)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   591
  | tryClose (G,  Const"*Goal*" $ L) = (unify([],G,L); eAssume_tac)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   592
  | tryClose (Const"Not" $ G,  L)    = (unify([],G,L); eContr_tac)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   593
  | tryClose (G,  Const"Not" $ L)    = (unify([],G,L); eContr_tac)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   594
  | tryClose _                       = raise UNIFY;
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   595
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   596
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   597
(*Were there Skolem terms in the premise?  Must NOT chase Vars*)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   598
fun hasSkolem (Skolem _)     = true
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   599
  | hasSkolem (Abs (_,body)) = hasSkolem body 
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   600
  | hasSkolem (f$t)          =  hasSkolem f orelse hasSkolem t
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   601
  | hasSkolem _              = false;
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   602
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   603
(*Attach the right "may duplicate" flag to new formulae: if they contain
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   604
  Skolem terms then allow duplication.*)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   605
fun joinMd md [] = []
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   606
  | joinMd md (G::Gs) = (G, hasSkolem G orelse md) :: joinMd md Gs;
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   607
2894
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
   608
(*Convert a Goal to an ordinary Not.  Used also in dup_intr, where a goal like
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
   609
  Ex(P) is duplicated as the assumption ~Ex(P). *)
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
   610
fun negOfGoal (Const"*Goal*" $ G) = negate G
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
   611
  | negOfGoal G                   = G;
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
   612
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
   613
fun negOfGoal2 (G,md) = (negOfGoal G, md);
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
   614
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
   615
(*Converts all Goals to Nots in the safe parts of a branch.  They could
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
   616
  have been moved there from the literals list after substitution (equalSubst).
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
   617
  There can be at most one--this function could be made more efficient.*)
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
   618
fun negOfGoals pairs = map (fn (Gs,haz) => (map negOfGoal2 Gs, haz)) pairs;
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
   619
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
   620
(*Tactic.  Convert *Goal* to negated assumption in FIRST position*)
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
   621
val negOfGoal_tac = rtac Data.ccontr THEN' rotate_tac ~1;
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
   622
2854
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   623
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   624
(** Backtracking and Pruning **)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   625
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   626
(*clashVar vars (n,trail) determines whether any of the last n elements
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   627
  of "trail" occur in "vars" OR in their instantiations*)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   628
fun clashVar [] = (fn _ => false)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   629
  | clashVar vars =
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   630
      let fun clash (0, _)     = false
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   631
	    | clash (_, [])    = false
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   632
	    | clash (n, v::vs) = exists (varOccur v) vars orelse clash(n-1,vs)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   633
      in  clash  end;
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   634
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   635
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   636
(*nbrs = # of branches just prior to closing this one.  Delete choice points
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   637
  for goals proved by the latest inference, provided NO variables in the
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   638
  next branch have been updated.*)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   639
fun prune (1, nxtVars, choices) = choices  (*DON'T prune at very end: allow 
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   640
					     backtracking over bad proofs*)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   641
  | prune (nbrs, nxtVars, choices) =
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   642
      let fun traceIt last =
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   643
		let val ll = length last
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   644
		    and lc = length choices
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   645
		in if !trace andalso ll<lc then
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   646
		    (writeln("PRUNING " ^ Int.toString(lc-ll) ^ " LEVELS"); 
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   647
		     last)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   648
		   else last
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   649
		end
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   650
	  fun pruneAux (last, _, _, []) = last
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   651
	    | pruneAux (last, ntrl, trl, ch' as (ntrl',nbrs',exn) :: choices) =
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   652
		if nbrs' < nbrs 
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   653
		then last  (*don't backtrack beyond first solution of goal*)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   654
		else if nbrs' > nbrs then pruneAux (last, ntrl, trl, choices)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   655
		else (* nbrs'=nbrs *)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   656
		     if clashVar nxtVars (ntrl-ntrl', trl) then last
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   657
		     else (*no clashes: can go back at least this far!*)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   658
			  pruneAux(choices, ntrl', List.drop(trl, ntrl-ntrl'), 
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   659
				   choices)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   660
  in  traceIt (pruneAux (choices, !ntrail, !trail, choices))  end;
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   661
2894
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
   662
fun nextVars ((br, lits, vars, lim) :: _) = map Var vars
2854
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   663
  | nextVars []                                 = [];
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   664
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   665
fun backtrack ((_, _, exn)::_) = raise exn
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   666
  | backtrack _                = raise PROVE;
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   667
2894
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
   668
(*Add the literal G, handling *Goal* and detecting duplicates.*)
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
   669
fun addLit (Const "*Goal*" $ G, lits) = 
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
   670
      (*New literal is a *Goal*, so change all other Goals to Nots*)
2854
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   671
      let fun bad (Const"*Goal*" $ _) = true
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   672
	    | bad (Const"Not" $ G')   = G aconv G'
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   673
	    | bad _                   = false;
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   674
	  fun change [] = []
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   675
	    | change (Const"*Goal*" $ G' :: lits) = 
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   676
		  if G aconv G' then change lits
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   677
		  else Const"Not" $ G' :: change lits
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   678
	    | change (Const"Not" $ G' :: lits)    = 
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   679
		  if G aconv G' then change lits
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   680
		  else Const"Not" $ G' :: change lits
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   681
	    | change (lit::lits) = lit :: change lits
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   682
      in
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   683
	Const "*Goal*" $ G :: (if exists bad lits then change lits else lits)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   684
      end
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   685
  | addLit (G,lits) = ins_term(G, lits)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   686
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   687
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   688
(*Tableau prover based on leanTaP.  Argument is a list of branches.  Each 
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   689
  branch contains a list of unexpanded formulae, a list of literals, and a 
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   690
  bound on unsafe expansions.*)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   691
fun prove (cs, brs, cont) =
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   692
 let val {safe0_netpair, safep_netpair, haz_netpair, ...} = Data.rep_claset cs
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   693
     val safeList = [safe0_netpair, safep_netpair]
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   694
     and hazList  = [haz_netpair]
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   695
     fun prv (tacs, trs, choices, []) = (cont (trs,choices,tacs))
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   696
       | prv (tacs, trs, choices, 
2894
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
   697
	      brs0 as (((G,md)::br, haz)::pairs, lits, vars, lim) :: brs) =
2854
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   698
	  let exception PRV (*backtrack to precisely this recursion!*)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   699
	      val ntrl = !ntrail 
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   700
	      val nbrs = length brs0
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   701
              val nxtVars = nextVars brs
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   702
	      val G = norm G
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   703
	      (*Make a new branch, decrementing "lim" if instantiations occur*)
2894
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
   704
	      fun newBr (vars',lim') prems =
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
   705
		  map (fn prem => 
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
   706
		       if (exists isGoal prem) 
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
   707
		       then (((joinMd md prem, []) :: 
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
   708
			      negOfGoals ((br, haz)::pairs)),
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
   709
			     map negOfGoal lits, 
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
   710
			     vars', lim') 
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
   711
		       else (((joinMd md prem, []) :: (br, haz) :: pairs),
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
   712
			     lits, vars', lim'))
2854
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   713
		  prems @
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   714
		  brs		  
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   715
	      (*Seek a matching rule.  If unifiable then add new premises
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   716
                to branch.*)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   717
	      fun deeper [] = raise NEWBRANCHES
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   718
		| deeper (((P,prems),tac)::grls) =
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   719
		    let val dummy = unify(add_term_vars(P,[]), P, G)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   720
			    (*P comes from the rule; G comes from the branch.*)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   721
                        val ntrl' = !ntrail
2894
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
   722
			val lim' = if ntrl < !ntrail then lim-3 else lim
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
   723
                        val vars  = vars_in_vars vars
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
   724
                        val vars' = foldr add_terms_vars (prems, vars)
2854
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   725
			val choices' = (ntrl, nbrs, PRV) :: choices
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   726
                    in
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   727
			if null prems then (*closed the branch: prune!*)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   728
			  prv(tac false :: tacs,	(*no duplication*)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   729
			      brs0::trs, 
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   730
			      prune (nbrs, nxtVars, choices'),
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   731
			      brs)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   732
			  handle PRV => 
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   733
			      (*reset Vars and try another rule*)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   734
			      (clearTo ntrl;  deeper grls)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   735
		        else 
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   736
			  prv(tac false :: tacs,	(*no duplication*)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   737
			      brs0::trs, choices',
2894
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
   738
			      newBr (vars',lim') prems)
2854
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   739
			  handle PRV => 
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   740
			      if ntrl < ntrl' then
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   741
				   (*Vars have been updated: must backtrack
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   742
				     even if not mentioned in other goals!
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   743
				     Reset Vars and try another rule*)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   744
				   (clearTo ntrl;  deeper grls)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   745
			      else (*backtrack to previous level*)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   746
				   backtrack choices
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   747
		    end
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   748
		    handle UNIFY => deeper grls
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   749
	      (*Try to close branch by unifying with head goal*)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   750
	      fun closeF [] = raise CLOSEF
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   751
		| closeF (L::Ls) = 
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   752
		    let val tacs' = tryClose(G,L)::tacs
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   753
			val choices' = prune (nbrs, nxtVars, 
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   754
					      (ntrl, nbrs, PRV) :: choices)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   755
		    in  prv (tacs', brs0::trs, choices', brs)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   756
			handle PRV => 
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   757
			    (*reset Vars and try another literal
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   758
			      [this handler is pruned if possible!]*)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   759
			 (clearTo ntrl;  closeF Ls)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   760
                    end
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   761
		    handle UNIFY => closeF Ls
2894
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
   762
	      fun closeFl [] = raise CLOSEF
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
   763
		| closeFl ((br, haz)::pairs) =
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
   764
		    closeF (map fst br)
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
   765
		      handle CLOSEF => closeF (map fst haz)
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
   766
			handle CLOSEF => closeFl pairs
2854
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   767
	  in if !trace then fullTrace := brs0 :: !fullTrace else ();
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   768
	     if lim<0 then backtrack choices
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   769
	     else
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   770
	     prv (Data.vars_gen_hyp_subst_tac false :: tacs, 
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   771
		  brs0::trs,  choices,
2894
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
   772
		  equalSubst (G, (br,haz)::pairs, lits, vars, lim) :: brs)
2854
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   773
	     handle DEST_EQ => closeF lits
2894
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
   774
	      handle CLOSEF => closeFl ((br,haz)::pairs)
2854
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   775
	        handle CLOSEF => 
2894
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
   776
		 deeper (netMkRules G vars safeList)
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
   777
		  handle NEWBRANCHES => 
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
   778
		   (case netMkRules G vars hazList of
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
   779
		       [] => (*no plausible rules: move G to literals*)
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
   780
			   prv (tacs, brs0::trs, choices,
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
   781
				((br,haz)::pairs, addLit(G,lits), vars, lim)
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
   782
				::brs)
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
   783
		    | _ => (*G admits some haz rules: try later*)
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
   784
			   prv (if isGoal G then negOfGoal_tac :: tacs
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
   785
				else tacs, 
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
   786
				brs0::trs,  choices,
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
   787
				((br, haz@[(negOfGoal G, md)])::pairs,
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
   788
				 lits, vars, lim)  ::  brs))
2854
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   789
	  end
2894
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
   790
       | prv (tacs, trs, choices, (([],haz)::(Gs,haz')::pairs, 
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
   791
				   lits, vars, lim) :: brs) =
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
   792
	     (*no more "safe" formulae: transfer haz down a level*)
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
   793
	   prv (tacs, trs, choices, ((Gs,haz@haz')::pairs, lits, vars, lim) 
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
   794
		:: brs)
2854
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   795
       | prv (tacs, trs, choices, 
2894
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
   796
	      brs0 as ([([], (H,md)::Hs)], lits, vars, lim) :: brs) =
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
   797
   	     (*no safe steps possible at any level: apply a haz rule*)
2854
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   798
	  let exception PRV (*backtrack to precisely this recursion!*)
2894
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
   799
	      val H = norm H
2854
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   800
	      val ntrl = !ntrail
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   801
	      fun newPrem (vars,dup) prem = 
2894
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
   802
		  ([(map (fn P => (P,false)) prem, []), (*may NOT duplicate*)
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
   803
		    ([], if dup then Hs @ [(negOfGoal H, md)] else Hs)],  
2854
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   804
		   lits,  
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   805
		   vars,  
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   806
		   (*Decrement "lim" if instantiations occur or the
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   807
		     formula is duplicated*)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   808
		   if ntrl < !ntrail then lim-3 
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   809
		   else if dup then lim-1 else lim)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   810
	      fun newBr x prems = map (newPrem x) prems  @  brs
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   811
	      (*Seek a matching rule.  If unifiable then add new premises
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   812
                to branch.*)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   813
	      fun deeper [] = raise NEWBRANCHES
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   814
		| deeper (((P,prems),tac)::grls) =
2894
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
   815
		    let val dummy = unify(add_term_vars(P,[]), P, H)
2854
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   816
			val ntrl' = !ntrail
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   817
                        val vars  = vars_in_vars vars
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   818
                        val vars' = foldr add_terms_vars (prems, vars)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   819
                        val dup = md andalso vars' <> vars
2894
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
   820
			(*duplicate H only if md and the premise has new vars*)
2854
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   821
                    in
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   822
		      prv(tac dup :: tacs, 
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   823
			  brs0::trs, 
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   824
			  (ntrl, length brs0, PRV) :: choices, 
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   825
			  newBr (vars', dup) prems)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   826
		     handle PRV => 
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   827
			 if ntrl < ntrl'       (*variables updated?*)
2883
fd1c0b8e9b61 Now exports declConsts!
paulson
parents: 2854
diff changeset
   828
                            orelse vars=vars'  (*pseudo-unsafe: no new Vars?*)
2854
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   829
			 then (*reset Vars and try another rule*)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   830
			      (clearTo ntrl;  deeper grls)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   831
			 else (*backtrack to previous level*)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   832
			      backtrack choices
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   833
		    end
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   834
		    handle UNIFY => deeper grls
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   835
	  in if !trace then fullTrace := brs0 :: !fullTrace else ();
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   836
	     if lim<1 then backtrack choices
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   837
	     else
2894
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
   838
	     deeper (netMkRules H vars hazList)
2854
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   839
	     handle NEWBRANCHES => 
2894
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
   840
		 (*cannot close branch: move H to literals*)
2854
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   841
		 prv (tacs,  brs0::trs,  choices,
2894
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
   842
		      ([([], Hs)], H::lits, vars, lim)::brs)
2854
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   843
	  end
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   844
       | prv (tacs, trs, choices, _ :: brs) = backtrack choices
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   845
 in prv ([], [], [(!ntrail, length brs, PROVE)], brs) end;
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   846
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   847
2883
fd1c0b8e9b61 Now exports declConsts!
paulson
parents: 2854
diff changeset
   848
(*Construct an initial branch.*)
2854
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   849
fun initBranch (ts,lim) = 
2894
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
   850
    ([(map (fn t => (t,true)) ts, [])],
d2ffee4f811b Re-organization of the order of haz rules
paulson
parents: 2883
diff changeset
   851
     [], add_terms_vars (ts,[]), lim);
2854
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   852
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   853
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   854
(*** Conversion & Skolemization of the Isabelle proof state ***)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   855
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   856
(*Make a list of all the parameters in a subgoal, even if nested*)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   857
local open Term 
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   858
in
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   859
fun discard_foralls (Const("all",_)$Abs(a,T,t)) = discard_foralls t
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   860
  | discard_foralls t = t;
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   861
end;
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   862
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   863
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   864
(*List of variables not appearing as arguments to the given parameter*)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   865
fun getVars []                  i = []
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   866
  | getVars ((_,(v,is))::alist) i =
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   867
	if i mem is then getVars alist i
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   868
	else v :: getVars alist i;
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   869
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   870
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   871
(*Conversion of a subgoal: Skolemize all parameters*)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   872
fun fromSubgoal tsig t =
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   873
  let val alist = ref []
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   874
      fun hdvar ((ix,(v,is))::_) = v
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   875
      fun from lev t =
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   876
	let val (ht,ts) = Term.strip_comb t
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   877
	    fun apply u = list_comb (u, map (from lev) ts)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   878
	    fun bounds [] = []
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   879
	      | bounds (Term.Bound i::ts) = 
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   880
		  if i<lev then error"Function Var's argument not a parameter"
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   881
		  else i-lev :: bounds ts
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   882
	      | bounds ts = error"Function Var's argument not a bound variable"
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   883
        in
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   884
	  case ht of 
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   885
	      t as Term.Const _ => apply (fromConst tsig t)	    
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   886
	    | Term.Free  (a,_) => apply (Free a)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   887
	    | Term.Bound i     => apply (Bound i)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   888
	    | Term.Var (ix,_) => 
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   889
		  (case (assoc_string_int(!alist,ix)) of
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   890
		       None => (alist := (ix, (ref None, bounds ts))
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   891
					  :: !alist;
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   892
				Var (hdvar(!alist)))
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   893
		     | Some(v,is) => if is=bounds ts then Var v
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   894
			    else error("Discrepancy among occurrences of ?"
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   895
				       ^ Syntax.string_of_vname ix))
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   896
	    | Term.Abs (a,_,body) => 
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   897
		  if null ts then Abs(a, from (lev+1) body)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   898
		  else error "fromSubgoal: argument not in normal form"
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   899
        end
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   900
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   901
      val npars = length (Logic.strip_params t)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   902
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   903
      (*Skolemize a subgoal from a proof state*)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   904
      fun skoSubgoal i t =
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   905
	  if i<npars then 
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   906
	      skoSubgoal (i+1)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   907
		(subst_bound (Skolem (gensym "SG_", getVars (!alist) i), 
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   908
			      t))
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   909
	  else t
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   910
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   911
  in  skoSubgoal 0 (from 0 (discard_foralls t))  end;
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   912
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   913
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   914
(*Tactic using tableau engine and proof reconstruction.  
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   915
 "lim" is depth limit.*)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   916
fun depth_tac cs lim i st = 
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   917
    (fullTrace:=[];  trail := [];  ntrail := 0;
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   918
     let val {tsig,...} = Sign.rep_sg (#sign (rep_thm st))
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   919
	 val skoprem = fromSubgoal tsig (List.nth(prems_of st, i-1))
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   920
         val hyps  = strip_imp_prems skoprem
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   921
         and concl = strip_imp_concl skoprem
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   922
         fun cont (_,choices,tacs) = 
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   923
	     (case Sequence.pull(EVERY' (rev tacs) i st) of
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   924
		  None => (writeln ("PROOF FAILED for depth " ^
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   925
				    Int.toString lim);
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   926
			   backtrack choices)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   927
		| cell => Sequence.seqof(fn()=> cell))
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   928
     in prove (cs, [initBranch (mkGoal concl :: hyps, lim)], cont)
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   929
     end
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   930
     handle Subscript => Sequence.null
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   931
	  | PROVE     => Sequence.null);
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   932
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   933
fun blast_tac cs = (DEEPEN (1,20) (depth_tac cs) 0);
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   934
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   935
fun Blast_tac i = blast_tac (!Data.claset) i;
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   936
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   937
end;
f03b1652fc6a Implementation of blast_tac: fast tableau prover
paulson
parents:
diff changeset
   938