src/HOL/Library/Sublist.thy
changeset 67614 560fbd6bc047
parent 67612 e4e57da0583a
parent 67613 ce654b0e6d69
child 68406 6beb45f6cf67
--- a/src/HOL/Library/Sublist.thy	Wed Feb 14 16:32:09 2018 +0100
+++ b/src/HOL/Library/Sublist.thy	Thu Feb 15 13:04:36 2018 +0100
@@ -298,7 +298,7 @@
   (is "_ \<Longrightarrow> \<exists>ps. ?P L ps")
 proof(induction "LEAST n. \<exists>xs \<in>L. n = length xs" arbitrary: L)
   case 0
-  have "[] : L" using "0.hyps" LeastI[of "\<lambda>n. \<exists>xs\<in>L. n = length xs"] \<open>L \<noteq> {}\<close>
+  have "[] \<in> L" using "0.hyps" LeastI[of "\<lambda>n. \<exists>xs\<in>L. n = length xs"] \<open>L \<noteq> {}\<close>
     by auto
   hence "?P L []" by(auto)
   thus ?case ..