File tree 28 files changed +28
-28
lines changed
Properties/BooleanAlgebra
28 files changed +28
-28
lines changed Original file line number Diff line number Diff line change @@ -16,7 +16,7 @@ open import Data.Unit
16
16
open import Data.Bool.Base using (Bool; true)
17
17
open import Data.Nat
18
18
open import Data.Sum using (inj₁; inj₂)
19
- open import Data.Product renaming (_×_ to _⟨×⟩_)
19
+ open import Data.Product.Base renaming (_×_ to _⟨×⟩_)
20
20
open import Data.Container using (Container; _▷_)
21
21
open import Data.Container.Combinator
22
22
open import Data.Container.FreeMonad as FreeMonad
Original file line number Diff line number Diff line change @@ -11,7 +11,7 @@ open import Algebra.Apartness.Bundles using (HeytingCommutativeRing)
11
11
module Algebra.Apartness.Properties.HeytingCommutativeRing
12
12
{c ℓ₁ ℓ₂} (HCR : HeytingCommutativeRing c ℓ₁ ℓ₂) where
13
13
14
- open import Data.Product using (_,_; proj₂)
14
+ open import Data.Product.Base using (_,_; proj₂)
15
15
open import Algebra using (CommutativeRing; RightIdentity)
16
16
17
17
open HeytingCommutativeRing HCR
Original file line number Diff line number Diff line change @@ -14,7 +14,7 @@ open import Algebra.Core using (Op₂)
14
14
open import Algebra.Definitions
15
15
open import Algebra.Structures
16
16
open import Relation.Binary.Construct.Add.Point.Equality renaming (_≈∙_ to lift≈)
17
- open import Data.Product using (_,_)
17
+ open import Data.Product.Base using (_,_)
18
18
open import Level using (Level; _⊔_)
19
19
open import Relation.Binary.Core
20
20
open import Relation.Binary.Definitions
Original file line number Diff line number Diff line change 10
10
module Algebra.Construct.Flip.Op where
11
11
12
12
open import Algebra
13
- import Data.Product as Prod
13
+ import Data.Product.Base as Prod
14
14
import Data.Sum as Sum
15
15
open import Function.Base using (flip)
16
16
open import Level using (Level)
Original file line number Diff line number Diff line change 8
8
9
9
open import Algebra
10
10
open import Data.Bool.Base using (false; true)
11
- open import Data.Product using (_×_; _,_; swap; map; uncurry′)
11
+ open import Data.Product.Base using (_×_; _,_; swap; map; uncurry′)
12
12
open import Function.Base using (_∘_)
13
13
open import Level using (Level; _⊔_)
14
14
open import Relation.Binary.Definitions using (Decidable)
Original file line number Diff line number Diff line change @@ -14,7 +14,7 @@ open import Algebra.Consequences.Base
14
14
open import Relation.Binary
15
15
open import Relation.Nullary using (¬_; yes; no)
16
16
open import Data.Sum.Base as Sum using (_⊎_; inj₁; inj₂; [_,_])
17
- open import Data.Product using (_×_; _,_)
17
+ open import Data.Product.Base using (_×_; _,_)
18
18
open import Level using (Level; _⊔_)
19
19
open import Relation.Binary.PropositionalEquality as P using (_≡_)
20
20
open import Relation.Unary using (Pred)
Original file line number Diff line number Diff line change @@ -10,7 +10,7 @@ open import Algebra.Core
10
10
open import Algebra.Bundles
11
11
open import Algebra.Construct.NaturalChoice.Base
12
12
open import Data.Sum using (inj₁; inj₂; [_,_])
13
- open import Data.Product using (_,_)
13
+ open import Data.Product.Base using (_,_)
14
14
open import Function.Base using (id)
15
15
open import Relation.Binary
16
16
import Algebra.Construct.NaturalChoice.MinOp as MinOp
Original file line number Diff line number Diff line change 9
9
10
10
{-# OPTIONS --cubical-compatible --safe #-}
11
11
12
- open import Data.Product as Prod
12
+ open import Data.Product.Base as Prod
13
13
open import Relation.Binary.Core
14
14
15
15
module Algebra.Construct.Subst.Equality
Original file line number Diff line number Diff line change @@ -11,7 +11,7 @@ module Algebra.Lattice.Morphism.Construct.Identity where
11
11
open import Algebra.Lattice.Bundles
12
12
open import Algebra.Lattice.Morphism.Structures
13
13
using ( module LatticeMorphisms )
14
- open import Data.Product using (_,_)
14
+ open import Data.Product.Base using (_,_)
15
15
open import Function.Base using (id)
16
16
open import Level using (Level)
17
17
open import Relation.Binary.Morphism.Construct.Identity using (isRelHomomorphism)
Original file line number Diff line number Diff line change @@ -15,7 +15,7 @@ open import Algebra.Lattice.Morphism.Structures
15
15
import Algebra.Consequences.Setoid as Consequences
16
16
import Algebra.Morphism.MagmaMonomorphism as MagmaMonomorphisms
17
17
import Algebra.Lattice.Properties.Lattice as LatticeProperties
18
- open import Data.Product using (_,_; map)
18
+ open import Data.Product.Base using (_,_; map)
19
19
open import Relation.Binary
20
20
import Relation.Binary.Morphism.RelMonomorphism as RelMonomorphisms
21
21
import Relation.Binary.Reasoning.Setoid as SetoidReasoning
Original file line number Diff line number Diff line change @@ -18,7 +18,7 @@ open import Effect.Applicative as Applicative
18
18
open import Effect.Monad
19
19
open import Data.Fin.Base using (Fin)
20
20
open import Data.Nat.Base
21
- open import Data.Product using (_,_; proj₁; proj₂)
21
+ open import Data.Product.Base using (_,_; proj₁; proj₂)
22
22
open import Data.Vec.Base as Vec using (Vec)
23
23
import Data.Vec.Effectful as VecCat
24
24
import Function.Identity.Effectful as IdCat
Original file line number Diff line number Diff line change 14
14
15
15
open import Algebra.Core
16
16
open import Algebra.Consequences.Setoid
17
- open import Data.Product using (proj₁; proj₂)
17
+ open import Data.Product.Base using (proj₁; proj₂)
18
18
open import Level using (_⊔_)
19
19
open import Relation.Binary using (Rel; Setoid; IsEquivalence)
20
20
Original file line number Diff line number Diff line change @@ -21,7 +21,7 @@ open import Algebra.Module.Morphism.Structures
21
21
; module ModuleMorphisms
22
22
)
23
23
open import Algebra.Morphism.Construct.Identity
24
- open import Data.Product using (_,_)
24
+ open import Data.Product.Base using (_,_)
25
25
open import Function.Base using (id)
26
26
open import Level using (Level)
27
27
Original file line number Diff line number Diff line change @@ -16,7 +16,7 @@ open import Algebra.Module.Core
16
16
import Algebra.Definitions as Defs
17
17
open import Algebra.Module.Definitions
18
18
open import Algebra.Structures
19
- open import Data.Product using (_,_; proj₁; proj₂)
19
+ open import Data.Product.Base using (_,_; proj₁; proj₂)
20
20
open import Level using (Level; _⊔_)
21
21
22
22
private
Original file line number Diff line number Diff line change @@ -10,7 +10,7 @@ module Algebra.Morphism.Consequences where
10
10
11
11
open import Algebra using (Magma)
12
12
open import Algebra.Morphism.Definitions
13
- open import Data.Product using (_,_)
13
+ open import Data.Product.Base using (_,_)
14
14
open import Function.Base using (id; _∘_)
15
15
open import Function.Definitions
16
16
import Relation.Binary.Reasoning.Setoid as EqR
Original file line number Diff line number Diff line change @@ -20,7 +20,7 @@ open import Algebra.Morphism.Structures
20
20
; module QuasigroupMorphisms
21
21
; module LoopMorphisms
22
22
)
23
- open import Data.Product using (_,_)
23
+ open import Data.Product.Base using (_,_)
24
24
open import Function.Base using (id)
25
25
open import Level using (Level)
26
26
open import Relation.Binary.Morphism.Construct.Identity using (isRelHomomorphism)
Original file line number Diff line number Diff line change @@ -24,7 +24,7 @@ open RawMonoid M₂ renaming (Carrier to B; _≈_ to _≈₂_; _∙_ to _◦_;
24
24
25
25
open import Algebra.Definitions
26
26
open import Algebra.Structures
27
- open import Data.Product using (map)
27
+ open import Data.Product.Base using (map)
28
28
import Relation.Binary.Reasoning.Setoid as SetoidReasoning
29
29
30
30
------------------------------------------------------------------------
Original file line number Diff line number Diff line change @@ -21,7 +21,7 @@ module Algebra.Ordered.Structures
21
21
open import Algebra.Core
22
22
open import Algebra.Definitions _≈_
23
23
open import Algebra.Structures _≈_
24
- open import Data.Product using (proj₁; proj₂)
24
+ open import Data.Product.Base using (proj₁; proj₂)
25
25
open import Function.Base using (flip)
26
26
open import Level using (_⊔_)
27
27
open import Relation.Binary.Definitions using (Transitive; Monotonic₁; Monotonic₂)
Original file line number Diff line number Diff line change @@ -30,7 +30,7 @@ open import Algebra.Structures _≈_
30
30
open import Relation.Binary
31
31
open import Function.Equality using (_⟨$⟩_)
32
32
open import Function.Equivalence using (_⇔_; module Equivalence )
33
- open import Data.Product using (_,_)
33
+ open import Data.Product.Base using (_,_)
34
34
35
35
------------------------------------------------------------------------
36
36
-- DEPRECATED NAMES
Original file line number Diff line number Diff line change 7
7
{-# OPTIONS --cubical-compatible --safe #-}
8
8
9
9
open import Algebra using (CommutativeMagma)
10
- open import Data.Product using (_×_; _,_; map)
10
+ open import Data.Product.Base using (_×_; _,_; map)
11
11
12
12
module Algebra.Properties.CommutativeMagma.Divisibility
13
13
{a ℓ} (CM : CommutativeMagma a ℓ)
Original file line number Diff line number Diff line change 7
7
{-# OPTIONS --cubical-compatible --safe #-}
8
8
9
9
open import Algebra using (CommutativeSemigroup)
10
- open import Data.Product using (_,_)
10
+ open import Data.Product.Base using (_,_)
11
11
import Relation.Binary.Reasoning.Setoid as EqReasoning
12
12
13
13
module Algebra.Properties.CommutativeSemigroup.Divisibility
Original file line number Diff line number Diff line change @@ -11,7 +11,7 @@ open import Algebra.Lattice.Bundles
11
11
open import Relation.Binary
12
12
open import Function.Base
13
13
open import Function.Bundles using (module Equivalence ; _⇔_)
14
- open import Data.Product using (_,_; swap)
14
+ open import Data.Product.Base using (_,_; swap)
15
15
16
16
module Algebra.Properties.Lattice {l₁ l₂} (L : Lattice l₁ l₂) where
17
17
Original file line number Diff line number Diff line change 7
7
{-# OPTIONS --cubical-compatible --safe #-}
8
8
9
9
open import Algebra using (Monoid)
10
- open import Data.Product using (_,_)
10
+ open import Data.Product.Base using (_,_)
11
11
open import Relation.Binary
12
12
13
13
module Algebra.Properties.Monoid.Divisibility
Original file line number Diff line number Diff line change 7
7
{-# OPTIONS --cubical-compatible --safe #-}
8
8
9
9
open import Algebra using (Semigroup)
10
- open import Data.Product using (_,_)
10
+ open import Data.Product.Base using (_,_)
11
11
open import Relation.Binary.Definitions using (Transitive)
12
12
13
13
module Algebra.Properties.Semigroup.Divisibility
Original file line number Diff line number Diff line change 8
8
9
9
open import Algebra using (Semiring)
10
10
import Algebra.Properties.Monoid.Divisibility as MonoidDivisibility
11
- open import Data.Product using (_,_)
11
+ open import Data.Product.Base using (_,_)
12
12
open import Data.Sum.Base using (_⊎_; inj₁; inj₂)
13
13
14
14
module Algebra.Properties.Semiring.Divisibility
Original file line number Diff line number Diff line change @@ -17,7 +17,7 @@ open import Data.Maybe.Base as Maybe
17
17
using (Maybe; decToMaybe; From-just; from-just)
18
18
open import Data.Nat as ℕ using (ℕ; zero; suc; _+_)
19
19
open import Data.Nat.GeneralisedArithmetic using (fold)
20
- open import Data.Product using (_×_; uncurry)
20
+ open import Data.Product.Base using (_×_; uncurry)
21
21
open import Data.Vec.Base using (Vec; []; _∷_; lookup; replicate)
22
22
23
23
open import Function.Base using (_∘_)
Original file line number Diff line number Diff line change @@ -15,7 +15,7 @@ open import Data.Fin.Base using (Fin; zero; suc)
15
15
open import Data.Maybe.Base as Maybe
16
16
using (Maybe; decToMaybe; From-just; from-just)
17
17
open import Data.Nat.Base as ℕ using (ℕ; zero; suc; _+_)
18
- open import Data.Product using (_×_; uncurry)
18
+ open import Data.Product.Base using (_×_; uncurry)
19
19
open import Data.Vec.Base using (Vec; []; _∷_; lookup; replicate)
20
20
21
21
open import Function.Base using (_∘_)
Original file line number Diff line number Diff line change @@ -12,7 +12,7 @@ import Algebra.Properties.Semiring.Mult as SemiringMultiplication
12
12
open import Data.Maybe.Base using (Maybe; just; nothing; map)
13
13
open import Algebra.Solver.Ring.AlmostCommutativeRing
14
14
open import Data.Nat.Base as ℕ
15
- open import Data.Product using (module Σ )
15
+ open import Data.Product.Base using (module Σ )
16
16
open import Function.Base using (id)
17
17
open import Relation.Binary.PropositionalEquality using (_≡_)
18
18
You can’t perform that action at this time.
0 commit comments