diff -r e13df75fee79 -r 9546828c0eb3 src/HOL/SPARK/Examples/Liseq/Longest_Increasing_Subsequence.thy --- a/src/HOL/SPARK/Examples/Liseq/Longest_Increasing_Subsequence.thy Sun Jan 16 15:26:47 2011 +0100 +++ b/src/HOL/SPARK/Examples/Liseq/Longest_Increasing_Subsequence.thy Sun Jan 16 15:31:22 2011 +0100 @@ -161,7 +161,7 @@ with assms have "Max js < i" by (auto simp add: iseq_def) with fin assms have "\j\js. j < i" - by (simp add: Max_less_iff) + by simp with assms show ?thesis by (simp add: iseq_def) qed