]> matita.cs.unibo.it Git - helm.git/blobdiff - matita/matita/contribs/lambdadelta/basic_2/reduction/cpr_cir.ma
some notation renamed and fixed
[helm.git] / matita / matita / contribs / lambdadelta / basic_2 / reduction / cpr_cir.ma
index d0e1e19ac6f525b691b00d2b50880b56aed233c9..99846d67ac4bafc17ee4a1f103b340d0d2ccd0f1 100644 (file)
@@ -17,7 +17,7 @@ include "basic_2/reduction/cpr.ma".
 
 (* CONTEXT-SENSITIVE PARALLEL REDUCTION FOR TERMS ***************************)
 
-(* Advanced forward lemmas on context-sensitive irreducible terms ***********)
+(* Advanced forward lemmas on irreducibility ********************************)
 
 lemma cpr_fwd_cir: ∀G,L,T1,T2. ⦃G, L⦄ ⊢ T1 ➡ T2 → ⦃G, L⦄ ⊢ ➡ 𝐈⦃T1⦄ → T2 = T1.
 #G #L #T1 #T2 #H elim H -G -L -T1 -T2