Skip to content
Merged
Show file tree
Hide file tree
Changes from all commits
Commits
File filter

Filter by extension

Filter by extension

Conversations
Failed to load comments.
Loading
Jump to
Jump to file
Failed to load files.
Loading
Diff view
Diff view
2 changes: 1 addition & 1 deletion src/Algebra/Lattice/Bundles/Raw.agda
Original file line number Diff line number Diff line change
Expand Up @@ -8,7 +8,7 @@

module Algebra.Lattice.Bundles.Raw where

open import Algebra.Core
open import Algebra.Core using (Op₂)
open import Algebra.Bundles.Raw using (RawMagma)
open import Level using (suc; _⊔_)
open import Relation.Binary.Core using (Rel)
Expand Down
4 changes: 3 additions & 1 deletion src/Algebra/Lattice/Construct/NaturalChoice/MaxOp.agda
Original file line number Diff line number Diff line change
Expand Up @@ -8,13 +8,15 @@
{-# OPTIONS --cubical-compatible --safe #-}

open import Algebra.Construct.NaturalChoice.Base
import Algebra.Lattice.Construct.NaturalChoice.MinOp as MinOp
using (MaxOperator; MaxOp⇒MinOp)
open import Relation.Binary.Bundles using (TotalPreorder)

module Algebra.Lattice.Construct.NaturalChoice.MaxOp
{a ℓ₁ ℓ₂} {O : TotalPreorder a ℓ₁ ℓ₂} (maxOp : MaxOperator O)
where

import Algebra.Lattice.Construct.NaturalChoice.MinOp as MinOp

private
module Min = MinOp (MaxOp⇒MinOp maxOp)

Expand Down
4 changes: 2 additions & 2 deletions src/Algebra/Lattice/Construct/NaturalChoice/MinMaxOp.agda
Original file line number Diff line number Diff line change
Expand Up @@ -6,8 +6,7 @@

{-# OPTIONS --cubical-compatible --safe #-}

open import Algebra.Lattice.Bundles
open import Algebra.Construct.NaturalChoice.Base
open import Algebra.Construct.NaturalChoice.Base using (MinOperator; MaxOperator)
open import Relation.Binary.Bundles using (TotalPreorder)

module Algebra.Lattice.Construct.NaturalChoice.MinMaxOp
Expand All @@ -22,6 +21,7 @@ open MaxOperator maxOp

open import Algebra.Lattice.Structures _≈_
open import Algebra.Construct.NaturalChoice.MinMaxOp minOp maxOp
open import Algebra.Lattice.Bundles using (Lattice; DistributiveLattice)
open import Relation.Binary.Reasoning.Preorder preorder

------------------------------------------------------------------------
Expand Down
7 changes: 3 additions & 4 deletions src/Algebra/Lattice/Construct/NaturalChoice/MinOp.agda
Original file line number Diff line number Diff line change
Expand Up @@ -7,9 +7,7 @@

{-# OPTIONS --cubical-compatible --safe #-}

open import Algebra.Bundles
open import Algebra.Lattice.Bundles
open import Algebra.Construct.NaturalChoice.Base
open import Algebra.Construct.NaturalChoice.Base using (MinOperator)
open import Relation.Binary.Bundles using (TotalPreorder)

module Algebra.Lattice.Construct.NaturalChoice.MinOp
Expand All @@ -18,8 +16,9 @@ module Algebra.Lattice.Construct.NaturalChoice.MinOp
open TotalPreorder O
open MinOperator minOp

open import Algebra.Lattice.Structures _≈_
open import Algebra.Construct.NaturalChoice.MinOp minOp
open import Algebra.Lattice.Bundles using (Semilattice)
open import Algebra.Lattice.Structures _≈_

------------------------------------------------------------------------
-- Structures
Expand Down