# HG changeset patch # User Shinji KONO # Date 1594706579 -32400 # Node ID 5e22b23ee3fd8710e29c639741235daae4919632 # Parent 811152bf2f472da163ddf3e862b816efd215fe92 ... diff -r 811152bf2f47 -r 5e22b23ee3fd README.md --- a/README.md Tue Jul 14 12:39:21 2020 +0900 +++ b/README.md Tue Jul 14 15:02:59 2020 +0900 @@ -85,27 +85,3 @@ They say the existing of the mappings can be proved in Classical Set Theory, but we simply assumes these non constructively. -## What have we done - -``` - Axioms of Ordinals - An implementation of countable Ordinal - ZF Axioms - Model of ZF based on OD/HOD - LEM axiom of choice from LEM - ODC LEM from axiom of choice - OPair classical ordered pair example - filter definition of filter and ideal - cardinal unfinished Cardinal number - BAlgebra boolean algebra of OD - -``` - - - - - - - - - diff -r 811152bf2f47 -r 5e22b23ee3fd zf-in-agda.html --- a/zf-in-agda.html Tue Jul 14 12:39:21 2020 +0900 +++ b/zf-in-agda.html Tue Jul 14 15:02:59 2020 +0900 @@ -341,7 +341,41 @@


-

A Model and a theory

+

Limit Ordinal

+If an ordinal is not a succesor of other, it is called limit ordinal. We need predicate to decide it. +

+ +

+     not-limit-p :  ( x : ord  ) → Dec ( ¬ ((y : ord) → ¬ (x ≡ osuc y) ))
+
+
+An ordinal may have an imeditate limit ordinal, we call it next x. Axiom of nrext is this. +

+ +

+    record IsNext {n : Level } (ord : Set n)  (o∅ : ord ) (osuc : ord → ord )  
+            (_o<_ : ord → ord → Set n) (next : ord → ord ) : Set (suc (suc n)) where
+       field
+         x<nx :    { y : ord } → (y o< next y )
+         osuc<nx : { x y : ord } → x o< next y → osuc x o< next y 
+         ¬nx<nx :  {x y : ord} → y o< x → x o< next y →  ¬ ((z : ord) → ¬ (x ≡ osuc z)) 
+
+
+We show some intresting lemma. +

+ +

+        next< : {x y z : Ordinal} → x o< next z  → y o< next x → y o< next z
+        nexto=n : {x y : Ordinal} → x o< next (osuc y)  → x o< next y 
+        nexto≡ : {x : Ordinal} → next x ≡ next (osuc x)  
+        next-is-limit : {x y : Ordinal} → ¬ (next x ≡ osuc y)
+
+
+These are proved from the axiom. Our countable ordinal satisfies these. +

+ +


+

A Model and a theory

Agda record is a type, so we can write it in the argument, but is it really exists?

If we have a value of the record, it simply exists, that is, we need to create all the existence @@ -358,7 +392,7 @@


-

postulate と module

+

postulate と module

Agda proofs are separated by modules, which are large records.

postulates are assumptions. We can assume a type without proofs. @@ -382,7 +416,7 @@


-

A ∨ B

+

A ∨ B

     data _∨_ (A B : Set) : Set where
@@ -411,7 +445,7 @@
 


-

Negation

+

Negation

        ⊥
@@ -447,7 +481,7 @@
 

-

Equality

+

Equality

All the value in Agda are terms. If we have the same normalized form, two terms are equal. @@ -481,7 +515,7 @@


-

Equivalence relation

+

Equivalence relation

@@ -498,7 +532,7 @@


-

Ordering

+

Ordering

Relation is a predicate on two value which has a same type. @@ -519,7 +553,7 @@


-

Quantifier

+

Quantifier

Handling quantifier in an intuitionistic logic requires special cares. @@ -543,7 +577,7 @@


-

Can we do math in this way?

+

Can we do math in this way?

Yes, we can. Actually we have Principia Mathematica by Russell and Whitehead (with out computer support).

In some sense, this story is a reprinting of the work, (but Principia Mathematica has a different formulation than ZF). @@ -556,7 +590,7 @@


-

Things which Agda cannot prove

+

