src/HOL/SVC_Oracle.ML
author paulson
Tue, 03 Aug 1999 13:15:54 +0200
changeset 7165 8c937127fd8c
parent 7162 8737390d1d0a
child 7187 676027b1d770
permissions -rw-r--r--
new examples file for SVC

(*  Title:      HOL/SVC_Oracle
    ID:         $Id$
    Author:     Lawrence C Paulson
    Copyright   1999  University of Cambridge

Installing the oracle for SVC (Stanford Validity Checker)

Based upon the work of Søren T. Heilmann
*)

(*Present the entire subgoal to the oracle, assumptions and all, but possibly
  abstracted.  Use via compose_tac, which performs no lifting but will
  instantiate variables.*)
fun svc_tac i st = 
  let val prem = List.nth (prems_of st, i-1)
      val th = invoke_oracle thy "svc_oracle" 
	             (#sign (rep_thm st), Svc.OracleExn prem)
   in 
      compose_tac (false, th, 0) i st
   end 
   handle Svc.OracleExn _ => Seq.empty
	| Subscript       => Seq.empty;