]> matita.cs.unibo.it Git - helm.git/blobdiff - matita/matita/lib/basics/list.ma
support for candidates of reducibility started ...
[helm.git] / matita / matita / lib / basics / list.ma
index 21dd7e3d1aa57597da06b06b7ba2c1c192b84be2..eaf89510a153c2f90e67c23c45caccf93a09f9d0 100644 (file)
@@ -72,7 +72,7 @@ ntheorem cons_append_commute:
 //; nqed. *)
 
 theorem append_cons:∀A.∀a:A.∀l,l1.l@(a::l1)=(l@[a])@l1.
-/2/ qed.
+#A #a #l #l1 >associative_append // qed.
 
 theorem nil_append_elim: ∀A.∀l1,l2: list A.∀P:?→?→Prop. 
   l1@l2=[] → P (nil A) (nil A) → P l1 l2.
@@ -214,5 +214,5 @@ qed.
 
 lemma length_ltl: ∀A,n,l. |ltl A l n| = |l| - n.
 #A #n elim n -n /2/
-#n #IHn * normalize /2/
+#n #IHn *; normalize /2/
 qed.