1 (**************************************************************************)
4 (* ||A|| A project by Andrea Asperti *)
6 (* ||I|| Developers: *)
7 (* ||T|| The HELM team. *)
8 (* ||A|| http://helm.cs.unibo.it *)
10 (* \ / This file is distributed under the terms of the *)
11 (* v GNU General Public License Version 2 *)
13 (**************************************************************************)
15 include "basic_2/reducibility/ltpr_ltpr.ma".
16 include "basic_2/computation/ltprs.ma".
18 (* CONTEXT-FREE PARALLEL COMPUTATION ON LOCAL ENVIRONMENTS ******************)
20 (* Advanced properties ******************************************************)
22 lemma ltprs_strip: ∀L1. ∀L:lenv. L ➡* L1 → ∀L2. L ➡ L2 →
23 ∃∃L0. L1 ➡ L0 & L2 ➡* L0.
26 (* Main properties **********************************************************)
28 theorem ltprs_conf: confluent … ltprs.
31 theorem ltprs_trans: Transitive … ltprs.