HomeHome Intuitionistic Logic Explorer
Theorem List (p. 134 of 135)
< Previous  Next >
Bad symbols? Try the
GIF version.

Mirrors  >  Metamath Home Page  >  ILE Home Page  >  Theorem List Contents  >  Recent Proofs       This page: Page List

Theorem List for Intuitionistic Logic Explorer - 13301-13400   *Has distinct variable group(s)
TypeLabelDescription
Statement
 
Theorembj-indind 13301* If 𝐴 is inductive and 𝐵 is "inductive in 𝐴", then (𝐴𝐵) is inductive. (Contributed by BJ, 25-Oct-2020.)
((Ind 𝐴 ∧ (∅ ∈ 𝐵 ∧ ∀𝑥𝐴 (𝑥𝐵 → suc 𝑥𝐵))) → Ind (𝐴𝐵))
 
Theorembj-dfom 13302 Alternate definition of ω, as the intersection of all the inductive sets. Proposal: make this the definition. (Contributed by BJ, 30-Nov-2019.)
ω = {𝑥 ∣ Ind 𝑥}
 
Theorembj-omind 13303 ω is an inductive class. (Contributed by BJ, 30-Nov-2019.)
Ind ω
 
Theorembj-omssind 13304 ω is included in all the inductive sets (but for the moment, we cannot prove that it is included in all the inductive classes). (Contributed by BJ, 30-Nov-2019.) (Proof modification is discouraged.)
(𝐴𝑉 → (Ind 𝐴 → ω ⊆ 𝐴))
 
Theorembj-ssom 13305* A characterization of subclasses of ω. (Contributed by BJ, 30-Nov-2019.) (Proof modification is discouraged.)
(∀𝑥(Ind 𝑥𝐴𝑥) ↔ 𝐴 ⊆ ω)
 
Theorembj-om 13306* A set is equal to ω if and only if it is the smallest inductive set. (Contributed by BJ, 30-Nov-2019.) (Proof modification is discouraged.)
(𝐴𝑉 → (𝐴 = ω ↔ (Ind 𝐴 ∧ ∀𝑥(Ind 𝑥𝐴𝑥))))
 
Theorembj-2inf 13307* Two formulations of the axiom of infinity (see ax-infvn 13310 and bj-omex 13311) . (Contributed by BJ, 30-Nov-2019.) (Proof modification is discouraged.)
(ω ∈ V ↔ ∃𝑥(Ind 𝑥 ∧ ∀𝑦(Ind 𝑦𝑥𝑦)))
 
11.2.8.3  The first three Peano postulates

The first three Peano postulates follow from constructive set theory (actually, from its core axioms). The proofs peano1 4516 and peano3 4518 already show this. In this section, we prove bj-peano2 13308 to complete this program. We also prove a preliminary version of the fifth Peano postulate from the core axioms.

 
Theorembj-peano2 13308 Constructive proof of peano2 4517. Temporary note: another possibility is to simply replace sucexg 4422 with bj-sucexg 13291 in the proof of peano2 4517. (Contributed by BJ, 18-Nov-2019.) (Proof modification is discouraged.)
(𝐴 ∈ ω → suc 𝐴 ∈ ω)
 
Theorempeano5set 13309* Version of peano5 4520 when ω ∩ 𝐴 is assumed to be a set, allowing a proof from the core axioms of CZF. (Contributed by BJ, 19-Nov-2019.) (Proof modification is discouraged.)
((ω ∩ 𝐴) ∈ 𝑉 → ((∅ ∈ 𝐴 ∧ ∀𝑥 ∈ ω (𝑥𝐴 → suc 𝑥𝐴)) → ω ⊆ 𝐴))
 
11.2.9  CZF: Infinity

In the absence of full separation, the axiom of infinity has to be stated more precisely, as the existence of the smallest class containing the empty set and the successor of each of its elements.

 
11.2.9.1  The set of natural numbers (finite ordinals)

In this section, we introduce the axiom of infinity in a constructive setting (ax-infvn 13310) and deduce that the class ω of finite ordinals is a set (bj-omex 13311).

 
Axiomax-infvn 13310* Axiom of infinity in a constructive setting. This asserts the existence of the special set we want (the set of natural numbers), instead of the existence of a set with some properties (ax-iinf 4510) from which one then proves, using full separation, that the wanted set exists (omex 4515). "vn" is for "von Neumann". (Contributed by BJ, 14-Nov-2019.)
𝑥(Ind 𝑥 ∧ ∀𝑦(Ind 𝑦𝑥𝑦))
 
Theorembj-omex 13311 Proof of omex 4515 from ax-infvn 13310. (Contributed by BJ, 14-Nov-2019.) (Proof modification is discouraged.)
ω ∈ V
 
11.2.9.2  Peano's fifth postulate

In this section, we give constructive proofs of two versions of Peano's fifth postulate.

 
Theorembdpeano5 13312* Bounded version of peano5 4520. (Contributed by BJ, 19-Nov-2019.) (Proof modification is discouraged.)
BOUNDED 𝐴       ((∅ ∈ 𝐴 ∧ ∀𝑥 ∈ ω (𝑥𝐴 → suc 𝑥𝐴)) → ω ⊆ 𝐴)
 
Theoremspeano5 13313* Version of peano5 4520 when 𝐴 is assumed to be a set, allowing a proof from the core axioms of CZF. (Contributed by BJ, 19-Nov-2019.) (Proof modification is discouraged.)
((𝐴𝑉 ∧ ∅ ∈ 𝐴 ∧ ∀𝑥 ∈ ω (𝑥𝐴 → suc 𝑥𝐴)) → ω ⊆ 𝐴)
 
11.2.9.3  Bounded induction and Peano's fourth postulate

In this section, we prove various versions of bounded induction from the basic axioms of CZF (in particular, without the axiom of set induction). We also prove Peano's fourth postulate. Together with the results from the previous sections, this proves from the core axioms of CZF (with infinity) that the set of finite ordinals satisfies the five Peano postulates and thus provides a model for the set of natural numbers.

 
Theoremfindset 13314* Bounded induction (principle of induction when 𝐴 is assumed to be a set) allowing a proof from basic constructive axioms. See find 4521 for a nonconstructive proof of the general case. See bdfind 13315 for a proof when 𝐴 is assumed to be bounded. (Contributed by BJ, 22-Nov-2019.) (Proof modification is discouraged.)
(𝐴𝑉 → ((𝐴 ⊆ ω ∧ ∅ ∈ 𝐴 ∧ ∀𝑥𝐴 suc 𝑥𝐴) → 𝐴 = ω))
 
