src/ZF/IMP/Assign.ML
author clasohm
Thu, 23 Mar 1995 15:39:13 +0100
changeset 971 f4815812665b
parent 482 3a4e092ba69c
permissions -rw-r--r--
fixed bug: parent theory wasn't loaded if .thy file was completly read before (regardless of the .ML file)

(*  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)]);