Skip to content

Commit

Permalink
Update Base.agda
Browse files Browse the repository at this point in the history
fixed the error
  • Loading branch information
anshwad10 authored Jan 13, 2025
1 parent b865c6f commit 7e13086
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion 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 : {ℓ ℓ'} {A : Type ℓ} {B : A Type ℓ'} ⦃ x : A ⦄ ⦃ _ : B x ⦄ Σ A B
Σ-instance ⦃ x ⦄ ⦃ y ⦄ = (x , y)

0 comments on commit 7e13086

Please sign in to comment.