Things which Agda cannot prove

The infamous Internal Parametricity is a limitation of Agda, it cannot prove so called Free Theorem, which @@ -586,7 +620,7 @@


-

Classical story of ZF Set Theory

+

Classical story of ZF Set Theory

@@ -603,7 +637,7 @@


-

Ordinals

+

Ordinals

Ordinals are our intuition of infinite things, which has ∅ and orders on the things. It also has a successor osuc.

@@ -623,7 +657,7 @@


-

Axiom of Ordinals

+

Axiom of Ordinals

Properties of infinite things. We request a transfinite induction, which states that if some properties are satisfied below all possible ordinals, the properties are true on all ordinals. @@ -651,7 +685,7 @@
-

Concrete Ordinals or Countable Ordinals

+

Concrete Ordinals or Countable Ordinals

We can define a list like structure with level, which is a kind of two dimensional infinite array. @@ -684,7 +718,7 @@


-

Model of Ordinals

+

Model of Ordinals

It is easy to show OrdinalD and its order satisfies the axioms of Ordinals. @@ -693,7 +727,7 @@


-

Debugging axioms using Model

+

Debugging axioms using Model

Whether axiom is correct or not can be checked by a validity on a mode.

If not, we may fix the axioms or the model, such as the definitions of the order. @@ -702,7 +736,7 @@


-

Countable Ordinals can contains uncountable set?

+

Countable Ordinals can contains uncountable set?

Yes, the ordinals contains any level of infinite Set in the axioms.

If we handle real-number in the model, only countable number of real-number is used. @@ -720,7 +754,7 @@


-

What is Set

+

What is Set

The word Set in Agda is not a Set of ZF Set, but it is a type (why it is named Set?).

From naive point view, a set i a list, but in Agda, elements have all the same type. @@ -730,7 +764,7 @@


-

We don't ask the contents of Set. It can be anything.

+

We don't ask the contents of Set. It can be anything.

From empty set φ, we can think a set contains a φ, and a pair of φ and the set, and so on, and all of them, and again we repeat this.

@@ -751,7 +785,7 @@


-

Ordinal Definable Set

+

Ordinal Definable Set

We can define a sbuset of Ordinals using predicates. What is a subset?

@@ -782,7 +816,7 @@


-

OD is not ZF Set

+

OD is not ZF Set

If we have 1 to 1 mapping between an OD and an Ordinal, OD contains several ODs and OD looks like a Set. The idea is to use an ordinal as a pointer to OD. Unfortunately this scheme does not work well. As we saw OD includes all Ordinals, which is a maximum of OD, but Ordinals has no maximum at all. So we have a contradction like @@ -800,7 +834,7 @@


-

HOD : Hereditarily Ordinal Definable

+

HOD : Hereditarily Ordinal Definable

What we need is a bounded OD, the containment is limited by an ordinal.

@@ -823,7 +857,7 @@


-

1 to 1 mapping between an HOD and an Ordinal

+

1 to 1 mapping between an HOD and an Ordinal

HOD is a predicate on Ordinals and the solution is bounded by some ordinal. If we have a mapping

@@ -859,7 +893,7 @@


-

Order preserving in the mapping of OD and Ordinal

+

Order preserving in the mapping of OD and Ordinal

Ordinals have the order and HOD has a natural order based on inclusion ( def / ∋ ).

@@ -891,7 +925,7 @@


-

Various Sets

+

Various Sets

In classical Set Theory, there is a hierarchy call L, which can be defined by a predicate.

@@ -906,7 +940,7 @@


-

Fixes on ZF to intuitionistic logic

+

Fixes on ZF to intuitionistic logic

We use ODs as Sets in ZF, and defines record ZF, that is, we have to define @@ -924,7 +958,7 @@


-

Pure logical axioms

+

Pure logical axioms

    empty, pair, select, ε-induction??infinity
@@ -959,7 +993,7 @@
 


-

Axiom of Pair

+

Axiom of Pair

In the Tanaka's book, axiom of pair is as follows.

@@ -986,7 +1020,7 @@


-

pair in OD

+

pair in OD

OD is an equation on Ordinals, we can simply write axiom of pair in the OD.

@@ -1001,7 +1035,7 @@


