Skip to content

Commit 4c5e885

Browse files
committed
Tidy up: s/Set/Type + flags + levels
1 parent 2d7cb5c commit 4c5e885

Some content is hidden

Large Commits have some content hidden by default. Use the searchbox below for content that may be hidden.

43 files changed

+84
-105
lines changed

Class/Applicative.agda

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -1,4 +1,4 @@
1-
{-# OPTIONS --without-K #-}
1+
{-# OPTIONS --cubical-compatible #-}
22
module Class.Applicative where
33

44
open import Class.Applicative.Core public

Class/Applicative/Core.agda

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -1,4 +1,4 @@
1-
{-# OPTIONS --without-K #-}
1+
{-# OPTIONS --cubical-compatible #-}
22
module Class.Applicative.Core where
33

44
open import Class.Prelude

Class/Applicative/Instances.agda

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -1,4 +1,4 @@
1-
{-# OPTIONS --without-K #-}
1+
{-# OPTIONS --cubical-compatible #-}
22
module Class.Applicative.Instances where
33

44
open import Class.Prelude

Class/Bifunctor.agda

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -1,4 +1,4 @@
1-
{-# OPTIONS --without-K #-}
1+
{-# OPTIONS --cubical-compatible #-}
22
module Class.Bifunctor where
33

44
open import Class.Prelude hiding (A; B; C)

Class/CommutativeMonoid.agda

Lines changed: 1 addition & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -1,5 +1,4 @@
1-
{-# OPTIONS --safe --without-K #-}
2-
1+
{-# OPTIONS --cubical-compatible #-}
32
module Class.CommutativeMonoid where
43

54
open import Class.CommutativeMonoid.Core public

Class/CommutativeMonoid/Core.agda

Lines changed: 5 additions & 4 deletions
Original file line numberDiff line numberDiff line change
@@ -1,12 +1,12 @@
1-
{-# OPTIONS --safe --without-K #-}
2-
1+
{-# OPTIONS --cubical-compatible #-}
32
module Class.CommutativeMonoid.Core where
43

5-
import Algebra as Alg
64
open import Class.Prelude
75
open import Class.Semigroup
86
open import Class.Monoid
97

8+
import Algebra as Alg
9+
1010
record CommutativeMonoid c ℓ Carrier : Type (lsuc (c ⊔ ℓ)) where
1111
infix 4 _≈_
1212
field
@@ -19,7 +19,8 @@ module Conversion {c ℓ} where
1919
toBundle : {Carrier} CommutativeMonoid c ℓ Carrier Alg.CommutativeMonoid c ℓ
2020
toBundle c = record { CommutativeMonoid c }
2121

22-
fromBundle : (m : Alg.CommutativeMonoid c ℓ) CommutativeMonoid c ℓ (Alg.CommutativeMonoid.Carrier m)
22+
fromBundle : (m : Alg.CommutativeMonoid c ℓ)
23+
CommutativeMonoid c ℓ (Alg.CommutativeMonoid.Carrier m)
2324
fromBundle c = record
2425
{ Alg.CommutativeMonoid c using (_≈_; isCommutativeMonoid)
2526
; semigroup = λ where ._◇_ Alg.CommutativeMonoid._∙_ c

Class/CommutativeMonoid/Instances.agda

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -1,4 +1,4 @@
1-
{-# OPTIONS --safe --without-K #-}
1+
{-# OPTIONS --cubical-compatible #-}
22

33
module Class.CommutativeMonoid.Instances where
44

Class/Core.agda

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -1,4 +1,4 @@
1-
{-# OPTIONS --without-K #-}
1+
{-# OPTIONS --cubical-compatible #-}
22
module Class.Core where
33

44
open import Class.Prelude

Class/Default.agda

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -2,7 +2,7 @@
22
-- Types with a default value.
33
------------------------------------------------------------------------
44

5-
{-# OPTIONS --without-K #-}
5+
{-# OPTIONS --cubical-compatible #-}
66
module Class.Default where
77

88
open import Class.Prelude

Class/Foldable.agda

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -1,4 +1,4 @@
1-
{-# OPTIONS --without-K #-}
1+
{-# OPTIONS --cubical-compatible #-}
22
module Class.Foldable where
33

44
open import Class.Foldable.Core public

0 commit comments

Comments
 (0)