mirror of
https://github.com/Smaug123/agdaproofs
synced 2025-10-15 08:28:39 +00:00
18 lines
356 B
Agda
18 lines
356 B
Agda
{-# OPTIONS --safe --warning=error #-}
|
||
|
||
open import LogicalFormulae
|
||
open import Naturals
|
||
open import Integers
|
||
open import Groups
|
||
open import Rings
|
||
open import Fields
|
||
open import PrimeNumbers
|
||
open import Setoids
|
||
open import Functions
|
||
open import FieldOfFractions
|
||
|
||
module Rationals where
|
||
|
||
ℚ : Field'
|
||
ℚ = encapsulateField (fieldOfFractions ℤIntDom)
|