-

Validity of Axiom of Pair

+

Validity of Axiom of Pair

Assuming ZFSet is OD, we are going to prove pair→ .

@@ -1042,7 +1076,7 @@


-

Equality of OD and Axiom of Extensionality

+

Equality of OD and Axiom of Extensionality

OD is defined by a predicates, if we compares normal form of the predicates, even if it contains the same elements, it may be different, which is no good as an equality of Sets. @@ -1104,7 +1138,7 @@

-

Validity of Axiom of Extensionality

+

Validity of Axiom of Extensionality

If we can derive (w ∋ A) ⇔ (w ∋ B) from od A == od B, the axiom becomes valid, but it seems impossible, so we assumes @@ -1125,7 +1159,110 @@


-

Non constructive assumptions so far

+

Axiom of infinity

+ +

+It means it has ω as a ZF Set. It is ususally written like this. +

+ +

+     ∃ A ( ∅ ∈ A ∧ ∀ x ∈ A ( x ∪ { x } ∈ A ) )
+
+
+x ∪ { x } is Union (x , (x , x)) in our notation. It contains existential quantifier, so we introduce a function +

+ +

+     infinite : ZFSet
+     infinity∅ :  ∅ ∈ infinite
+     infinity :  ∀( x : ZFSet  ) → x ∈ infinite →  ( x ∪ { x }) ∈ infinite 
+
+
+ +
+

ω in HOD

+ +

+To define an OD which arrows od→ord (Union (x , (x , x))) as a predicate, we can use Agda data structure. +

+ +

+    data infinite-d  : ( x : Ordinal  ) → Set n where
+        iφ :  infinite-d o∅
+        isuc : {x : Ordinal  } →   infinite-d  x  →
+                infinite-d  (od→ord ( Union (ord→od x , (ord→od x , ord→od x ) ) ))
+
+
+It has simular structure as Data.Nat in Agda, and it defines a correspendence of HOD and the data structure. Now +we can define HOD like this. +

+ +

+    infinite : HOD 
+    infinite = record { od = record { def = λ x → infinite-d x } ; odmax = ? ; <odmax = ? } 
+
+
+So what is the bound of ω? Analyzing the definition, it depends on the value of od→ord (x , x), which +cannot know the aboslute value. This is because we don't have constructive definition of od→ord : HOD → Ordinal. +

+We need some restriction on the HOD-Ordinal mapping. Simple one is this. +

+ +

+        ωmax : Ordinal
+        <ωmax : {y : Ordinal} → infinite-d y → y o< ωmax
+
+
+It depends on infinite-d and put no assuption on the other similar construction. A more general one may be +

+ +

+        hod-ord< :  {x : HOD } → Set n
+        hod-ord< {x} =  od→ord x o< next (odmax x)
+
+
+next : Ordinal → Ordinal means imediate next limit ordinal of x. It supress unecessary space between address of HOD and +its bound. +

+In other words, the space between address of HOD and its bound is arbitrary, it is possible to assume ω has no bound. +This is the reason of necessity of Axiom of infinite. +

+ +


+

increment pase of address of HOD

+The address of HOD may have obvious bound, but it is defined in a relative way. +

+ +

+    pair-xx<xy : {x y : HOD} → od→ord (x , x) o< osuc (od→ord (x , y) )
+    pair<y : {x y : HOD } → y ∋ x  → od→ord (x , x) o< osuc (od→ord y)
+
+
+Basicaly, we cannot know the concrete address of HOD other than empty set. +

+Assuming, previous assuption, we have +

+ +

+    pair-ord< : {x : HOD } → ( {y : HOD } → od→ord y o< next (odmax y) ) → od→ord ( x , x ) o< next (od→ord x)
+    pair-ord< {x} ho< = subst (λ k → od→ord (x , x) o< k ) lemmab0 lemmab1  where
+           lemmab0 : next (odmax (x , x)) ≡ next (od→ord x)
+
+
+So the address of ( x , x) and Union (x , (x , x)) is restricted in the limit ordinal. This makes ω bound. +

+We also notice that if we have od→ord (x , x) ≡ osuc (od→ord x), c<→o< can be drived from ⊆→o≤ . +

