src/HOL/Library/Dlist.thy
changeset 40122 1d8ad2ff3e01
parent 39915 ecf97cf3d248
child 40603 963ee2331d20
--- a/src/HOL/Library/Dlist.thy	Mon Oct 25 13:34:57 2010 +0200
+++ b/src/HOL/Library/Dlist.thy	Mon Oct 25 13:34:58 2010 +0200
@@ -143,11 +143,11 @@
   proof (induct xs)
     case Nil from empty show ?case by (simp add: empty_def)
   next
-    case (insert x xs)
+    case (Cons x xs)
     then have "\<not> member (Dlist xs) x" and "P (Dlist xs)"
       by (simp_all add: member_def List.member_def)
     with insrt have "P (insert x (Dlist xs))" .
-    with insert show ?case by (simp add: insert_def distinct_remdups_id)
+    with Cons show ?case by (simp add: insert_def distinct_remdups_id)
   qed
   with dxs show "P dxs" by simp
 qed