src/HOL/IMP/Denotation.ML
author nipkow
Tue, 23 Jan 1996 10:59:35 +0100
changeset 1447 bc2c0acbbf29
parent 1266 3ae9fe3c0f68
child 1465 5d7a7e439cec
permissions -rw-r--r--
Added a verified verification-condition generator.

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