Theorembdfind 13315* Bounded induction (principle of induction when 𝐴 is assumed to be bounded), proved from basic constructive axioms. See find 4521 for a nonconstructive proof of the general case. See findset 13314 for a proof when 𝐴 is assumed to be a set. (Contributed by BJ, 22-Nov-2019.) (Proof modification is discouraged.)
BOUNDED 𝐴       ((𝐴 ⊆ ω ∧ ∅ ∈ 𝐴 ∧ ∀𝑥𝐴 suc 𝑥𝐴) → 𝐴 = ω)
 
Theorembj-bdfindis 13316* Bounded induction (principle of induction for bounded formulas), using implicit substitutions (the biconditional versions of the hypotheses are implicit substitutions, and we have weakened them to implications). Constructive proof (from CZF). See finds 4522 for a proof of full induction in IZF. From this version, it is easy to prove bounded versions of finds 4522, finds2 4523, finds1 4524. (Contributed by BJ, 21-Nov-2019.) (Proof modification is discouraged.)
BOUNDED 𝜑    &   𝑥𝜓    &   𝑥𝜒    &   𝑥𝜃    &   (𝑥 = ∅ → (𝜓𝜑))    &   (𝑥 = 𝑦 → (𝜑𝜒))    &   (𝑥 = suc 𝑦 → (𝜃𝜑))       ((𝜓 ∧ ∀𝑦 ∈ ω (𝜒𝜃)) → ∀𝑥 ∈ ω 𝜑)
 
Theorembj-bdfindisg 13317* Version of bj-bdfindis 13316 using a class term in the consequent. Constructive proof (from CZF). See the comment of bj-bdfindis 13316 for explanations. (Contributed by BJ, 21-Nov-2019.) (Proof modification is discouraged.)
BOUNDED 𝜑    &   𝑥𝜓    &   𝑥𝜒    &   𝑥𝜃    &   (𝑥 = ∅ → (𝜓𝜑))    &   (𝑥 = 𝑦 → (𝜑𝜒))    &   (𝑥 = suc 𝑦 → (𝜃𝜑))    &   𝑥𝐴    &   𝑥𝜏    &   (𝑥 = 𝐴 → (𝜑𝜏))       ((𝜓 ∧ ∀𝑦 ∈ ω (𝜒𝜃)) → (𝐴 ∈ ω → 𝜏))
 
Theorembj-bdfindes 13318 Bounded induction (principle of induction for bounded formulas), using explicit substitutions. Constructive proof (from CZF). See the comment of bj-bdfindis 13316 for explanations. From this version, it is easy to prove the bounded version of findes 4525. (Contributed by BJ, 21-Nov-2019.) (Proof modification is discouraged.)
BOUNDED 𝜑       (([∅ / 𝑥]𝜑 ∧ ∀𝑥 ∈ ω (𝜑[suc 𝑥 / 𝑥]𝜑)) → ∀𝑥 ∈ ω 𝜑)
 
Theorembj-nn0suc0 13319* Constructive proof of a variant of nn0suc 4526. For a constructive proof of nn0suc 4526, see bj-nn0suc 13333. (Contributed by BJ, 19-Nov-2019.) (Proof modification is discouraged.)
(𝐴 ∈ ω → (𝐴 = ∅ ∨ ∃𝑥𝐴 𝐴 = suc 𝑥))
 
Theorembj-nntrans 13320 A natural number is a transitive set. (Contributed by BJ, 22-Nov-2019.) (Proof modification is discouraged.)
(𝐴 ∈ ω → (𝐵𝐴𝐵𝐴))
 
Theorembj-nntrans2 13321 A natural number is a transitive set. (Contributed by BJ, 22-Nov-2019.) (Proof modification is discouraged.)
(𝐴 ∈ ω → Tr 𝐴)
 
Theorembj-nnelirr 13322 A natural number does not belong to itself. Version of elirr 4464 for natural numbers, which does not require ax-setind 4460. (Contributed by BJ, 24-Nov-2019.) (Proof modification is discouraged.)
(𝐴 ∈ ω → ¬ 𝐴𝐴)
 
Theorembj-nnen2lp 13323 A version of en2lp 4477 for natural numbers, which does not require ax-setind 4460.

Note: using this theorem and bj-nnelirr 13322, one can remove dependency on ax-setind 4460 from nntri2 6398 and nndcel 6404; one can actually remove more dependencies from these. (Contributed by BJ, 28-Nov-2019.) (Proof modification is discouraged.)

((𝐴 ∈ ω ∧ 𝐵 ∈ ω) → ¬ (𝐴𝐵𝐵𝐴))
 
Theorembj-peano4 13324 Remove from peano4 4519 dependency on ax-setind 4460. Therefore, it only requires core constructive axioms (albeit more of them). (Contributed by BJ, 28-Nov-2019.) (Proof modification is discouraged.)
((𝐴 ∈ ω ∧ 𝐵 ∈ ω) → (suc 𝐴 = suc 𝐵𝐴 = 𝐵))
 
Theorembj-omtrans 13325 The set ω is transitive. A natural number is included in ω. Constructive proof of elnn 4527.

The idea is to use bounded induction with the formula 𝑥 ⊆ ω. This formula, in a logic with terms, is bounded. So in our logic without terms, we need to temporarily replace it with 𝑥𝑎 and then deduce the original claim. (Contributed by BJ, 29-Dec-2019.) (Proof modification is discouraged.)

(𝐴 ∈ ω → 𝐴 ⊆ ω)
 
Theorembj-omtrans2 13326 The set ω is transitive. (Contributed by BJ, 29-Dec-2019.) (Proof modification is discouraged.)
Tr ω
 
Theorembj-nnord 13327 A natural number is an ordinal. Constructive proof of nnord 4533. Can also be proved from bj-nnelon 13328 if the latter is proved from bj-omssonALT 13332. (Contributed by BJ, 27-Oct-2020.) (Proof modification is discouraged.)
(𝐴 ∈ ω → Ord 𝐴)
 
Theorembj-nnelon 13328 A natural number is an ordinal. Constructive proof of nnon 4531. Can also be proved from bj-omssonALT 13332. (Contributed by BJ, 27-Oct-2020.) (Proof modification is discouraged.)
(𝐴 ∈ ω → 𝐴 ∈ On)
 
Theorembj-omord 13329 The set ω is an ordinal. Constructive proof of ordom 4528. (Contributed by BJ, 29-Dec-2019.) (Proof modification is discouraged.)
Ord ω
 
