Coherent data #
In this file, we define the type of coherent data below a particular proper type index.
Main declarations #
ConNF.ModelDataData
: Coherent data below a given levelα
.
TODO: We're going to try allowing model data at level ⊥
to vary. That is, we use
(β : TypeIndex) → [LeLevel β] → ModelData β
instead of (β : Λ) → [LeLevel β] → ModelData β
.
Instances
theorem
ConNF.PreCoherentData.ext
{inst✝ : Params}
{inst✝¹ : Level}
{x y : PreCoherentData}
(data : LeData.data = LeData.data)
(positions : HEq LeData.positions LeData.positions)
(allPermSderiv : HEq (@allPermSderiv inst✝ inst✝¹ x) (@allPermSderiv inst✝ inst✝¹ y))
(singleton : HEq (@singleton inst✝ inst✝¹ x) (@singleton inst✝ inst✝¹ y))
:
instance
ConNF.instDerivativeAllPerm
[Params]
[Level]
[PreCoherentData]
{β γ : TypeIndex}
[LeLevel β]
[LeLevel γ]
:
Derivative (AllPerm β) (AllPerm γ) β γ
Equations
- One or more equations did not get rendered due to their size.
Note that in earlier versions of the proof we additionally used the following assumption.
typedMem_tSetForget {β : Λ} {γ : TypeIndex} [LeLevel β] [LeLevel γ]
(hγ : γ < β) (x : TSet β) (y : StrSet γ) :
y ∈[hγ] xᵁ → ∃ z : TSet γ, y = zᵁ
- allPerm_of_smulFuzz {γ : Λ} [LeLevel ↑γ] (ρs : {δ : TypeIndex} → [inst : LtLevel δ] → δ < ↑γ → AllPerm δ) (h : ∀ {δ : TypeIndex} {ε : Λ} [inst : LtLevel δ] [inst_1 : LtLevel ↑ε] (hδ : δ < ↑γ) (hε : ↑ε < ↑γ) (hδε : δ ≠ ↑ε) (t : Tangle δ), (ρs hε)ᵁ ↘. • fuzz hδε t = fuzz hδε (ρs hδ • t)) : ∃ (ρ : AllPerm ↑γ), ∀ (δ : TypeIndex) [inst : LtLevel δ] (hδ : δ < ↑γ), ρ ↘ hδ = ρs hδ
Instances
theorem
ConNF.CoherentData.ext
{inst✝ : Params}
{inst✝¹ : Level}
{x y : CoherentData}
(data : LeData.data = LeData.data)
(positions : HEq LeData.positions LeData.positions)
(allPermSderiv :
HEq (@PreCoherentData.allPermSderiv inst✝ inst✝¹ toPreCoherentData)
(@PreCoherentData.allPermSderiv inst✝ inst✝¹ toPreCoherentData))
(singleton : HEq (@singleton inst✝ inst✝¹ toPreCoherentData) (@singleton inst✝ inst✝¹ toPreCoherentData))
: