src/HOL/UNITY/Comp/TimerArray.thy
changeset 35416 d8d7d1b785af
parent 18556 dc39832e9280
child 36866 426d5781bb25
--- a/src/HOL/UNITY/Comp/TimerArray.thy	Wed Feb 24 11:55:52 2010 +0100
+++ b/src/HOL/UNITY/Comp/TimerArray.thy	Mon Mar 01 13:40:23 2010 +0100
@@ -1,5 +1,4 @@
 (*  Title:      HOL/UNITY/TimerArray.thy
-    ID:         $Id$
     Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
     Copyright   1998  University of Cambridge
 
@@ -10,14 +9,13 @@
 
 types 'a state = "nat * 'a"   (*second component allows new variables*)
 
-constdefs
-  count  :: "'a state => nat"
+definition count :: "'a state => nat" where
     "count s == fst s"
   
-  decr  :: "('a state * 'a state) set"
+definition decr  :: "('a state * 'a state) set" where
     "decr == UN n uu. {((Suc n, uu), (n,uu))}"
   
-  Timer :: "'a state program"
+definition Timer :: "'a state program" where
     "Timer == mk_total_program (UNIV, {decr}, UNIV)"