Theorembj-omelon 13330 The set ω is an ordinal. Constructive proof of omelon 4530. (Contributed by BJ, 29-Dec-2019.) (Proof modification is discouraged.)
ω ∈ On
 
Theorembj-omsson 13331 Constructive proof of omsson 4534. See also bj-omssonALT 13332. (Contributed by BJ, 27-Oct-2020.) (Proof modification is discouraged.) (New usage is discouraged.
ω ⊆ On
 
Theorembj-omssonALT 13332 Alternate proof of bj-omsson 13331. (Contributed by BJ, 27-Oct-2020.) (Proof modification is discouraged.) (New usage is discouraged.)
ω ⊆ On
 
Theorembj-nn0suc 13333* Proof of (biconditional form of) nn0suc 4526 from the core axioms of CZF. See also bj-nn0sucALT 13347. As a characterization of the elements of ω, this could be labeled "elom". (Contributed by BJ, 19-Nov-2019.) (Proof modification is discouraged.)
(𝐴 ∈ ω ↔ (𝐴 = ∅ ∨ ∃𝑥 ∈ ω 𝐴 = suc 𝑥))
 
11.2.10  CZF: Set induction

In this section, we add the axiom of set induction to the core axioms of CZF.

 
11.2.10.1  Set induction

In this section, we prove some variants of the axiom of set induction.

 
Theoremsetindft 13334* Axiom of set-induction with a disjoint variable condition replaced with a non-freeness hypothesis (Contributed by BJ, 22-Nov-2019.)
(∀𝑥𝑦𝜑 → (∀𝑥(∀𝑦𝑥 [𝑦 / 𝑥]𝜑𝜑) → ∀𝑥𝜑))
 
Theoremsetindf 13335* Axiom of set-induction with a disjoint variable condition replaced with a non-freeness hypothesis (Contributed by BJ, 22-Nov-2019.)
𝑦𝜑       (∀𝑥(∀𝑦𝑥 [𝑦 / 𝑥]𝜑𝜑) → ∀𝑥𝜑)
 
Theoremsetindis 13336* Axiom of set induction using implicit substitutions. (Contributed by BJ, 22-Nov-2019.)
𝑥𝜓    &   𝑥𝜒    &   𝑦𝜑    &   𝑦𝜓    &   (𝑥 = 𝑧 → (𝜑𝜓))    &   (𝑥 = 𝑦 → (𝜒𝜑))       (∀𝑦(∀𝑧𝑦 𝜓𝜒) → ∀𝑥𝜑)
 
Axiomax-bdsetind 13337* Axiom of bounded set induction. (Contributed by BJ, 28-Nov-2019.)
BOUNDED 𝜑       (∀𝑎(∀𝑦𝑎 [𝑦 / 𝑎]𝜑𝜑) → ∀𝑎𝜑)
 
Theorembdsetindis 13338* Axiom of bounded set induction using implicit substitutions. (Contributed by BJ, 22-Nov-2019.) (Proof modification is discouraged.)
BOUNDED 𝜑    &   𝑥𝜓    &   𝑥𝜒    &   𝑦𝜑    &   𝑦𝜓    &   (𝑥 = 𝑧 → (𝜑𝜓))    &   (𝑥 = 𝑦 → (𝜒𝜑))       (∀𝑦(∀𝑧𝑦 𝜓𝜒) → ∀𝑥𝜑)
 
Theorembj-inf2vnlem1 13339* Lemma for bj-inf2vn 13343. Remark: unoptimized proof (have to use more deduction style). (Contributed by BJ, 8-Dec-2019.) (Proof modification is discouraged.)
(∀𝑥(𝑥𝐴 ↔ (𝑥 = ∅ ∨ ∃𝑦𝐴 𝑥 = suc 𝑦)) → Ind 𝐴)
 
Theorembj-inf2vnlem2 13340* Lemma for bj-inf2vnlem3 13341 and bj-inf2vnlem4 13342. Remark: unoptimized proof (have to use more deduction style). (Contributed by BJ, 8-Dec-2019.) (Proof modification is discouraged.)
(∀𝑥𝐴 (𝑥 = ∅ ∨ ∃𝑦𝐴 𝑥 = suc 𝑦) → (Ind 𝑍 → ∀𝑢(∀𝑡𝑢 (𝑡𝐴𝑡𝑍) → (𝑢𝐴𝑢𝑍))))
 
Theorembj-inf2vnlem3 13341* Lemma for bj-inf2vn 13343. (Contributed by BJ, 8-Dec-2019.) (Proof modification is discouraged.)
BOUNDED 𝐴    &   BOUNDED 𝑍       (∀𝑥𝐴 (𝑥 = ∅ ∨ ∃𝑦𝐴 𝑥 = suc 𝑦) → (Ind 𝑍𝐴𝑍))
 
Theorembj-inf2vnlem4 13342* Lemma for bj-inf2vn2 13344. (Contributed by BJ, 8-Dec-2019.) (Proof modification is discouraged.)
(∀𝑥𝐴 (𝑥 = ∅ ∨ ∃𝑦𝐴 𝑥 = suc 𝑦) → (Ind 𝑍𝐴𝑍))
 
Theorembj-inf2vn 13343* A sufficient condition for ω to be a set. See bj-inf2vn2 13344 for the unbounded version from full set induction. (Contributed by BJ, 8-Dec-2019.) (Proof modification is discouraged.)
BOUNDED 𝐴       (𝐴𝑉 → (∀𝑥(𝑥𝐴 ↔ (𝑥 = ∅ ∨ ∃𝑦𝐴 𝑥 = suc 𝑦)) → 𝐴 = ω))
 
Theorembj-inf2vn2 13344* A sufficient condition for ω to be a set; unbounded version of bj-inf2vn 13343. (Contributed by BJ, 8-Dec-2019.) (Proof modification is discouraged.)
(𝐴𝑉 → (∀𝑥(𝑥𝐴 ↔ (𝑥 = ∅ ∨ ∃𝑦𝐴 𝑥 = suc 𝑦)) → 𝐴 = ω))
 
Axiomax-inf2 13345* Another axiom of infinity in a constructive setting (see ax-infvn 13310). (Contributed by BJ, 14-Nov-2019.) (New usage is discouraged.)
𝑎𝑥(𝑥𝑎 ↔ (𝑥 = ∅ ∨ ∃𝑦𝑎 𝑥 = suc 𝑦))
 
Theorembj-omex2 13346 Using bounded set induction and the strong axiom of infinity, ω is a set, that is, we recover ax-infvn 13310 (see bj-2inf 13307 for the equivalence of the latter with bj-omex 13311). (Contributed by BJ, 8-Dec-2019.) (Proof modification is discouraged.) (New usage is discouraged.)
ω ∈ V
 
Theorembj-nn0sucALT 13347* Alternate proof of bj-nn0suc 13333, also constructive but from ax-inf2 13345, hence requiring ax-bdsetind 13337. (Contributed by BJ, 8-Dec-2019.) (Proof modification is discouraged.) (New usage is discouraged.)
(𝐴 ∈ ω ↔ (𝐴 = ∅ ∨ ∃𝑥 ∈ ω 𝐴 = suc 𝑥))
 
11.2.10.2  Full induction

In this section, using the axiom of set induction, we prove full induction on the set of natural numbers.

 
Theorembj-findis 13348* Principle of induction, using implicit substitutions (the biconditional versions of the hypotheses are implicit substitutions, and we have weakened them to implications). Constructive proof (from CZF). See bj-bdfindis 13316 for a bounded version not requiring ax-setind 4460. See finds 4522 for a proof in IZF. From this version, it is easy to prove of finds 4522, finds2 4523, finds1 4524. (Contributed by BJ, 22-Dec-2019.) (Proof modification is discouraged.)
𝑥𝜓    &   𝑥𝜒    &   𝑥𝜃    &   (𝑥 = ∅ → (𝜓𝜑))    &   (𝑥 = 𝑦 → (𝜑𝜒))    &   (𝑥 = suc 𝑦 → (𝜃𝜑))       ((𝜓 ∧ ∀𝑦 ∈ ω (𝜒𝜃)) → ∀𝑥 ∈ ω 𝜑)
 
Theorembj-findisg 13349* Version of bj-findis 13348 using a class term in the consequent. Constructive proof (from CZF). See the comment of bj-findis 13348 for explanations. (Contributed by BJ, 21-Nov-2019.) (Proof modification is discouraged.)
𝑥𝜓    &   𝑥𝜒    &   𝑥𝜃    &   (𝑥 = ∅ → (𝜓𝜑))    &   (𝑥 = 𝑦 → (𝜑𝜒))    &   (𝑥 = suc 𝑦 → (𝜃𝜑))    &   𝑥𝐴    &   𝑥𝜏    &   (𝑥 = 𝐴 → (𝜑𝜏))       ((𝜓 ∧ ∀𝑦 ∈ ω (𝜒𝜃)) → (𝐴 ∈ ω → 𝜏))
 
Theorembj-findes 13350 Principle of induction, using explicit substitutions. Constructive proof (from CZF). See the comment of bj-findis 13348 for explanations. From this version, it is easy to prove findes 4525. (Contributed by BJ, 21-Nov-2019.) (Proof modification is discouraged.)
(([∅ / 𝑥]𝜑 ∧ ∀𝑥 ∈ ω (𝜑[suc 𝑥 / 𝑥]𝜑)) → ∀𝑥 ∈ ω 𝜑)
 
11.2.11  CZF: Strong collection

In this section, we state the axiom scheme of strong collection, which is part of CZF set theory.

 
Axiomax-strcoll 13351* Axiom scheme of strong collection. It is stated with all possible disjoint variable conditions, to show that this weak form is sufficient. The antecedent means that 𝜑 represents a multivalued function on 𝑎, or equivalently a collection of nonempty classes indexed by 𝑎, and the axiom asserts the existence of a set 𝑏 which "collects" at least one element in the image of each 𝑥𝑎 and which is made only of such elements. That second conjunct is what makes it "strong", compared to the axiom scheme of collection ax-coll 4051. (Contributed by BJ, 5-Oct-2019.)
𝑎(∀𝑥𝑎𝑦𝜑 → ∃𝑏(∀𝑥𝑎𝑦𝑏 𝜑 ∧ ∀𝑦𝑏𝑥𝑎 𝜑))
 
Theoremstrcoll2 13352* Version of ax-strcoll 13351 with one disjoint variable condition removed and without initial universal quantifier. (Contributed by BJ, 5-Oct-2019.)
(∀𝑥𝑎𝑦𝜑 → ∃𝑏(∀𝑥𝑎𝑦𝑏 𝜑 ∧ ∀𝑦𝑏𝑥𝑎 𝜑))
 
Theoremstrcollnft 13353* Closed form of strcollnf 13354. (Contributed by BJ, 21-Oct-2019.)
(∀𝑥𝑦𝑏𝜑 → (∀𝑥𝑎𝑦𝜑 → ∃𝑏(∀𝑥𝑎𝑦𝑏 𝜑 ∧ ∀𝑦𝑏𝑥𝑎 𝜑)))
 
Theoremstrcollnf 13354* Version of ax-strcoll 13351 with one disjoint variable condition removed, the other disjoint variable condition replaced with a non-freeness hypothesis, and without initial universal quantifier. Version of strcoll2 13352 with the disjoint variable condition on 𝑏, 𝜑 replaced with a non-freeness hypothesis.

This proof aims to demonstrate a standard technique, but strcoll2 13352 will generally suffice: since the theorem asserts the existence of a set 𝑏, supposing that that setvar does not occur in the already defined 𝜑 is not a big constraint. (Contributed by BJ, 21-Oct-2019.)

𝑏𝜑       (∀𝑥𝑎𝑦𝜑 → ∃𝑏(∀𝑥𝑎𝑦𝑏 𝜑 ∧ ∀𝑦𝑏𝑥𝑎 𝜑))
 
TheoremstrcollnfALT 13355* Alternate proof of strcollnf 13354, not using strcollnft 13353. (Contributed by BJ, 5-Oct-2019.) (Proof modification is discouraged.) (New usage is discouraged.)
𝑏𝜑       (∀𝑥𝑎𝑦𝜑 → ∃𝑏(∀𝑥𝑎𝑦𝑏 𝜑 ∧ ∀𝑦𝑏𝑥𝑎 𝜑))
 
11.2.12  CZF: Subset collection

In this section, we state the axiom scheme of subset collection, which is part of CZF set theory.

 
Axiomax-sscoll 13356* Axiom scheme of subset collection. It is stated with all possible disjoint variable conditions, to show that this weak form is sufficient. The antecedent means that 𝜑 represents a multivalued function from 𝑎 to 𝑏, or equivalently a collection of nonempty subsets of 𝑏 indexed by 𝑎, and the consequent asserts the existence of a subset of 𝑐 which "collects" at least one element in the image of each 𝑥𝑎 and which is made only of such elements. The axiom asserts the existence, for any sets 𝑎, 𝑏, of a set 𝑐 such that that implication holds for any value of the parameter 𝑧 of 𝜑. (Contributed by BJ, 5-Oct-2019.)
𝑎𝑏𝑐𝑧(∀𝑥𝑎𝑦𝑏 𝜑 → ∃𝑑𝑐 (∀𝑥𝑎𝑦𝑑 𝜑 ∧ ∀𝑦𝑑𝑥𝑎 𝜑))
 
Theoremsscoll2 13357* Version of ax-sscoll 13356 with two disjoint variable conditions removed and without initial universal quantifiers. (Contributed by BJ, 5-Oct-2019.)
𝑐𝑧(∀𝑥𝑎𝑦𝑏 𝜑 → ∃𝑑𝑐 (∀𝑥𝑎𝑦𝑑 𝜑 ∧ ∀𝑦𝑑𝑥𝑎 𝜑))
 
11.2.13  Real numbers
 
Axiomax-ddkcomp 13358 Axiom of Dedekind completeness for Dedekind real numbers: every inhabited upper-bounded located set of reals has a real upper bound. Ideally, this axiom should be "proved" as "axddkcomp" for the real numbers constructed from IZF, and then the axiom ax-ddkcomp 13358 should be used in place of construction specific results. In particular, axcaucvg 7732 should be proved from it. (Contributed by BJ, 24-Oct-2021.)
(((𝐴 ⊆ ℝ ∧ ∃𝑥 𝑥𝐴) ∧ ∃𝑥 ∈ ℝ ∀𝑦𝐴 𝑦 < 𝑥 ∧ ∀𝑥 ∈ ℝ ∀𝑦 ∈ ℝ (𝑥 < 𝑦 → (∃𝑧𝐴 𝑥 < 𝑧 ∨ ∀𝑧𝐴 𝑧 < 𝑦))) → ∃𝑥 ∈ ℝ (∀𝑦𝐴 𝑦𝑥 ∧ ((𝐵𝑅 ∧ ∀𝑦𝐴 𝑦𝐵) → 𝑥𝐵)))
 
11.3  Mathbox for Jim Kingdon
 
11.3.1  Natural numbers
 
Theoremel2oss1o 13359 Being an element of ordinal two implies being a subset of ordinal one. The converse is equivalent to excluded middle by ss1oel2o 13360. (Contributed by Jim Kingdon, 8-Aug-2022.)
(𝐴 ∈ 2o𝐴 ⊆ 1o)
 
Theoremss1oel2o 13360 Any subset of ordinal one being an element of ordinal two is equivalent to excluded middle. A variation of exmid01 4129 which more directly illustrates the contrast with el2oss1o 13359. (Contributed by Jim Kingdon, 8-Aug-2022.)
(EXMID ↔ ∀𝑥(𝑥 ⊆ 1o𝑥 ∈ 2o))
 
Theorempw1dom2 13361 The power set of 1o dominates 2o. Also see pwpw0ss 3739 which is similar. (Contributed by Jim Kingdon, 21-Sep-2022.)
2o ≼ 𝒫 1o
 
Theoremnnti 13362 Ordering on a natural number generates a tight apartness. (Contributed by Jim Kingdon, 7-Aug-2022.)
(𝜑𝐴 ∈ ω)       ((𝜑 ∧ (𝑢𝐴𝑣𝐴)) → (𝑢 = 𝑣 ↔ (¬ 𝑢 E 𝑣 ∧ ¬ 𝑣 E 𝑢)))
 
Theorem012of 13363 Mapping zero and one between 0 and ω style integers. (Contributed by Jim Kingdon, 28-Jun-2024.)
𝐺 = frec((𝑥 ∈ ℤ ↦ (𝑥 + 1)), 0)       (𝐺 ↾ {0, 1}):{0, 1}⟶2o
 
Theorem2o01f 13364 Mapping zero and one between ω and 0 style integers. (Contributed by Jim Kingdon, 28-Jun-2024.)
𝐺 = frec((𝑥 ∈ ℤ ↦ (𝑥 + 1)), 0)       (𝐺 ↾ 2o):2o⟶{0, 1}
 
11.3.2  The power set of a singleton
 
Theorempwtrufal 13365 A subset of the singleton {∅} cannot be anything other than or {∅}. Removing the double negation would change the meaning, as seen at exmid01 4129. If we view a subset of a singleton as a truth value (as seen in theorems like exmidexmid 4128), then this theorem states there are no truth values other than true and false, as described in section 1.1 of [Bauer], p. 481. (Contributed by Mario Carneiro and Jim Kingdon, 11-Sep-2023.)
(𝐴 ⊆ {∅} → ¬ ¬ (𝐴 = ∅ ∨ 𝐴 = {∅}))
 
Theorempwle2 13366* An exercise related to 𝑁 copies of a singleton and the power set of a singleton (where the latter can also be thought of as representing truth values). Posed as an exercise by Martin Escardo online. (Contributed by Jim Kingdon, 3-Sep-2023.)
𝑇 = 𝑥𝑁 ({𝑥} × 1o)       ((𝑁 ∈ ω ∧ 𝐺:𝑇1-1→𝒫 1o) → 𝑁 ⊆ 2o)
 
Theorempwf1oexmid 13367* An exercise related to 𝑁 copies of a singleton and the power set of a singleton (where the latter can also be thought of as representing truth values). Posed as an exercise by Martin Escardo online. (Contributed by Jim Kingdon, 3-Sep-2023.)
𝑇 = 𝑥𝑁 ({𝑥} × 1o)       ((𝑁 ∈ ω ∧ 𝐺:𝑇1-1→𝒫 1o) → (ran 𝐺 = 𝒫 1o ↔ (𝑁 = 2oEXMID)))
 
Theoremexmid1stab 13368* If any proposition is stable, excluded middle follows. We are thinking of 𝑥 as a proposition and 𝑥 = {∅} as "x is true". (Contributed by Jim Kingdon, 28-Nov-2023.)
((𝜑𝑥 ⊆ {∅}) → STAB 𝑥 = {∅})       (𝜑EXMID)
 
Theoremsubctctexmid 13369* If every subcountable set is countable and Markov's principle holds, excluded middle follows. Proposition 2.6 of [BauerSwan], p. 14:4. The proof is taken from that paper. (Contributed by Jim Kingdon, 29-Nov-2023.)
(𝜑 → ∀𝑥(∃𝑠(𝑠 ⊆ ω ∧ ∃𝑓 𝑓:𝑠onto𝑥) → ∃𝑔 𝑔:ω–onto→(𝑥 ⊔ 1o)))    &   (𝜑 → ω ∈ Markov)       (𝜑EXMID)
 
Theoremsssneq 13370* Any two elements of a subset of a singleton are equal. (Contributed by Jim Kingdon, 28-May-2024.)
(𝐴 ⊆ {𝐵} → ∀𝑦𝐴𝑧𝐴 𝑦 = 𝑧)
 
Theorempw1nct 13371* A condition which ensures that the powerset of a singleton is not countable. The antecedent here can be referred to as the uniformity principle. Based on Mastodon posts by Andrej Bauer and Rahul Chhabra. (Contributed by Jim Kingdon, 29-May-2024.)
(∀𝑟(𝑟 ⊆ (𝒫 1o × ω) → (∀𝑝 ∈ 𝒫 1o𝑛 ∈ ω 𝑝𝑟𝑛 → ∃𝑚 ∈ ω ∀𝑞 ∈ 𝒫 1o𝑞𝑟𝑚)) → ¬ ∃𝑓 𝑓:ω–onto→(𝒫 1o ⊔ 1o))
 
11.3.3  Omniscience of NN+oo
 
Theorem0nninf 13372 The zero element of (the constant sequence equal to ). (Contributed by Jim Kingdon, 14-Jul-2022.)
(ω × {∅}) ∈ ℕ
 
Theoremnninff 13373 An element of is a sequence of zeroes and ones. (Contributed by Jim Kingdon, 4-Aug-2022.)
(𝐴 ∈ ℕ𝐴:ω⟶2o)
 
Theoremnnsf 13374* Domain and range of 𝑆. Part of Definition 3.3 of [PradicBrown2022], p. 5. (Contributed by Jim Kingdon, 30-Jul-2022.)
𝑆 = (𝑝 ∈ ℕ ↦ (𝑖 ∈ ω ↦ if(𝑖 = ∅, 1o, (𝑝 𝑖))))       𝑆:ℕ⟶ℕ
 
Theorempeano4nninf 13375* The successor function on is one to one. Half of Lemma 3.4 of [PradicBrown2022], p. 5. (Contributed by Jim Kingdon, 31-Jul-2022.)
𝑆 = (𝑝 ∈ ℕ ↦ (𝑖 ∈ ω ↦ if(𝑖 = ∅, 1o, (𝑝 𝑖))))       𝑆:ℕ1-1→ℕ
 
Theorempeano3nninf 13376* The successor function on is never zero. Half of Lemma 3.4 of [PradicBrown2022], p. 5. (Contributed by Jim Kingdon, 1-Aug-2022.)
𝑆 = (𝑝 ∈ ℕ ↦ (𝑖 ∈ ω ↦ if(𝑖 = ∅, 1o, (𝑝 𝑖))))       (𝐴 ∈ ℕ → (𝑆𝐴) ≠ (𝑥 ∈ ω ↦ ∅))
 
Theoremnninfalllemn 13377* Lemma for nninfall 13379. Mapping of a natural number to an element of . (Contributed by Jim Kingdon, 4-Aug-2022.)
(𝜑𝑃 ∈ ℕ)    &   (𝜑𝑁 ∈ ω)    &   (𝜑 → ∀𝑥𝑁 (𝑃𝑥) = 1o)    &   (𝜑 → (𝑃𝑁) = ∅)       (𝜑𝑃 = (𝑖 ∈ ω ↦ if(𝑖𝑁, 1o, ∅)))
 
Theoremnninfalllem1 13378* Lemma for nninfall 13379. (Contributed by Jim Kingdon, 1-Aug-2022.)
(𝜑𝑄 ∈ (2o𝑚))    &   (𝜑 → (𝑄‘(𝑥 ∈ ω ↦ 1o)) = 1o)    &   (𝜑 → ∀𝑛 ∈ ω (𝑄‘(𝑖 ∈ ω ↦ if(𝑖𝑛, 1o, ∅))) = 1o)    &   (𝜑𝑃 ∈ ℕ)    &   (𝜑 → (𝑄𝑃) = ∅)       (𝜑 → ∀𝑛 ∈ ω (𝑃𝑛) = 1o)
 
Theoremnninfall 13379* Given a decidable predicate on , showing it holds for natural numbers and the point at infinity suffices to show it holds everywhere. The sense in which 𝑄 is a decidable predicate is that it assigns a value of either or 1o (which can be thought of as false and true) to every element of . Lemma 3.5 of [PradicBrown2022], p. 5. (Contributed by Jim Kingdon, 1-Aug-2022.)
(𝜑𝑄 ∈ (2o𝑚))    &   (𝜑 → (𝑄‘(𝑥 ∈ ω ↦ 1o)) = 1o)    &   (𝜑 → ∀𝑛 ∈ ω (𝑄‘(𝑖 ∈ ω ↦ if(𝑖𝑛, 1o, ∅))) = 1o)       (𝜑 → ∀𝑝 ∈ ℕ (𝑄𝑝) = 1o)
 
Theoremnninfex 13380 is a set. (Contributed by Jim Kingdon, 10-Aug-2022.)
∈ V
 
Theoremnninfsellemdc 13381* Lemma for nninfself 13384. Showing that the selection function is well defined. (Contributed by Jim Kingdon, 8-Aug-2022.)
((𝑄 ∈ (2o𝑚) ∧ 𝑁 ∈ ω) → DECID𝑘 ∈ suc 𝑁(𝑄‘(𝑖 ∈ ω ↦ if(𝑖𝑘, 1o, ∅))) = 1o)
 
Theoremnninfsellemcl 13382* Lemma for nninfself 13384. (Contributed by Jim Kingdon, 8-Aug-2022.)
((𝑄 ∈ (2o𝑚) ∧ 𝑁 ∈ ω) → if(∀𝑘 ∈ suc 𝑁(𝑄‘(𝑖 ∈ ω ↦ if(𝑖𝑘, 1o, ∅))) = 1o, 1o, ∅) ∈ 2o)
 
Theoremnninfsellemsuc 13383* Lemma for nninfself 13384. (Contributed by Jim Kingdon, 6-Aug-2022.)
((𝑄 ∈ (2o𝑚) ∧ 𝐽 ∈ ω) → if(∀𝑘 ∈ suc suc 𝐽(𝑄‘(𝑖 ∈ ω ↦ if(𝑖𝑘, 1o, ∅))) = 1o, 1o, ∅) ⊆ if(∀𝑘 ∈ suc 𝐽(𝑄‘(𝑖 ∈ ω ↦ if(𝑖𝑘, 1o, ∅))) = 1o, 1o, ∅))
 
Theoremnninfself 13384* Domain and range of the selection function for . (Contributed by Jim Kingdon, 6-Aug-2022.)
𝐸 = (𝑞 ∈ (2o𝑚) ↦ (𝑛 ∈ ω ↦ if(∀𝑘 ∈ suc 𝑛(𝑞‘(𝑖 ∈ ω ↦ if(𝑖𝑘, 1o, ∅))) = 1o, 1o, ∅)))       𝐸:(2o𝑚)⟶ℕ
 
Theoremnninfsellemeq 13385* Lemma for nninfsel 13388. (Contributed by Jim Kingdon, 9-Aug-2022.)
𝐸 = (𝑞 ∈ (2o𝑚) ↦ (𝑛 ∈ ω ↦ if(∀𝑘 ∈ suc 𝑛(𝑞‘(𝑖 ∈ ω ↦ if(𝑖𝑘, 1o, ∅))) = 1o, 1o, ∅)))    &   (𝜑𝑄 ∈ (2o𝑚))    &   (𝜑 → (𝑄‘(𝐸𝑄)) = 1o)    &   (𝜑𝑁 ∈ ω)    &   (𝜑 → ∀𝑘𝑁 (𝑄‘(𝑖 ∈ ω ↦ if(𝑖𝑘, 1o, ∅))) = 1o)    &   (𝜑 → (𝑄‘(𝑖 ∈ ω ↦ if(𝑖𝑁, 1o, ∅))) = ∅)       (𝜑 → (𝐸𝑄) = (𝑖 ∈ ω ↦ if(𝑖𝑁, 1o, ∅)))
 
Theoremnninfsellemqall 13386* Lemma for nninfsel 13388. (Contributed by Jim Kingdon, 9-Aug-2022.)
𝐸 = (𝑞 ∈ (2o𝑚) ↦ (𝑛 ∈ ω ↦ if(∀𝑘 ∈ suc 𝑛(𝑞‘(𝑖 ∈ ω ↦ if(𝑖𝑘, 1o, ∅))) = 1o, 1o, ∅)))    &   (𝜑𝑄 ∈ (2o𝑚))    &   (𝜑 → (𝑄‘(𝐸𝑄)) = 1o)    &   (𝜑𝑁 ∈ ω)       (𝜑 → (𝑄‘(𝑖 ∈ ω ↦ if(𝑖𝑁, 1o, ∅))) = 1o)
 
Theoremnninfsellemeqinf 13387* Lemma for nninfsel 13388. (Contributed by Jim Kingdon, 9-Aug-2022.)
𝐸 = (𝑞 ∈ (2o𝑚) ↦ (𝑛 ∈ ω ↦ if(∀𝑘 ∈ suc 𝑛(𝑞‘(𝑖 ∈ ω ↦ if(𝑖𝑘, 1o, ∅))) = 1o, 1o, ∅)))    &   (𝜑𝑄 ∈ (2o𝑚))    &   (𝜑 → (𝑄‘(𝐸𝑄)) = 1o)       (𝜑 → (𝐸𝑄) = (𝑖 ∈ ω ↦ 1o))
 
Theoremnninfsel 13388* 𝐸 is a selection function for . Theorem 3.6 of [PradicBrown2022], p. 5. (Contributed by Jim Kingdon, 9-Aug-2022.)
𝐸 = (𝑞 ∈ (2o𝑚) ↦ (𝑛 ∈ ω ↦ if(∀𝑘 ∈ suc 𝑛(𝑞‘(𝑖 ∈ ω ↦ if(𝑖𝑘, 1o, ∅))) = 1o, 1o, ∅)))    &   (𝜑𝑄 ∈ (2o𝑚))    &   (𝜑 → (𝑄‘(𝐸𝑄)) = 1o)       (𝜑 → ∀𝑝 ∈ ℕ (𝑄𝑝) = 1o)
 
Theoremnninfomnilem 13389* Lemma for nninfomni 13390. (Contributed by Jim Kingdon, 10-Aug-2022.)
𝐸 = (𝑞 ∈ (2o𝑚) ↦ (𝑛 ∈ ω ↦ if(∀𝑘 ∈ suc 𝑛(𝑞‘(𝑖 ∈ ω ↦ if(𝑖𝑘, 1o, ∅))) = 1o, 1o, ∅)))        ∈ Omni
 
Theoremnninfomni 13390 is omniscient. Corollary 3.7 of [PradicBrown2022], p. 5. (Contributed by Jim Kingdon, 10-Aug-2022.)
∈ Omni
 
Theoremnninffeq 13391* Equality of two functions on which agree at every integer and at the point at infinity. From an online post by Martin Escardo. (Contributed by Jim Kingdon, 4-Aug-2023.)
(𝜑𝐹:ℕ⟶ℕ0)    &   (𝜑𝐺:ℕ⟶ℕ0)    &   (𝜑 → (𝐹‘(𝑥 ∈ ω ↦ 1o)) = (𝐺‘(𝑥 ∈ ω ↦ 1o)))    &   (𝜑 → ∀𝑛 ∈ ω (𝐹‘(𝑖 ∈ ω ↦ if(𝑖𝑛, 1o, ∅))) = (𝐺‘(𝑖 ∈ ω ↦ if(𝑖𝑛, 1o, ∅))))       (𝜑𝐹 = 𝐺)
 
11.3.4  Schroeder-Bernstein Theorem
 
Theoremexmidsbthrlem 13392* Lemma for exmidsbthr 13393. (Contributed by Jim Kingdon, 11-Aug-2022.)
𝑆 = (𝑝 ∈ ℕ ↦ (𝑖 ∈ ω ↦ if(𝑖 = ∅, 1o, (𝑝 𝑖))))       (∀𝑥𝑦((𝑥𝑦𝑦𝑥) → 𝑥𝑦) → EXMID)
 
Theoremexmidsbthr 13393* The Schroeder-Bernstein Theorem implies excluded middle. Theorem 1 of [PradicBrown2022], p. 1. (Contributed by Jim Kingdon, 11-Aug-2022.)
(∀𝑥𝑦((𝑥𝑦𝑦𝑥) → 𝑥𝑦) → EXMID)
 
Theoremexmidsbth 13394* The Schroeder-Bernstein Theorem is equivalent to excluded middle. This is Metamath 100 proof #25. The forward direction (isbth 6863) is the proof of the Schroeder-Bernstein Theorem from the Metamath Proof Explorer database (in which excluded middle holds), but adapted to use EXMID as an antecedent rather than being unconditionally true, as in the non-intuitionist proof at https://us.metamath.org/mpeuni/sbth.html 6863.

The reverse direction (exmidsbthr 13393) is the one which establishes that Schroeder-Bernstein implies excluded middle. This resolves the question of whether we will be able to prove Schroeder-Bernstein from our axioms in the negative. (Contributed by Jim Kingdon, 13-Aug-2022.)

(EXMID ↔ ∀𝑥𝑦((𝑥𝑦𝑦𝑥) → 𝑥𝑦))
 
Theoremsbthomlem 13395 Lemma for sbthom 13396. (Contributed by Mario Carneiro and Jim Kingdon, 13-Jul-2023.)
(𝜑 → ω ∈ Omni)    &   (𝜑𝑌 ⊆ {∅})    &   (𝜑𝐹:ω–1-1-onto→(𝑌 ⊔ ω))       (𝜑 → (𝑌 = ∅ ∨ 𝑌 = {∅}))
 
Theoremsbthom 13396 Schroeder-Bernstein is not possible even for ω. We know by exmidsbth 13394 that full Schroeder-Bernstein will not be provable but what about the case where one of the sets is ω? That case plus the Limited Principle of Omniscience (LPO) implies excluded middle, so we will not be able to prove it. (Contributed by Mario Carneiro and Jim Kingdon, 10-Jul-2023.)
((∀𝑥((𝑥 ≼ ω ∧ ω ≼ 𝑥) → 𝑥 ≈ ω) ∧ ω ∈ Omni) → EXMID)
 
11.3.5  Real and complex numbers
 
Theoremqdencn 13397* The set of complex numbers whose real and imaginary parts are rational is dense in the complex plane. This is a two dimensional analogue to qdenre 11006 (and also would hold for ℝ × ℝ with the usual metric; this is not about complex numbers in particular). (Contributed by Jim Kingdon, 18-Oct-2021.)
𝑄 = {𝑧 ∈ ℂ ∣ ((ℜ‘𝑧) ∈ ℚ ∧ (ℑ‘𝑧) ∈ ℚ)}       ((𝐴 ∈ ℂ ∧ 𝐵 ∈ ℝ+) → ∃𝑥𝑄 (abs‘(𝑥𝐴)) < 𝐵)
 
Theoremrefeq 13398* Equality of two real functions which agree at negative numbers, positive numbers, and zero. This holds even without real trichotomy. From an online post by Martin Escardo. (Contributed by Jim Kingdon, 9-Jul-2023.)
(𝜑𝐹:ℝ⟶ℝ)    &   (𝜑𝐺:ℝ⟶ℝ)    &   (𝜑 → ∀𝑥 ∈ ℝ (𝑥 < 0 → (𝐹𝑥) = (𝐺𝑥)))    &   (𝜑 → ∀𝑥 ∈ ℝ (0 < 𝑥 → (𝐹𝑥) = (𝐺𝑥)))    &   (𝜑 → (𝐹‘0) = (𝐺‘0))       (𝜑𝐹 = 𝐺)
 
Theoremtriap 13399 Two ways of stating real number trichotomy. (Contributed by Jim Kingdon, 23-Aug-2023.)
((𝐴 ∈ ℝ ∧ 𝐵 ∈ ℝ) → ((𝐴 < 𝐵𝐴 = 𝐵𝐵 < 𝐴) ↔ DECID 𝐴 # 𝐵))
 
Theoremisomninnlem 13400* Lemma for isomninn 13401. The result, with a hypothesis to provide a convenient notation. (Contributed by Jim Kingdon, 30-Aug-2023.)
𝐺 = frec((𝑥 ∈ ℤ ↦ (𝑥 + 1)), 0)       (𝐴𝑉 → (𝐴 ∈ Omni ↔ ∀𝑓 ∈ ({0, 1} ↑𝑚 𝐴)(∃𝑥𝐴 (𝑓𝑥) = 0 ∨ ∀𝑥𝐴 (𝑓𝑥) = 1)))
    < Previous  Next >

Page List
Jump to page: Contents  1 1-100 2 101-200 3 201-300 4 301-400 5 401-500 6 501-600 7 601-700 8 701-800 9 801-900 10 901-1000 11 1001-1100 12 1101-1200 13 1201-1300 14 1301-1400 15 1401-1500 16 1501-1600 17 1601-1700 18 1701-1800 19 1801-1900 20 1901-2000 21 2001-2100 22 2101-2200 23 2201-2300 24 2301-2400 25 2401-2500 26 2501-2600 27 2601-2700 28 2701-2800 29 2801-2900 30 2901-3000 31 3001-3100 32 3101-3200 33 3201-3300 34 3301-3400 35 3401-3500 36 3501-3600 37 3601-3700 38 3701-3800 39 3801-3900 40 3901-4000 41 4001-4100 42 4101-4200 43 4201-4300 44 4301-4400 45 4401-4500 46 4501-4600 47 4601-4700 48 4701-4800 49 4801-4900 50 4901-5000 51 5001-5100 52 5101-5200 53 5201-5300 54 5301-5400 55 5401-5500 56 5501-5600 57 5601-5700 58 5701-5800 59 5801-5900 60 5901-6000 61 6001-6100 62 6101-6200 63 6201-6300 64 6301-6400 65 6401-6500 66 6501-6600 67 6601-6700 68 6701-6800 69 6801-6900 70 6901-7000 71 7001-7100 72 7101-7200 73 7201-7300 74 7301-7400 75 7401-7500 76 7501-7600 77 7601-7700 78 7701-7800 79 7801-7900 80 7901-8000 81 8001-8100 82 8101-8200 83 8201-8300 84 8301-8400 85 8401-8500 86 8501-8600 87 8601-8700 88 8701-8800 89 8801-8900 90 8901-9000 91 9001-9100 92 9101-9200 93 9201-9300 94 9301-9400 95 9401-9500 96 9501-9600 97 9601-9700 98 9701-9800 99 9801-9900 100 9901-10000 101 10001-10100 102 10101-10200 103 10201-10300 104 10301-10400 105 10401-10500 106 10501-10600 107 10601-10700 108 10701-10800 109 10801-10900 110 10901-11000 111 11001-11100 112 11101-11200 113 11201-11300 114 11301-11400 115 11401-11500 116 11501-11600 117 11601-11700 118 11701-11800 119 11801-11900 120 11901-12000 121 12001-12100 122 12101-12200 123 12201-12300 124 12301-12400 125 12401-12500 126 12501-12600 127 12601-12700 128 12701-12800 129 12801-12900 130 12901-13000 131 13001-13100 132 13101-13200 133 13201-13300 134 13301-13400 135 13401-13441
  Copyright terms: Public domain < Previous  Next >