mirror of
https://github.com/Smaug123/agdaproofs
synced 2025-10-16 17:08:39 +00:00
More rings stuff (#83)
This commit is contained in:
@@ -18,5 +18,8 @@ open import Agda.Primitive using (Level; lzero; lsuc; _⊔_)
|
||||
|
||||
module Rings.Ideals.Prime.Definition {a b : _} {A : Set a} {S : Setoid {a} {b} A} {_+_ _*_ : A → A → A} {R : Ring S _+_ _*_} {c : _} {pred : A → Set c} (i : Ideal R pred) where
|
||||
|
||||
PrimeIdeal : Set (a ⊔ c)
|
||||
PrimeIdeal = {a b : A} → pred (a * b) → ((pred a) → False) → pred b
|
||||
record PrimeIdeal : Set (a ⊔ c) where
|
||||
field
|
||||
isPrime : {a b : A} → pred (a * b) → ((pred a) → False) → pred b
|
||||
notContained : A
|
||||
notContainedIsNotContained : (pred notContained) → False
|
||||
|
Reference in New Issue
Block a user