Files
agdaproofs/Numbers/Integers/Integers.agda
2019-11-17 17:37:10 +00:00

25 lines
900 B
Agda
Raw Permalink Blame History

This file contains ambiguous Unicode characters

This file contains Unicode characters that might be confused with other characters. If you think that this is intentional, you can safely ignore this warning. Use the Escape button to reveal them.

{-# OPTIONS --safe --warning=error --without-K #-}
open import Numbers.Naturals.Definition
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_) public
open import Numbers.Integers.RingStructure.IntegralDomain public using (IntDom) public
open import Numbers.Integers.RingStructure.Ring public using (Ring) public
open Numbers.Integers.Order using (_<Z_ ; OrderedRing) public
_-Z_ :
a -Z b = a +Z (Group.inverse Group b)
_^Z_ :
a ^Z zero = nonneg 1
a ^Z succ b = a *Z (a ^Z b)