]> matita.cs.unibo.it Git - helm.git/blobdiff - matita/matita/contribs/lambdadelta/basic_2/reduction/cnr.ma
- name changes in the rediction rules
[helm.git] / matita / matita / contribs / lambdadelta / basic_2 / reduction / cnr.ma
index e0e84742f9c9668328d5ce8886536bf9b90a21af..d68be168026e618aa715a8ce8f09a25961ff8b26 100644 (file)
@@ -69,9 +69,9 @@ lemma cnr_inv_appl: ∀G,L,V,T. ⦃G, L⦄ ⊢ ➡ 𝐍⦃ⓐV.T⦄ → ∧∧ 
 ]
 qed-.
 
-lemma cnr_inv_tau: ∀G,L,V,T. ⦃G, L⦄ ⊢ ➡ 𝐍⦃ⓝV.T⦄ → ⊥.
+lemma cnr_inv_eps: ∀G,L,V,T. ⦃G, L⦄ ⊢ ➡ 𝐍⦃ⓝV.T⦄ → ⊥.
 #G #L #V #T #H lapply (H T ?) -H
-/2 width=4 by cpr_tau, discr_tpair_xy_y/
+/2 width=4 by cpr_eps, discr_tpair_xy_y/
 qed-.
 
 (* Basic properties *********************************************************)