]> matita.cs.unibo.it Git - helm.git/blobdiff - matita/matita/contribs/lambdadelta/basic_2/rt_computation/fsb_fpbg.ma
commit in ground_2, static_2, basic_2, apps_2
[helm.git] / matita / matita / contribs / lambdadelta / basic_2 / rt_computation / fsb_fpbg.ma
index 07a9aad5eec9d8e0a714d1d7649c7bc85243e915..cd2c4124815b517af7783d98d82d5843562fd9e7 100644 (file)
@@ -64,3 +64,12 @@ lemma fsb_ind_fpbg: ∀h,o. ∀Q:relation3 genv lenv term.
 #h #o #Q #IH #G1 #L1 #T1 #H @(fsb_ind_fpbg_fpbs … H) -H
 /3 width=1 by/
 qed-.
+
+(* Inversion lemmas with proper parallel rst-computation for closures *******)
+
+lemma fsb_fpbg_refl_false (h) (o) (G) (L) (T):
+                          ≥[h,o] 𝐒⦃G, L, T⦄ → ⦃G, L, T⦄ >[h,o] ⦃G, L, T⦄ → ⊥.
+#h #o #G #L #T #H
+@(fsb_ind_fpbg … H) -G -L -T #G1 #L1 #T1 #_ #IH #H
+/2 width=5 by/
+qed-.