Skip to content

Commit

Permalink
add a 'beta' for the fundamental thm of id
Browse files Browse the repository at this point in the history
  • Loading branch information
felixwellen committed Dec 7, 2022
1 parent b2a0c41 commit ddb192d
Showing 1 changed file with 8 additions and 0 deletions.
8 changes: 8 additions & 0 deletions Cubical/Foundations/Equiv/Fiberwise.agda
Original file line number Diff line number Diff line change
Expand Up @@ -89,3 +89,11 @@ fundamentalTheoremOfId : {A : Type ℓ} (Eq : A → A → Type ℓ')
((x : A) isContr (Σ[ y ∈ A ] Eq x y))
(x y : A) (x ≡ y) ≃ (Eq x y)
fundamentalTheoremOfId Eq eqRefl eqContr x = recognizeId (Eq x) (eqRefl x) (eqContr x)

fundamentalTheoremOfIdβ :
{A : Type ℓ} (Eq : A A Type ℓ')
(eqRefl : (x : A) Eq x x)
(eqContr : (x : A) isContr (Σ[ y ∈ A ] Eq x y))
(x : A)
fst (fundamentalTheoremOfId Eq eqRefl eqContr x x) refl ≡ eqRefl x
fundamentalTheoremOfIdβ Eq eqRefl eqContr x = JRefl (λ y p Eq x y) (eqRefl x)

0 comments on commit ddb192d

Please sign in to comment.