diff -r 851c90b23a9e -r ea13ff5a26d1 src/HOL/UNITY/Comp/TimerArray.thy --- /dev/null Thu Jan 01 00:00:00 1970 +0000 +++ b/src/HOL/UNITY/Comp/TimerArray.thy Mon Mar 05 15:32:54 2001 +0100 @@ -0,0 +1,23 @@ +(* Title: HOL/UNITY/TimerArray.thy + ID: $Id$ + Author: Lawrence C Paulson, Cambridge University Computer Laboratory + Copyright 1998 University of Cambridge + +A trivial example of reasoning about an array of processes +*) + +TimerArray = PPROD + + +types 'a state = "nat * 'a" (*second component allows new variables*) + +constdefs + count :: "'a state => nat" + "count s == fst s" + + decr :: "('a state * 'a state) set" + "decr == UN n uu. {((Suc n, uu), (n,uu))}" + + Timer :: 'a state program + "Timer == mk_program (UNIV, {decr}, UNIV)" + +end