]> matita.cs.unibo.it Git - helm.git/blobdiff - matita/matita/contribs/lambdadelta/basic_2/reducibility/cpr.ma
commit completed! some bugs fixed and some instances of auto resized
[helm.git] / matita / matita / contribs / lambdadelta / basic_2 / reducibility / cpr.ma
index 22fbfc148440b49c722985a6ae9a518598942845..fffaad09885f4efc87d7786831839ed4ec902f83 100644 (file)
@@ -28,7 +28,7 @@ interpretation
 (* Basic properties *********************************************************)
 
 lemma cpr_intro: ∀L,T1,T,T2,d,e. T1 ➡ T → L ⊢ T ▶* [d, e] T2 → L ⊢ T1 ➡ T2.
-/4 width=3/ qed-.
+/3 width=5/ qed-.
 
 (* Basic_1: was by definition: pr2_free *)
 lemma cpr_tpr: ∀T1,T2. T1 ➡ T2 → ∀L. L ⊢ T1 ➡ T2.