X-Git-Url: http://matita.cs.unibo.it/gitweb/?a=blobdiff_plain;ds=inline;f=matita%2Fmatita%2Fcontribs%2Flambda%2Fterm.ma;h=92a838fb4cbe8b8f3bccdef807e66a817f20b307;hb=5ca47b58902b9f2583ad1354b860c04ea62df46c;hp=660830d2784222dac9bc681e15b5d144aaf24edc;hpb=2199f327081f49b21bdcd23d702b5e07ea4f58ce;p=helm.git diff --git a/matita/matita/contribs/lambda/term.ma b/matita/matita/contribs/lambda/term.ma index 660830d27..92a838fb4 100644 --- a/matita/matita/contribs/lambda/term.ma +++ b/matita/matita/contribs/lambda/term.ma @@ -18,11 +18,11 @@ include "preamble.ma". (* TERM STRUCTURE ***********************************************************) -(* Policy: term metavariables: A, B, C, D, M, N - de Bruijn indexes : i, j +(* Policy: term metavariables : A, B, C, D, M, N + depth metavariables: i, j *) inductive term: Type[0] ≝ -| VRef: nat → term (* variable reference by index *) +| VRef: nat → term (* variable reference by depth *) | Abst: term → term (* function formation *) | Appl: term → term → term (* function application *) . @@ -47,7 +47,7 @@ notation "hvbox( 𝛌 . term 46 A )" notation "hvbox( @ term 46 C . break term 46 A )" non associative with precedence 46 for @{ 'Application $C $A }. - +(* definition appl_compatible_dx: predicate (relation term) ≝ λR. ∀B,A1,A2. R A1 A2 → R (@B.A1) (@B.A2). @@ -55,3 +55,4 @@ lemma star_appl_compatible_dx: ∀R. appl_compatible_dx R → appl_compatible_dx (star … R). #R #HR #B #A1 #A2 #H elim H -A2 // /3 width=3/ qed. +*)