Coding functions #
In this file, we define coding functions.
Main declarations #
ConNF.CodingFunction
: The type of coding functions.
theorem
ConNF.Support.orbitRel_isEquivalence
[Params]
[Level]
[CoherentData]
{β : TypeIndex}
[LeLevel β]
:
Equations
- ConNF.Support.setoid β = { r := ConNF.Support.orbitRel, iseqv := ⋯ }
Equations
Instances For
def
ConNF.Support.orbit
[Params]
[Level]
[CoherentData]
{β : TypeIndex}
[LeLevel β]
(S : Support β)
:
Instances For
theorem
ConNF.SupportOrbit.out_orbit
[Params]
[Level]
[CoherentData]
{β : TypeIndex}
[LeLevel β]
(o : SupportOrbit β)
:
theorem
ConNF.SupportOrbit.exists_support
[Params]
[Level]
[CoherentData]
{β : TypeIndex}
[LeLevel β]
(o : SupportOrbit β)
:
- rel_coinjective : self.rel.Coinjective
Instances For
theorem
ConNF.CodingFunction.ext'
[Params]
[Level]
[CoherentData]
{β : TypeIndex}
[LeLevel β]
{χ₁ χ₂ : CodingFunction β}
(h : ∀ (S : Support β) (x : TSet β), χ₁.rel S x ↔ χ₂.rel S x)
:
theorem
ConNF.CodingFunction.ext_aux
[Params]
[Level]
[CoherentData]
{β : TypeIndex}
[LeLevel β]
{χ₁ χ₂ : CodingFunction β}
{S : Support β}
{x : TSet β}
(h₁ : χ₁.rel S x)
(h₂ : χ₂.rel S x)
:
theorem
ConNF.CodingFunction.ext
[Params]
[Level]
[CoherentData]
{β : TypeIndex}
[LeLevel β]
{χ₁ χ₂ : CodingFunction β}
(S : Support β)
(x : TSet β)
(h₁ : χ₁.rel S x)
(h₂ : χ₂.rel S x)
:
Equations
- One or more equations did not get rendered due to their size.