Skip to content

Commit

Permalink
Update Base.agda
Browse files Browse the repository at this point in the history
  • Loading branch information
anshwad10 authored Jan 13, 2025
1 parent 36f8b9f commit b865c6f
Showing 1 changed file with 2 additions and 2 deletions.
4 changes: 2 additions & 2 deletions Cubical/Data/Sigma/Base.agda
Original file line number Diff line number Diff line change
Expand Up @@ -54,5 +54,5 @@ syntax ∃!-syntax A (λ x → B) = ∃![ x ∈ A ] B
-- Instance

instance
Σ-instance : {ℓ ℓ'} {A : Type ℓ} {B : A Type ℓ'} {{ x : A }} {{ B x }} Σ A B
Σ-instance {{ x }} {{ y }} = (x , y)
Σ-instance : {ℓ ℓ'} {A : Type ℓ} {B : A Type ℓ'} x : A ⦄ ⦃ B x Σ A B
Σ-instance x ⦄ ⦃ y = (x , y)

0 comments on commit b865c6f

Please sign in to comment.