src/HOL/UNITY/Comp/TimerArray.thy
changeset 61943 7fba644ed827
parent 42463 f270e3e18be5
child 67613 ce654b0e6d69
--- a/src/HOL/UNITY/Comp/TimerArray.thy	Sun Dec 27 21:46:36 2015 +0100
+++ b/src/HOL/UNITY/Comp/TimerArray.thy	Sun Dec 27 22:07:17 2015 +0100
@@ -42,7 +42,7 @@
 lemma TimerArray_leadsTo_zero:
      "finite I  
       ==> (plam i: I. Timer) : UNIV leadsTo {(s,uu). ALL i:I. s i = 0}"
-apply (erule_tac A'1 = "%i. lift_set i ({0} <*> UNIV)" 
+apply (erule_tac A'1 = "%i. lift_set i ({0} \<times> UNIV)" 
        in finite_stable_completion [THEN leadsTo_weaken])
 apply auto
 (*Safety property, already reduced to the single Timer case*)
@@ -51,7 +51,7 @@
 (*Progress property for the array of Timers*)
 apply (rule_tac f = "sub i o fst" in lessThan_induct)
 apply (case_tac "m")
-(*Annoying need to massage the conditions to have the form (... <*> UNIV)*)
+(*Annoying need to massage the conditions to have the form (... \<times> UNIV)*)
 apply (auto intro: subset_imp_leadsTo 
         simp add: insert_absorb 
                   lift_set_Un_distrib [symmetric] lessThan_Suc [symmetric]