Home | Intuitionistic Logic Explorer Theorem List (p. 139 of 141) | < Previous Next > |
Browser slow? Try the
Unicode version. |
||
Mirrors > Metamath Home Page > ILE Home Page > Theorem List Contents > Recent Proofs This page: Page List |
Type | Label | Description |
---|---|---|
Statement | ||
Theorem | fmelpw1o 13801 |
With a formula
one can associate an element of ,
which
can therefore be thought of as the set of "truth values" (but
recall that
there are no other genuine truth values than and , by
nndc 846, which translate to and respectively by iftrue 3530
and iffalse 3533, giving pwtrufal 13990).
As proved in if0ab 13800, the associated element of is the extension, in , of the formula . (Contributed by BJ, 15-Aug-2024.) |
Theorem | bj-charfun 13802* | Properties of the characteristic function on the class of the class . (Contributed by BJ, 15-Aug-2024.) |
Theorem | bj-charfundc 13803* | Properties of the characteristic function on the class of the class , provided membership in is decidable in . (Contributed by BJ, 6-Aug-2024.) |
DECID | ||
Theorem | bj-charfundcALT 13804* | Alternate proof of bj-charfundc 13803. It was expected to be much shorter since it uses bj-charfun 13802 for the main part of the proof and the rest is basic computations, but these turn out to be lengthy, maybe because of the limited library of available lemmas. (Contributed by BJ, 15-Aug-2024.) (Proof modification is discouraged.) (New usage is discouraged.) |
DECID | ||
Theorem | bj-charfunr 13805* |
If a class has a
"weak" characteristic function on a class ,
then negated membership in is decidable (in other words,
membership in
is testable) in .
The hypothesis imposes that be a set. As usual, it could be formulated as to deal with general classes, but that extra generality would not make the theorem much more useful. The theorem would still hold if the codomain of were any class with testable equality to the point where is sent. (Contributed by BJ, 6-Aug-2024.) |
DECID | ||
Theorem | bj-charfunbi 13806* |
In an ambient set , if
membership in is
stable, then it is
decidable if and only if has a characteristic function.
This characterization can be applied to singletons when the set has stable equality, which is the case as soon as it has a tight apartness relation. (Contributed by BJ, 6-Aug-2024.) |
STAB DECID | ||
This section develops constructive Zermelo--Fraenkel set theory (CZF) on top of intuitionistic logic. It is a constructive theory in the sense that its logic is intuitionistic and it is predicative. "Predicative" means that new sets can be constructed only from already constructed sets. In particular, the axiom of separation ax-sep 4105 is not predicative (because we cannot allow all formulas to define a subset) and is replaced in CZF by bounded separation ax-bdsep 13879. Because this axiom is weaker than full separation, the axiom of replacement or collection ax-coll 4102 of ZF and IZF has to be strengthened in CZF to the axiom of strong collection ax-strcoll 13977 (which is a theorem of IZF), and the axiom of infinity needs a more precise version, the von Neumann axiom of infinity ax-infvn 13936. Similarly, the axiom of powerset ax-pow 4158 is not predicative (checking whether a set is included in another requires to universally quantifier over that "not yet constructed" set) and is replaced in CZF by the axiom of fullness or the axiom of subset collection ax-sscoll 13982. In an intuitionistic context, the axiom of regularity is stated in IZF as well as in CZF as the axiom of set induction ax-setind 4519. It is sometimes interesting to study the weakening of CZF where that axiom is replaced by bounded set induction ax-bdsetind 13963. For more details on CZF, a useful set of notes is Peter Aczel and Michael Rathjen, CST Book draft. (available at http://www1.maths.leeds.ac.uk/~rathjen/book.pdf 13963) and an interesting article is Michael Shulman, Comparing material and structural set theories, Annals of Pure and Applied Logic, Volume 170, Issue 4 (Apr. 2019), 465--504. https://doi.org/10.48550/arXiv.1808.05204 13963 I also thank Michael Rathjen and Michael Shulman for useful hints in the formulation of some results. | ||
The present definition of bounded formulas emerged from a discussion on GitHub between Jim Kingdon, Mario Carneiro and I, started 23-Sept-2019 (see https://github.com/metamath/set.mm/issues/1173 and links therein). In order to state certain axiom schemes of Constructive Zermelo–Fraenkel (CZF) set theory, like the axiom scheme of bounded (or restricted, or Δ0) separation, it is necessary to distinguish certain formulas, called bounded (or restricted, or Δ0) formulas. The necessity of considering bounded formulas also arises in several theories of bounded arithmetic, both classical or intuitionistic, for instance to state the axiom scheme of Δ0-induction. To formalize this in Metamath, there are several choices to make. A first choice is to either create a new type for bounded formulas, or to create a predicate on formulas that indicates whether they are bounded. In the first case, one creates a new type "wff0" with a new set of metavariables (ph0 ...) and an axiom "$a wff ph0 " ensuring that bounded formulas are formulas, so that one can reuse existing theorems, and then axioms take the form "$a wff0 ( ph0 -> ps0 )", etc. In the second case, one introduces a predicate "BOUNDED " with the intended meaning that "BOUNDED " is a formula meaning that is a bounded formula. We choose the second option, since the first would complicate the grammar, risking to make it ambiguous. (TODO: elaborate.) A second choice is to view "bounded" either as a syntactic or a semantic property. For instance, is not syntactically bounded since it has an unbounded universal quantifier, but it is semantically bounded since it is equivalent to which is bounded. We choose the second option, so that formulas using defined symbols can be proved bounded. A third choice is in the form of the axioms, either in closed form or in inference form. One cannot state all the axioms in closed form, especially ax-bd0 13808. Indeed, if we posited it in closed form, then we could prove for instance BOUNDED and BOUNDED which is problematic (with the law of excluded middle, this would entail that all formulas are bounded, but even without it, too many formulas could be proved bounded...). (TODO: elaborate.) Having ax-bd0 13808 in inference form ensures that a formula can be proved bounded only if it is equivalent *for all values of the free variables* to a syntactically bounded one. The other axioms (ax-bdim 13809 through ax-bdsb 13817) can be written either in closed or inference form. The fact that ax-bd0 13808 is an inference is enough to ensure that the closed forms cannot be "exploited" to prove that some unbounded formulas are bounded. (TODO: check.) However, we state all the axioms in inference form to make it clear that we do not exploit any over-permissiveness. Finally, note that our logic has no terms, only variables. Therefore, we cannot prove for instance that is a bounded formula. However, since can be defined as "the such that PHI" a proof using the fact that is bounded can be converted to a proof in iset.mm by replacing with everywhere and prepending the antecedent PHI, since is bounded by ax-bdel 13816. For a similar method, see bj-omtrans 13951. Note that one cannot add an axiom BOUNDED since by bdph 13845 it would imply that every formula is bounded. | ||
Syntax | wbd 13807 | Syntax for the predicate BOUNDED. |
BOUNDED | ||
Axiom | ax-bd0 13808 | If two formulas are equivalent, then boundedness of one implies boundedness of the other. (Contributed by BJ, 3-Oct-2019.) |
BOUNDED BOUNDED | ||
Axiom | ax-bdim 13809 | An implication between two bounded formulas is bounded. (Contributed by BJ, 25-Sep-2019.) |
BOUNDED BOUNDED BOUNDED | ||
Axiom | ax-bdan 13810 | The conjunction of two bounded formulas is bounded. (Contributed by BJ, 25-Sep-2019.) |
BOUNDED BOUNDED BOUNDED | ||
Axiom | ax-bdor 13811 | The disjunction of two bounded formulas is bounded. (Contributed by BJ, 25-Sep-2019.) |
BOUNDED BOUNDED BOUNDED | ||
Axiom | ax-bdn 13812 | The negation of a bounded formula is bounded. (Contributed by BJ, 25-Sep-2019.) |
BOUNDED BOUNDED | ||
Axiom | ax-bdal 13813* | A bounded universal quantification of a bounded formula is bounded. Note the disjoint variable condition on . (Contributed by BJ, 25-Sep-2019.) |
BOUNDED BOUNDED | ||
Axiom | ax-bdex 13814* | A bounded existential quantification of a bounded formula is bounded. Note the disjoint variable condition on . (Contributed by BJ, 25-Sep-2019.) |
BOUNDED BOUNDED | ||
Axiom | ax-bdeq 13815 | An atomic formula is bounded (equality predicate). (Contributed by BJ, 3-Oct-2019.) |
BOUNDED | ||
Axiom | ax-bdel 13816 | An atomic formula is bounded (membership predicate). (Contributed by BJ, 3-Oct-2019.) |
BOUNDED | ||
Axiom | ax-bdsb 13817 | A formula resulting from proper substitution in a bounded formula is bounded. This probably cannot be proved from the other axioms, since neither the definiens in df-sb 1756, nor probably any other equivalent formula, is syntactically bounded. (Contributed by BJ, 3-Oct-2019.) |
BOUNDED BOUNDED | ||
Theorem | bdeq 13818 | Equality property for the predicate BOUNDED. (Contributed by BJ, 3-Oct-2019.) |
BOUNDED BOUNDED | ||
Theorem | bd0 13819 | A formula equivalent to a bounded one is bounded. See also bd0r 13820. (Contributed by BJ, 3-Oct-2019.) |
BOUNDED BOUNDED | ||
Theorem | bd0r 13820 | A formula equivalent to a bounded one is bounded. Stated with a commuted (compared with bd0 13819) biconditional in the hypothesis, to work better with definitions ( is the definiendum that one wants to prove bounded). (Contributed by BJ, 3-Oct-2019.) |
BOUNDED BOUNDED | ||
Theorem | bdbi 13821 | A biconditional between two bounded formulas is bounded. (Contributed by BJ, 3-Oct-2019.) |
BOUNDED BOUNDED BOUNDED | ||
Theorem | bdstab 13822 | Stability of a bounded formula is bounded. (Contributed by BJ, 3-Oct-2019.) |
BOUNDED BOUNDED STAB | ||
Theorem | bddc 13823 | Decidability of a bounded formula is bounded. (Contributed by BJ, 3-Oct-2019.) |
BOUNDED BOUNDED DECID | ||
Theorem | bd3or 13824 | A disjunction of three bounded formulas is bounded. (Contributed by BJ, 3-Oct-2019.) |
BOUNDED BOUNDED BOUNDED BOUNDED | ||
Theorem | bd3an 13825 | A conjunction of three bounded formulas is bounded. (Contributed by BJ, 3-Oct-2019.) |
BOUNDED BOUNDED BOUNDED BOUNDED | ||
Theorem | bdth 13826 | A truth (a (closed) theorem) is a bounded formula. (Contributed by BJ, 6-Oct-2019.) |
BOUNDED | ||
Theorem | bdtru 13827 | The truth value is bounded. (Contributed by BJ, 3-Oct-2019.) |
BOUNDED | ||
Theorem | bdfal 13828 | The truth value is bounded. (Contributed by BJ, 3-Oct-2019.) |
BOUNDED | ||
Theorem | bdnth 13829 | A falsity is a bounded formula. (Contributed by BJ, 6-Oct-2019.) |
BOUNDED | ||
Theorem | bdnthALT 13830 | Alternate proof of bdnth 13829 not using bdfal 13828. Then, bdfal 13828 can be proved from this theorem, using fal 1355. The total number of proof steps would be 17 (for bdnthALT 13830) + 3 = 20, which is more than 8 (for bdfal 13828) + 9 (for bdnth 13829) = 17. (Contributed by BJ, 6-Oct-2019.) (Proof modification is discouraged.) (New usage is discouraged.) |
BOUNDED | ||
Theorem | bdxor 13831 | The exclusive disjunction of two bounded formulas is bounded. (Contributed by BJ, 3-Oct-2019.) |
BOUNDED BOUNDED BOUNDED | ||
Theorem | bj-bdcel 13832* | Boundedness of a membership formula. (Contributed by BJ, 8-Dec-2019.) |
BOUNDED BOUNDED | ||
Theorem | bdab 13833 | Membership in a class defined by class abstraction using a bounded formula, is a bounded formula. (Contributed by BJ, 3-Oct-2019.) |
BOUNDED BOUNDED | ||
Theorem | bdcdeq 13834 | Conditional equality of a bounded formula is a bounded formula. (Contributed by BJ, 16-Oct-2019.) |
BOUNDED BOUNDED CondEq | ||
In line with our definitions of classes as extensions of predicates, it is useful to define a predicate for bounded classes, which is done in df-bdc 13836. Note that this notion is only a technical device which can be used to shorten proofs of (semantic) boundedness of formulas. As will be clear by the end of this subsection (see for instance bdop 13870), one can prove the boundedness of any concrete term using only setvars and bounded formulas, for instance, BOUNDED BOUNDED . The proofs are long since one has to prove boundedness at each step of the construction, without being able to prove general theorems like BOUNDED BOUNDED . | ||
Syntax | wbdc 13835 | Syntax for the predicate BOUNDED. |
BOUNDED | ||
Definition | df-bdc 13836* | Define a bounded class as one such that membership in this class is a bounded formula. (Contributed by BJ, 3-Oct-2019.) |
BOUNDED BOUNDED | ||
Theorem | bdceq 13837 | Equality property for the predicate BOUNDED. (Contributed by BJ, 3-Oct-2019.) |
BOUNDED BOUNDED | ||
Theorem | bdceqi 13838 | A class equal to a bounded one is bounded. Note the use of ax-ext 2152. See also bdceqir 13839. (Contributed by BJ, 3-Oct-2019.) |
BOUNDED BOUNDED | ||
Theorem | bdceqir 13839 | A class equal to a bounded one is bounded. Stated with a commuted (compared with bdceqi 13838) equality in the hypothesis, to work better with definitions ( is the definiendum that one wants to prove bounded; see comment of bd0r 13820). (Contributed by BJ, 3-Oct-2019.) |
BOUNDED BOUNDED | ||
Theorem | bdel 13840* | The belonging of a setvar in a bounded class is a bounded formula. (Contributed by BJ, 3-Oct-2019.) |
BOUNDED BOUNDED | ||
Theorem | bdeli 13841* | Inference associated with bdel 13840. Its converse is bdelir 13842. (Contributed by BJ, 3-Oct-2019.) |
BOUNDED BOUNDED | ||
Theorem | bdelir 13842* | Inference associated with df-bdc 13836. Its converse is bdeli 13841. (Contributed by BJ, 3-Oct-2019.) |
BOUNDED BOUNDED | ||
Theorem | bdcv 13843 | A setvar is a bounded class. (Contributed by BJ, 3-Oct-2019.) |
BOUNDED | ||
Theorem | bdcab 13844 | A class defined by class abstraction using a bounded formula is bounded. (Contributed by BJ, 6-Oct-2019.) |
BOUNDED BOUNDED | ||
Theorem | bdph 13845 | A formula which defines (by class abstraction) a bounded class is bounded. (Contributed by BJ, 6-Oct-2019.) |
BOUNDED BOUNDED | ||
Theorem | bds 13846* | Boundedness of a formula resulting from implicit substitution in a bounded formula. Note that the proof does not use ax-bdsb 13817; therefore, using implicit instead of explicit substitution when boundedness is important, one might avoid using ax-bdsb 13817. (Contributed by BJ, 19-Nov-2019.) |
BOUNDED BOUNDED | ||
Theorem | bdcrab 13847* | A class defined by restricted abstraction from a bounded class and a bounded formula is bounded. (Contributed by BJ, 3-Oct-2019.) |
BOUNDED BOUNDED BOUNDED | ||
Theorem | bdne 13848 | Inequality of two setvars is a bounded formula. (Contributed by BJ, 16-Oct-2019.) |
BOUNDED | ||
Theorem | bdnel 13849* | Non-membership of a setvar in a bounded formula is a bounded formula. (Contributed by BJ, 16-Oct-2019.) |
BOUNDED BOUNDED | ||
Theorem | bdreu 13850* |
Boundedness of existential uniqueness.
Remark regarding restricted quantifiers: the formula need not be bounded even if and are. Indeed, is bounded by bdcvv 13852, and (in minimal propositional calculus), so by bd0 13819, if were bounded when is bounded, then would be bounded as well when is bounded, which is not the case. The same remark holds with . (Contributed by BJ, 16-Oct-2019.) |
BOUNDED BOUNDED | ||
Theorem | bdrmo 13851* | Boundedness of existential at-most-one. (Contributed by BJ, 16-Oct-2019.) |
BOUNDED BOUNDED | ||
Theorem | bdcvv 13852 | The universal class is bounded. The formulation may sound strange, but recall that here, "bounded" means "Δ0". (Contributed by BJ, 3-Oct-2019.) |
BOUNDED | ||
Theorem | bdsbc 13853 | A formula resulting from proper substitution of a setvar for a setvar in a bounded formula is bounded. See also bdsbcALT 13854. (Contributed by BJ, 16-Oct-2019.) |
BOUNDED BOUNDED | ||
Theorem | bdsbcALT 13854 | Alternate proof of bdsbc 13853. (Contributed by BJ, 16-Oct-2019.) (Proof modification is discouraged.) (New usage is discouraged.) |
BOUNDED BOUNDED | ||
Theorem | bdccsb 13855 | A class resulting from proper substitution of a setvar for a setvar in a bounded class is bounded. (Contributed by BJ, 16-Oct-2019.) |
BOUNDED BOUNDED | ||
Theorem | bdcdif 13856 | The difference of two bounded classes is bounded. (Contributed by BJ, 3-Oct-2019.) |
BOUNDED BOUNDED BOUNDED | ||
Theorem | bdcun 13857 | The union of two bounded classes is bounded. (Contributed by BJ, 3-Oct-2019.) |
BOUNDED BOUNDED BOUNDED | ||
Theorem | bdcin 13858 | The intersection of two bounded classes is bounded. (Contributed by BJ, 3-Oct-2019.) |
BOUNDED BOUNDED BOUNDED | ||
Theorem | bdss 13859 | The inclusion of a setvar in a bounded class is a bounded formula. Note: apparently, we cannot prove from the present axioms that equality of two bounded classes is a bounded formula. (Contributed by BJ, 3-Oct-2019.) |
BOUNDED BOUNDED | ||
Theorem | bdcnul 13860 | The empty class is bounded. See also bdcnulALT 13861. (Contributed by BJ, 3-Oct-2019.) |
BOUNDED | ||
Theorem | bdcnulALT 13861 | Alternate proof of bdcnul 13860. Similarly, for the next few theorems proving boundedness of a class, one can either use their definition followed by bdceqir 13839, or use the corresponding characterizations of its elements followed by bdelir 13842. (Contributed by BJ, 3-Oct-2019.) (Proof modification is discouraged.) (New usage is discouraged.) |
BOUNDED | ||
Theorem | bdeq0 13862 | Boundedness of the formula expressing that a setvar is equal to the empty class. (Contributed by BJ, 21-Nov-2019.) |
BOUNDED | ||
Theorem | bj-bd0el 13863 | Boundedness of the formula "the empty set belongs to the setvar ". (Contributed by BJ, 30-Nov-2019.) |
BOUNDED | ||
Theorem | bdcpw 13864 | The power class of a bounded class is bounded. (Contributed by BJ, 3-Oct-2019.) |
BOUNDED BOUNDED | ||
Theorem | bdcsn 13865 | The singleton of a setvar is bounded. (Contributed by BJ, 16-Oct-2019.) |
BOUNDED | ||
Theorem | bdcpr 13866 | The pair of two setvars is bounded. (Contributed by BJ, 16-Oct-2019.) |
BOUNDED | ||
Theorem | bdctp 13867 | The unordered triple of three setvars is bounded. (Contributed by BJ, 16-Oct-2019.) |
BOUNDED | ||
Theorem | bdsnss 13868* | Inclusion of a singleton of a setvar in a bounded class is a bounded formula. (Contributed by BJ, 16-Oct-2019.) |
BOUNDED BOUNDED | ||
Theorem | bdvsn 13869* | Equality of a setvar with a singleton of a setvar is a bounded formula. (Contributed by BJ, 16-Oct-2019.) |
BOUNDED | ||
Theorem | bdop 13870 | The ordered pair of two setvars is a bounded class. (Contributed by BJ, 21-Nov-2019.) |
BOUNDED | ||
Theorem | bdcuni 13871 | The union of a setvar is a bounded class. (Contributed by BJ, 15-Oct-2019.) |
BOUNDED | ||
Theorem | bdcint 13872 | The intersection of a setvar is a bounded class. (Contributed by BJ, 16-Oct-2019.) |
BOUNDED | ||
Theorem | bdciun 13873* | The indexed union of a bounded class with a setvar indexing set is a bounded class. (Contributed by BJ, 16-Oct-2019.) |
BOUNDED BOUNDED | ||
Theorem | bdciin 13874* | The indexed intersection of a bounded class with a setvar indexing set is a bounded class. (Contributed by BJ, 16-Oct-2019.) |
BOUNDED BOUNDED | ||
Theorem | bdcsuc 13875 | The successor of a setvar is a bounded class. (Contributed by BJ, 16-Oct-2019.) |
BOUNDED | ||
Theorem | bdeqsuc 13876* | Boundedness of the formula expressing that a setvar is equal to the successor of another. (Contributed by BJ, 21-Nov-2019.) |
BOUNDED | ||
Theorem | bj-bdsucel 13877 | Boundedness of the formula "the successor of the setvar belongs to the setvar ". (Contributed by BJ, 30-Nov-2019.) |
BOUNDED | ||
Theorem | bdcriota 13878* | A class given by a restricted definition binder is bounded, under the given hypotheses. (Contributed by BJ, 24-Nov-2019.) |
BOUNDED BOUNDED | ||
In this section, we state the axiom scheme of bounded separation, which is part of CZF set theory. | ||
Axiom | ax-bdsep 13879* | Axiom scheme of bounded (or restricted, or Δ0) separation. It is stated with all possible disjoint variable conditions, to show that this weak form is sufficient. For the full axiom of separation, see ax-sep 4105. (Contributed by BJ, 5-Oct-2019.) |
BOUNDED | ||
Theorem | bdsep1 13880* | Version of ax-bdsep 13879 without initial universal quantifier. (Contributed by BJ, 5-Oct-2019.) |
BOUNDED | ||
Theorem | bdsep2 13881* | Version of ax-bdsep 13879 with one disjoint variable condition removed and without initial universal quantifier. Use bdsep1 13880 when sufficient. (Contributed by BJ, 5-Oct-2019.) |
BOUNDED | ||
Theorem | bdsepnft 13882* | Closed form of bdsepnf 13883. Version of ax-bdsep 13879 with one disjoint variable condition removed, the other disjoint variable condition replaced by a nonfreeness antecedent, and without initial universal quantifier. Use bdsep1 13880 when sufficient. (Contributed by BJ, 19-Oct-2019.) |
BOUNDED | ||
Theorem | bdsepnf 13883* | Version of ax-bdsep 13879 with one disjoint variable condition removed, the other disjoint variable condition replaced by a nonfreeness hypothesis, and without initial universal quantifier. See also bdsepnfALT 13884. Use bdsep1 13880 when sufficient. (Contributed by BJ, 5-Oct-2019.) |
BOUNDED | ||
Theorem | bdsepnfALT 13884* | Alternate proof of bdsepnf 13883, not using bdsepnft 13882. (Contributed by BJ, 5-Oct-2019.) (Proof modification is discouraged.) (New usage is discouraged.) |
BOUNDED | ||
Theorem | bdzfauscl 13885* | Closed form of the version of zfauscl 4107 for bounded formulas using bounded separation. (Contributed by BJ, 13-Nov-2019.) |
BOUNDED | ||
Theorem | bdbm1.3ii 13886* | Bounded version of bm1.3ii 4108. (Contributed by BJ, 5-Oct-2019.) (Proof modification is discouraged.) |
BOUNDED | ||
Theorem | bj-axemptylem 13887* | Lemma for bj-axempty 13888 and bj-axempty2 13889. (Contributed by BJ, 25-Oct-2020.) (Proof modification is discouraged.) Use ax-nul 4113 instead. (New usage is discouraged.) |
Theorem | bj-axempty 13888* | Axiom of the empty set from bounded separation. It is provable from bounded separation since the intuitionistic FOL used in iset.mm assumes a nonempty universe. See axnul 4112. (Contributed by BJ, 25-Oct-2020.) (Proof modification is discouraged.) Use ax-nul 4113 instead. (New usage is discouraged.) |
Theorem | bj-axempty2 13889* | Axiom of the empty set from bounded separation, alternate version to bj-axempty 13888. (Contributed by BJ, 27-Oct-2020.) (Proof modification is discouraged.) Use ax-nul 4113 instead. (New usage is discouraged.) |
Theorem | bj-nalset 13890* | nalset 4117 from bounded separation. (Contributed by BJ, 18-Nov-2019.) (Proof modification is discouraged.) |
Theorem | bj-vprc 13891 | vprc 4119 from bounded separation. (Contributed by BJ, 18-Nov-2019.) (Proof modification is discouraged.) |
Theorem | bj-nvel 13892 | nvel 4120 from bounded separation. (Contributed by BJ, 18-Nov-2019.) (Proof modification is discouraged.) |
Theorem | bj-vnex 13893 | vnex 4118 from bounded separation. (Contributed by BJ, 18-Nov-2019.) (Proof modification is discouraged.) |
Theorem | bdinex1 13894 | Bounded version of inex1 4121. (Contributed by BJ, 13-Nov-2019.) (Proof modification is discouraged.) |
BOUNDED | ||
Theorem | bdinex2 13895 | Bounded version of inex2 4122. (Contributed by BJ, 13-Nov-2019.) (Proof modification is discouraged.) |
BOUNDED | ||
Theorem | bdinex1g 13896 | Bounded version of inex1g 4123. (Contributed by BJ, 13-Nov-2019.) (Proof modification is discouraged.) |
BOUNDED | ||
Theorem | bdssex 13897 | Bounded version of ssex 4124. (Contributed by BJ, 13-Nov-2019.) (Proof modification is discouraged.) |
BOUNDED | ||
Theorem | bdssexi 13898 | Bounded version of ssexi 4125. (Contributed by BJ, 13-Nov-2019.) (Proof modification is discouraged.) |
BOUNDED | ||
Theorem | bdssexg 13899 | Bounded version of ssexg 4126. (Contributed by BJ, 13-Nov-2019.) (Proof modification is discouraged.) |
BOUNDED | ||
Theorem | bdssexd 13900 | Bounded version of ssexd 4127. (Contributed by BJ, 13-Nov-2019.) (Proof modification is discouraged.) |
BOUNDED |
< Previous Next > |
Copyright terms: Public domain | < Previous Next > |