Skip to content

Commit

Permalink
Cleaner proof
Browse files Browse the repository at this point in the history
  • Loading branch information
LuuBluum committed Sep 9, 2024
1 parent ab1e96c commit 2a34d83
Showing 1 changed file with 5 additions and 7 deletions.
12 changes: 5 additions & 7 deletions Cubical/Relation/Binary/Order/Poset/Mappings.agda
Original file line number Diff line number Diff line change
Expand Up @@ -426,13 +426,11 @@ Involution→EqualResidual : (P : Poset ℓ ℓ')
(res : hasResidual P P f)
f ∘ f ≡ idfun ⟨ P ⟩
f ≡ (residual P P f res)
Involution→EqualResidual P f (isf , f⁺ , isf⁺ , f⁺∘f , f∘f⁺) inv
= funExt λ x anti (f x) (f⁺ x)
(subst (λ g f x ≤ f⁺ (g x)) inv (f⁺∘f (f x)))
(subst (λ g g (f⁺ x) ≤ f x) inv (IsIsotone.pres≤ isf _ _ (f∘f⁺ x)))
where pos = PosetStr.isPoset (snd P)
_≤_ = PosetStr._≤_ (snd P)
anti = IsPoset.is-antisym pos
Involution→EqualResidual P f res inv
= sym (cong₂ (λ g h g ∘ f⁺ ∘ h) (sym inv) (sym inv) ∙
cong (λ g f ∘ g ∘ f) (AbsorbResidual P P f res) ∙
cong (f ∘_) inv)
where f⁺ = res .snd .fst

Res : Poset ℓ ℓ' Semigroup (ℓ-max ℓ ℓ')
fst (Res E) = Σ[ f ∈ (⟨ E ⟩ ⟨ E ⟩) ] hasResidual E E f
Expand Down

0 comments on commit 2a34d83

Please sign in to comment.