]> matita.cs.unibo.it Git - helm.git/blobdiff - matita/matita/contribs/lambdadelta/ground/arith/arith_2a.ma
milestone update in ground
[helm.git] / matita / matita / contribs / lambdadelta / ground / arith / arith_2a.ma
index b5ff26116ef36e2b41f8e3c4abd9a51fc374f45c..92224c4c9560d1f51b5c54e52c144fda38b2ec00 100644 (file)
@@ -87,7 +87,7 @@ lemma lt_plus_SO_to_le: ∀x,y. x < y + (𝟏) → x ≤ y.
 
 (* Iterators ****************************************************************)
 
-lemma iter_SO: ∀B:Type[0]. ∀f:B→B. ∀b,l. f^(l+𝟏) b = f (f^l b).
+lemma iter_SO: ∀B:Type[0]. ∀f:B→B. ∀b,l. (f^(l+𝟏)) b = f ((f^l) b).
 #B #f #b #l
 <niter_succ //
 qed.