]> matita.cs.unibo.it Git - helm.git/blobdiff - matita/matita/contribs/lambdadelta/basic_2/grammar/lenv_weight.ma
xoa: change in naming convenctions for existential quantifies
[helm.git] / matita / matita / contribs / lambdadelta / basic_2 / grammar / lenv_weight.ma
index 59e2e6172bc24a83e79d60cdb537e2e403087cae..537d32e5611f2e0ce975080963469a13a36df74a 100644 (file)
@@ -29,11 +29,5 @@ interpretation "weight (local environment)" 'Weight L = (lw L).
 lemma lw_pair: ∀I,L,V. #{L} < #{(L.ⓑ{I}V)}.
 /3 width=1/ qed.
 
-(* Basic eliminators ********************************************************)
-
-axiom lw_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 *)