Parallel composition of kernels #
Two kernels κ : Kernel α β
and η : Kernel γ δ
can be applied in parallel to give a kernel
κ ∥ₖ η
from α × γ
to β × δ
: (κ ∥ₖ η) (a, c) = (κ a).prod (η c)
.
Main definitions #
parallelComp (κ : Kernel α β) (η : Kernel γ δ) : Kernel (α × γ) (β × δ)
: parallel composition of two s-finite kernels. We define a notationκ ∥ₖ η = parallelComp κ η
.∫⁻ bd, g bd ∂(κ ∥ₖ η) ac = ∫⁻ b, ∫⁻ d, g (b, d) ∂η ac.2 ∂κ ac.1
Main statements #
parallelComp_comp_copy
:(κ ∥ₖ η) ∘ₖ (copy α) = κ ×ₖ η
deterministic_comp_copy
: for a deterministic kernel, copying then applying the kernel to the two copies is the same as first applying the kernel then copying. That is, ifκ
is a deterministic kernel,(κ ∥ₖ κ) ∘ₖ copy α = copy β ∘ₖ κ
.
Notations #
κ ∥ₖ η = ProbabilityTheory.Kernel.parallelComp κ η
Implementation notes #
Our formalization of kernels is centered around the composition-product: the product and then the
parallel composition are defined as special cases of the composition-product.
We could have alternatively used the building blocks of kernels seen as a Markov category:
composition, parallel composition (or tensor product) and the deterministic kernels id
, copy
,
swap
and discard
. The product and composition-product could then be built from these.
Parallel product of two kernels.
Equations
- κ.parallelComp η = (ProbabilityTheory.Kernel.prodMkRight γ κ).prod (ProbabilityTheory.Kernel.prodMkLeft α η)
Instances For
Parallel product of two kernels.
Equations
- One or more equations did not get rendered due to their size.
Instances For
For a deterministic kernel, copying then applying the kernel to the two copies is the same as first applying the kernel then copying.