diff -r 827cac8abecc -r 026e7c6a6d08 src/HOL/UNITY/Simple/Common.thy --- a/src/HOL/UNITY/Simple/Common.thy Mon Sep 21 16:11:36 2009 +0200 +++ b/src/HOL/UNITY/Simple/Common.thy Tue Sep 22 15:36:55 2009 +0200 @@ -1,5 +1,4 @@ (* Title: HOL/UNITY/Common - ID: $Id$ Author: Lawrence C Paulson, Cambridge University Computer Laboratory Copyright 1998 University of Cambridge @@ -10,7 +9,9 @@ From Misra, "A Logic for Concurrent Programming" (1994), sections 5.1 and 13.1. *) -theory Common imports "../UNITY_Main" begin +theory Common +imports "../UNITY_Main" +begin consts ftime :: "nat=>nat" @@ -65,7 +66,7 @@ lemma "mk_total_program (UNIV, {range(%t.(t, max (ftime t) (gtime t)))}, UNIV) \ {m} co (maxfg m)" apply (simp add: mk_total_program_def) -apply (simp add: constrains_def maxfg_def gasc) +apply (simp add: constrains_def maxfg_def gasc min_max.sup_absorb2) done (*This one is t := t+1 if t {m} co (maxfg m)" apply (simp add: mk_total_program_def) -apply (simp add: constrains_def maxfg_def gasc) +apply (simp add: constrains_def maxfg_def gasc min_max.sup_absorb2) done