src/HOL/UNITY/Comp/Priority.thy
changeset 46911 6d2a2f0e904e
parent 45600 1bbbac9a0cb0
child 57492 74bf65a1910a
--- a/src/HOL/UNITY/Comp/Priority.thy	Tue Mar 13 21:17:37 2012 +0100
+++ b/src/HOL/UNITY/Comp/Priority.thy	Tue Mar 13 22:49:02 2012 +0100
@@ -143,16 +143,12 @@
 
 
 text{* p15: universal property: all Components well behave  *}
-lemma system_well_behaves [rule_format]:
-     "\<forall>i. system \<in> Highest i co Highest i Un Lowest i"
-apply clarify
-apply (simp add: system_def Component_def mk_total_program_def totalize_JN, 
-       safety, auto)
-done
+lemma system_well_behaves: "system \<in> Highest i co Highest i Un Lowest i"
+  by (simp add: system_def Component_def mk_total_program_def totalize_JN, safety, auto)
 
 
 lemma Acyclic_eq: "Acyclic = (\<Inter>i. {s. i\<notin>above i s})"
-by (auto simp add: Acyclic_def acyclic_def trancl_converse)
+  by (auto simp add: Acyclic_def acyclic_def trancl_converse)
 
 
 lemmas system_co =