src/HOL/UNITY/TimerArray.thy
author wenzelm
Thu, 14 Oct 1999 15:03:34 +0200
changeset 7865 d9be8bc5624e
parent 7537 875754b599df
child 8251 9be357df93d4
permissions -rw-r--r--
support thumbpdf (via 'png' output format);

(*  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 +

constdefs
  decr  :: "(nat*nat) set"
    "decr == UN n. {(Suc n, n)}"
  
  Timer :: nat program
    "Timer == mk_program (UNIV, {decr})"

end