X-Git-Url: http://matita.cs.unibo.it/gitweb/?a=blobdiff_plain;f=matita%2Fmatita%2Flib%2Flambda%2Fpaths%2Flabeled_st_reduction.ma;h=60e2c28f8df4c9e2919bb5060a1adb7739c4e8a4;hb=613d8642b1154dde0c026cbdcd96568910198251;hp=2f93b35afda99911f8c82f7df482c457e1b18e07;hpb=aa9654656f7d0aeb9345e0b86a9e35f861687580;p=helm.git diff --git a/matita/matita/lib/lambda/paths/labeled_st_reduction.ma b/matita/matita/lib/lambda/paths/labeled_st_reduction.ma index 2f93b35af..60e2c28f8 100644 --- a/matita/matita/lib/lambda/paths/labeled_st_reduction.ma +++ b/matita/matita/lib/lambda/paths/labeled_st_reduction.ma @@ -12,9 +12,14 @@ (* *) (**************************************************************************) -include "subterms/booleanized.ma". -include "paths/labeled_sequential_reduction.ma". -include "paths/standard_order.ma". +include "lambda/subterms/booleanized.ma". +include "lambda/paths/labeled_sequential_reduction.ma". +include "lambda/paths/standard_order.ma". + +include "lambda/notation/relations/std_3.ma". + +include "lambda/xoa/ex_4_1.ma". +include "lambda/xoa/ex_3_4.ma". (* PATH-LABELED STANDARD REDUCTION ON SUBTERMS (SINGLE STEP) ****************) @@ -31,10 +36,6 @@ inductive pl_st: path → relation subterms ≝ interpretation "path-labeled standard reduction" 'Std F p G = (pl_st p F G). -notation "hvbox( F break Ⓡ ↦ [ term 46 p ] break term 46 G )" - non associative with precedence 45 - for @{ 'Std $F $p $G }. - lemma pl_st_fwd_pl_sred: ∀p,F1,F2. F1 Ⓡ↦[p] F2 → ⇓F1 ↦[p] ⇓F2. #p #F1 #F2 #H elim H -p -F1 -F2 normalize /2 width=1/ qed-.