+ +

+    ⊆→o≤→c<→o< : ({x : HOD} → od→ord (x , x) ≡ osuc (od→ord x) )
+       →  ({y z : HOD  }   → ({x : Ordinal} → def (od y) x → def (od z) x ) → od→ord y o< osuc (od→ord z) )
+       →   {x y : HOD  }   → def (od y) ( od→ord x ) → od→ord x o< od→ord y 
+
+
+ +
+

Non constructive assumptions so far

@@ -1143,7 +1280,7 @@


-

Axiom which have negation form

+

Axiom which have negation form

@@ -1167,7 +1304,7 @@


-

Union

+

Union

The original form of the Axiom of Union is

@@ -1183,25 +1320,28 @@ union← : ( X z : ZFSet ) → (X∋z : Union X ∋ z ) → ¬ ( (u : ZFSet ) → ¬ ((X ∋ u) ∧ (u ∋ z ))) -The definition of Union in OD is like this. +The definition of Union in HOD is like this.

-    Union : OD  → OD   
-    Union U = record { def = λ x → ¬ (∀ (u : Ordinal ) → ¬ ((def U u) ∧ (def (ord→od u) x)))  }
+    Union : HOD  → HOD   
+    Union U = record { od = record { def = λ x → ¬ (∀ (u : Ordinal ) → ¬ ((odef U u) ∧ (odef (ord→od u) x)))  }
+       ; odmax = osuc (od→ord U) ; <odmax = ?  } 
 
 
+The bound of Union is evident, but its proof is rather complicated. +

Proof of validity is straight forward.

-         union→ :  (X z u : OD) → (X ∋ u) ∧ (u ∋ z) → Union X ∋ z
+         union→ :  (X z u : HOD) → (X ∋ u) ∧ (u ∋ z) → Union X ∋ z
          union→ X z u xx not = ⊥-elim ( not (od→ord u) ( record { proj1 = proj1 xx
-              ; proj2 = subst ( λ k → def k (od→ord z)) (sym oiso) (proj2 xx) } ))
-         union← :  (X z : OD) (X∋z : Union X ∋ z) →  ¬  ( (u : OD ) → ¬ ((X ∋  u) ∧ (u ∋ z )))
+              ; proj2 = subst ( λ k → odef k (od→ord z)) (sym oiso) (proj2 xx) } ))
+         union← :  (X z : HOD) (X∋z : Union X ∋ z) →  ¬  ( (u : HOD ) → ¬ ((X ∋  u) ∧ (u ∋ z )))
          union← X z UX∋z =  FExists _ lemma UX∋z where
-              lemma : {y : Ordinal} → def X y ∧ def (ord→od y) (od→ord z) → ¬ ((u : OD) → ¬ (X ∋ u) ∧ (u ∋ z))
-              lemma {y} xx not = not (ord→od y) record { proj1 = subst ( λ k → def X k ) (sym diso) (proj1 xx ) ; proj2 = proj2 xx }
+              lemma : {y : Ordinal} → odef X y ∧ odef (ord→od y) (od→ord z) → ¬ ((u : HOD) → ¬ (X ∋ u) ∧ (u ∋ z))
+              lemma {y} xx not = not (ord→od y) record { proj1 = subst ( λ k → odef X k ) (sym diso) (proj1 xx ) ; proj2 = proj2 xx } 
 
 
where @@ -1219,7 +1359,7 @@


-

Axiom of replacement

+

Axiom of replacement

We can replace the elements of a set by a function and it becomes a set. From the book,

@@ -1231,7 +1371,7 @@

-     Replace : OD  → (OD  → OD  ) → OD
+     Replace : HOD  → (HOD  → HOD  ) → HOD
 
 
The axioms becomes as follows. @@ -1251,19 +1391,26 @@ in-codomain X ψ = record { def = λ x → ¬ ( (y : Ordinal ) → ¬ ( def X y ∧ ( x ≡ od→ord (ψ (ord→od y ))))) } -Besides this upper bounds is required. +in-codomain is a logical relation-ship, and it is written in OD.

