Skip to content

Commit

Permalink
Remove the instance
Browse files Browse the repository at this point in the history
  • Loading branch information
anshwad10 authored Jan 13, 2025
1 parent ae50c10 commit 933df36
Showing 1 changed file with 0 additions and 6 deletions.
6 changes: 0 additions & 6 deletions Cubical/Data/Sigma/Base.agda
Original file line number Diff line number Diff line change
Expand Up @@ -50,9 +50,3 @@ infix 2 ∃!-syntax
∃!-syntax = ∃!

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)

0 comments on commit 933df36

Please sign in to comment.