]> matita.cs.unibo.it Git - helm.git/blobdiff - matita/matita/contribs/lambdadelta/basic_2/grammar/lenv_weight.ma
- new syntax for let rec/corec with flavor specifier (tested on lambdadelta/ground_2/)
[helm.git] / matita / matita / contribs / lambdadelta / basic_2 / grammar / lenv_weight.ma
index 537d32e5611f2e0ce975080963469a13a36df74a..c9d79e5f5195ffc74e9ee8445b531b8c62f8a6c6 100644 (file)
@@ -17,17 +17,18 @@ include "basic_2/grammar/lenv.ma".
 
 (* WEIGHT OF A LOCAL ENVIRONMENT ********************************************)
 
-let rec lw L ≝ match L with
+rec definition lw L ≝ match L with
 [ LAtom       ⇒ 0
-| LPair L _ V ⇒ lw L + #{V}
+| LPair L _ V ⇒ lw L + {V}
 ].
 
 interpretation "weight (local environment)" 'Weight L = (lw L).
 
 (* Basic properties *********************************************************)
 
-lemma lw_pair: ∀I,L,V. #{L} < #{(L.ⓑ{I}V)}.
-/3 width=1/ qed.
+lemma lw_pair: ∀I,L,V. ♯{L} < ♯{L.ⓑ{I}V}.
+/3 width=1 by lt_plus_to_minus_r, monotonic_lt_plus_r/ qed.
 
-(* Basic_1: removed theorems 2: clt_cong clt_head clt_thead *)
+(* Basic_1: removed theorems 4: clt_cong clt_head clt_thead clt_wf_ind *)
+(* Basic_1: removed local theorems 1: clt_wf__q_ind *)
 (* Basic_1: note: clt_thead should be renamed clt_ctail *)