-    Replace : OD  → (OD  → OD  ) → OD 
-    Replace X ψ = record { def = λ x → (x o< sup-o  ( λ x → od→ord (ψ (ord→od x )))) ∧ def (in-codomain X ψ) x }
+    Replace : HOD  → (HOD  → HOD) → HOD 
+    Replace X ψ = record { od = record { def = λ x → (x o< sup-o X (λ y X∋y → od→ord (ψ (ord→od y)))) ∧ def (in-codomain X ψ) x }
+       ; odmax = rmax ; <odmax = rmax<} where 
+          rmax : Ordinal
+          rmax = sup-o X (λ y X∋y → od→ord (ψ (ord→od y)))
+          rmax< :  {y : Ordinal} → (y o< rmax) ∧ def (in-codomain X ψ) y → y o< rmax
+          rmax< lt = proj1 lt
 
 
-We omit the proof of the validity, but it is rather straight forward. +The bbound of Replace is defined by supremum, that is, it is not limited in a limit ordinal of original ZF Set. +

+Once we have a bound, validity of the axiom is an easy task to check the logical relation-ship.


-

Validity of Power Set Axiom

+

Validity of Power Set Axiom

The original Power Set Axiom is this.

@@ -1300,15 +1447,17 @@

-    ZFSubset : (A x : OD  ) → OD 
-    ZFSubset A x =  record { def = λ y → def A y ∧  def x y }  
+   ZFSubset : (A x : HOD  ) → HOD 
+   ZFSubset A x =  record { od = record { def = λ y → odef A y ∧  odef x y } ; odmax = omin (odmax A) (odmax x) ; <odmax = lemma }  where 
+     lemma : {y : Ordinal} → def (od A) y ∧ def (od x) y → y o< omin (odmax A) (odmax x)
+     lemma {y} and = min1 (<odmax A (proj1 and)) (<odmax x (proj2 and))
 
 
We can prove,

-    ( {y : OD } → x ∋ y → ZFSubset A x ∋  y ) ⇔  ( x ⊆ A  ) 
+    ( {y : HOD } → x ∋ y → ZFSubset A x ∋  y ) ⇔  ( x ⊆ A  ) 
 
 
We only have upper bound as an ordinal, but we have an obvious OD based on the order of Ordinals, @@ -1334,27 +1483,27 @@

-     ∩-≡ :  { a b : OD  } → ({x : OD  } → (a ∋ x → b ∋ x)) → a == ( b ∩ a )
+     ∩-≡ :  { a b : HOD  } → ({x : HOD  } → (a ∋ x → b ∋ x)) → od a == od ( b ∩ a )
 
 
In case of Ord a intro of Power Set axiom becomes valid.

-    ord-power← : (a : Ordinal ) (t : OD) → ({x : OD} → (t ∋ x → (Ord a) ∋ x)) → Def (Ord a) ∋ t
+    ord-power← : (a : Ordinal ) (t : HOD) → ({x : HOD} → (t ∋ x → (Ord a) ∋ x)) → OPwr (Ord a) ∋ t
 
 
Using this, we can prove,

-         power→ :  ( A t : OD) → Power A ∋ t → {x : OD} → t ∋ x → ¬ ¬ (A ∋ x)
-         power← :  (A t : OD) → ({x : OD} → (t ∋ x → A ∋ x)) → Power A ∋ t
+         power→ :  ( A t : HOD) → Power A ∋ t → {x : HOD} → t ∋ x → ¬ ¬ (A ∋ x)
+         power← :  (A t : HOD) → ({x : HOD} → (t ∋ x → A ∋ x)) → Power A ∋ t
 
 

-

Axiom of regularity, Axiom of choice, ε-induction

+

Axiom of regularity, Axiom of choice, ε-induction

Axiom of regularity requires non self intersectable elements (which is called minimum), if we @@ -1365,9 +1514,9 @@

