mirror of
https://github.com/Smaug123/agdaproofs
synced 2025-10-15 00:18:39 +00:00
Move equiv rels (#46)
This commit is contained in:
@@ -13,6 +13,7 @@ open import Setoids.Orders
|
||||
open import Functions
|
||||
open import Fields.FieldOfFractions
|
||||
open import Fields.FieldOfFractionsOrder
|
||||
open import Sets.EquivalenceRelations
|
||||
|
||||
module Numbers.Rationals where
|
||||
|
||||
@@ -41,7 +42,7 @@ module Numbers.Rationals where
|
||||
a =Q b = Setoid._∼_ (fieldOfFractionsSetoid ℤIntDom) a b
|
||||
|
||||
reflQ : {x : ℚ} → (x =Q x)
|
||||
reflQ {x} = Reflexive.reflexive (Equivalence.reflexiveEq (Setoid.eq (fieldOfFractionsSetoid ℤIntDom))) {x}
|
||||
reflQ {x} = Equivalence.reflexive (Setoid.eq (fieldOfFractionsSetoid ℤIntDom)) {x}
|
||||
|
||||
_≤Q_ : ℚ → ℚ → Set
|
||||
a ≤Q b = (a <Q b) || (a =Q b)
|
||||
|
Reference in New Issue
Block a user