]> matita.cs.unibo.it Git - helm.git/blobdiff - matita/matita/lib/basics/lists/listb.ma
FinOpt
[helm.git] / matita / matita / lib / basics / lists / listb.ma
index 640f1391cc469e515b2e16f1b73917ed3dad5e5e..ac72b008bee54237a9360bb2830545ab5ec7b853 100644 (file)
@@ -103,6 +103,15 @@ lemma memb_compose: ∀S1,S2,S3,op,a1,a2,l1,l2.
   ]
 qed.
 
+lemma mem_to_memb: ∀S:DeqSet.∀a,l. mem S a l → memb S a l = true.
+#S #a #l elim l normalize
+  [@False_ind
+  |#hd #tl #Hind *
+    [#eqa >(\b eqa) %
+    |#Hmem cases (a==hd) // normalize /2/
+    ]
+  ]
+qed.
 (**************** unicity test *****************)
 
 let rec uniqueb (S:DeqSet) l on l : bool ≝