First Git commit

This commit is contained in:
Smaug123
2019-01-04 20:45:34 +00:00
commit a435e3764e
39 changed files with 9074 additions and 0 deletions

17
IntegralDomains.agda Normal file
View File

@@ -0,0 +1,17 @@
{-# OPTIONS --safe --warning=error #-}
open import LogicalFormulae
open import Groups
open import Naturals
open import Orders
open import Setoids
open import Functions
open import Rings
open import Agda.Primitive using (Level; lzero; lsuc; _⊔_)
module IntegralDomains where
record IntegralDomain {n m : _} {A : Set n} {S : Setoid {n} {m} A} {_+_ : A A A} {_*_ : A A A} (R : Ring S _+_ _*_) : Set (lsuc m n) where
field
intDom : {a b : A} Setoid.__ S (a * b) (Ring.0R R) (Setoid.__ S a (Ring.0R R)) || (Setoid.__ S b (Ring.0R R))
nontrivial : Setoid.__ S (Ring.1R R) (Ring.0R R) False