-  minimal : (x : OD  ) → ¬ (x == od∅ )→ OD
-  x∋minimal : (x : OD  ) → ( ne : ¬ (x == od∅ ) ) → def x ( od→ord ( minimal x ne ) )
-  minimal-1 : (x : OD  ) → ( ne : ¬ (x == od∅ ) ) → (y : OD ) → ¬ ( def (minimal x ne) (od→ord y)) ∧ (def x (od→ord  y) )
+  minimal : (x : HOD  ) → ¬ (x == od∅ )→ OD
+  x∋minimal : (x : HOD  ) → ( ne : ¬ (x == od∅ ) ) → def x ( od→ord ( minimal x ne ) )
+  minimal-1 : (x : HOD  ) → ( ne : ¬ (x == od∅ ) ) → (y : HOD ) → ¬ ( def (minimal x ne) (od→ord y)) ∧ (def x (od→ord  y) )
 
 
We can avoid this using ε-induction (a predicate is valid on all set if the predicate is true on some element of set). @@ -1375,9 +1524,9 @@

-    ε-induction : { ψ : OD  → Set (suc n)}
-       → ( {x : OD } → ({ y : OD } →  x ∋ y → ψ y ) → ψ x )
-       → (x : OD ) → ψ x
+    ε-induction : { ψ : HOD  → Set (suc n)}
+       → ( {x : HOD } → ({ y : HOD } →  x ∋ y → ψ y ) → ψ x )
+       → (x : HOD ) → ψ x
 
 
In our model, we assumes the mapping between Ordinals and OD, this is actually the TransFinite induction in Ordinals. @@ -1401,8 +1550,8 @@


-

Axiom of choice and Law of Excluded Middle

-In our model, since OD has a mapping to Ordinals, it has evident order, which means well ordering theorem is valid, +

Axiom of choice and Law of Excluded Middle

+In our model, since HOD has a mapping to Ordinals, it has evident order, which means well ordering theorem is valid, but it don't have correct form of the axiom yet. They say well ordering axiom is equivalent to the axiom of choice, but it requires law of the exclude middle.

@@ -1412,7 +1561,7 @@

-    ppp :  { p : Set n } { a : OD  } → record { def = λ x → p } ∋ a → p
+    ppp :  { p : Set n } { a : HOD  } → record { def = λ x → p } ∋ a → p
     ppp  {p} {a} d = d
 
 
@@ -1421,51 +1570,59 @@


-

Relation-ship among ZF axiom

+

Relation-ship among ZF axiom


-

Non constructive assumption in our model

-mapping between OD and Ordinals +

Non constructive assumption in our model

+mapping between HOD and Ordinals

-  od→ord : OD  → Ordinal
+  od→ord : HOD  → Ordinal
   ord→od : Ordinal  → OD
-  oiso   :  {x : OD }      → ord→od ( od→ord x ) ≡ x
+  oiso   :  {x : HOD }      → ord→od ( od→ord x ) ≡ x
   diso   :  {x : Ordinal } → od→ord ( ord→od x ) ≡ x
-  c<→o<  :  {x y : OD  }   → def y ( od→ord x ) → od→ord x o< od→ord y
+  c<→o<  :  {x y : HOD  }   → def y ( od→ord x ) → od→ord x o< od→ord y
+  ⊆→o≤   :  {y z : HOD  }   → ({x : Ordinal} → def (od y) x → def (od z) x ) → od→ord y o< osuc (od→ord z)
 
 
Equivalence on OD

-  ==→o≡ : { x y : OD  } → (x == y) → x ≡ y
+  ==→o≡ : { x y : HOD  } → (od x == od y) → x ≡ y
 
 
Upper bound

-  sup-o  :  ( Ordinal  → Ordinal ) →  Ordinal
-  sup-o< :  { ψ : Ordinal  →  Ordinal } → ∀ {x : Ordinal } → ψ x  o<  sup-o ψ
+  sup-o  :  (A : HOD) → (     ( x : Ordinal ) → def (od A) x →  Ordinal ) →  Ordinal 
+  sup-o< :  (A : HOD) → { ψ : ( x : Ordinal ) → def (od A) x →  Ordinal } → ∀ {x : Ordinal } → (lt : def (od A) x ) → ψ x lt o<  sup-o A ψ 
+
+
+In order to have bounded ω, +

+ +

+  hod-ord< : {x : HOD} →  od→ord x o< next (odmax x)
 
 
Axiom of choice and strong axiom of regularity.

