src/HOL/IMP/Denotation.ML
author lcp
Tue, 25 Apr 1995 11:14:03 +0200
changeset 1072 0140ff702b23
parent 924 806721cfbf46
child 1266 3ae9fe3c0f68
permissions -rw-r--r--
updated version

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

open Denotation;

(**** Rewrite Rules for A,B,C ****)

val A_simps =
     [A_nat,A_loc,A_op1,A_op2];

val B_simps = map (fn t => t RS eq_reflection)
     [B_true,B_false,B_op,B_not,B_and,B_or]

val C_simps = map (fn t => t RS eq_reflection)
  [C_skip,C_assign,C_comp,C_if,C_while]; 

(**** mono (Gamma(b,c)) ****)

qed_goalw "Gamma_mono" Denotation.thy [mono_def,Gamma_def]
	"mono (Gamma b c)"
     (fn _ => [(best_tac comp_cs 1)]);