src/ZF/IMP/Assign.ML
author paulson
Fri, 10 Apr 1998 13:15:28 +0200
changeset 4804 02b7c759159b
parent 482 3a4e092ba69c
permissions -rw-r--r--
Fixed bug in inductive sections to allow disjunctive premises; added tracing flag trace_induct

(*  Title: 	ZF/IMP/Assign.ML
    ID:         $Id$
    Author: 	Heiko Loetzbeyer & Robert Sandner, TUM
    Copyright   1994 TUM
*)

open Assign;

val assign_type = prove_goalw Assign.thy [assign_def]
	"[| sigma:loc -> nat; n:nat |] ==> sigma[n/x] : loc -> nat"
    (fn prems => [(fast_tac  
                   (ZF_cs addIs [apply_type,lam_type,if_type]@prems) 1)]);