src/HOL/MicroJava/DFA/SemilatAlg.thy
changeset 67613 ce654b0e6d69
parent 61994 133a8a888ae8
child 68249 949d93804740
--- a/src/HOL/MicroJava/DFA/SemilatAlg.thy	Tue Feb 13 14:24:50 2018 +0100
+++ b/src/HOL/MicroJava/DFA/SemilatAlg.thy	Thu Feb 15 12:11:00 2018 +0100
@@ -18,7 +18,7 @@
 | "(x#xs) ++_f y = xs ++_f (x +_f y)"
 
 definition bounded :: "'s step_type \<Rightarrow> nat \<Rightarrow> bool" where
-"bounded step n == !p<n. !s. !(q,t):set(step p s). q<n"  
+"bounded step n == \<forall>p<n. \<forall>s. \<forall>(q,t)\<in>set(step p s). q<n"  
 
 definition pres_type :: "'s step_type \<Rightarrow> nat \<Rightarrow> 's set \<Rightarrow> bool" where
 "pres_type step n A == \<forall>s\<in>A. \<forall>p<n. \<forall>(q,s')\<in>set (step p s). s' \<in> A"
@@ -36,7 +36,7 @@
   by (unfold mono_def, blast)
 
 lemma boundedD: 
-  "\<lbrakk> bounded step n; p < n; (q,t) : set (step p xs) \<rbrakk> \<Longrightarrow> q < n" 
+  "\<lbrakk> bounded step n; p < n; (q,t) \<in> set (step p xs) \<rbrakk> \<Longrightarrow> q < n" 
   by (unfold bounded_def, blast)
 
 lemma lesubstep_type_refl [simp, intro]: