]> matita.cs.unibo.it Git - helm.git/blobdiff - matita/matita/contribs/lambda_delta/basic_2/reducibility/cpr_lift.ma
- nDestructTac: Sys.break handled in two places
[helm.git] / matita / matita / contribs / lambda_delta / basic_2 / reducibility / cpr_lift.ma
index 120946cb1bd483f723e0a1d49dd90717f32f6e37..dedb174e6e4b72c3dafa91e0fea2c14c039f3407 100644 (file)
@@ -88,7 +88,7 @@ elim (tpr_inv_appl1 … H1) -H1 *
 qed-.
 
 (* Note: the main property of simple terms *)
-lemma cpr_inv_appl1_simple: ∀L,V1,T1,U. L ⊢ ⓐV1. T1 ➡ U → 𝐒[T1] →
+lemma cpr_inv_appl1_simple: ∀L,V1,T1,U. L ⊢ ⓐV1. T1 ➡ U → 𝐒⦃T1⦄ →
                             ∃∃V2,T2. L ⊢ V1 ➡ V2 & L ⊢ T1 ➡ T2 &
                                      U = ⓐV2. T2.
 #L #V1 #T1 #U #H #HT1