src/HOL/TLA/Stfun.ML
author wenzelm
Mon, 08 Feb 1999 13:02:56 +0100
changeset 6255 db63752140c7
parent 4089 96fba19bcbe2
child 12607 16b63730cfbb
permissions -rw-r--r--
updated (Stephan Merz);

(* 
    File:	 Stfun.ML
    Author:      Stephan Merz
    Copyright:   1998 University of Munich

Lemmas and tactics for states and state functions.
*)

(*  [| basevars v; !!x. v x = c ==> Q |] ==> Q  *)
bind_thm("baseE", (standard (basevars RS exE)));

(* -------------------------------------------------------------------------------
   The following shows that there should not be duplicates in a "stvars" tuple:

Goal "!!v. basevars (v::bool stfun, v) ==> False";
by (etac baseE 1);
by (subgoal_tac "(LIFT (v,v)) x = (True, False)" 1); 
by (atac 2);
by (Asm_full_simp_tac 1);

------------------------------------------------------------------------------- *)