mirror of
https://github.com/Smaug123/agdaproofs
synced 2025-10-14 07:58:41 +00:00
Split out Integers and remove use of K (#39)
This commit is contained in:
17
Numbers/Integers/Integers.agda
Normal file
17
Numbers/Integers/Integers.agda
Normal file
@@ -0,0 +1,17 @@
|
||||
{-# OPTIONS --safe --warning=error --without-K #-}
|
||||
|
||||
open import Numbers.Integers.Definition
|
||||
open import Numbers.Integers.Addition
|
||||
open import Numbers.Integers.Multiplication
|
||||
open import Numbers.Integers.Order
|
||||
open import Groups.Definition
|
||||
|
||||
module Numbers.Integers.Integers where
|
||||
|
||||
open Numbers.Integers.Definition using (ℤ ; nonneg ; negSucc) public
|
||||
open Numbers.Integers.Addition using (_+Z_ ; ℤGroup ; ℤAbGrp) public
|
||||
open Numbers.Integers.Multiplication using (_*Z_ ; ℤIntDom ; ℤRing) public
|
||||
open Numbers.Integers.Order using (_<Z_ ; ℤOrderedRing) public
|
||||
|
||||
_-Z_ : ℤ → ℤ → ℤ
|
||||
a -Z b = a +Z (Group.inverse ℤGroup b)
|
Reference in New Issue
Block a user