src/HOL/UNITY/Guar.thy
changeset 46577 e5438c5797ae
parent 45477 11d9c2768729
child 58889 5b7a9633cfa8
--- a/src/HOL/UNITY/Guar.thy	Tue Feb 21 17:08:32 2012 +0100
+++ b/src/HOL/UNITY/Guar.thy	Tue Feb 21 17:09:17 2012 +0100
@@ -17,7 +17,7 @@
 begin
 
 instance program :: (type) order
-proof qed (auto simp add: program_less_le dest: component_antisym intro: component_refl component_trans)
+  by default (auto simp add: program_less_le dest: component_antisym intro: component_trans)
 
 text{*Existential and Universal properties.  I formalize the two-program
       case, proving equivalence with Chandy and Sanders's n-ary definitions*}