lemma
authorhaftmann
Thu, 11 Mar 2021 07:05:29 +0000
changeset 73410 7b59d2945e54
parent 73409 fbd69f277699
child 73411 1f1366966296
lemma
src/HOL/Library/Permutations.thy
--- a/src/HOL/Library/Permutations.thy	Thu Mar 11 11:22:25 2021 +0100
+++ b/src/HOL/Library/Permutations.thy	Thu Mar 11 07:05:29 2021 +0000
@@ -62,6 +62,10 @@
 lemma permutes_subset: "p permutes S \<Longrightarrow> S \<subseteq> T \<Longrightarrow> p permutes T"
   unfolding permutes_def by blast
 
+lemma permutes_imp_permutes_insert:
+  \<open>p permutes insert x S\<close> if \<open>p permutes S\<close>
+  using that by (rule permutes_subset) auto
+
 lemma permutes_empty[simp]: "p permutes {} \<longleftrightarrow> p = id"
   by (auto simp add: fun_eq_iff permutes_def)