![]() |
Metamath
Proof Explorer Theorem List (p. 345 of 473) | < Previous Next > |
Bad symbols? Try the
GIF version. |
||
Mirrors > Metamath Home Page > MPE Home Page > Theorem List Contents > Recent Proofs This page: Page List |
Color key: | ![]() (1-29807) |
![]() (29808-31330) |
![]() (31331-47223) |
Type | Label | Description |
---|---|---|
Statement | ||
Theorem | mulsid1 34401 | Surreal one is an identity element for multiplication. (Contributed by Scott Fenton, 4-Feb-2025.) |
⊢ (𝐴 ∈ No → (𝐴 ·s 1s ) = 𝐴) | ||
Theorem | mulsid2 34402 | Surreal one is an identity element for multiplication. (Contributed by Scott Fenton, 4-Feb-2025.) |
⊢ (𝐴 ∈ No → ( 1s ·s 𝐴) = 𝐴) | ||
Theorem | mulsproplem1 34403* | Lemma for surreal multiplication properties. In the next few lemmas, we aim to prove two properties of surreal multiplication at the same time. Here, we instantiate some quantifiers. (Contributed by Scott Fenton, 7-Feb-2025.) |
⊢ (𝜑 → ∀𝑥 ∈ No ∀𝑦 ∈ No ∀𝑧 ∈ No ∀𝑤 ∈ No (((( bday ‘𝑥) +no ( bday ‘𝑦)) +no (( bday ‘𝑧) +no ( bday ‘𝑤))) ∈ ((( bday ‘𝐴) +no ( bday ‘𝐵)) +no (( bday ‘𝐶) +no ( bday ‘𝐷))) → ((𝑥 ·s 𝑦) ∈ No ∧ ((𝑥 <s 𝑦 ∧ 𝑧 <s 𝑤) → ((𝑦 ·s 𝑧) -s (𝑥 ·s 𝑧)) <s ((𝑦 ·s 𝑤) − (𝑥 ·s 𝑤)))))) & ⊢ (𝜑 → 𝑋 ∈ No ) & ⊢ (𝜑 → 𝑌 ∈ No ) & ⊢ (𝜑 → 𝑍 ∈ No ) & ⊢ (𝜑 → 𝑊 ∈ No ) & ⊢ (𝜑 → ((( bday ‘𝑋) +no ( bday ‘𝑌)) +no (( bday ‘𝑍) +no ( bday ‘𝑊))) ∈ ((( bday ‘𝐴) +no ( bday ‘𝐵)) +no (( bday ‘𝐶) +no ( bday ‘𝐷)))) ⇒ ⊢ (𝜑 → ((𝑋 ·s 𝑌) ∈ No ∧ ((𝑋 <s 𝑌 ∧ 𝑍 <s 𝑊) → ((𝑌 ·s 𝑍) -s (𝑋 ·s 𝑍)) <s ((𝑌 ·s 𝑊) − (𝑋 ·s 𝑊))))) | ||
Theorem | mulsproplem2 34404* | Lemma for surreal multiplication properties. Show that the core expression involved in surreal multiplication's recursive definition is a surreal under the inductive hypothesis. (Contributed by Scott Fenton, 7-Feb-2025.) |
⊢ (𝜑 → ∀𝑥 ∈ No ∀𝑦 ∈ No ∀𝑧 ∈ No ∀𝑤 ∈ No (((( bday ‘𝑥) +no ( bday ‘𝑦)) +no (( bday ‘𝑧) +no ( bday ‘𝑤))) ∈ ((( bday ‘𝐴) +no ( bday ‘𝐵)) +no (( bday ‘𝐶) +no ( bday ‘𝐷))) → ((𝑥 ·s 𝑦) ∈ No ∧ ((𝑥 <s 𝑦 ∧ 𝑧 <s 𝑤) → ((𝑦 ·s 𝑧) -s (𝑥 ·s 𝑧)) <s ((𝑦 ·s 𝑤) − (𝑥 ·s 𝑤)))))) & ⊢ (𝜑 → 𝐴 ∈ No ) & ⊢ (𝜑 → 𝐵 ∈ No ) & ⊢ (𝜑 → 𝑋 ∈ ( O ‘( bday ‘𝐴))) & ⊢ (𝜑 → 𝑌 ∈ ( O ‘( bday ‘𝐵))) ⇒ ⊢ (𝜑 → (((𝑋 ·s 𝐵) +s (𝐴 ·s 𝑌)) -s (𝑋 ·s 𝑌)) ∈ No ) | ||
Syntax | ctxp 34405 | Declare the syntax for tail Cartesian product. |
class (𝐴 ⊗ 𝐵) | ||
Syntax | cpprod 34406 | Declare the syntax for the parallel product. |
class pprod(𝑅, 𝑆) | ||
Syntax | csset 34407 | Declare the subset relationship class. |
class SSet | ||
Syntax | ctrans 34408 | Declare the transitive set class. |
class Trans | ||
Syntax | cbigcup 34409 | Declare the set union relationship. |
class Bigcup | ||
Syntax | cfix 34410 | Declare the syntax for the fixpoints of a class. |
class Fix 𝐴 | ||
Syntax | climits 34411 | Declare the class of limit ordinals. |
class Limits | ||
Syntax | cfuns 34412 | Declare the syntax for the class of all function. |
class Funs | ||
Syntax | csingle 34413 | Declare the syntax for the singleton function. |
class Singleton | ||
Syntax | csingles 34414 | Declare the syntax for the class of all singletons. |
class Singletons | ||
Syntax | cimage 34415 | Declare the syntax for the image functor. |
class Image𝐴 | ||
Syntax | ccart 34416 | Declare the syntax for the cartesian function. |
class Cart | ||
Syntax | cimg 34417 | Declare the syntax for the image function. |
class Img | ||
Syntax | cdomain 34418 | Declare the syntax for the domain function. |
class Domain | ||
Syntax | crange 34419 | Declare the syntax for the range function. |
class Range | ||
Syntax | capply 34420 | Declare the syntax for the application function. |
class Apply | ||
Syntax | ccup 34421 | Declare the syntax for the cup function. |
class Cup | ||
Syntax | ccap 34422 | Declare the syntax for the cap function. |
class Cap | ||
Syntax | csuccf 34423 | Declare the syntax for the successor function. |
class Succ | ||
Syntax | cfunpart 34424 | Declare the syntax for the functional part functor. |
class Funpart𝐹 | ||
Syntax | cfullfn 34425 | Declare the syntax for the full function functor. |
class FullFun𝐹 | ||
Syntax | crestrict 34426 | Declare the syntax for the restriction function. |
class Restrict | ||
Syntax | cub 34427 | Declare the syntax for the upper bound relationship functor. |
class UB𝑅 | ||
Syntax | clb 34428 | Declare the syntax for the lower bound relationship functor. |
class LB𝑅 | ||
Definition | df-txp 34429 | Define the tail cross of two classes. Membership in this class is defined by txpss3v 34453 and brtxp 34455. (Contributed by Scott Fenton, 31-Mar-2012.) |
⊢ (𝐴 ⊗ 𝐵) = ((◡(1st ↾ (V × V)) ∘ 𝐴) ∩ (◡(2nd ↾ (V × V)) ∘ 𝐵)) | ||
Definition | df-pprod 34430 | Define the parallel product of two classes. Membership in this class is defined by pprodss4v 34459 and brpprod 34460. (Contributed by Scott Fenton, 11-Apr-2014.) |
⊢ pprod(𝐴, 𝐵) = ((𝐴 ∘ (1st ↾ (V × V))) ⊗ (𝐵 ∘ (2nd ↾ (V × V)))) | ||
Definition | df-sset 34431 | Define the subset class. For the value, see brsset 34464. (Contributed by Scott Fenton, 31-Mar-2012.) |
⊢ SSet = ((V × V) ∖ ran ( E ⊗ (V ∖ E ))) | ||
Definition | df-trans 34432 | Define the class of all transitive sets. (Contributed by Scott Fenton, 31-Mar-2012.) |
⊢ Trans = (V ∖ ran (( E ∘ E ) ∖ E )) | ||
Definition | df-bigcup 34433 | Define the Bigcup function, which, per fvbigcup 34477, carries a set to its union. (Contributed by Scott Fenton, 11-Apr-2012.) |
⊢ Bigcup = ((V × V) ∖ ran ((V ⊗ E ) △ (( E ∘ E ) ⊗ V))) | ||
Definition | df-fix 34434 | Define the class of all fixpoints of a relationship. (Contributed by Scott Fenton, 11-Apr-2012.) |
⊢ Fix 𝐴 = dom (𝐴 ∩ I ) | ||
Definition | df-limits 34435 | Define the class of all limit ordinals. (Contributed by Scott Fenton, 11-Apr-2012.) |
⊢ Limits = ((On ∩ Fix Bigcup ) ∖ {∅}) | ||
Definition | df-funs 34436 | Define the class of all functions. See elfuns 34490 for membership. (Contributed by Scott Fenton, 18-Feb-2013.) |
⊢ Funs = (𝒫 (V × V) ∖ Fix ( E ∘ ((1st ⊗ ((V ∖ I ) ∘ 2nd )) ∘ ◡ E ))) | ||
Definition | df-singleton 34437 | Define the singleton function. See brsingle 34492 for its value. (Contributed by Scott Fenton, 4-Apr-2014.) |
⊢ Singleton = ((V × V) ∖ ran ((V ⊗ E ) △ ( I ⊗ V))) | ||
Definition | df-singles 34438 | Define the class of all singletons. See elsingles 34493 for membership. (Contributed by Scott Fenton, 19-Feb-2013.) |
⊢ Singletons = ran Singleton | ||
Definition | df-image 34439 | Define the image functor. This function takes a set 𝐴 to a function 𝑥 ↦ (𝐴 “ 𝑥), providing that the latter exists. See imageval 34505 for the derivation. (Contributed by Scott Fenton, 27-Mar-2014.) |
⊢ Image𝐴 = ((V × V) ∖ ran ((V ⊗ E ) △ (( E ∘ ◡𝐴) ⊗ V))) | ||
Definition | df-cart 34440 | Define the cartesian product function. See brcart 34507 for its value. (Contributed by Scott Fenton, 11-Apr-2014.) |
⊢ Cart = (((V × V) × V) ∖ ran ((V ⊗ E ) △ (pprod( E , E ) ⊗ V))) | ||
Definition | df-img 34441 | Define the image function. See brimg 34512 for its value. (Contributed by Scott Fenton, 12-Apr-2014.) |
⊢ Img = (Image((2nd ∘ 1st ) ↾ (1st ↾ (V × V))) ∘ Cart) | ||
Definition | df-domain 34442 | Define the domain function. See brdomain 34508 for its value. (Contributed by Scott Fenton, 11-Apr-2014.) |
⊢ Domain = Image(1st ↾ (V × V)) | ||
Definition | df-range 34443 | Define the range function. See brrange 34509 for its value. (Contributed by Scott Fenton, 11-Apr-2014.) |
⊢ Range = Image(2nd ↾ (V × V)) | ||
Definition | df-cup 34444 | Define the little cup function. See brcup 34514 for its value. (Contributed by Scott Fenton, 14-Apr-2014.) |
⊢ Cup = (((V × V) × V) ∖ ran ((V ⊗ E ) △ (((◡1st ∘ E ) ∪ (◡2nd ∘ E )) ⊗ V))) | ||
Definition | df-cap 34445 | Define the little cap function. See brcap 34515 for its value. (Contributed by Scott Fenton, 17-Apr-2014.) |
⊢ Cap = (((V × V) × V) ∖ ran ((V ⊗ E ) △ (((◡1st ∘ E ) ∩ (◡2nd ∘ E )) ⊗ V))) | ||
Definition | df-restrict 34446 | Define the restriction function. See brrestrict 34524 for its value. (Contributed by Scott Fenton, 17-Apr-2014.) |
⊢ Restrict = (Cap ∘ (1st ⊗ (Cart ∘ (2nd ⊗ (Range ∘ 1st ))))) | ||
Definition | df-succf 34447 | Define the successor function. See brsuccf 34516 for its value. (Contributed by Scott Fenton, 14-Apr-2014.) |
⊢ Succ = (Cup ∘ ( I ⊗ Singleton)) | ||
Definition | df-apply 34448 | Define the application function. See brapply 34513 for its value. (Contributed by Scott Fenton, 12-Apr-2014.) |
⊢ Apply = (( Bigcup ∘ Bigcup ) ∘ (((V × V) ∖ ran ((V ⊗ E ) △ (( E ↾ Singletons ) ⊗ V))) ∘ ((Singleton ∘ Img) ∘ pprod( I , Singleton)))) | ||
Definition | df-funpart 34449 | Define the functional part of a class 𝐹. This is the maximal part of 𝐹 that is a function. See funpartfun 34518 and funpartfv 34520 for the meaning of this statement. (Contributed by Scott Fenton, 16-Apr-2014.) |
⊢ Funpart𝐹 = (𝐹 ↾ dom ((Image𝐹 ∘ Singleton) ∩ (V × Singletons ))) | ||
Definition | df-fullfun 34450 | Define the full function over 𝐹. This is a function with domain V that always agrees with 𝐹 for its value. (Contributed by Scott Fenton, 17-Apr-2014.) |
⊢ FullFun𝐹 = (Funpart𝐹 ∪ ((V ∖ dom Funpart𝐹) × {∅})) | ||
Definition | df-ub 34451 | Define the upper bound relationship functor. See brub 34529 for value. (Contributed by Scott Fenton, 3-May-2018.) |
⊢ UB𝑅 = ((V × V) ∖ ((V ∖ 𝑅) ∘ ◡ E )) | ||
Definition | df-lb 34452 | Define the lower bound relationship functor. See brlb 34530 for value. (Contributed by Scott Fenton, 3-May-2018.) |
⊢ LB𝑅 = UB◡𝑅 | ||
Theorem | txpss3v 34453 | A tail Cartesian product is a subset of the class of ordered triples. (Contributed by Scott Fenton, 31-Mar-2012.) |
⊢ (𝐴 ⊗ 𝐵) ⊆ (V × (V × V)) | ||
Theorem | txprel 34454 | A tail Cartesian product is a relationship. (Contributed by Scott Fenton, 31-Mar-2012.) |
⊢ Rel (𝐴 ⊗ 𝐵) | ||
Theorem | brtxp 34455 | Characterize a ternary relation over a tail Cartesian product. Together with txpss3v 34453, this completely defines membership in a tail cross. (Contributed by Scott Fenton, 31-Mar-2012.) (Proof shortened by Peter Mazsa, 2-Oct-2022.) |
⊢ 𝑋 ∈ V & ⊢ 𝑌 ∈ V & ⊢ 𝑍 ∈ V ⇒ ⊢ (𝑋(𝐴 ⊗ 𝐵)〈𝑌, 𝑍〉 ↔ (𝑋𝐴𝑌 ∧ 𝑋𝐵𝑍)) | ||
Theorem | brtxp2 34456* | The binary relation over a tail cross when the second argument is not an ordered pair. (Contributed by Scott Fenton, 14-Apr-2014.) (Revised by Mario Carneiro, 3-May-2015.) |
⊢ 𝐴 ∈ V ⇒ ⊢ (𝐴(𝑅 ⊗ 𝑆)𝐵 ↔ ∃𝑥∃𝑦(𝐵 = 〈𝑥, 𝑦〉 ∧ 𝐴𝑅𝑥 ∧ 𝐴𝑆𝑦)) | ||
Theorem | dfpprod2 34457 | Expanded definition of parallel product. (Contributed by Scott Fenton, 3-May-2014.) |
⊢ pprod(𝐴, 𝐵) = ((◡(1st ↾ (V × V)) ∘ (𝐴 ∘ (1st ↾ (V × V)))) ∩ (◡(2nd ↾ (V × V)) ∘ (𝐵 ∘ (2nd ↾ (V × V))))) | ||
Theorem | pprodcnveq 34458 | A converse law for parallel product. (Contributed by Scott Fenton, 3-May-2014.) |
⊢ pprod(𝑅, 𝑆) = ◡pprod(◡𝑅, ◡𝑆) | ||
Theorem | pprodss4v 34459 | The parallel product is a subclass of ((V × V) × (V × V)). (Contributed by Scott Fenton, 11-Apr-2014.) (Revised by Mario Carneiro, 19-Apr-2014.) (Proof shortened by Peter Mazsa, 2-Oct-2022.) |
⊢ pprod(𝐴, 𝐵) ⊆ ((V × V) × (V × V)) | ||
Theorem | brpprod 34460 | Characterize a quaternary relation over a tail Cartesian product. Together with pprodss4v 34459, this completely defines membership in a parallel product. (Contributed by Scott Fenton, 11-Apr-2014.) (Revised by Mario Carneiro, 19-Apr-2014.) |
⊢ 𝑋 ∈ V & ⊢ 𝑌 ∈ V & ⊢ 𝑍 ∈ V & ⊢ 𝑊 ∈ V ⇒ ⊢ (〈𝑋, 𝑌〉pprod(𝐴, 𝐵)〈𝑍, 𝑊〉 ↔ (𝑋𝐴𝑍 ∧ 𝑌𝐵𝑊)) | ||
Theorem | brpprod3a 34461* | Condition for parallel product when the last argument is not an ordered pair. (Contributed by Scott Fenton, 11-Apr-2014.) (Revised by Mario Carneiro, 19-Apr-2014.) |
⊢ 𝑋 ∈ V & ⊢ 𝑌 ∈ V & ⊢ 𝑍 ∈ V ⇒ ⊢ (〈𝑋, 𝑌〉pprod(𝑅, 𝑆)𝑍 ↔ ∃𝑧∃𝑤(𝑍 = 〈𝑧, 𝑤〉 ∧ 𝑋𝑅𝑧 ∧ 𝑌𝑆𝑤)) | ||
Theorem | brpprod3b 34462* | Condition for parallel product when the first argument is not an ordered pair. (Contributed by Scott Fenton, 3-May-2014.) |
⊢ 𝑋 ∈ V & ⊢ 𝑌 ∈ V & ⊢ 𝑍 ∈ V ⇒ ⊢ (𝑋pprod(𝑅, 𝑆)〈𝑌, 𝑍〉 ↔ ∃𝑧∃𝑤(𝑋 = 〈𝑧, 𝑤〉 ∧ 𝑧𝑅𝑌 ∧ 𝑤𝑆𝑍)) | ||
Theorem | relsset 34463 | The subset class is a binary relation. (Contributed by Scott Fenton, 31-Mar-2012.) |
⊢ Rel SSet | ||
Theorem | brsset 34464 | For sets, the SSet binary relation is equivalent to the subset relationship. (Contributed by Scott Fenton, 31-Mar-2012.) |
⊢ 𝐵 ∈ V ⇒ ⊢ (𝐴 SSet 𝐵 ↔ 𝐴 ⊆ 𝐵) | ||
Theorem | idsset 34465 | I is equal to the intersection of SSet and its converse. (Contributed by Scott Fenton, 31-Mar-2012.) |
⊢ I = ( SSet ∩ ◡ SSet ) | ||
Theorem | eltrans 34466 | Membership in the class of all transitive sets. (Contributed by Scott Fenton, 31-Mar-2012.) |
⊢ 𝐴 ∈ V ⇒ ⊢ (𝐴 ∈ Trans ↔ Tr 𝐴) | ||
Theorem | dfon3 34467 | A quantifier-free definition of On. (Contributed by Scott Fenton, 5-Apr-2012.) |
⊢ On = (V ∖ ran (( SSet ∩ ( Trans × V)) ∖ ( I ∪ E ))) | ||
Theorem | dfon4 34468 | Another quantifier-free definition of On. (Contributed by Scott Fenton, 4-May-2014.) |
⊢ On = (V ∖ (( SSet ∖ ( I ∪ E )) “ Trans )) | ||
Theorem | brtxpsd 34469* | Expansion of a common form used in quantifier-free definitions. (Contributed by Scott Fenton, 17-Apr-2014.) (Revised by Mario Carneiro, 19-Apr-2014.) |
⊢ 𝐴 ∈ V & ⊢ 𝐵 ∈ V ⇒ ⊢ (¬ 𝐴ran ((V ⊗ E ) △ (𝑅 ⊗ V))𝐵 ↔ ∀𝑥(𝑥 ∈ 𝐵 ↔ 𝑥𝑅𝐴)) | ||
Theorem | brtxpsd2 34470* | Another common abbreviation for quantifier-free definitions. (Contributed by Scott Fenton, 21-Apr-2014.) |
⊢ 𝐴 ∈ V & ⊢ 𝐵 ∈ V & ⊢ 𝑅 = (𝐶 ∖ ran ((V ⊗ E ) △ (𝑆 ⊗ V))) & ⊢ 𝐴𝐶𝐵 ⇒ ⊢ (𝐴𝑅𝐵 ↔ ∀𝑥(𝑥 ∈ 𝐵 ↔ 𝑥𝑆𝐴)) | ||
Theorem | brtxpsd3 34471* | A third common abbreviation for quantifier-free definitions. (Contributed by Scott Fenton, 3-May-2014.) |
⊢ 𝐴 ∈ V & ⊢ 𝐵 ∈ V & ⊢ 𝑅 = (𝐶 ∖ ran ((V ⊗ E ) △ (𝑆 ⊗ V))) & ⊢ 𝐴𝐶𝐵 & ⊢ (𝑥 ∈ 𝑋 ↔ 𝑥𝑆𝐴) ⇒ ⊢ (𝐴𝑅𝐵 ↔ 𝐵 = 𝑋) | ||
Theorem | relbigcup 34472 | The Bigcup relationship is a relationship. (Contributed by Scott Fenton, 11-Apr-2012.) |
⊢ Rel Bigcup | ||
Theorem | brbigcup 34473 | Binary relation over Bigcup . (Contributed by Scott Fenton, 11-Apr-2012.) |
⊢ 𝐵 ∈ V ⇒ ⊢ (𝐴 Bigcup 𝐵 ↔ ∪ 𝐴 = 𝐵) | ||
Theorem | dfbigcup2 34474 | Bigcup using maps-to notation. (Contributed by Scott Fenton, 16-Apr-2012.) |
⊢ Bigcup = (𝑥 ∈ V ↦ ∪ 𝑥) | ||
Theorem | fobigcup 34475 | Bigcup maps the universe onto itself. (Contributed by Scott Fenton, 16-Apr-2012.) |
⊢ Bigcup :V–onto→V | ||
Theorem | fnbigcup 34476 | Bigcup is a function over the universal class. (Contributed by Scott Fenton, 11-Apr-2012.) |
⊢ Bigcup Fn V | ||
Theorem | fvbigcup 34477 | For sets, Bigcup yields union. (Contributed by Scott Fenton, 11-Apr-2012.) |
⊢ 𝐴 ∈ V ⇒ ⊢ ( Bigcup ‘𝐴) = ∪ 𝐴 | ||
Theorem | elfix 34478 | Membership in the fixpoints of a class. (Contributed by Scott Fenton, 11-Apr-2012.) |
⊢ 𝐴 ∈ V ⇒ ⊢ (𝐴 ∈ Fix 𝑅 ↔ 𝐴𝑅𝐴) | ||
Theorem | elfix2 34479 | Alternative membership in the fixpoint of a class. (Contributed by Scott Fenton, 11-Apr-2012.) |
⊢ Rel 𝑅 ⇒ ⊢ (𝐴 ∈ Fix 𝑅 ↔ 𝐴𝑅𝐴) | ||
Theorem | dffix2 34480 | The fixpoints of a class in terms of its range. (Contributed by Scott Fenton, 16-Apr-2012.) |
⊢ Fix 𝐴 = ran (𝐴 ∩ I ) | ||
Theorem | fixssdm 34481 | The fixpoints of a class are a subset of its domain. (Contributed by Scott Fenton, 16-Apr-2012.) |
⊢ Fix 𝐴 ⊆ dom 𝐴 | ||
Theorem | fixssrn 34482 | The fixpoints of a class are a subset of its range. (Contributed by Scott Fenton, 16-Apr-2012.) |
⊢ Fix 𝐴 ⊆ ran 𝐴 | ||
Theorem | fixcnv 34483 | The fixpoints of a class are the same as those of its converse. (Contributed by Scott Fenton, 16-Apr-2012.) |
⊢ Fix 𝐴 = Fix ◡𝐴 | ||
Theorem | fixun 34484 | The fixpoint operator distributes over union. (Contributed by Scott Fenton, 16-Apr-2012.) |
⊢ Fix (𝐴 ∪ 𝐵) = ( Fix 𝐴 ∪ Fix 𝐵) | ||
Theorem | ellimits 34485 | Membership in the class of all limit ordinals. (Contributed by Scott Fenton, 11-Apr-2012.) |
⊢ 𝐴 ∈ V ⇒ ⊢ (𝐴 ∈ Limits ↔ Lim 𝐴) | ||
Theorem | limitssson 34486 | The class of all limit ordinals is a subclass of the class of all ordinals. (Contributed by Scott Fenton, 11-Apr-2012.) |
⊢ Limits ⊆ On | ||
Theorem | dfom5b 34487 | A quantifier-free definition of ω that does not depend on ax-inf 9573. (Note: label was changed from dfom5 9585 to dfom5b 34487 to prevent naming conflict. NM, 12-Feb-2013.) (Contributed by Scott Fenton, 11-Apr-2012.) |
⊢ ω = (On ∩ ∩ Limits ) | ||
Theorem | sscoid 34488 | A condition for subset and composition with identity. (Contributed by Scott Fenton, 13-Apr-2018.) |
⊢ (𝐴 ⊆ ( I ∘ 𝐵) ↔ (Rel 𝐴 ∧ 𝐴 ⊆ 𝐵)) | ||
Theorem | dffun10 34489 | Another potential definition of functionality. Based on statements in http://people.math.gatech.edu/~belinfan/research/autoreas/otter/sum/fs/. (Contributed by Scott Fenton, 30-Aug-2017.) |
⊢ (Fun 𝐹 ↔ 𝐹 ⊆ ( I ∘ (V ∖ ((V ∖ I ) ∘ 𝐹)))) | ||
Theorem | elfuns 34490 | Membership in the class of all functions. (Contributed by Scott Fenton, 18-Feb-2013.) |
⊢ 𝐹 ∈ V ⇒ ⊢ (𝐹 ∈ Funs ↔ Fun 𝐹) | ||
Theorem | elfunsg 34491 | Closed form of elfuns 34490. (Contributed by Scott Fenton, 2-May-2014.) |
⊢ (𝐹 ∈ 𝑉 → (𝐹 ∈ Funs ↔ Fun 𝐹)) | ||
Theorem | brsingle 34492 | The binary relation form of the singleton function. (Contributed by Scott Fenton, 4-Apr-2014.) (Revised by Mario Carneiro, 19-Apr-2014.) |
⊢ 𝐴 ∈ V & ⊢ 𝐵 ∈ V ⇒ ⊢ (𝐴Singleton𝐵 ↔ 𝐵 = {𝐴}) | ||
Theorem | elsingles 34493* | Membership in the class of all singletons. (Contributed by Scott Fenton, 19-Feb-2013.) |
⊢ (𝐴 ∈ Singletons ↔ ∃𝑥 𝐴 = {𝑥}) | ||
Theorem | fnsingle 34494 | The singleton relationship is a function over the universe. (Contributed by Scott Fenton, 4-Apr-2014.) (Revised by Mario Carneiro, 19-Apr-2014.) |
⊢ Singleton Fn V | ||
Theorem | fvsingle 34495 | The value of the singleton function. (Contributed by Scott Fenton, 4-Apr-2014.) (Revised by Mario Carneiro, 19-Apr-2014.) (Revised by Scott Fenton, 13-Apr-2018.) |
⊢ (Singleton‘𝐴) = {𝐴} | ||
Theorem | dfsingles2 34496* | Alternate definition of the class of all singletons. (Contributed by Scott Fenton, 20-Nov-2013.) (Revised by Mario Carneiro, 19-Apr-2014.) |
⊢ Singletons = {𝑥 ∣ ∃𝑦 𝑥 = {𝑦}} | ||
Theorem | snelsingles 34497 | A singleton is a member of the class of all singletons. (Contributed by Scott Fenton, 19-Feb-2013.) |
⊢ 𝐴 ∈ V ⇒ ⊢ {𝐴} ∈ Singletons | ||
Theorem | dfiota3 34498 | A definition of iota using minimal quantifiers. (Contributed by Scott Fenton, 19-Feb-2013.) |
⊢ (℩𝑥𝜑) = ∪ ∪ ({{𝑥 ∣ 𝜑}} ∩ Singletons ) | ||
Theorem | dffv5 34499 | Another quantifier-free definition of function value. (Contributed by Scott Fenton, 19-Feb-2013.) |
⊢ (𝐹‘𝐴) = ∪ ∪ ({(𝐹 “ {𝐴})} ∩ Singletons ) | ||
Theorem | unisnif 34500 | Express union of singleton in terms of if. (Contributed by Scott Fenton, 27-Mar-2014.) (Revised by Mario Carneiro, 19-Apr-2014.) |
⊢ ∪ {𝐴} = if(𝐴 ∈ V, 𝐴, ∅) |
< Previous Next > |
Copyright terms: Public domain | < Previous Next > |