]> matita.cs.unibo.it Git - helm.git/blobdiff - matita/matita/contribs/lambdadelta/basic_2/computation/fpbs.ma
some improvements towards an alternative definition of fpbs ...
[helm.git] / matita / matita / contribs / lambdadelta / basic_2 / computation / fpbs.ma
index ebebb4577274f4aac0baa2f10d32aba296b20d2e..00f4a93aa34b55e34826eea836905fdc08ce61fe 100644 (file)
@@ -29,7 +29,7 @@ interpretation "'big tree' parallel computation (closure)"
 (* Basic eliminators ********************************************************)
 
 lemma fpbs_ind: ∀h,g,G1,L1,T1. ∀R:relation3 genv lenv term. R G1 L1 T1 →
-                (∀L,G2,G,L2,T,T2. ⦃G1, L1, T1⦄ ≥[h, g] ⦃G, L, T⦄ → ⦃G, L, T⦄ ≽[h, g] ⦃G2, L2, T2⦄ → R G L T → R G2 L2 T2) →
+                (∀G,G2,L,L2,T,T2. ⦃G1, L1, T1⦄ ≥[h, g] ⦃G, L, T⦄ → ⦃G, L, T⦄ ≽[h, g] ⦃G2, L2, T2⦄ → R G L T → R G2 L2 T2) →
                 ∀G2,L2,T2. ⦃G1, L1, T1⦄ ≥[h, g] ⦃G2, L2, T2⦄ → R G2 L2 T2.
 /3 width=8 by tri_TC_star_ind/ qed-.