Skip to content

Commit

Permalink
some cleanup
Browse files Browse the repository at this point in the history
  • Loading branch information
marcinjangrzybowski committed Feb 6, 2024
1 parent 51e1b29 commit 88c23b0
Showing 1 changed file with 0 additions and 3 deletions.
3 changes: 0 additions & 3 deletions Cubical/Foundations/Powerset.agda
Original file line number Diff line number Diff line change
Expand Up @@ -50,9 +50,6 @@ A ⊆ B = ∀ x → x ∈ A → x ∈ B
subst-∈ : (A : ℙ X) {x y : X} x ≡ y x ∈ A y ∈ A
subst-∈ A = subst (_∈ A)

subst-∈' : (A : ℙ X) {x y : X} x ∈ A x ≡ y y ∈ A
subst-∈' A x p = subst (_∈ A) p x

⊆-refl-consequence : (A B : ℙ X) A ≡ B (A ⊆ B) × (B ⊆ A)
⊆-refl-consequence A B p = subst (A ⊆_) p (⊆-refl A)
, subst (B ⊆_) (sym p) (⊆-refl B)
Expand Down

0 comments on commit 88c23b0

Please sign in to comment.