-  minimal : (x : OD  ) → ¬ (x == od∅ )→ OD
-  x∋minimal : (x : OD  ) → ( ne : ¬ (x == od∅ ) ) → def x ( od→ord ( minimal x ne ) )
-  minimal-1 : (x : OD  ) → ( ne : ¬ (x == od∅ ) ) → (y : OD ) → ¬ ( def (minimal x ne) (od→ord y)) ∧ (def x (od→ord  y) )
+  minimal : (x : HOD  ) → ¬ (x =h= od∅ )→ HOD 
+  x∋minimal : (x : HOD  ) → ( ne : ¬ (x =h= od∅ ) ) → odef x ( od→ord ( minimal x ne ) )
+  minimal-1 : (x : HOD  ) → ( ne : ¬ (x =h= od∅ ) ) → (y : HOD ) → ¬ ( odef (minimal x ne) (od→ord y)) ∧ (odef x (od→ord  y) )
 
 

-

So it this correct?

+

So it this correct?

Our axiom are syntactically the same in the text book, but negations are slightly different. @@ -1476,7 +1633,7 @@

Except the upper bound, axioms are simple logical relation.

-Proof of existence of mapping between OD and Ordinals are not obvious. We don't know we prove it or not. +Proof of existence of mapping between HOD and Ordinals are not obvious. We don't know we prove it or not.

Existence of the Upper bounds is a pure assumption, if we have not limit on Ordinals, it may contradicts, but we don't have explicit upper limit on Ordinals. @@ -1485,7 +1642,7 @@


-

How to use Agda Set Theory

+

How to use Agda Set Theory

Assuming record ZF, classical set theory can be developed. If necessary, axiom of choice can be postulated or assuming law of excluded middle.

@@ -1496,7 +1653,7 @@


-

Topos and Set Theory

+

Topos and Set Theory

Topos is a mathematical structure in Category Theory, which is a Cartesian closed category which has a sub-object classifier.

@@ -1514,7 +1671,7 @@


-

Cardinal number and Continuum hypothesis

+

Cardinal number and Continuum hypothesis

Axiom of choice is required to define cardinal number

definition of cardinal number is not yet done @@ -1532,7 +1689,7 @@


-

Filter

+

Filter

filter is a dual of ideal on boolean algebra or lattice. Existence on natural number @@ -1540,13 +1697,13 @@

-    record Filter  ( L : OD  ) : Set (suc n) where
+    record Filter  ( L : HOD  ) : Set (suc n) where
        field
            filter : OD
            proper : ¬ ( filter ∋ od∅ )
            inL :  filter ⊆ L 
-           filter1 : { p q : OD } →  q ⊆ L  → filter ∋ p →  p ⊆ q  → filter ∋ q
-           filter2 : { p q : OD } → filter ∋ p →  filter ∋ q  → filter ∋ (p ∩ q)
+           filter1 : { p q : HOD } →  q ⊆ L  → filter ∋ p →  p ⊆ q  → filter ∋ q
+           filter2 : { p q : HOD } → filter ∋ p →  filter ∋ q  → filter ∋ (p ∩ q)
 
 
We may construct a model of non standard analysis or set theory. @@ -1555,7 +1712,7 @@


-

Programming Mathematics

+

Programming Mathematics

Mathematics is a functional programming in Agda where proof is a value of a variable. The mathematical structure are

@@ -1580,7 +1737,7 @@


-

link

+

link

Summer school of foundation of mathematics (in Japanese)
https://www.sci.shizuoka.ac.jp/~math/yorioka/ss2019/

