Skip to content

Commit

Permalink
fixed knock-on ambiguity bugs
Browse files Browse the repository at this point in the history
  • Loading branch information
jamesmckinna committed Oct 2, 2024
1 parent 3923598 commit deaf59e
Show file tree
Hide file tree
Showing 2 changed files with 2 additions and 2 deletions.
2 changes: 1 addition & 1 deletion src/Relation/Binary/Bundles.agda
Original file line number Diff line number Diff line change
Expand Up @@ -395,4 +395,4 @@ record ApartnessRelation c ℓ₁ ℓ₂ : Set (suc (c ⊔ ℓ₁ ⊔ ℓ₂)) w

open RawApartnessRelation rawApartnessRelation public
hiding (Carrier; _≈_ ; _#_)

2 changes: 1 addition & 1 deletion src/Relation/Binary/Properties/Poset.agda
Original file line number Diff line number Diff line change
Expand Up @@ -25,7 +25,7 @@ open Poset P renaming (Carrier to A)

import Relation.Binary.Construct.NonStrictToStrict _≈_ _≤_ as ToStrict
import Relation.Binary.Properties.Preorder preorder as PreorderProperties
open Eq using (_≉_)


------------------------------------------------------------------------
-- The _≥_ relation is also a poset.
Expand Down

0 comments on commit deaf59e

Please sign in to comment.