]> matita.cs.unibo.it Git - helm.git/blobdiff - helm/software/matita/library/list/list.ma
Dummy dependent types are no longer cleaned in inductive type arities.
[helm.git] / helm / software / matita / library / list / list.ma
index a180cbabc8b5d4dfcd7a6d0aea16440adde1ef97..ad44bd63a287846d917a08d278b57f01378fd205 100644 (file)
@@ -186,13 +186,13 @@ qed.
 
 lemma eq_map : ∀A,B,f,g,l. (∀x.f x = g x) → map A B f l = map A B g l.
 intros (A B f g l Efg); elim l; simplify; [1: reflexivity ];
-rewrite > (Efg t); rewrite > H; reflexivity;  
+rewrite > (Efg a); rewrite > H; reflexivity;  
 qed.
 
 lemma le_length_filter : \forall A,l,p.length A (filter A l p) \leq length A l.
 intros;elim l
   [simplify;apply le_n
-  |simplify;apply (bool_elim ? (p t));intro
+  |simplify;apply (bool_elim ? (p a));intro
      [simplify;apply le_S_S;assumption
      |simplify;apply le_S;assumption]]
 qed.
\ No newline at end of file