Foundation of axiomatic set theory (in Japanese)
https://www.sci.shizuoka.ac.jp/~math/yorioka/ss2019/sakai0.pdf @@ -1613,55 +1770,59 @@

  • A ∧ B
  • record
  • Mathematical structure -
  • A Model and a theory -
  • postulate と module -
  • A ∨ B -
  • Negation -
  • Equality -
  • Equivalence relation -
  • Ordering -
  • Quantifier -
  • Can we do math in this way? -
  • Things which Agda cannot prove -
  • Classical story of ZF Set Theory -
  • Ordinals -
  • Axiom of Ordinals -
  • Concrete Ordinals or Countable Ordinals -
  • Model of Ordinals -
  • Debugging axioms using Model -
  • Countable Ordinals can contains uncountable set? -
  • What is Set -
  • We don't ask the contents of Set. It can be anything. -
  • Ordinal Definable Set -
  • OD is not ZF Set -
  • HOD : Hereditarily Ordinal Definable -
  • 1 to 1 mapping between an HOD and an Ordinal -
  • Order preserving in the mapping of OD and Ordinal -
  • Various Sets -
  • Fixes on ZF to intuitionistic logic -
  • Pure logical axioms -
  • Axiom of Pair -
  • pair in OD -
  • Validity of Axiom of Pair -
  • Equality of OD and Axiom of Extensionality -
  • Validity of Axiom of Extensionality -
  • Non constructive assumptions so far -
  • Axiom which have negation form -
  • Union -
  • Axiom of replacement -
  • Validity of Power Set Axiom -
  • Axiom of regularity, Axiom of choice, ε-induction -
  • Axiom of choice and Law of Excluded Middle -
  • Relation-ship among ZF axiom -
  • Non constructive assumption in our model -
  • So it this correct? -
  • How to use Agda Set Theory -
  • Topos and Set Theory -
  • Cardinal number and Continuum hypothesis -
  • Filter -
  • Programming Mathematics -
  • link +
  • Limit Ordinal +
  • A Model and a theory +
  • postulate と module +
  • A ∨ B +
  • Negation +
  • Equality +
  • Equivalence relation +
  • Ordering +
  • Quantifier +
  • Can we do math in this way? +
  • Things which Agda cannot prove +
  • Classical story of ZF Set Theory +
  • Ordinals +
  • Axiom of Ordinals +
  • Concrete Ordinals or Countable Ordinals +
  • Model of Ordinals +
  • Debugging axioms using Model +
  • Countable Ordinals can contains uncountable set? +
  • What is Set +
  • We don't ask the contents of Set. It can be anything. +
  • Ordinal Definable Set +
  • OD is not ZF Set +
  • HOD : Hereditarily Ordinal Definable +
  • 1 to 1 mapping between an HOD and an Ordinal +
  • Order preserving in the mapping of OD and Ordinal +
  • Various Sets +
  • Fixes on ZF to intuitionistic logic +
  • Pure logical axioms +
  • Axiom of Pair +
  • pair in OD +
  • Validity of Axiom of Pair +
  • Equality of OD and Axiom of Extensionality +
  • Validity of Axiom of Extensionality +
  • Axiom of infinity +
  • ω in HOD +
  • increment pase of address of HOD +
  • Non constructive assumptions so far +
  • Axiom which have negation form +
  • Union +
  • Axiom of replacement +
  • Validity of Power Set Axiom +
  • Axiom of regularity, Axiom of choice, ε-induction +
  • Axiom of choice and Law of Excluded Middle +
  • Relation-ship among ZF axiom +
  • Non constructive assumption in our model +
  • So it this correct? +
  • How to use Agda Set Theory +
  • Topos and Set Theory +
  • Cardinal number and Continuum hypothesis +
  • Filter +
  • Programming Mathematics +
  • link -
    Shinji KONO / Tue Jul 7 15:44:35 2020 +
    Shinji KONO / Tue Jul 14 15:02:38 2020 diff -r 811152bf2f47 -r 5e22b23ee3fd zf-in-agda.ind --- a/zf-in-agda.ind Tue Jul 14 12:39:21 2020 +0900 +++ b/zf-in-agda.ind Tue Jul 14 15:02:59 2020 +0900 @@ -234,6 +234,30 @@ Fields of Ordinal is existential objects in the mathematical structure. +-- Limit Ordinal + +If an ordinal is not a succesor of other, it is called limit ordinal. We need predicate to decide it. + + not-limit-p : ( x : ord ) → Dec ( ¬ ((y : ord) → ¬ (x ≡ osuc y) )) + +An ordinal may have an imeditate limit ordinal, we call it next x. Axiom of nrext is this. + + record IsNext {n : Level } (ord : Set n) (o∅ : ord ) (osuc : ord → ord ) + (_o<_ : ord → ord → Set n) (next : ord → ord ) : Set (suc (suc n)) where + field + x