fixed dodgy intro! attributes
authorpaulson <lp15@cam.ac.uk>
Tue, 25 Jan 2022 14:13:33 +0000
changeset 75008 43b3d5318d72
parent 75007 2e16798b6f2b
child 75009 d2f97439f53e
fixed dodgy intro! attributes
src/HOL/Library/More_List.thy
--- a/src/HOL/Library/More_List.thy	Tue Jan 25 09:57:44 2022 +0100
+++ b/src/HOL/Library/More_List.thy	Tue Jan 25 14:13:33 2022 +0000
@@ -91,11 +91,11 @@
 where
   "no_leading P xs \<longleftrightarrow> (xs \<noteq> [] \<longrightarrow> \<not> P (hd xs))"
 
-lemma no_leading_Nil [simp, intro!]:
+lemma no_leading_Nil [iff]:
   "no_leading P []"
   by (simp add: no_leading_def)
 
-lemma no_leading_Cons [simp, intro!]:
+lemma no_leading_Cons [iff]:
   "no_leading P (x # xs) \<longleftrightarrow> \<not> P x"
   by (simp add: no_leading_def)
 
@@ -148,7 +148,7 @@
   "no_trailing P xs \<longleftrightarrow> (xs \<noteq> [] \<longrightarrow> \<not> P (last xs))"
   by (induct xs) simp_all
 
-lemma no_trailing_Nil [simp, intro!]:
+lemma no_trailing_Nil [iff]:
   "no_trailing P []"
   by simp