File tree Expand file tree Collapse file tree 1 file changed +3
-4
lines changed
Expand file tree Collapse file tree 1 file changed +3
-4
lines changed Original file line number Diff line number Diff line change @@ -39,8 +39,7 @@ open import Relation.Binary.PropositionalEquality.Properties
3939 using (module ≡-Reasoning )
4040open import Relation.Nullary.Negation.Core using (¬_)
4141import Relation.Nullary.Indexed as I
42- open import Relation.Unary using (⟨_⟩⊢_)
43- open import Relation.Unary.Properties using (⟨_⟩⊢ˡ; ⟨_⟩⊢ʳ)
42+ open import Relation.Unary.Properties using (⟨_⟩⊢⁻_; ⟨_⟩⊢⁺_)
4443
4544private
4645 variable
@@ -361,7 +360,7 @@ Related-cong {A = A} {B = B} {C = C} {D = D} A≈B C≈D = mk⇔
361360-- Relating a predicate to an existentially quantified one with the
362361-- restriction that the quantified variable is equal to the given one
363362
364- ∃-≡ : ∀ (P : A → Set b) {x} → P x ↔ (⟨ id ⟩⊢ P) x
365- ∃-≡ P {x} = mk↔ₛ′ (⟨ id ⟩⊢ˡ id) (⟨ id ⟩⊢ʳ id)
363+ ∃-≡ : ∀ (P : A → Set b) {x} → P x ↔ (∃[ y ] y ≡ x × P y)
364+ ∃-≡ P {x} = mk↔ₛ′ (⟨ id ⟩⊢⁻ id) (⟨ id ⟩⊢⁺ id)
366365 (λ where (_ , refl , _) → refl) (λ where _ → refl)
367366
You can’t perform that action at this time.
0 commit comments