Move things around, add more to fields (#16)

This commit is contained in:
Patrick Stevens
2019-01-10 22:36:55 +00:00
committed by GitHub
parent 02434c01f9
commit 9e22ba78f5
31 changed files with 288 additions and 102 deletions

32
Numbers/Reals.agda Normal file
View File

@@ -0,0 +1,32 @@
{-# OPTIONS --safe --warning=error #-}
open import Fields
open import Rings
open import Functions
open import Orders
open import LogicalFormulae
open import Rationals
open import Naturals
open import Agda.Primitive using (Level; lzero; lsuc; _⊔_)
module Reals where
record Subset {m n : _} (A : Set m) (B : Set n) : Set (m n) where
field
inj : A B
injInj : Injection inj
--record RealField {n : _} {A : Set n} {R : Ring A} {F : Field R} : Set _ where
-- field
-- orderedField : OrderedField F
-- open OrderedField orderedField
-- open TotalOrder ord
-- open Ring R
-- field
-- complete : {c : _} {C : Set c} → (S : Subset C A) → (upperBound : A) → ({s : C} → (Subset.inj S s) < upperBound) → Sg A (λ lub → ({s : C} → (Subset.inj S s) < lub) && ({s : C} → (Subset.inj S s) < upperBound → (Subset.inj S s) < lub))
record Real : Set where
field
f :
converges : {ε : } Sg (λ x {y : } x <N y (f x) +Q (f y) <Q ε)