File tree Expand file tree Collapse file tree 7 files changed +39
-40
lines changed Expand file tree Collapse file tree 7 files changed +39
-40
lines changed Original file line number Diff line number Diff line change 9
9
10
10
module Algebra.Construct.Add.Identity where
11
11
12
- open import Algebra.Bundles
12
+ open import Algebra.Bundles using (Semigroup; Monoid)
13
13
open import Algebra.Core using (Op₂)
14
14
open import Algebra.Definitions
15
- open import Algebra.Structures
15
+ using (Congruent₂; Associative; LeftIdentity; RightIdentity; Identity)
16
+ open import Algebra.Structures using (IsMagma; IsSemigroup; IsMonoid)
16
17
open import Relation.Binary.Construct.Add.Point.Equality renaming (_≈∙_ to lift≈)
17
18
open import Data.Product.Base using (_,_)
18
19
open import Level using (Level; _⊔_)
19
- open import Relation.Binary.Core
20
- open import Relation.Binary.Definitions
21
- open import Relation.Binary.Structures
22
- open import Relation.Nullary.Construct.Add.Point
20
+ open import Relation.Binary.Core using (Rel)
21
+ open import Relation.Binary.Definitions using (Reflexive)
22
+ open import Relation.Binary.Structures using (IsEquivalence)
23
+ open import Relation.Nullary.Construct.Add.Point using (Pointed; [_]; ∙)
23
24
24
25
private
25
26
variable
@@ -101,3 +102,4 @@ monoid : Semigroup a (a ⊔ ℓ) → Monoid a (a ⊔ ℓ)
101
102
monoid S = record
102
103
{ isMonoid = isMonoid S.isSemigroup
103
104
} where module S = Semigroup S
105
+
Original file line number Diff line number Diff line change 7
7
8
8
{-# OPTIONS --cubical-compatible --safe #-}
9
9
10
- open import Algebra.Core
10
+ open import Algebra.Core using (Op₂)
11
11
open import Level as L hiding (_⊔_)
12
12
open import Function.Base using (flip)
13
13
open import Relation.Binary.Bundles using (TotalPreorder)
Original file line number Diff line number Diff line change @@ -11,9 +11,8 @@ open import Relation.Binary.Bundles using (TotalOrder)
11
11
module Algebra.Construct.NaturalChoice.Max
12
12
{a ℓ₁ ℓ₂} (totalOrder : TotalOrder a ℓ₁ ℓ₂) where
13
13
14
- open import Algebra.Core
15
- open import Algebra.Definitions
16
- open import Algebra.Construct.NaturalChoice.Base
14
+ open import Algebra.Core using (Op₂)
15
+ open import Algebra.Construct.NaturalChoice.Base using (MaxOperator)
17
16
open import Relation.Binary.Construct.Flip.EqAndOrd using ()
18
17
renaming (totalOrder to flip)
19
18
Original file line number Diff line number Diff line change 7
7
8
8
{-# OPTIONS --cubical-compatible --safe #-}
9
9
10
- open import Algebra.Core
11
- open import Algebra.Construct.NaturalChoice.Base
12
- import Algebra.Construct.NaturalChoice.MinOp as MinOp
13
- open import Function.Base using (flip)
14
- open import Relation.Binary.Core using (_Preserves_⟶_)
10
+ open import Algebra.Construct.NaturalChoice.Base using (MaxOperator; MaxOp⇒MinOp)
15
11
open import Relation.Binary.Bundles using (TotalPreorder)
16
- open import Relation.Binary.Construct.Flip.EqAndOrd using ()
17
- renaming (totalPreorder to flipOrder)
18
12
19
13
module Algebra.Construct.NaturalChoice.MaxOp
20
14
{a ℓ₁ ℓ₂} {O : TotalPreorder a ℓ₁ ℓ₂} (maxOp : MaxOperator O)
21
15
where
22
16
23
- open TotalPreorder O renaming (Carrier to A; _≲_ to _≤_)
17
+ import Algebra.Construct.NaturalChoice.MinOp as MinOp
18
+ open import Algebra.Core using (Op₂)
19
+ open import Function.Base using (flip)
24
20
open MaxOperator maxOp
21
+ open import Relation.Binary.Core using (_Preserves_⟶_)
22
+ open import Relation.Binary.Construct.Flip.EqAndOrd using ()
23
+ renaming (totalPreorder to flipOrder)
24
+ open TotalPreorder O renaming (Carrier to A; _≲_ to _≤_)
25
25
26
26
-- Max is just min with a flipped order
27
27
Original file line number Diff line number Diff line change 6
6
7
7
{-# OPTIONS --cubical-compatible --safe #-}
8
8
9
- open import Algebra.Core
10
- open import Algebra.Bundles
11
- open import Algebra.Construct.NaturalChoice.Base
12
- open import Data.Sum.Base using (inj₁; inj₂; [_,_])
13
- open import Data.Product.Base using (_,_)
14
- open import Function.Base using (id)
15
9
open import Relation.Binary.Bundles using (TotalOrder)
16
- import Algebra.Construct.NaturalChoice.MinOp as MinOp
17
10
18
11
module Algebra.Construct.NaturalChoice.Min
19
12
{a ℓ₁ ℓ₂} (O : TotalOrder a ℓ₁ ℓ₂)
20
13
where
21
14
15
+ open import Algebra.Core using (Op₂)
16
+ open import Algebra.Construct.NaturalChoice.Base
17
+ import Algebra.Construct.NaturalChoice.MinOp as MinOp
18
+ open import Data.Sum.Base using (inj₁; inj₂; [_,_])
19
+ open import Data.Product.Base using (_,_)
20
+ open import Function.Base using (id)
22
21
open TotalOrder O renaming (Carrier to A)
23
22
24
23
------------------------------------------------------------------------
Original file line number Diff line number Diff line change 7
7
8
8
{-# OPTIONS --cubical-compatible --safe #-}
9
9
10
- open import Algebra.Core
11
- open import Algebra.Bundles
12
- open import Algebra.Construct.NaturalChoice.Base
13
- open import Data.Sum.Base as Sum using (inj₁; inj₂; [_,_])
14
- open import Data.Product.Base using (_,_)
15
- open import Function.Base using (id; _∘_; flip)
16
- open import Relation.Binary.Core using (_Preserves_⟶_)
10
+ open import Algebra.Construct.NaturalChoice.Base using (MinOperator; MaxOperator)
17
11
open import Relation.Binary.Bundles using (TotalPreorder)
18
- open import Relation.Binary.Consequences
19
12
20
13
module Algebra.Construct.NaturalChoice.MinMaxOp
21
14
{a ℓ₁ ℓ₂} {O : TotalPreorder a ℓ₁ ℓ₂}
22
15
(minOp : MinOperator O)
23
16
(maxOp : MaxOperator O)
24
17
where
25
18
19
+ open import Data.Sum.Base as Sum using (inj₁; inj₂; [_,_])
20
+ open import Data.Product.Base using (_,_)
21
+ open import Function.Base using (id; _∘_; flip)
22
+ open import Relation.Binary.Core using (_Preserves_⟶_)
23
+
26
24
open TotalPreorder O renaming
27
25
( Carrier to A
28
26
; _≲_ to _≤_
Original file line number Diff line number Diff line change 7
7
8
8
{-# OPTIONS --cubical-compatible --safe #-}
9
9
10
- open import Algebra.Core
10
+ open import Relation.Binary.Bundles using (TotalPreorder)
11
+ open import Algebra.Construct.NaturalChoice.Base using (MinOperator; MinOp⇒MaxOp)
12
+
13
+ module Algebra.Construct.NaturalChoice.MinOp
14
+ {a ℓ₁ ℓ₂} {O : TotalPreorder a ℓ₁ ℓ₂} (minOp : MinOperator O) where
15
+
16
+ open import Algebra.Core using (Op₂)
11
17
open import Algebra.Bundles
12
- open import Algebra.Construct.NaturalChoice.Base
18
+ using (RawMagma; Magma; Semigroup; Band; CommutativeSemigroup; SelectiveMagma; Monoid)
13
19
open import Data.Sum.Base as Sum using (inj₁; inj₂; [_,_])
14
20
open import Data.Product.Base using (_,_)
15
21
open import Function.Base using (id; _∘_)
16
22
open import Relation.Binary.Core using (_Preserves_⟶_; _Preserves₂_⟶_⟶_)
17
- open import Relation.Binary.Bundles using (TotalPreorder)
18
23
open import Relation.Binary.Definitions using (Maximum; Minimum)
19
- open import Relation.Binary.Consequences
20
-
21
- module Algebra.Construct.NaturalChoice.MinOp
22
- {a ℓ₁ ℓ₂} {O : TotalPreorder a ℓ₁ ℓ₂} (minOp : MinOperator O) where
23
24
24
25
open TotalPreorder O renaming
25
26
( Carrier to A
You can’t perform that action at this time.
0 commit comments