]> matita.cs.unibo.it Git - helm.git/blobdiff - matita/matita/contribs/lambda_delta/basic_2/grammar/lenv_weight.ma
- some work on context equivalence of atomic arity assignment
[helm.git] / matita / matita / contribs / lambda_delta / basic_2 / grammar / lenv_weight.ma
index 990b5c5d07639c7d2060638967778e39e130461a..48ef29453580c3c168a8bcbe60d981de54056a0f 100644 (file)
@@ -24,5 +24,16 @@ let rec lw L ≝ match L with
 
 interpretation "weight (local environment)" 'Weight L = (lw L).
 
+(* Basic properties *********************************************************)
+
+lemma lw_pair: ∀I,L,V. #[L] < #[(L.ⓑ{I}V)].
+/3 width=1/ qed.
+
+(* Basic eliminators ********************************************************)
+
+axiom lw_wf_ind: ∀R:predicate lenv.
+                 (∀L2. (∀L1. #[L1] < #[L2] → R L1) → R L2) →
+                 ∀L. R L.
+
 (* Basic_1: removed theorems 2: clt_cong clt_head clt_thead *)
 (* Basic_1: note: clt_thead should be renamed clt_ctail *)