lemma dlist_ext
authorhaftmann
Thu, 22 Apr 2010 09:30:36 +0200
changeset 36274 42bd879dc1b0
parent 36273 283c84ee7db9
child 36275 c6ca9e258269
lemma dlist_ext
src/HOL/Library/Dlist.thy
--- a/src/HOL/Library/Dlist.thy	Wed Apr 21 21:11:26 2010 +0200
+++ b/src/HOL/Library/Dlist.thy	Thu Apr 22 09:30:36 2010 +0200
@@ -47,6 +47,11 @@
   show "[] \<in> ?dlist" by simp
 qed
 
+lemma dlist_ext:
+  assumes "list_of_dlist xs = list_of_dlist ys"
+  shows "xs = ys"
+  using assms by (simp add: list_of_dlist_inject)
+
 
 text {* Formal, totalized constructor for @{typ "'a dlist"}: *}