]> matita.cs.unibo.it Git - helm.git/blobdiff - matita/matita/contribs/lambdadelta/basic_2/static/lfdeq_lfdeq.ma
update in ground_2 and basic_2
[helm.git] / matita / matita / contribs / lambdadelta / basic_2 / static / lfdeq_lfdeq.ma
index 2fae91f3901c2fff1cd7d727966ba89365bc4834..e88b4397cd768bc3e1e837dcee4ffcb667106c86 100644 (file)
@@ -23,7 +23,7 @@ include "basic_2/static/lfdeq_length.ma".
 
 (* Basic_2A1: uses: lleq_sym *)
 lemma lfdeq_sym: ∀h,o,T. symmetric … (lfdeq h o T).
-/3 width=3 by lfdeq_fle_comp, lfxs_sym, tdeq_sym/ qed-.
+/3 width=3 by lfdeq_fsle_comp, lfxs_sym, tdeq_sym/ qed-.
 
 (* Basic_2A1: uses: lleq_dec *)
 lemma lfdeq_dec: ∀h,o,L1,L2. ∀T:term. Decidable (L1 ≛[h, o, T] L2).