merged
authornipkow
Wed, 08 Nov 2023 21:45:02 +0100
changeset 78923 ab85d87dc2be
parent 78921 2fee5fba3116 (current diff)
parent 78922 9e43ab263d33 (diff)
child 78924 0481c84f6919
merged
--- a/src/HOL/Library/NList.thy	Wed Nov 08 20:31:29 2023 +0100
+++ b/src/HOL/Library/NList.thy	Wed Nov 08 21:45:02 2023 +0100
@@ -20,6 +20,9 @@
 lemma nlistsE_length [simp]: "xs \<in> nlists n A \<Longrightarrow> size xs = n"
   by (simp add: nlists_def)
 
+lemma in_nlists_UNIV: "xs \<in> nlists k UNIV \<longleftrightarrow> length xs = k"
+unfolding nlists_def by(auto)
+
 lemma less_lengthI: "\<lbrakk> xs \<in> nlists n A; p < n \<rbrakk> \<Longrightarrow> p < size xs"
 by (simp)