X-Git-Url: http://matita.cs.unibo.it/gitweb/?p=helm.git;a=blobdiff_plain;f=matita%2Fmatita%2Fcontribs%2Flambdadelta%2Fground%2Farith%2Farith_2a.ma;h=a136174bc8b209fc0c813c013b3382cdca587938;hp=b5ff26116ef36e2b41f8e3c4abd9a51fc374f45c;hb=48cd63fc7f4415925582eae224a36a9c1bb3cc06;hpb=888840f6b3a71d3d686b53b702d362ab90ab0038 diff --git a/matita/matita/contribs/lambdadelta/ground/arith/arith_2a.ma b/matita/matita/contribs/lambdadelta/ground/arith/arith_2a.ma index b5ff26116..a136174bc 100644 --- a/matita/matita/contribs/lambdadelta/ground/arith/arith_2a.ma +++ b/matita/matita/contribs/lambdadelta/ground/arith/arith_2a.ma @@ -12,16 +12,12 @@ (* *) (**************************************************************************) -include "ground/notation/functions/two_0.ma". +include "ground/arith/pnat_two.ma". include "ground/arith/nat_le_minus_plus.ma". include "ground/arith/nat_lt.ma". (* ARITHMETICAL PROPERTIES FOR λδ-2A ****************************************) -interpretation - "zero (non-negative integers)" - 'Two = (ninj (psucc punit)). - (* Equalities ***************************************************************) lemma plus_n_2: ∀n. (n + 𝟐) = n + 𝟏 + 𝟏. @@ -87,7 +83,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