File tree Expand file tree Collapse file tree 1 file changed +0
-8
lines changed Expand file tree Collapse file tree 1 file changed +0
-8
lines changed Original file line number Diff line number Diff line change 1515
1616{-# OPTIONS --cubical-compatible --safe #-}
1717
18- <<<<<<< HEAD
1918open import Relation.Binary.Core using (Rel)
20- =======
21- open import Relation.Binary.Core using (Rel; _Preserves_⟶_; _Preserves₂_⟶_⟶_)
22- >>>>>>> f0e0101df (chore: move imports around in Algebra.Definitions)
2319
2420module Algebra.Definitions
2521 {a ℓ} {A : Set a} -- The underlying set
@@ -29,13 +25,9 @@ module Algebra.Definitions
2925open import Algebra.Core using (Op₁; Op₂)
3026open import Data.Product.Base using (_×_; ∃-syntax)
3127open import Data.Sum.Base using (_⊎_)
32- <<<<<<< HEAD
3328open import Relation.Binary.Definitions using (Monotonic₁; Monotonic₂)
3429open import Relation.Nullary.Negation.Core using (¬_)
3530
36- =======
37- open import Relation.Nullary.Negation.Core using (¬_)
38- >>>>>>> f0e0101df (chore: move imports around in Algebra.Definitions)
3931
4032------------------------------------------------------------------------
4133-- Properties of operations
You can’t perform that action at this time.
0 commit comments