Home | Metamath
Proof Explorer Theorem List (p. 342 of 466) | < 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: | Metamath Proof Explorer
(1-29289) |
Hilbert Space Explorer
(29290-30812) |
Users' Mathboxes
(30813-46532) |
Type | Label | Description |
---|---|---|
Statement | ||
Theorem | cofcutr 34101* | If 𝑋 is the cut of 𝐴 and 𝐵, then 𝐴 is cofinal with ( L ‘𝑋) and 𝐵 is coinitial with ( R ‘𝑋). Theorem 2.9 of [Gonshor] p. 12. (Contributed by Scott Fenton, 25-Sep-2024.) |
⊢ ((𝐴 <<s 𝐵 ∧ 𝑋 = (𝐴 |s 𝐵)) → (∀𝑥 ∈ ( L ‘𝑋)∃𝑦 ∈ 𝐴 𝑥 ≤s 𝑦 ∧ ∀𝑧 ∈ ( R ‘𝑋)∃𝑤 ∈ 𝐵 𝑤 ≤s 𝑧)) | ||
Theorem | cofcutrtime 34102* | If 𝑋 is the cut of 𝐴 and 𝐵 and all of 𝐴 and 𝐵 are older than 𝑋, then ( L ‘𝑋) is cofinal with 𝐴 and ( R ‘𝑋) is coinitial with 𝐵. Note: we will call a cut where all of the elements of the cut are older than the cut itself a "timely" cut. Part of Theorem 4.02(12) of [Alling] p. 125. (Contributed by Scott Fenton, 27-Sep-2024.) |
⊢ (((𝐴 ∪ 𝐵) ⊆ ( O ‘( bday ‘𝑋)) ∧ 𝐴 <<s 𝐵 ∧ 𝑋 = (𝐴 |s 𝐵)) → (∀𝑥 ∈ 𝐴 ∃𝑦 ∈ ( L ‘𝑋)𝑥 ≤s 𝑦 ∧ ∀𝑧 ∈ 𝐵 ∃𝑤 ∈ ( R ‘𝑋)𝑤 ≤s 𝑧)) | ||
Syntax | cnorec 34103 | Declare the syntax for surreal recursion of one variable. |
class norec (𝐹) | ||
Definition | df-norec 34104* | Define the recursion generator for surreal functions of one variable. This generator creates a recursive function of surreals from their value on their left and right sets. (Contributed by Scott Fenton, 19-Aug-2024.) |
⊢ norec (𝐹) = frecs({〈𝑥, 𝑦〉 ∣ 𝑥 ∈ (( L ‘𝑦) ∪ ( R ‘𝑦))}, No , 𝐹) | ||
Theorem | lrrecval 34105* | The next step in the development of the surreals is to establish induction and recursion across left and right sets. To that end, we are going to develop a relationship 𝑅 that is founded, partial, and set-like across the surreals. This first theorem just establishes the value of 𝑅. (Contributed by Scott Fenton, 19-Aug-2024.) |
⊢ 𝑅 = {〈𝑥, 𝑦〉 ∣ 𝑥 ∈ (( L ‘𝑦) ∪ ( R ‘𝑦))} ⇒ ⊢ ((𝐴 ∈ No ∧ 𝐵 ∈ No ) → (𝐴𝑅𝐵 ↔ 𝐴 ∈ (( L ‘𝐵) ∪ ( R ‘𝐵)))) | ||
Theorem | lrrecval2 34106* | Next, we establish an alternate expression for 𝑅. (Contributed by Scott Fenton, 19-Aug-2024.) |
⊢ 𝑅 = {〈𝑥, 𝑦〉 ∣ 𝑥 ∈ (( L ‘𝑦) ∪ ( R ‘𝑦))} ⇒ ⊢ ((𝐴 ∈ No ∧ 𝐵 ∈ No ) → (𝐴𝑅𝐵 ↔ ( bday ‘𝐴) ∈ ( bday ‘𝐵))) | ||
Theorem | lrrecpo 34107* | Now, we establish that 𝑅 is a partial ordering on No . (Contributed by Scott Fenton, 19-Aug-2024.) |
⊢ 𝑅 = {〈𝑥, 𝑦〉 ∣ 𝑥 ∈ (( L ‘𝑦) ∪ ( R ‘𝑦))} ⇒ ⊢ 𝑅 Po No | ||
Theorem | lrrecse 34108* | Next, we show that 𝑅 is set-like over No . (Contributed by Scott Fenton, 19-Aug-2024.) |
⊢ 𝑅 = {〈𝑥, 𝑦〉 ∣ 𝑥 ∈ (( L ‘𝑦) ∪ ( R ‘𝑦))} ⇒ ⊢ 𝑅 Se No | ||
Theorem | lrrecfr 34109* | Now we show that 𝑅 is founded over No . (Contributed by Scott Fenton, 19-Aug-2024.) |
⊢ 𝑅 = {〈𝑥, 𝑦〉 ∣ 𝑥 ∈ (( L ‘𝑦) ∪ ( R ‘𝑦))} ⇒ ⊢ 𝑅 Fr No | ||
Theorem | lrrecpred 34110* | Finally, we calculate the value of the predecessor class over 𝑅. (Contributed by Scott Fenton, 19-Aug-2024.) |
⊢ 𝑅 = {〈𝑥, 𝑦〉 ∣ 𝑥 ∈ (( L ‘𝑦) ∪ ( R ‘𝑦))} ⇒ ⊢ (𝐴 ∈ No → Pred(𝑅, No , 𝐴) = (( L ‘𝐴) ∪ ( R ‘𝐴))) | ||
Theorem | noinds 34111* | Induction principle for a single surreal. If a property passes from a surreal's left and right sets to the surreal itself, then it holds for all surreals. (Contributed by Scott Fenton, 19-Aug-2024.) |
⊢ (𝑥 = 𝑦 → (𝜑 ↔ 𝜓)) & ⊢ (𝑥 = 𝐴 → (𝜑 ↔ 𝜒)) & ⊢ (𝑥 ∈ No → (∀𝑦 ∈ (( L ‘𝑥) ∪ ( R ‘𝑥))𝜓 → 𝜑)) ⇒ ⊢ (𝐴 ∈ No → 𝜒) | ||
Theorem | norecfn 34112 | Surreal recursion over one variable is a function over the surreals. (Contributed by Scott Fenton, 19-Aug-2024.) |
⊢ 𝐹 = norec (𝐺) ⇒ ⊢ 𝐹 Fn No | ||
Theorem | norecov 34113 | Calculate the value of the surreal recursion operation. (Contributed by Scott Fenton, 19-Aug-2024.) |
⊢ 𝐹 = norec (𝐺) ⇒ ⊢ (𝐴 ∈ No → (𝐹‘𝐴) = (𝐴𝐺(𝐹 ↾ (( L ‘𝐴) ∪ ( R ‘𝐴))))) | ||
Syntax | cnorec2 34114 | Declare the syntax for surreal recursion on two arguments. |
class norec2 (𝐹) | ||
Definition | df-norec2 34115* | Define surreal recursion on two variables. This function is key to the development of most of surreal numbers. (Contributed by Scott Fenton, 20-Aug-2024.) |
⊢ norec2 (𝐹) = frecs({〈𝑎, 𝑏〉 ∣ (𝑎 ∈ ( No × No ) ∧ 𝑏 ∈ ( No × No ) ∧ (((1st ‘𝑎){〈𝑐, 𝑑〉 ∣ 𝑐 ∈ (( L ‘𝑑) ∪ ( R ‘𝑑))} (1st ‘𝑏) ∨ (1st ‘𝑎) = (1st ‘𝑏)) ∧ ((2nd ‘𝑎){〈𝑐, 𝑑〉 ∣ 𝑐 ∈ (( L ‘𝑑) ∪ ( R ‘𝑑))} (2nd ‘𝑏) ∨ (2nd ‘𝑎) = (2nd ‘𝑏)) ∧ 𝑎 ≠ 𝑏))}, ( No × No ), 𝐹) | ||
Theorem | noxpordpo 34116* | To get through most of the textbook defintions in surreal numbers we will need recursion on two variables. This set of theorems sets up the preconditions for double recursion. This theorem establishes the partial ordering. (Contributed by Scott Fenton, 19-Aug-2024.) |
⊢ 𝑅 = {〈𝑎, 𝑏〉 ∣ 𝑎 ∈ (( L ‘𝑏) ∪ ( R ‘𝑏))} & ⊢ 𝑆 = {〈𝑥, 𝑦〉 ∣ (𝑥 ∈ ( No × No ) ∧ 𝑦 ∈ ( No × No ) ∧ (((1st ‘𝑥)𝑅(1st ‘𝑦) ∨ (1st ‘𝑥) = (1st ‘𝑦)) ∧ ((2nd ‘𝑥)𝑅(2nd ‘𝑦) ∨ (2nd ‘𝑥) = (2nd ‘𝑦)) ∧ 𝑥 ≠ 𝑦))} ⇒ ⊢ 𝑆 Po ( No × No ) | ||
Theorem | noxpordfr 34117* | Next we establish the foundedness of the relationship. (Contributed by Scott Fenton, 19-Aug-2024.) |
⊢ 𝑅 = {〈𝑎, 𝑏〉 ∣ 𝑎 ∈ (( L ‘𝑏) ∪ ( R ‘𝑏))} & ⊢ 𝑆 = {〈𝑥, 𝑦〉 ∣ (𝑥 ∈ ( No × No ) ∧ 𝑦 ∈ ( No × No ) ∧ (((1st ‘𝑥)𝑅(1st ‘𝑦) ∨ (1st ‘𝑥) = (1st ‘𝑦)) ∧ ((2nd ‘𝑥)𝑅(2nd ‘𝑦) ∨ (2nd ‘𝑥) = (2nd ‘𝑦)) ∧ 𝑥 ≠ 𝑦))} ⇒ ⊢ 𝑆 Fr ( No × No ) | ||
Theorem | noxpordse 34118* | Next we establish the set-like nature of the relationship. (Contributed by Scott Fenton, 19-Aug-2024.) |
⊢ 𝑅 = {〈𝑎, 𝑏〉 ∣ 𝑎 ∈ (( L ‘𝑏) ∪ ( R ‘𝑏))} & ⊢ 𝑆 = {〈𝑥, 𝑦〉 ∣ (𝑥 ∈ ( No × No ) ∧ 𝑦 ∈ ( No × No ) ∧ (((1st ‘𝑥)𝑅(1st ‘𝑦) ∨ (1st ‘𝑥) = (1st ‘𝑦)) ∧ ((2nd ‘𝑥)𝑅(2nd ‘𝑦) ∨ (2nd ‘𝑥) = (2nd ‘𝑦)) ∧ 𝑥 ≠ 𝑦))} ⇒ ⊢ 𝑆 Se ( No × No ) | ||
Theorem | noxpordpred 34119* | Next we calculate the predecessor class of the relationship. (Contributed by Scott Fenton, 19-Aug-2024.) |
⊢ 𝑅 = {〈𝑎, 𝑏〉 ∣ 𝑎 ∈ (( L ‘𝑏) ∪ ( R ‘𝑏))} & ⊢ 𝑆 = {〈𝑥, 𝑦〉 ∣ (𝑥 ∈ ( No × No ) ∧ 𝑦 ∈ ( No × No ) ∧ (((1st ‘𝑥)𝑅(1st ‘𝑦) ∨ (1st ‘𝑥) = (1st ‘𝑦)) ∧ ((2nd ‘𝑥)𝑅(2nd ‘𝑦) ∨ (2nd ‘𝑥) = (2nd ‘𝑦)) ∧ 𝑥 ≠ 𝑦))} ⇒ ⊢ ((𝐴 ∈ No ∧ 𝐵 ∈ No ) → Pred(𝑆, ( No × No ), 〈𝐴, 𝐵〉) = ((((( L ‘𝐴) ∪ ( R ‘𝐴)) ∪ {𝐴}) × ((( L ‘𝐵) ∪ ( R ‘𝐵)) ∪ {𝐵})) ∖ {〈𝐴, 𝐵〉})) | ||
Theorem | no2indslem 34120* | Double induction on surreals with explicit notation for the relationships. (Contributed by Scott Fenton, 22-Aug-2024.) |
⊢ 𝑅 = {〈𝑎, 𝑏〉 ∣ 𝑎 ∈ (( L ‘𝑏) ∪ ( R ‘𝑏))} & ⊢ 𝑆 = {〈𝑐, 𝑑〉 ∣ (𝑐 ∈ ( No × No ) ∧ 𝑑 ∈ ( No × No ) ∧ (((1st ‘𝑐)𝑅(1st ‘𝑑) ∨ (1st ‘𝑐) = (1st ‘𝑑)) ∧ ((2nd ‘𝑐)𝑅(2nd ‘𝑑) ∨ (2nd ‘𝑐) = (2nd ‘𝑑)) ∧ 𝑐 ≠ 𝑑))} & ⊢ (𝑥 = 𝑧 → (𝜑 ↔ 𝜓)) & ⊢ (𝑦 = 𝑤 → (𝜓 ↔ 𝜒)) & ⊢ (𝑥 = 𝑧 → (𝜃 ↔ 𝜒)) & ⊢ (𝑥 = 𝐴 → (𝜑 ↔ 𝜏)) & ⊢ (𝑦 = 𝐵 → (𝜏 ↔ 𝜂)) & ⊢ ((𝑥 ∈ No ∧ 𝑦 ∈ No ) → ((∀𝑧 ∈ (( L ‘𝑥) ∪ ( R ‘𝑥))∀𝑤 ∈ (( L ‘𝑦) ∪ ( R ‘𝑦))𝜒 ∧ ∀𝑧 ∈ (( L ‘𝑥) ∪ ( R ‘𝑥))𝜓 ∧ ∀𝑤 ∈ (( L ‘𝑦) ∪ ( R ‘𝑦))𝜃) → 𝜑)) ⇒ ⊢ ((𝐴 ∈ No ∧ 𝐵 ∈ No ) → 𝜂) | ||
Theorem | no2inds 34121* | Double induction on surreals. The many substitution instances are to cover all possible cases. (Contributed by Scott Fenton, 22-Aug-2024.) |
⊢ (𝑥 = 𝑧 → (𝜑 ↔ 𝜓)) & ⊢ (𝑦 = 𝑤 → (𝜓 ↔ 𝜒)) & ⊢ (𝑥 = 𝑧 → (𝜃 ↔ 𝜒)) & ⊢ (𝑥 = 𝐴 → (𝜑 ↔ 𝜏)) & ⊢ (𝑦 = 𝐵 → (𝜏 ↔ 𝜂)) & ⊢ ((𝑥 ∈ No ∧ 𝑦 ∈ No ) → ((∀𝑧 ∈ (( L ‘𝑥) ∪ ( R ‘𝑥))∀𝑤 ∈ (( L ‘𝑦) ∪ ( R ‘𝑦))𝜒 ∧ ∀𝑧 ∈ (( L ‘𝑥) ∪ ( R ‘𝑥))𝜓 ∧ ∀𝑤 ∈ (( L ‘𝑦) ∪ ( R ‘𝑦))𝜃) → 𝜑)) ⇒ ⊢ ((𝐴 ∈ No ∧ 𝐵 ∈ No ) → 𝜂) | ||
Theorem | norec2fn 34122 | The double-recursion operator on surreals yields a function on pairs of surreals. (Contributed by Scott Fenton, 20-Aug-2024.) |
⊢ 𝐹 = norec2 (𝐺) ⇒ ⊢ 𝐹 Fn ( No × No ) | ||
Theorem | norec2ov 34123 | The value of the double-recursion surreal function. (Contributed by Scott Fenton, 20-Aug-2024.) |
⊢ 𝐹 = norec2 (𝐺) ⇒ ⊢ ((𝐴 ∈ No ∧ 𝐵 ∈ No ) → (𝐴𝐹𝐵) = (〈𝐴, 𝐵〉𝐺(𝐹 ↾ ((((( L ‘𝐴) ∪ ( R ‘𝐴)) ∪ {𝐴}) × ((( L ‘𝐵) ∪ ( R ‘𝐵)) ∪ {𝐵})) ∖ {〈𝐴, 𝐵〉})))) | ||
Theorem | no3inds 34124* | Triple induction over surreal numbers. (Contributed by Scott Fenton, 9-Oct-2024.) |
⊢ (𝑎 = 𝑑 → (𝜑 ↔ 𝜓)) & ⊢ (𝑏 = 𝑒 → (𝜓 ↔ 𝜒)) & ⊢ (𝑐 = 𝑓 → (𝜒 ↔ 𝜃)) & ⊢ (𝑎 = 𝑑 → (𝜏 ↔ 𝜃)) & ⊢ (𝑏 = 𝑒 → (𝜂 ↔ 𝜏)) & ⊢ (𝑏 = 𝑒 → (𝜁 ↔ 𝜃)) & ⊢ (𝑐 = 𝑓 → (𝜎 ↔ 𝜏)) & ⊢ (𝑎 = 𝑋 → (𝜑 ↔ 𝜌)) & ⊢ (𝑏 = 𝑌 → (𝜌 ↔ 𝜇)) & ⊢ (𝑐 = 𝑍 → (𝜇 ↔ 𝜆)) & ⊢ ((𝑎 ∈ No ∧ 𝑏 ∈ No ∧ 𝑐 ∈ No ) → (((∀𝑑 ∈ (( L ‘𝑎) ∪ ( R ‘𝑎))∀𝑒 ∈ (( L ‘𝑏) ∪ ( R ‘𝑏))∀𝑓 ∈ (( L ‘𝑐) ∪ ( R ‘𝑐))𝜃 ∧ ∀𝑑 ∈ (( L ‘𝑎) ∪ ( R ‘𝑎))∀𝑒 ∈ (( L ‘𝑏) ∪ ( R ‘𝑏))𝜒 ∧ ∀𝑑 ∈ (( L ‘𝑎) ∪ ( R ‘𝑎))∀𝑓 ∈ (( L ‘𝑐) ∪ ( R ‘𝑐))𝜁) ∧ (∀𝑑 ∈ (( L ‘𝑎) ∪ ( R ‘𝑎))𝜓 ∧ ∀𝑒 ∈ (( L ‘𝑏) ∪ ( R ‘𝑏))∀𝑓 ∈ (( L ‘𝑐) ∪ ( R ‘𝑐))𝜏 ∧ ∀𝑒 ∈ (( L ‘𝑏) ∪ ( R ‘𝑏))𝜎) ∧ ∀𝑓 ∈ (( L ‘𝑐) ∪ ( R ‘𝑐))𝜂) → 𝜑)) ⇒ ⊢ ((𝑋 ∈ No ∧ 𝑌 ∈ No ∧ 𝑍 ∈ No ) → 𝜆) | ||
Syntax | cadds 34125 | Declare the syntax for surreal addition. |
class +s | ||
Syntax | cnegs 34126 | Declare the syntax for surreal negation. |
class -us | ||
Syntax | csubs 34127 | Declare the syntax for surreal subtraction. |
class -s | ||
Definition | df-adds 34128* | Define surreal addition. This is the first of the field operations on the surreals. Definition from [Conway] p. 5. Definition from [Gonshor] p. 13. (Contributed by Scott Fenton, 20-Aug-2024.) |
⊢ +s = norec2 ((𝑥 ∈ V, 𝑎 ∈ V ↦ (({𝑦 ∣ ∃𝑙 ∈ ( L ‘(1st ‘𝑥))𝑦 = (𝑙𝑎(2nd ‘𝑥))} ∪ {𝑧 ∣ ∃𝑙 ∈ ( L ‘(2nd ‘𝑥))𝑧 = ((1st ‘𝑥)𝑎𝑙)}) |s ({𝑦 ∣ ∃𝑟 ∈ ( R ‘(1st ‘𝑥))𝑦 = (𝑟𝑎(2nd ‘𝑥))} ∪ {𝑧 ∣ ∃𝑟 ∈ ( R ‘(2nd ‘𝑥))𝑧 = ((1st ‘𝑥)𝑎𝑟)})))) | ||
Definition | df-negs 34129* | Define surreal negation. Definition from [Conway] p. 5. (Contributed by Scott Fenton, 20-Aug-2024.) |
⊢ -us = norec ((𝑥 ∈ V, 𝑛 ∈ V ↦ ((𝑛 “ ( R ‘𝑥)) |s (𝑛 “ ( L ‘𝑥))))) | ||
Definition | df-subs 34130* | Define surreal subtraction. (Contributed by Scott Fenton, 20-Aug-2024.) |
⊢ -s = (𝑥 ∈ No , 𝑦 ∈ No ↦ (𝑥 +s ( -us ‘𝑦))) | ||
Theorem | negsfn 34131 | Surreal negation is a function over surreals. (Contributed by Scott Fenton, 20-Aug-2024.) |
⊢ -us Fn No | ||
Theorem | negsval 34132 | The value of the surreal negation function. (Contributed by Scott Fenton, 20-Aug-2024.) |
⊢ (𝐴 ∈ No → ( -us ‘𝐴) = (( -us “ ( R ‘𝐴)) |s ( -us “ ( L ‘𝐴)))) | ||
Theorem | negs0s 34133 | Negative surreal zero is surreal zero. (Contributed by Scott Fenton, 20-Aug-2024.) |
⊢ ( -us ‘ 0s ) = 0s | ||
Theorem | addsfn 34134 | Surreal addition is a function over pairs of surreals. (Contributed by Scott Fenton, 20-Aug-2024.) |
⊢ +s Fn ( No × No ) | ||
Theorem | addsval 34135* | The value of surreal addition. Definition from [Conway] p. 5. (Contributed by Scott Fenton, 20-Aug-2024.) |
⊢ ((𝐴 ∈ No ∧ 𝐵 ∈ No ) → (𝐴 +s 𝐵) = (({𝑦 ∣ ∃𝑙 ∈ ( L ‘𝐴)𝑦 = (𝑙 +s 𝐵)} ∪ {𝑧 ∣ ∃𝑙 ∈ ( L ‘𝐵)𝑧 = (𝐴 +s 𝑙)}) |s ({𝑦 ∣ ∃𝑟 ∈ ( R ‘𝐴)𝑦 = (𝑟 +s 𝐵)} ∪ {𝑧 ∣ ∃𝑟 ∈ ( R ‘𝐵)𝑧 = (𝐴 +s 𝑟)}))) | ||
Theorem | addsid1 34136 | Surreal addition to zero is identity. Part of Theorem 3 of [Conway] p. 17. (Contributed by Scott Fenton, 20-Aug-2024.) |
⊢ (𝐴 ∈ No → (𝐴 +s 0s ) = 𝐴) | ||
Theorem | addsid1d 34137 | Surreal addition to zero is identity. Part of Theorem 3 of [Conway] p. 17. (Contributed by Scott Fenton, 20-Aug-2024.) |
⊢ (𝜑 → 𝐴 ∈ No ) ⇒ ⊢ (𝜑 → (𝐴 +s 0s ) = 𝐴) | ||
Theorem | addscom 34138 | Surreal addition commutes. Part of Theorem 3 of [Conway] p. 17. (Contributed by Scott Fenton, 20-Aug-2024.) |
⊢ ((𝐴 ∈ No ∧ 𝐵 ∈ No ) → (𝐴 +s 𝐵) = (𝐵 +s 𝐴)) | ||
Theorem | addscomd 34139 | Surreal addition commutes. Part of Theorem 3 of [Conway] p. 17. (Contributed by Scott Fenton, 20-Aug-2024.) |
⊢ (𝜑 → 𝐴 ∈ No ) & ⊢ (𝜑 → 𝐵 ∈ No ) ⇒ ⊢ (𝜑 → (𝐴 +s 𝐵) = (𝐵 +s 𝐴)) | ||
Theorem | addscllem1 34140 | Lemma for addscl (future) Alternate expression for surreal addition. (Contributed by Scott Fenton, 23-Aug-2024.) |
⊢ ((𝐴 ∈ No ∧ 𝐵 ∈ No ) → (𝐴 +s 𝐵) = ((( +s “ (( L ‘𝐴) × {𝐵})) ∪ ( +s “ ({𝐴} × ( L ‘𝐵)))) |s (( +s “ (( R ‘𝐴) × {𝐵})) ∪ ( +s “ ({𝐴} × ( R ‘𝐵)))))) | ||
Syntax | ctxp 34141 | Declare the syntax for tail Cartesian product. |
class (𝐴 ⊗ 𝐵) | ||
Syntax | cpprod 34142 | Declare the syntax for the parallel product. |
class pprod(𝑅, 𝑆) | ||
Syntax | csset 34143 | Declare the subset relationship class. |
class SSet | ||
Syntax | ctrans 34144 | Declare the transitive set class. |
class Trans | ||
Syntax | cbigcup 34145 | Declare the set union relationship. |
class Bigcup | ||
Syntax | cfix 34146 | Declare the syntax for the fixpoints of a class. |
class Fix 𝐴 | ||
Syntax | climits 34147 | Declare the class of limit ordinals. |
class Limits | ||
Syntax | cfuns 34148 | Declare the syntax for the class of all function. |
class Funs | ||
Syntax | csingle 34149 | Declare the syntax for the singleton function. |
class Singleton | ||
Syntax | csingles 34150 | Declare the syntax for the class of all singletons. |
class Singletons | ||
Syntax | cimage 34151 | Declare the syntax for the image functor. |
class Image𝐴 | ||
Syntax | ccart 34152 | Declare the syntax for the cartesian function. |
class Cart | ||
Syntax | cimg 34153 | Declare the syntax for the image function. |
class Img | ||
Syntax | cdomain 34154 | Declare the syntax for the domain function. |
class Domain | ||
Syntax | crange 34155 | Declare the syntax for the range function. |
class Range | ||
Syntax | capply 34156 | Declare the syntax for the application function. |
class Apply | ||
Syntax | ccup 34157 | Declare the syntax for the cup function. |
class Cup | ||
Syntax | ccap 34158 | Declare the syntax for the cap function. |
class Cap | ||
Syntax | csuccf 34159 | Declare the syntax for the successor function. |
class Succ | ||
Syntax | cfunpart 34160 | Declare the syntax for the functional part functor. |
class Funpart𝐹 | ||
Syntax | cfullfn 34161 | Declare the syntax for the full function functor. |
class FullFun𝐹 | ||
Syntax | crestrict 34162 | Declare the syntax for the restriction function. |
class Restrict | ||
Syntax | cub 34163 | Declare the syntax for the upper bound relationship functor. |
class UB𝑅 | ||
Syntax | clb 34164 | Declare the syntax for the lower bound relationship functor. |
class LB𝑅 | ||
Definition | df-txp 34165 | Define the tail cross of two classes. Membership in this class is defined by txpss3v 34189 and brtxp 34191. (Contributed by Scott Fenton, 31-Mar-2012.) |
⊢ (𝐴 ⊗ 𝐵) = ((◡(1st ↾ (V × V)) ∘ 𝐴) ∩ (◡(2nd ↾ (V × V)) ∘ 𝐵)) | ||
Definition | df-pprod 34166 | Define the parallel product of two classes. Membership in this class is defined by pprodss4v 34195 and brpprod 34196. (Contributed by Scott Fenton, 11-Apr-2014.) |
⊢ pprod(𝐴, 𝐵) = ((𝐴 ∘ (1st ↾ (V × V))) ⊗ (𝐵 ∘ (2nd ↾ (V × V)))) | ||
Definition | df-sset 34167 | Define the subset class. For the value, see brsset 34200. (Contributed by Scott Fenton, 31-Mar-2012.) |
⊢ SSet = ((V × V) ∖ ran ( E ⊗ (V ∖ E ))) | ||
Definition | df-trans 34168 | Define the class of all transitive sets. (Contributed by Scott Fenton, 31-Mar-2012.) |
⊢ Trans = (V ∖ ran (( E ∘ E ) ∖ E )) | ||
Definition | df-bigcup 34169 | Define the Bigcup function, which, per fvbigcup 34213, 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 34170 | Define the class of all fixpoints of a relationship. (Contributed by Scott Fenton, 11-Apr-2012.) |
⊢ Fix 𝐴 = dom (𝐴 ∩ I ) | ||
Definition | df-limits 34171 | Define the class of all limit ordinals. (Contributed by Scott Fenton, 11-Apr-2012.) |
⊢ Limits = ((On ∩ Fix Bigcup ) ∖ {∅}) | ||
Definition | df-funs 34172 | Define the class of all functions. See elfuns 34226 for membership. (Contributed by Scott Fenton, 18-Feb-2013.) |
⊢ Funs = (𝒫 (V × V) ∖ Fix ( E ∘ ((1st ⊗ ((V ∖ I ) ∘ 2nd )) ∘ ◡ E ))) | ||
Definition | df-singleton 34173 | Define the singleton function. See brsingle 34228 for its value. (Contributed by Scott Fenton, 4-Apr-2014.) |
⊢ Singleton = ((V × V) ∖ ran ((V ⊗ E ) △ ( I ⊗ V))) | ||
Definition | df-singles 34174 | Define the class of all singletons. See elsingles 34229 for membership. (Contributed by Scott Fenton, 19-Feb-2013.) |
⊢ Singletons = ran Singleton | ||
Definition | df-image 34175 | Define the image functor. This function takes a set 𝐴 to a function 𝑥 ↦ (𝐴 “ 𝑥), providing that the latter exists. See imageval 34241 for the derivation. (Contributed by Scott Fenton, 27-Mar-2014.) |
⊢ Image𝐴 = ((V × V) ∖ ran ((V ⊗ E ) △ (( E ∘ ◡𝐴) ⊗ V))) | ||
Definition | df-cart 34176 | Define the cartesian product function. See brcart 34243 for its value. (Contributed by Scott Fenton, 11-Apr-2014.) |
⊢ Cart = (((V × V) × V) ∖ ran ((V ⊗ E ) △ (pprod( E , E ) ⊗ V))) | ||
Definition | df-img 34177 | Define the image function. See brimg 34248 for its value. (Contributed by Scott Fenton, 12-Apr-2014.) |
⊢ Img = (Image((2nd ∘ 1st ) ↾ (1st ↾ (V × V))) ∘ Cart) | ||
Definition | df-domain 34178 | Define the domain function. See brdomain 34244 for its value. (Contributed by Scott Fenton, 11-Apr-2014.) |
⊢ Domain = Image(1st ↾ (V × V)) | ||
Definition | df-range 34179 | Define the range function. See brrange 34245 for its value. (Contributed by Scott Fenton, 11-Apr-2014.) |
⊢ Range = Image(2nd ↾ (V × V)) | ||
Definition | df-cup 34180 | Define the little cup function. See brcup 34250 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 34181 | Define the little cap function. See brcap 34251 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 34182 | Define the restriction function. See brrestrict 34260 for its value. (Contributed by Scott Fenton, 17-Apr-2014.) |
⊢ Restrict = (Cap ∘ (1st ⊗ (Cart ∘ (2nd ⊗ (Range ∘ 1st ))))) | ||
Definition | df-succf 34183 | Define the successor function. See brsuccf 34252 for its value. (Contributed by Scott Fenton, 14-Apr-2014.) |
⊢ Succ = (Cup ∘ ( I ⊗ Singleton)) | ||
Definition | df-apply 34184 | Define the application function. See brapply 34249 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 34185 | Define the functional part of a class 𝐹. This is the maximal part of 𝐹 that is a function. See funpartfun 34254 and funpartfv 34256 for the meaning of this statement. (Contributed by Scott Fenton, 16-Apr-2014.) |
⊢ Funpart𝐹 = (𝐹 ↾ dom ((Image𝐹 ∘ Singleton) ∩ (V × Singletons ))) | ||
Definition | df-fullfun 34186 | 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 34187 | Define the upper bound relationship functor. See brub 34265 for value. (Contributed by Scott Fenton, 3-May-2018.) |
⊢ UB𝑅 = ((V × V) ∖ ((V ∖ 𝑅) ∘ ◡ E )) | ||
Definition | df-lb 34188 | Define the lower bound relationship functor. See brlb 34266 for value. (Contributed by Scott Fenton, 3-May-2018.) |
⊢ LB𝑅 = UB◡𝑅 | ||
Theorem | txpss3v 34189 | 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 34190 | A tail Cartesian product is a relationship. (Contributed by Scott Fenton, 31-Mar-2012.) |
⊢ Rel (𝐴 ⊗ 𝐵) | ||
Theorem | brtxp 34191 | Characterize a ternary relation over a tail Cartesian product. Together with txpss3v 34189, 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 34192* | 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 34193 | 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 34194 | A converse law for parallel product. (Contributed by Scott Fenton, 3-May-2014.) |
⊢ pprod(𝑅, 𝑆) = ◡pprod(◡𝑅, ◡𝑆) | ||
Theorem | pprodss4v 34195 | 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 34196 | Characterize a quaternary relation over a tail Cartesian product. Together with pprodss4v 34195, 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 34197* | 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 34198* | 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 34199 | The subset class is a binary relation. (Contributed by Scott Fenton, 31-Mar-2012.) |
⊢ Rel SSet | ||
Theorem | brsset 34200 | For sets, the SSet binary relation is equivalent to the subset relationship. (Contributed by Scott Fenton, 31-Mar-2012.) |
⊢ 𝐵 ∈ V ⇒ ⊢ (𝐴 SSet 𝐵 ↔ 𝐴 ⊆ 𝐵) |
< Previous Next > |
Copyright terms: Public domain | < Previous Next > |