Skip to content
Merged
Show file tree
Hide file tree
Changes from 1 commit
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
7 changes: 7 additions & 0 deletions CHANGELOG.md
Original file line number Diff line number Diff line change
Expand Up @@ -32,6 +32,13 @@ New modules
Additions to existing modules
-----------------------------

* Exporting more `Raw` substructures from `Algebra.Bundles.Ring`:
```agda
rawNearSemiring : RawNearSemiring _ _
rawRingWithoutOne : RawRingWithoutOne _ _
+-rawGroup : RawGroup _ _
```

* In `Data.Fin.Properties`:
```agda
nonZeroIndex : Fin n → ℕ.NonZero n
Expand Down
6 changes: 6 additions & 0 deletions src/Algebra/Bundles.agda
Original file line number Diff line number Diff line change
Expand Up @@ -961,6 +961,9 @@ record Ring c ℓ : Set (suc (c ⊔ ℓ)) where
; semiringWithoutAnnihilatingZero
)

open NearSemiring nearSemiring public
using (rawNearSemiring)

open AbelianGroup +-abelianGroup public
using () renaming (group to +-group; invertibleMagma to +-invertibleMagma; invertibleUnitalMagma to +-invertibleUnitalMagma)

Expand All @@ -974,6 +977,9 @@ record Ring c ℓ : Set (suc (c ⊔ ℓ)) where
; 1# = 1#
}

open RawRing rawRing public
using (rawRingWithoutOne; +-rawGroup)


record CommutativeRing c ℓ : Set (suc (c ⊔ ℓ)) where
infix 8 -_
Expand Down