| Metamath
Proof Explorer Theorem List (p. 184 of 498) | < 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-30880) |
(30881-32403) |
(32404-49791) |
| Type | Label | Description |
|---|---|---|
| Statement | ||
| Theorem | joindmss 18301 | Subset property of domain of join. (Contributed by NM, 12-Sep-2018.) |
| ⊢ 𝐵 = (Base‘𝐾) & ⊢ ∨ = (join‘𝐾) & ⊢ (𝜑 → 𝐾 ∈ 𝑉) ⇒ ⊢ (𝜑 → dom ∨ ⊆ (𝐵 × 𝐵)) | ||
| Theorem | joinval2lem 18302* | Lemma for joinval2 18303 and joineu 18304. (Contributed by NM, 12-Sep-2018.) TODO: combine this through joineu 18304 into joinlem 18305? |
| ⊢ 𝐵 = (Base‘𝐾) & ⊢ ≤ = (le‘𝐾) & ⊢ ∨ = (join‘𝐾) & ⊢ (𝜑 → 𝐾 ∈ 𝑉) & ⊢ (𝜑 → 𝑋 ∈ 𝐵) & ⊢ (𝜑 → 𝑌 ∈ 𝐵) ⇒ ⊢ ((𝑋 ∈ 𝐵 ∧ 𝑌 ∈ 𝐵) → ((∀𝑦 ∈ {𝑋, 𝑌}𝑦 ≤ 𝑥 ∧ ∀𝑧 ∈ 𝐵 (∀𝑦 ∈ {𝑋, 𝑌}𝑦 ≤ 𝑧 → 𝑥 ≤ 𝑧)) ↔ ((𝑋 ≤ 𝑥 ∧ 𝑌 ≤ 𝑥) ∧ ∀𝑧 ∈ 𝐵 ((𝑋 ≤ 𝑧 ∧ 𝑌 ≤ 𝑧) → 𝑥 ≤ 𝑧)))) | ||
| Theorem | joinval2 18303* | Value of join for a poset with LUB expanded. (Contributed by NM, 16-Sep-2011.) (Revised by NM, 11-Sep-2018.) |
| ⊢ 𝐵 = (Base‘𝐾) & ⊢ ≤ = (le‘𝐾) & ⊢ ∨ = (join‘𝐾) & ⊢ (𝜑 → 𝐾 ∈ 𝑉) & ⊢ (𝜑 → 𝑋 ∈ 𝐵) & ⊢ (𝜑 → 𝑌 ∈ 𝐵) ⇒ ⊢ (𝜑 → (𝑋 ∨ 𝑌) = (℩𝑥 ∈ 𝐵 ((𝑋 ≤ 𝑥 ∧ 𝑌 ≤ 𝑥) ∧ ∀𝑧 ∈ 𝐵 ((𝑋 ≤ 𝑧 ∧ 𝑌 ≤ 𝑧) → 𝑥 ≤ 𝑧)))) | ||
| Theorem | joineu 18304* | Uniqueness of join of elements in the domain. (Contributed by NM, 12-Sep-2018.) |
| ⊢ 𝐵 = (Base‘𝐾) & ⊢ ≤ = (le‘𝐾) & ⊢ ∨ = (join‘𝐾) & ⊢ (𝜑 → 𝐾 ∈ 𝑉) & ⊢ (𝜑 → 𝑋 ∈ 𝐵) & ⊢ (𝜑 → 𝑌 ∈ 𝐵) & ⊢ (𝜑 → 〈𝑋, 𝑌〉 ∈ dom ∨ ) ⇒ ⊢ (𝜑 → ∃!𝑥 ∈ 𝐵 ((𝑋 ≤ 𝑥 ∧ 𝑌 ≤ 𝑥) ∧ ∀𝑧 ∈ 𝐵 ((𝑋 ≤ 𝑧 ∧ 𝑌 ≤ 𝑧) → 𝑥 ≤ 𝑧))) | ||
| Theorem | joinlem 18305* | Lemma for join properties. (Contributed by NM, 16-Sep-2011.) (Revised by NM, 12-Sep-2018.) |
| ⊢ 𝐵 = (Base‘𝐾) & ⊢ ≤ = (le‘𝐾) & ⊢ ∨ = (join‘𝐾) & ⊢ (𝜑 → 𝐾 ∈ 𝑉) & ⊢ (𝜑 → 𝑋 ∈ 𝐵) & ⊢ (𝜑 → 𝑌 ∈ 𝐵) & ⊢ (𝜑 → 〈𝑋, 𝑌〉 ∈ dom ∨ ) ⇒ ⊢ (𝜑 → ((𝑋 ≤ (𝑋 ∨ 𝑌) ∧ 𝑌 ≤ (𝑋 ∨ 𝑌)) ∧ ∀𝑧 ∈ 𝐵 ((𝑋 ≤ 𝑧 ∧ 𝑌 ≤ 𝑧) → (𝑋 ∨ 𝑌) ≤ 𝑧))) | ||
| Theorem | lejoin1 18306 | A join's first argument is less than or equal to the join. (Contributed by NM, 16-Sep-2011.) |
| ⊢ 𝐵 = (Base‘𝐾) & ⊢ ≤ = (le‘𝐾) & ⊢ ∨ = (join‘𝐾) & ⊢ (𝜑 → 𝐾 ∈ 𝑉) & ⊢ (𝜑 → 𝑋 ∈ 𝐵) & ⊢ (𝜑 → 𝑌 ∈ 𝐵) & ⊢ (𝜑 → 〈𝑋, 𝑌〉 ∈ dom ∨ ) ⇒ ⊢ (𝜑 → 𝑋 ≤ (𝑋 ∨ 𝑌)) | ||
| Theorem | lejoin2 18307 | A join's second argument is less than or equal to the join. (Contributed by NM, 16-Sep-2011.) |
| ⊢ 𝐵 = (Base‘𝐾) & ⊢ ≤ = (le‘𝐾) & ⊢ ∨ = (join‘𝐾) & ⊢ (𝜑 → 𝐾 ∈ 𝑉) & ⊢ (𝜑 → 𝑋 ∈ 𝐵) & ⊢ (𝜑 → 𝑌 ∈ 𝐵) & ⊢ (𝜑 → 〈𝑋, 𝑌〉 ∈ dom ∨ ) ⇒ ⊢ (𝜑 → 𝑌 ≤ (𝑋 ∨ 𝑌)) | ||
| Theorem | joinle 18308 | A join is less than or equal to a third value iff each argument is less than or equal to the third value. (Contributed by NM, 16-Sep-2011.) |
| ⊢ 𝐵 = (Base‘𝐾) & ⊢ ≤ = (le‘𝐾) & ⊢ ∨ = (join‘𝐾) & ⊢ (𝜑 → 𝐾 ∈ Poset) & ⊢ (𝜑 → 𝑋 ∈ 𝐵) & ⊢ (𝜑 → 𝑌 ∈ 𝐵) & ⊢ (𝜑 → 𝑍 ∈ 𝐵) & ⊢ (𝜑 → 〈𝑋, 𝑌〉 ∈ dom ∨ ) ⇒ ⊢ (𝜑 → ((𝑋 ≤ 𝑍 ∧ 𝑌 ≤ 𝑍) ↔ (𝑋 ∨ 𝑌) ≤ 𝑍)) | ||
| Theorem | meetfval 18309* | Value of meet function for a poset. (Contributed by NM, 12-Sep-2011.) (Revised by NM, 9-Sep-2018.) TODO: prove meetfval2 18310 first to reduce net proof size (existence part)? |
| ⊢ 𝐺 = (glb‘𝐾) & ⊢ ∧ = (meet‘𝐾) ⇒ ⊢ (𝐾 ∈ 𝑉 → ∧ = {〈〈𝑥, 𝑦〉, 𝑧〉 ∣ {𝑥, 𝑦}𝐺𝑧}) | ||
| Theorem | meetfval2 18310* | Value of meet function for a poset. (Contributed by NM, 12-Sep-2011.) (Revised by NM, 9-Sep-2018.) |
| ⊢ 𝐺 = (glb‘𝐾) & ⊢ ∧ = (meet‘𝐾) ⇒ ⊢ (𝐾 ∈ 𝑉 → ∧ = {〈〈𝑥, 𝑦〉, 𝑧〉 ∣ ({𝑥, 𝑦} ∈ dom 𝐺 ∧ 𝑧 = (𝐺‘{𝑥, 𝑦}))}) | ||
| Theorem | meetdm 18311* | Domain of meet function for a poset-type structure. (Contributed by NM, 16-Sep-2018.) |
| ⊢ 𝐺 = (glb‘𝐾) & ⊢ ∧ = (meet‘𝐾) ⇒ ⊢ (𝐾 ∈ 𝑉 → dom ∧ = {〈𝑥, 𝑦〉 ∣ {𝑥, 𝑦} ∈ dom 𝐺}) | ||
| Theorem | meetdef 18312 | Two ways to say that a meet is defined. (Contributed by NM, 9-Sep-2018.) |
| ⊢ 𝐺 = (glb‘𝐾) & ⊢ ∧ = (meet‘𝐾) & ⊢ (𝜑 → 𝐾 ∈ 𝑉) & ⊢ (𝜑 → 𝑋 ∈ 𝑊) & ⊢ (𝜑 → 𝑌 ∈ 𝑍) ⇒ ⊢ (𝜑 → (〈𝑋, 𝑌〉 ∈ dom ∧ ↔ {𝑋, 𝑌} ∈ dom 𝐺)) | ||
| Theorem | meetval 18313 | Meet value. Since both sides evaluate to ∅ when they don't exist, for convenience we drop the {𝑋, 𝑌} ∈ dom 𝐺 requirement. (Contributed by NM, 9-Sep-2018.) |
| ⊢ 𝐺 = (glb‘𝐾) & ⊢ ∧ = (meet‘𝐾) & ⊢ (𝜑 → 𝐾 ∈ 𝑉) & ⊢ (𝜑 → 𝑋 ∈ 𝑊) & ⊢ (𝜑 → 𝑌 ∈ 𝑍) ⇒ ⊢ (𝜑 → (𝑋 ∧ 𝑌) = (𝐺‘{𝑋, 𝑌})) | ||
| Theorem | meetcl 18314 | Closure of meet of elements in the domain. (Contributed by NM, 12-Sep-2018.) |
| ⊢ 𝐵 = (Base‘𝐾) & ⊢ ∧ = (meet‘𝐾) & ⊢ (𝜑 → 𝐾 ∈ 𝑉) & ⊢ (𝜑 → 𝑋 ∈ 𝐵) & ⊢ (𝜑 → 𝑌 ∈ 𝐵) & ⊢ (𝜑 → 〈𝑋, 𝑌〉 ∈ dom ∧ ) ⇒ ⊢ (𝜑 → (𝑋 ∧ 𝑌) ∈ 𝐵) | ||
| Theorem | meetdmss 18315 | Subset property of domain of meet. (Contributed by NM, 12-Sep-2018.) |
| ⊢ 𝐵 = (Base‘𝐾) & ⊢ ∧ = (meet‘𝐾) & ⊢ (𝜑 → 𝐾 ∈ 𝑉) ⇒ ⊢ (𝜑 → dom ∧ ⊆ (𝐵 × 𝐵)) | ||
| Theorem | meetval2lem 18316* | Lemma for meetval2 18317 and meeteu 18318. (Contributed by NM, 12-Sep-2018.) TODO: combine this through meeteu 18318 into meetlem 18319? |
| ⊢ 𝐵 = (Base‘𝐾) & ⊢ ≤ = (le‘𝐾) & ⊢ ∧ = (meet‘𝐾) & ⊢ (𝜑 → 𝐾 ∈ 𝑉) & ⊢ (𝜑 → 𝑋 ∈ 𝐵) & ⊢ (𝜑 → 𝑌 ∈ 𝐵) ⇒ ⊢ ((𝑋 ∈ 𝐵 ∧ 𝑌 ∈ 𝐵) → ((∀𝑦 ∈ {𝑋, 𝑌}𝑥 ≤ 𝑦 ∧ ∀𝑧 ∈ 𝐵 (∀𝑦 ∈ {𝑋, 𝑌}𝑧 ≤ 𝑦 → 𝑧 ≤ 𝑥)) ↔ ((𝑥 ≤ 𝑋 ∧ 𝑥 ≤ 𝑌) ∧ ∀𝑧 ∈ 𝐵 ((𝑧 ≤ 𝑋 ∧ 𝑧 ≤ 𝑌) → 𝑧 ≤ 𝑥)))) | ||
| Theorem | meetval2 18317* | Value of meet for a poset with LUB expanded. (Contributed by NM, 16-Sep-2011.) (Revised by NM, 11-Sep-2018.) |
| ⊢ 𝐵 = (Base‘𝐾) & ⊢ ≤ = (le‘𝐾) & ⊢ ∧ = (meet‘𝐾) & ⊢ (𝜑 → 𝐾 ∈ 𝑉) & ⊢ (𝜑 → 𝑋 ∈ 𝐵) & ⊢ (𝜑 → 𝑌 ∈ 𝐵) ⇒ ⊢ (𝜑 → (𝑋 ∧ 𝑌) = (℩𝑥 ∈ 𝐵 ((𝑥 ≤ 𝑋 ∧ 𝑥 ≤ 𝑌) ∧ ∀𝑧 ∈ 𝐵 ((𝑧 ≤ 𝑋 ∧ 𝑧 ≤ 𝑌) → 𝑧 ≤ 𝑥)))) | ||
| Theorem | meeteu 18318* | Uniqueness of meet of elements in the domain. (Contributed by NM, 12-Sep-2018.) |
| ⊢ 𝐵 = (Base‘𝐾) & ⊢ ≤ = (le‘𝐾) & ⊢ ∧ = (meet‘𝐾) & ⊢ (𝜑 → 𝐾 ∈ 𝑉) & ⊢ (𝜑 → 𝑋 ∈ 𝐵) & ⊢ (𝜑 → 𝑌 ∈ 𝐵) & ⊢ (𝜑 → 〈𝑋, 𝑌〉 ∈ dom ∧ ) ⇒ ⊢ (𝜑 → ∃!𝑥 ∈ 𝐵 ((𝑥 ≤ 𝑋 ∧ 𝑥 ≤ 𝑌) ∧ ∀𝑧 ∈ 𝐵 ((𝑧 ≤ 𝑋 ∧ 𝑧 ≤ 𝑌) → 𝑧 ≤ 𝑥))) | ||
| Theorem | meetlem 18319* | Lemma for meet properties. (Contributed by NM, 16-Sep-2011.) (Revised by NM, 12-Sep-2018.) |
| ⊢ 𝐵 = (Base‘𝐾) & ⊢ ≤ = (le‘𝐾) & ⊢ ∧ = (meet‘𝐾) & ⊢ (𝜑 → 𝐾 ∈ 𝑉) & ⊢ (𝜑 → 𝑋 ∈ 𝐵) & ⊢ (𝜑 → 𝑌 ∈ 𝐵) & ⊢ (𝜑 → 〈𝑋, 𝑌〉 ∈ dom ∧ ) ⇒ ⊢ (𝜑 → (((𝑋 ∧ 𝑌) ≤ 𝑋 ∧ (𝑋 ∧ 𝑌) ≤ 𝑌) ∧ ∀𝑧 ∈ 𝐵 ((𝑧 ≤ 𝑋 ∧ 𝑧 ≤ 𝑌) → 𝑧 ≤ (𝑋 ∧ 𝑌)))) | ||
| Theorem | lemeet1 18320 | A meet's first argument is less than or equal to the meet. (Contributed by NM, 16-Sep-2011.) (Revised by NM, 12-Sep-2018.) |
| ⊢ 𝐵 = (Base‘𝐾) & ⊢ ≤ = (le‘𝐾) & ⊢ ∧ = (meet‘𝐾) & ⊢ (𝜑 → 𝐾 ∈ 𝑉) & ⊢ (𝜑 → 𝑋 ∈ 𝐵) & ⊢ (𝜑 → 𝑌 ∈ 𝐵) & ⊢ (𝜑 → 〈𝑋, 𝑌〉 ∈ dom ∧ ) ⇒ ⊢ (𝜑 → (𝑋 ∧ 𝑌) ≤ 𝑋) | ||
| Theorem | lemeet2 18321 | A meet's second argument is less than or equal to the meet. (Contributed by NM, 16-Sep-2011.) (Revised by NM, 12-Sep-2018.) |
| ⊢ 𝐵 = (Base‘𝐾) & ⊢ ≤ = (le‘𝐾) & ⊢ ∧ = (meet‘𝐾) & ⊢ (𝜑 → 𝐾 ∈ 𝑉) & ⊢ (𝜑 → 𝑋 ∈ 𝐵) & ⊢ (𝜑 → 𝑌 ∈ 𝐵) & ⊢ (𝜑 → 〈𝑋, 𝑌〉 ∈ dom ∧ ) ⇒ ⊢ (𝜑 → (𝑋 ∧ 𝑌) ≤ 𝑌) | ||
| Theorem | meetle 18322 | A meet is less than or equal to a third value iff each argument is less than or equal to the third value. (Contributed by NM, 16-Sep-2011.) (Revised by NM, 12-Sep-2018.) |
| ⊢ 𝐵 = (Base‘𝐾) & ⊢ ≤ = (le‘𝐾) & ⊢ ∧ = (meet‘𝐾) & ⊢ (𝜑 → 𝐾 ∈ Poset) & ⊢ (𝜑 → 𝑋 ∈ 𝐵) & ⊢ (𝜑 → 𝑌 ∈ 𝐵) & ⊢ (𝜑 → 𝑍 ∈ 𝐵) & ⊢ (𝜑 → 〈𝑋, 𝑌〉 ∈ dom ∧ ) ⇒ ⊢ (𝜑 → ((𝑍 ≤ 𝑋 ∧ 𝑍 ≤ 𝑌) ↔ 𝑍 ≤ (𝑋 ∧ 𝑌))) | ||
| Theorem | joincomALT 18323 | The join of a poset is commutative. (This may not be a theorem under other definitions of meet.) (Contributed by NM, 16-Sep-2011.) (New usage is discouraged.) (Proof modification is discouraged.) |
| ⊢ 𝐵 = (Base‘𝐾) & ⊢ ∨ = (join‘𝐾) ⇒ ⊢ ((𝐾 ∈ 𝑉 ∧ 𝑋 ∈ 𝐵 ∧ 𝑌 ∈ 𝐵) → (𝑋 ∨ 𝑌) = (𝑌 ∨ 𝑋)) | ||
| Theorem | joincom 18324 | The join of a poset is commutative. (The antecedent 〈𝑋, 𝑌〉 ∈ dom ∨ ∧ 〈𝑌, 𝑋〉 ∈ dom ∨ i.e., "the joins exist" could be omitted as an artifact of our particular join definition, but other definitions may require it.) (Contributed by NM, 16-Sep-2011.) (Revised by NM, 12-Sep-2018.) |
| ⊢ 𝐵 = (Base‘𝐾) & ⊢ ∨ = (join‘𝐾) ⇒ ⊢ (((𝐾 ∈ Poset ∧ 𝑋 ∈ 𝐵 ∧ 𝑌 ∈ 𝐵) ∧ (〈𝑋, 𝑌〉 ∈ dom ∨ ∧ 〈𝑌, 𝑋〉 ∈ dom ∨ )) → (𝑋 ∨ 𝑌) = (𝑌 ∨ 𝑋)) | ||
| Theorem | meetcomALT 18325 | The meet of a poset is commutative. (This may not be a theorem under other definitions of meet.) (Contributed by NM, 17-Sep-2011.) (New usage is discouraged.) (Proof modification is discouraged.) |
| ⊢ 𝐵 = (Base‘𝐾) & ⊢ ∧ = (meet‘𝐾) ⇒ ⊢ ((𝐾 ∈ 𝑉 ∧ 𝑋 ∈ 𝐵 ∧ 𝑌 ∈ 𝐵) → (𝑋 ∧ 𝑌) = (𝑌 ∧ 𝑋)) | ||
| Theorem | meetcom 18326 | The meet of a poset is commutative. (The antecedent 〈𝑋, 𝑌〉 ∈ dom ∧ ∧ 〈𝑌, 𝑋〉 ∈ dom ∧ i.e., "the meets exist" could be omitted as an artifact of our particular join definition, but other definitions may require it.) (Contributed by NM, 17-Sep-2011.) (Revised by NM, 12-Sep-2018.) |
| ⊢ 𝐵 = (Base‘𝐾) & ⊢ ∧ = (meet‘𝐾) ⇒ ⊢ (((𝐾 ∈ Poset ∧ 𝑋 ∈ 𝐵 ∧ 𝑌 ∈ 𝐵) ∧ (〈𝑋, 𝑌〉 ∈ dom ∧ ∧ 〈𝑌, 𝑋〉 ∈ dom ∧ )) → (𝑋 ∧ 𝑌) = (𝑌 ∧ 𝑋)) | ||
| Theorem | join0 18327 | Lemma for odumeet 18332. (Contributed by Stefan O'Rear, 29-Jan-2015.) |
| ⊢ (join‘∅) = ∅ | ||
| Theorem | meet0 18328 | Lemma for odujoin 18330. (Contributed by Stefan O'Rear, 29-Jan-2015.) TODO (df-riota 7310 update): This proof increased from 152 bytes to 547 bytes after the df-riota 7310 change. Any way to shorten it? join0 18327 also. |
| ⊢ (meet‘∅) = ∅ | ||
| Theorem | odulub 18329 | Least upper bounds in a dual order are greatest lower bounds in the original order. (Contributed by Stefan O'Rear, 29-Jan-2015.) |
| ⊢ 𝐷 = (ODual‘𝑂) & ⊢ 𝐿 = (glb‘𝑂) ⇒ ⊢ (𝑂 ∈ 𝑉 → 𝐿 = (lub‘𝐷)) | ||
| Theorem | odujoin 18330 | Joins in a dual order are meets in the original. (Contributed by Stefan O'Rear, 29-Jan-2015.) |
| ⊢ 𝐷 = (ODual‘𝑂) & ⊢ ∧ = (meet‘𝑂) ⇒ ⊢ ∧ = (join‘𝐷) | ||
| Theorem | oduglb 18331 | Greatest lower bounds in a dual order are least upper bounds in the original order. (Contributed by Stefan O'Rear, 29-Jan-2015.) |
| ⊢ 𝐷 = (ODual‘𝑂) & ⊢ 𝑈 = (lub‘𝑂) ⇒ ⊢ (𝑂 ∈ 𝑉 → 𝑈 = (glb‘𝐷)) | ||
| Theorem | odumeet 18332 | Meets in a dual order are joins in the original. (Contributed by Stefan O'Rear, 29-Jan-2015.) |
| ⊢ 𝐷 = (ODual‘𝑂) & ⊢ ∨ = (join‘𝑂) ⇒ ⊢ ∨ = (meet‘𝐷) | ||
| Theorem | poslubmo 18333* | Least upper bounds in a poset are unique if they exist. (Contributed by Stefan O'Rear, 31-Jan-2015.) (Revised by NM, 16-Jun-2017.) |
| ⊢ ≤ = (le‘𝐾) & ⊢ 𝐵 = (Base‘𝐾) ⇒ ⊢ ((𝐾 ∈ Poset ∧ 𝑆 ⊆ 𝐵) → ∃*𝑥 ∈ 𝐵 (∀𝑦 ∈ 𝑆 𝑦 ≤ 𝑥 ∧ ∀𝑧 ∈ 𝐵 (∀𝑦 ∈ 𝑆 𝑦 ≤ 𝑧 → 𝑥 ≤ 𝑧))) | ||
| Theorem | posglbmo 18334* | Greatest lower bounds in a poset are unique if they exist. (Contributed by NM, 20-Sep-2018.) |
| ⊢ ≤ = (le‘𝐾) & ⊢ 𝐵 = (Base‘𝐾) ⇒ ⊢ ((𝐾 ∈ Poset ∧ 𝑆 ⊆ 𝐵) → ∃*𝑥 ∈ 𝐵 (∀𝑦 ∈ 𝑆 𝑥 ≤ 𝑦 ∧ ∀𝑧 ∈ 𝐵 (∀𝑦 ∈ 𝑆 𝑧 ≤ 𝑦 → 𝑧 ≤ 𝑥))) | ||
| Theorem | poslubd 18335* | Properties which determine the least upper bound in a poset. (Contributed by Stefan O'Rear, 31-Jan-2015.) |
| ⊢ ≤ = (le‘𝐾) & ⊢ 𝐵 = (Base‘𝐾) & ⊢ 𝑈 = (lub‘𝐾) & ⊢ (𝜑 → 𝐾 ∈ Poset) & ⊢ (𝜑 → 𝑆 ⊆ 𝐵) & ⊢ (𝜑 → 𝑇 ∈ 𝐵) & ⊢ ((𝜑 ∧ 𝑥 ∈ 𝑆) → 𝑥 ≤ 𝑇) & ⊢ ((𝜑 ∧ 𝑦 ∈ 𝐵 ∧ ∀𝑥 ∈ 𝑆 𝑥 ≤ 𝑦) → 𝑇 ≤ 𝑦) ⇒ ⊢ (𝜑 → (𝑈‘𝑆) = 𝑇) | ||
| Theorem | poslubdg 18336* | Properties which determine the least upper bound in a poset. (Contributed by Stefan O'Rear, 31-Jan-2015.) |
| ⊢ ≤ = (le‘𝐾) & ⊢ (𝜑 → 𝐵 = (Base‘𝐾)) & ⊢ (𝜑 → 𝑈 = (lub‘𝐾)) & ⊢ (𝜑 → 𝐾 ∈ Poset) & ⊢ (𝜑 → 𝑆 ⊆ 𝐵) & ⊢ (𝜑 → 𝑇 ∈ 𝐵) & ⊢ ((𝜑 ∧ 𝑥 ∈ 𝑆) → 𝑥 ≤ 𝑇) & ⊢ ((𝜑 ∧ 𝑦 ∈ 𝐵 ∧ ∀𝑥 ∈ 𝑆 𝑥 ≤ 𝑦) → 𝑇 ≤ 𝑦) ⇒ ⊢ (𝜑 → (𝑈‘𝑆) = 𝑇) | ||
| Theorem | posglbdg 18337* | Properties which determine the greatest lower bound in a poset. (Contributed by Stefan O'Rear, 31-Jan-2015.) |
| ⊢ ≤ = (le‘𝐾) & ⊢ (𝜑 → 𝐵 = (Base‘𝐾)) & ⊢ (𝜑 → 𝐺 = (glb‘𝐾)) & ⊢ (𝜑 → 𝐾 ∈ Poset) & ⊢ (𝜑 → 𝑆 ⊆ 𝐵) & ⊢ (𝜑 → 𝑇 ∈ 𝐵) & ⊢ ((𝜑 ∧ 𝑥 ∈ 𝑆) → 𝑇 ≤ 𝑥) & ⊢ ((𝜑 ∧ 𝑦 ∈ 𝐵 ∧ ∀𝑥 ∈ 𝑆 𝑦 ≤ 𝑥) → 𝑦 ≤ 𝑇) ⇒ ⊢ (𝜑 → (𝐺‘𝑆) = 𝑇) | ||
| Syntax | ctos 18338 | Extend class notation with the class of all tosets. |
| class Toset | ||
| Definition | df-toset 18339* | Define the class of totally ordered sets (tosets). (Contributed by FL, 17-Nov-2014.) |
| ⊢ Toset = {𝑓 ∈ Poset ∣ [(Base‘𝑓) / 𝑏][(le‘𝑓) / 𝑟]∀𝑥 ∈ 𝑏 ∀𝑦 ∈ 𝑏 (𝑥𝑟𝑦 ∨ 𝑦𝑟𝑥)} | ||
| Theorem | istos 18340* | The predicate "is a toset". (Contributed by FL, 17-Nov-2014.) |
| ⊢ 𝐵 = (Base‘𝐾) & ⊢ ≤ = (le‘𝐾) ⇒ ⊢ (𝐾 ∈ Toset ↔ (𝐾 ∈ Poset ∧ ∀𝑥 ∈ 𝐵 ∀𝑦 ∈ 𝐵 (𝑥 ≤ 𝑦 ∨ 𝑦 ≤ 𝑥))) | ||
| Theorem | tosso 18341 | Write the totally ordered set structure predicate in terms of the proper class strict order predicate. (Contributed by Mario Carneiro, 8-Feb-2015.) |
| ⊢ 𝐵 = (Base‘𝐾) & ⊢ ≤ = (le‘𝐾) & ⊢ < = (lt‘𝐾) ⇒ ⊢ (𝐾 ∈ 𝑉 → (𝐾 ∈ Toset ↔ ( < Or 𝐵 ∧ ( I ↾ 𝐵) ⊆ ≤ ))) | ||
| Theorem | tospos 18342 | A Toset is a Poset. (Contributed by Thierry Arnoux, 20-Jan-2018.) |
| ⊢ (𝐹 ∈ Toset → 𝐹 ∈ Poset) | ||
| Theorem | tleile 18343 | In a Toset, any two elements are comparable. (Contributed by Thierry Arnoux, 11-Feb-2018.) |
| ⊢ 𝐵 = (Base‘𝐾) & ⊢ ≤ = (le‘𝐾) ⇒ ⊢ ((𝐾 ∈ Toset ∧ 𝑋 ∈ 𝐵 ∧ 𝑌 ∈ 𝐵) → (𝑋 ≤ 𝑌 ∨ 𝑌 ≤ 𝑋)) | ||
| Theorem | tltnle 18344 | In a Toset, "less than" is equivalent to the negation of the converse of "less than or equal to", see pltnle 18260. (Contributed by Thierry Arnoux, 11-Feb-2018.) |
| ⊢ 𝐵 = (Base‘𝐾) & ⊢ ≤ = (le‘𝐾) & ⊢ < = (lt‘𝐾) ⇒ ⊢ ((𝐾 ∈ Toset ∧ 𝑋 ∈ 𝐵 ∧ 𝑌 ∈ 𝐵) → (𝑋 < 𝑌 ↔ ¬ 𝑌 ≤ 𝑋)) | ||
| Syntax | cp0 18345 | Extend class notation with poset zero. |
| class 0. | ||
| Syntax | cp1 18346 | Extend class notation with poset unit. |
| class 1. | ||
| Definition | df-p0 18347 | Define poset zero. (Contributed by NM, 12-Oct-2011.) |
| ⊢ 0. = (𝑝 ∈ V ↦ ((glb‘𝑝)‘(Base‘𝑝))) | ||
| Definition | df-p1 18348 | Define poset unit. (Contributed by NM, 22-Oct-2011.) |
| ⊢ 1. = (𝑝 ∈ V ↦ ((lub‘𝑝)‘(Base‘𝑝))) | ||
| Theorem | p0val 18349 | Value of poset zero. (Contributed by NM, 12-Oct-2011.) |
| ⊢ 𝐵 = (Base‘𝐾) & ⊢ 𝐺 = (glb‘𝐾) & ⊢ 0 = (0.‘𝐾) ⇒ ⊢ (𝐾 ∈ 𝑉 → 0 = (𝐺‘𝐵)) | ||
| Theorem | p1val 18350 | Value of poset zero. (Contributed by NM, 22-Oct-2011.) |
| ⊢ 𝐵 = (Base‘𝐾) & ⊢ 𝑈 = (lub‘𝐾) & ⊢ 1 = (1.‘𝐾) ⇒ ⊢ (𝐾 ∈ 𝑉 → 1 = (𝑈‘𝐵)) | ||
| Theorem | p0le 18351 | Any element is less than or equal to a poset's upper bound (if defined). (Contributed by NM, 22-Oct-2011.) (Revised by NM, 13-Sep-2018.) |
| ⊢ 𝐵 = (Base‘𝐾) & ⊢ 𝐺 = (glb‘𝐾) & ⊢ ≤ = (le‘𝐾) & ⊢ 0 = (0.‘𝐾) & ⊢ (𝜑 → 𝐾 ∈ 𝑉) & ⊢ (𝜑 → 𝑋 ∈ 𝐵) & ⊢ (𝜑 → 𝐵 ∈ dom 𝐺) ⇒ ⊢ (𝜑 → 0 ≤ 𝑋) | ||
| Theorem | ple1 18352 | Any element is less than or equal to a poset's upper bound (if defined). (Contributed by NM, 22-Oct-2011.) (Revised by NM, 13-Sep-2018.) |
| ⊢ 𝐵 = (Base‘𝐾) & ⊢ 𝑈 = (lub‘𝐾) & ⊢ ≤ = (le‘𝐾) & ⊢ 1 = (1.‘𝐾) & ⊢ (𝜑 → 𝐾 ∈ 𝑉) & ⊢ (𝜑 → 𝑋 ∈ 𝐵) & ⊢ (𝜑 → 𝐵 ∈ dom 𝑈) ⇒ ⊢ (𝜑 → 𝑋 ≤ 1 ) | ||
| Theorem | resspos 18353 | The restriction of a Poset is a Poset. (Contributed by Thierry Arnoux, 20-Jan-2018.) |
| ⊢ ((𝐹 ∈ Poset ∧ 𝐴 ∈ 𝑉) → (𝐹 ↾s 𝐴) ∈ Poset) | ||
| Theorem | resstos 18354 | The restriction of a Toset is a Toset. (Contributed by Thierry Arnoux, 20-Jan-2018.) |
| ⊢ ((𝐹 ∈ Toset ∧ 𝐴 ∈ 𝑉) → (𝐹 ↾s 𝐴) ∈ Toset) | ||
| Syntax | clat 18355 | Extend class notation with the class of all lattices. |
| class Lat | ||
| Definition | df-lat 18356 | Define the class of all lattices. A lattice is a poset in which the join and meet of any two elements always exists. (Contributed by NM, 18-Oct-2012.) (Revised by NM, 12-Sep-2018.) |
| ⊢ Lat = {𝑝 ∈ Poset ∣ (dom (join‘𝑝) = ((Base‘𝑝) × (Base‘𝑝)) ∧ dom (meet‘𝑝) = ((Base‘𝑝) × (Base‘𝑝)))} | ||
| Theorem | islat 18357 | The predicate "is a lattice". (Contributed by NM, 18-Oct-2012.) (Revised by NM, 12-Sep-2018.) |
| ⊢ 𝐵 = (Base‘𝐾) & ⊢ ∨ = (join‘𝐾) & ⊢ ∧ = (meet‘𝐾) ⇒ ⊢ (𝐾 ∈ Lat ↔ (𝐾 ∈ Poset ∧ (dom ∨ = (𝐵 × 𝐵) ∧ dom ∧ = (𝐵 × 𝐵)))) | ||
| Theorem | odulatb 18358 | Being a lattice is self-dual. (Contributed by Stefan O'Rear, 29-Jan-2015.) |
| ⊢ 𝐷 = (ODual‘𝑂) ⇒ ⊢ (𝑂 ∈ 𝑉 → (𝑂 ∈ Lat ↔ 𝐷 ∈ Lat)) | ||
| Theorem | odulat 18359 | Being a lattice is self-dual. (Contributed by Stefan O'Rear, 29-Jan-2015.) |
| ⊢ 𝐷 = (ODual‘𝑂) ⇒ ⊢ (𝑂 ∈ Lat → 𝐷 ∈ Lat) | ||
| Theorem | latcl2 18360 | The join and meet of any two elements exist. (Contributed by NM, 14-Sep-2018.) |
| ⊢ 𝐵 = (Base‘𝐾) & ⊢ ∨ = (join‘𝐾) & ⊢ ∧ = (meet‘𝐾) & ⊢ (𝜑 → 𝐾 ∈ Lat) & ⊢ (𝜑 → 𝑋 ∈ 𝐵) & ⊢ (𝜑 → 𝑌 ∈ 𝐵) ⇒ ⊢ (𝜑 → (〈𝑋, 𝑌〉 ∈ dom ∨ ∧ 〈𝑋, 𝑌〉 ∈ dom ∧ )) | ||
| Theorem | latlem 18361 | Lemma for lattice properties. (Contributed by NM, 14-Sep-2011.) |
| ⊢ 𝐵 = (Base‘𝐾) & ⊢ ∨ = (join‘𝐾) & ⊢ ∧ = (meet‘𝐾) ⇒ ⊢ ((𝐾 ∈ Lat ∧ 𝑋 ∈ 𝐵 ∧ 𝑌 ∈ 𝐵) → ((𝑋 ∨ 𝑌) ∈ 𝐵 ∧ (𝑋 ∧ 𝑌) ∈ 𝐵)) | ||
| Theorem | latpos 18362 | A lattice is a poset. (Contributed by NM, 17-Sep-2011.) |
| ⊢ (𝐾 ∈ Lat → 𝐾 ∈ Poset) | ||
| Theorem | latjcl 18363 | Closure of join operation in a lattice. (chjcom 31468 analog.) (Contributed by NM, 14-Sep-2011.) |
| ⊢ 𝐵 = (Base‘𝐾) & ⊢ ∨ = (join‘𝐾) ⇒ ⊢ ((𝐾 ∈ Lat ∧ 𝑋 ∈ 𝐵 ∧ 𝑌 ∈ 𝐵) → (𝑋 ∨ 𝑌) ∈ 𝐵) | ||
| Theorem | latmcl 18364 | Closure of meet operation in a lattice. (incom 4162 analog.) (Contributed by NM, 14-Sep-2011.) |
| ⊢ 𝐵 = (Base‘𝐾) & ⊢ ∧ = (meet‘𝐾) ⇒ ⊢ ((𝐾 ∈ Lat ∧ 𝑋 ∈ 𝐵 ∧ 𝑌 ∈ 𝐵) → (𝑋 ∧ 𝑌) ∈ 𝐵) | ||
| Theorem | latref 18365 | A lattice ordering is reflexive. (ssid 3960 analog.) (Contributed by NM, 8-Oct-2011.) |
| ⊢ 𝐵 = (Base‘𝐾) & ⊢ ≤ = (le‘𝐾) ⇒ ⊢ ((𝐾 ∈ Lat ∧ 𝑋 ∈ 𝐵) → 𝑋 ≤ 𝑋) | ||
| Theorem | latasymb 18366 | A lattice ordering is asymmetric. (eqss 3953 analog.) (Contributed by NM, 22-Oct-2011.) |
| ⊢ 𝐵 = (Base‘𝐾) & ⊢ ≤ = (le‘𝐾) ⇒ ⊢ ((𝐾 ∈ Lat ∧ 𝑋 ∈ 𝐵 ∧ 𝑌 ∈ 𝐵) → ((𝑋 ≤ 𝑌 ∧ 𝑌 ≤ 𝑋) ↔ 𝑋 = 𝑌)) | ||
| Theorem | latasym 18367 | A lattice ordering is asymmetric. (eqss 3953 analog.) (Contributed by NM, 8-Oct-2011.) |
| ⊢ 𝐵 = (Base‘𝐾) & ⊢ ≤ = (le‘𝐾) ⇒ ⊢ ((𝐾 ∈ Lat ∧ 𝑋 ∈ 𝐵 ∧ 𝑌 ∈ 𝐵) → ((𝑋 ≤ 𝑌 ∧ 𝑌 ≤ 𝑋) → 𝑋 = 𝑌)) | ||
| Theorem | lattr 18368 | A lattice ordering is transitive. (sstr 3946 analog.) (Contributed by NM, 17-Nov-2011.) |
| ⊢ 𝐵 = (Base‘𝐾) & ⊢ ≤ = (le‘𝐾) ⇒ ⊢ ((𝐾 ∈ Lat ∧ (𝑋 ∈ 𝐵 ∧ 𝑌 ∈ 𝐵 ∧ 𝑍 ∈ 𝐵)) → ((𝑋 ≤ 𝑌 ∧ 𝑌 ≤ 𝑍) → 𝑋 ≤ 𝑍)) | ||
| Theorem | latasymd 18369 | Deduce equality from lattice ordering. (eqssd 3955 analog.) (Contributed by NM, 18-Nov-2011.) |
| ⊢ 𝐵 = (Base‘𝐾) & ⊢ ≤ = (le‘𝐾) & ⊢ (𝜑 → 𝐾 ∈ Lat) & ⊢ (𝜑 → 𝑋 ∈ 𝐵) & ⊢ (𝜑 → 𝑌 ∈ 𝐵) & ⊢ (𝜑 → 𝑋 ≤ 𝑌) & ⊢ (𝜑 → 𝑌 ≤ 𝑋) ⇒ ⊢ (𝜑 → 𝑋 = 𝑌) | ||
| Theorem | lattrd 18370 | A lattice ordering is transitive. Deduction version of lattr 18368. (Contributed by NM, 3-Sep-2012.) |
| ⊢ 𝐵 = (Base‘𝐾) & ⊢ ≤ = (le‘𝐾) & ⊢ (𝜑 → 𝐾 ∈ Lat) & ⊢ (𝜑 → 𝑋 ∈ 𝐵) & ⊢ (𝜑 → 𝑌 ∈ 𝐵) & ⊢ (𝜑 → 𝑍 ∈ 𝐵) & ⊢ (𝜑 → 𝑋 ≤ 𝑌) & ⊢ (𝜑 → 𝑌 ≤ 𝑍) ⇒ ⊢ (𝜑 → 𝑋 ≤ 𝑍) | ||
| Theorem | latjcom 18371 | The join of a lattice commutes. (chjcom 31468 analog.) (Contributed by NM, 16-Sep-2011.) |
| ⊢ 𝐵 = (Base‘𝐾) & ⊢ ∨ = (join‘𝐾) ⇒ ⊢ ((𝐾 ∈ Lat ∧ 𝑋 ∈ 𝐵 ∧ 𝑌 ∈ 𝐵) → (𝑋 ∨ 𝑌) = (𝑌 ∨ 𝑋)) | ||
| Theorem | latlej1 18372 | A join's first argument is less than or equal to the join. (chub1 31469 analog.) (Contributed by NM, 17-Sep-2011.) |
| ⊢ 𝐵 = (Base‘𝐾) & ⊢ ≤ = (le‘𝐾) & ⊢ ∨ = (join‘𝐾) ⇒ ⊢ ((𝐾 ∈ Lat ∧ 𝑋 ∈ 𝐵 ∧ 𝑌 ∈ 𝐵) → 𝑋 ≤ (𝑋 ∨ 𝑌)) | ||
| Theorem | latlej2 18373 | A join's second argument is less than or equal to the join. (chub2 31470 analog.) (Contributed by NM, 17-Sep-2011.) |
| ⊢ 𝐵 = (Base‘𝐾) & ⊢ ≤ = (le‘𝐾) & ⊢ ∨ = (join‘𝐾) ⇒ ⊢ ((𝐾 ∈ Lat ∧ 𝑋 ∈ 𝐵 ∧ 𝑌 ∈ 𝐵) → 𝑌 ≤ (𝑋 ∨ 𝑌)) | ||
| Theorem | latjle12 18374 | A join is less than or equal to a third value iff each argument is less than or equal to the third value. (chlub 31471 analog.) (Contributed by NM, 17-Sep-2011.) |
| ⊢ 𝐵 = (Base‘𝐾) & ⊢ ≤ = (le‘𝐾) & ⊢ ∨ = (join‘𝐾) ⇒ ⊢ ((𝐾 ∈ Lat ∧ (𝑋 ∈ 𝐵 ∧ 𝑌 ∈ 𝐵 ∧ 𝑍 ∈ 𝐵)) → ((𝑋 ≤ 𝑍 ∧ 𝑌 ≤ 𝑍) ↔ (𝑋 ∨ 𝑌) ≤ 𝑍)) | ||
| Theorem | latleeqj1 18375 | "Less than or equal to" in terms of join. (chlejb1 31474 analog.) (Contributed by NM, 21-Oct-2011.) |
| ⊢ 𝐵 = (Base‘𝐾) & ⊢ ≤ = (le‘𝐾) & ⊢ ∨ = (join‘𝐾) ⇒ ⊢ ((𝐾 ∈ Lat ∧ 𝑋 ∈ 𝐵 ∧ 𝑌 ∈ 𝐵) → (𝑋 ≤ 𝑌 ↔ (𝑋 ∨ 𝑌) = 𝑌)) | ||
| Theorem | latleeqj2 18376 | "Less than or equal to" in terms of join. (chlejb2 31475 analog.) (Contributed by NM, 14-Nov-2011.) |
| ⊢ 𝐵 = (Base‘𝐾) & ⊢ ≤ = (le‘𝐾) & ⊢ ∨ = (join‘𝐾) ⇒ ⊢ ((𝐾 ∈ Lat ∧ 𝑋 ∈ 𝐵 ∧ 𝑌 ∈ 𝐵) → (𝑋 ≤ 𝑌 ↔ (𝑌 ∨ 𝑋) = 𝑌)) | ||
| Theorem | latjlej1 18377 | Add join to both sides of a lattice ordering. (chlej1i 31435 analog.) (Contributed by NM, 8-Nov-2011.) |
| ⊢ 𝐵 = (Base‘𝐾) & ⊢ ≤ = (le‘𝐾) & ⊢ ∨ = (join‘𝐾) ⇒ ⊢ ((𝐾 ∈ Lat ∧ (𝑋 ∈ 𝐵 ∧ 𝑌 ∈ 𝐵 ∧ 𝑍 ∈ 𝐵)) → (𝑋 ≤ 𝑌 → (𝑋 ∨ 𝑍) ≤ (𝑌 ∨ 𝑍))) | ||
| Theorem | latjlej2 18378 | Add join to both sides of a lattice ordering. (chlej2i 31436 analog.) (Contributed by NM, 8-Nov-2011.) |
| ⊢ 𝐵 = (Base‘𝐾) & ⊢ ≤ = (le‘𝐾) & ⊢ ∨ = (join‘𝐾) ⇒ ⊢ ((𝐾 ∈ Lat ∧ (𝑋 ∈ 𝐵 ∧ 𝑌 ∈ 𝐵 ∧ 𝑍 ∈ 𝐵)) → (𝑋 ≤ 𝑌 → (𝑍 ∨ 𝑋) ≤ (𝑍 ∨ 𝑌))) | ||
| Theorem | latjlej12 18379 | Add join to both sides of a lattice ordering. (chlej12i 31437 analog.) (Contributed by NM, 8-Nov-2011.) |
| ⊢ 𝐵 = (Base‘𝐾) & ⊢ ≤ = (le‘𝐾) & ⊢ ∨ = (join‘𝐾) ⇒ ⊢ ((𝐾 ∈ Lat ∧ (𝑋 ∈ 𝐵 ∧ 𝑌 ∈ 𝐵) ∧ (𝑍 ∈ 𝐵 ∧ 𝑊 ∈ 𝐵)) → ((𝑋 ≤ 𝑌 ∧ 𝑍 ≤ 𝑊) → (𝑋 ∨ 𝑍) ≤ (𝑌 ∨ 𝑊))) | ||
| Theorem | latnlej 18380 | An idiom to express that a lattice element differs from two others. (Contributed by NM, 28-May-2012.) |
| ⊢ 𝐵 = (Base‘𝐾) & ⊢ ≤ = (le‘𝐾) & ⊢ ∨ = (join‘𝐾) ⇒ ⊢ ((𝐾 ∈ Lat ∧ (𝑋 ∈ 𝐵 ∧ 𝑌 ∈ 𝐵 ∧ 𝑍 ∈ 𝐵) ∧ ¬ 𝑋 ≤ (𝑌 ∨ 𝑍)) → (𝑋 ≠ 𝑌 ∧ 𝑋 ≠ 𝑍)) | ||
| Theorem | latnlej1l 18381 | An idiom to express that a lattice element differs from two others. (Contributed by NM, 19-Jul-2012.) |
| ⊢ 𝐵 = (Base‘𝐾) & ⊢ ≤ = (le‘𝐾) & ⊢ ∨ = (join‘𝐾) ⇒ ⊢ ((𝐾 ∈ Lat ∧ (𝑋 ∈ 𝐵 ∧ 𝑌 ∈ 𝐵 ∧ 𝑍 ∈ 𝐵) ∧ ¬ 𝑋 ≤ (𝑌 ∨ 𝑍)) → 𝑋 ≠ 𝑌) | ||
| Theorem | latnlej1r 18382 | An idiom to express that a lattice element differs from two others. (Contributed by NM, 19-Jul-2012.) |
| ⊢ 𝐵 = (Base‘𝐾) & ⊢ ≤ = (le‘𝐾) & ⊢ ∨ = (join‘𝐾) ⇒ ⊢ ((𝐾 ∈ Lat ∧ (𝑋 ∈ 𝐵 ∧ 𝑌 ∈ 𝐵 ∧ 𝑍 ∈ 𝐵) ∧ ¬ 𝑋 ≤ (𝑌 ∨ 𝑍)) → 𝑋 ≠ 𝑍) | ||
| Theorem | latnlej2 18383 | An idiom to express that a lattice element differs from two others. (Contributed by NM, 10-Jul-2012.) |
| ⊢ 𝐵 = (Base‘𝐾) & ⊢ ≤ = (le‘𝐾) & ⊢ ∨ = (join‘𝐾) ⇒ ⊢ ((𝐾 ∈ Lat ∧ (𝑋 ∈ 𝐵 ∧ 𝑌 ∈ 𝐵 ∧ 𝑍 ∈ 𝐵) ∧ ¬ 𝑋 ≤ (𝑌 ∨ 𝑍)) → (¬ 𝑋 ≤ 𝑌 ∧ ¬ 𝑋 ≤ 𝑍)) | ||
| Theorem | latnlej2l 18384 | An idiom to express that a lattice element differs from two others. (Contributed by NM, 19-Jul-2012.) |
| ⊢ 𝐵 = (Base‘𝐾) & ⊢ ≤ = (le‘𝐾) & ⊢ ∨ = (join‘𝐾) ⇒ ⊢ ((𝐾 ∈ Lat ∧ (𝑋 ∈ 𝐵 ∧ 𝑌 ∈ 𝐵 ∧ 𝑍 ∈ 𝐵) ∧ ¬ 𝑋 ≤ (𝑌 ∨ 𝑍)) → ¬ 𝑋 ≤ 𝑌) | ||
| Theorem | latnlej2r 18385 | An idiom to express that a lattice element differs from two others. (Contributed by NM, 19-Jul-2012.) |
| ⊢ 𝐵 = (Base‘𝐾) & ⊢ ≤ = (le‘𝐾) & ⊢ ∨ = (join‘𝐾) ⇒ ⊢ ((𝐾 ∈ Lat ∧ (𝑋 ∈ 𝐵 ∧ 𝑌 ∈ 𝐵 ∧ 𝑍 ∈ 𝐵) ∧ ¬ 𝑋 ≤ (𝑌 ∨ 𝑍)) → ¬ 𝑋 ≤ 𝑍) | ||
| Theorem | latjidm 18386 | Lattice join is idempotent. Analogue of unidm 4110. (Contributed by NM, 8-Oct-2011.) |
| ⊢ 𝐵 = (Base‘𝐾) & ⊢ ∨ = (join‘𝐾) ⇒ ⊢ ((𝐾 ∈ Lat ∧ 𝑋 ∈ 𝐵) → (𝑋 ∨ 𝑋) = 𝑋) | ||
| Theorem | latmcom 18387 | The join of a lattice commutes. (Contributed by NM, 6-Nov-2011.) |
| ⊢ 𝐵 = (Base‘𝐾) & ⊢ ∧ = (meet‘𝐾) ⇒ ⊢ ((𝐾 ∈ Lat ∧ 𝑋 ∈ 𝐵 ∧ 𝑌 ∈ 𝐵) → (𝑋 ∧ 𝑌) = (𝑌 ∧ 𝑋)) | ||
| Theorem | latmle1 18388 | A meet is less than or equal to its first argument. (Contributed by NM, 21-Oct-2011.) |
| ⊢ 𝐵 = (Base‘𝐾) & ⊢ ≤ = (le‘𝐾) & ⊢ ∧ = (meet‘𝐾) ⇒ ⊢ ((𝐾 ∈ Lat ∧ 𝑋 ∈ 𝐵 ∧ 𝑌 ∈ 𝐵) → (𝑋 ∧ 𝑌) ≤ 𝑋) | ||
| Theorem | latmle2 18389 | A meet is less than or equal to its second argument. (Contributed by NM, 21-Oct-2011.) |
| ⊢ 𝐵 = (Base‘𝐾) & ⊢ ≤ = (le‘𝐾) & ⊢ ∧ = (meet‘𝐾) ⇒ ⊢ ((𝐾 ∈ Lat ∧ 𝑋 ∈ 𝐵 ∧ 𝑌 ∈ 𝐵) → (𝑋 ∧ 𝑌) ≤ 𝑌) | ||
| Theorem | latlem12 18390 | An element is less than or equal to a meet iff the element is less than or equal to each argument of the meet. (Contributed by NM, 21-Oct-2011.) |
| ⊢ 𝐵 = (Base‘𝐾) & ⊢ ≤ = (le‘𝐾) & ⊢ ∧ = (meet‘𝐾) ⇒ ⊢ ((𝐾 ∈ Lat ∧ (𝑋 ∈ 𝐵 ∧ 𝑌 ∈ 𝐵 ∧ 𝑍 ∈ 𝐵)) → ((𝑋 ≤ 𝑌 ∧ 𝑋 ≤ 𝑍) ↔ 𝑋 ≤ (𝑌 ∧ 𝑍))) | ||
| Theorem | latleeqm1 18391 | "Less than or equal to" in terms of meet. (Contributed by NM, 7-Nov-2011.) |
| ⊢ 𝐵 = (Base‘𝐾) & ⊢ ≤ = (le‘𝐾) & ⊢ ∧ = (meet‘𝐾) ⇒ ⊢ ((𝐾 ∈ Lat ∧ 𝑋 ∈ 𝐵 ∧ 𝑌 ∈ 𝐵) → (𝑋 ≤ 𝑌 ↔ (𝑋 ∧ 𝑌) = 𝑋)) | ||
| Theorem | latleeqm2 18392 | "Less than or equal to" in terms of meet. (Contributed by NM, 7-Nov-2011.) |
| ⊢ 𝐵 = (Base‘𝐾) & ⊢ ≤ = (le‘𝐾) & ⊢ ∧ = (meet‘𝐾) ⇒ ⊢ ((𝐾 ∈ Lat ∧ 𝑋 ∈ 𝐵 ∧ 𝑌 ∈ 𝐵) → (𝑋 ≤ 𝑌 ↔ (𝑌 ∧ 𝑋) = 𝑋)) | ||
| Theorem | latmlem1 18393 | Add meet to both sides of a lattice ordering. (Contributed by NM, 10-Nov-2011.) |
| ⊢ 𝐵 = (Base‘𝐾) & ⊢ ≤ = (le‘𝐾) & ⊢ ∧ = (meet‘𝐾) ⇒ ⊢ ((𝐾 ∈ Lat ∧ (𝑋 ∈ 𝐵 ∧ 𝑌 ∈ 𝐵 ∧ 𝑍 ∈ 𝐵)) → (𝑋 ≤ 𝑌 → (𝑋 ∧ 𝑍) ≤ (𝑌 ∧ 𝑍))) | ||
| Theorem | latmlem2 18394 | Add meet to both sides of a lattice ordering. (sslin 4196 analog.) (Contributed by NM, 10-Nov-2011.) |
| ⊢ 𝐵 = (Base‘𝐾) & ⊢ ≤ = (le‘𝐾) & ⊢ ∧ = (meet‘𝐾) ⇒ ⊢ ((𝐾 ∈ Lat ∧ (𝑋 ∈ 𝐵 ∧ 𝑌 ∈ 𝐵 ∧ 𝑍 ∈ 𝐵)) → (𝑋 ≤ 𝑌 → (𝑍 ∧ 𝑋) ≤ (𝑍 ∧ 𝑌))) | ||
| Theorem | latmlem12 18395 | Add join to both sides of a lattice ordering. (ss2in 4198 analog.) (Contributed by NM, 10-Nov-2011.) |
| ⊢ 𝐵 = (Base‘𝐾) & ⊢ ≤ = (le‘𝐾) & ⊢ ∧ = (meet‘𝐾) ⇒ ⊢ ((𝐾 ∈ Lat ∧ (𝑋 ∈ 𝐵 ∧ 𝑌 ∈ 𝐵) ∧ (𝑍 ∈ 𝐵 ∧ 𝑊 ∈ 𝐵)) → ((𝑋 ≤ 𝑌 ∧ 𝑍 ≤ 𝑊) → (𝑋 ∧ 𝑍) ≤ (𝑌 ∧ 𝑊))) | ||
| Theorem | latnlemlt 18396 | Negation of "less than or equal to" expressed in terms of meet and less-than. (nssinpss 4220 analog.) (Contributed by NM, 5-Feb-2012.) |
| ⊢ 𝐵 = (Base‘𝐾) & ⊢ ≤ = (le‘𝐾) & ⊢ < = (lt‘𝐾) & ⊢ ∧ = (meet‘𝐾) ⇒ ⊢ ((𝐾 ∈ Lat ∧ 𝑋 ∈ 𝐵 ∧ 𝑌 ∈ 𝐵) → (¬ 𝑋 ≤ 𝑌 ↔ (𝑋 ∧ 𝑌) < 𝑋)) | ||
| Theorem | latnle 18397 | Equivalent expressions for "not less than" in a lattice. (chnle 31476 analog.) (Contributed by NM, 16-Nov-2011.) |
| ⊢ 𝐵 = (Base‘𝐾) & ⊢ ≤ = (le‘𝐾) & ⊢ < = (lt‘𝐾) & ⊢ ∨ = (join‘𝐾) ⇒ ⊢ ((𝐾 ∈ Lat ∧ 𝑋 ∈ 𝐵 ∧ 𝑌 ∈ 𝐵) → (¬ 𝑌 ≤ 𝑋 ↔ 𝑋 < (𝑋 ∨ 𝑌))) | ||
| Theorem | latmidm 18398 | Lattice meet is idempotent. Analogue of inidm 4180. (Contributed by NM, 8-Nov-2011.) |
| ⊢ 𝐵 = (Base‘𝐾) & ⊢ ∧ = (meet‘𝐾) ⇒ ⊢ ((𝐾 ∈ Lat ∧ 𝑋 ∈ 𝐵) → (𝑋 ∧ 𝑋) = 𝑋) | ||
| Theorem | latabs1 18399 | Lattice absorption law. From definition of lattice in [Kalmbach] p. 14. (chabs1 31478 analog.) (Contributed by NM, 8-Nov-2011.) |
| ⊢ 𝐵 = (Base‘𝐾) & ⊢ ∨ = (join‘𝐾) & ⊢ ∧ = (meet‘𝐾) ⇒ ⊢ ((𝐾 ∈ Lat ∧ 𝑋 ∈ 𝐵 ∧ 𝑌 ∈ 𝐵) → (𝑋 ∨ (𝑋 ∧ 𝑌)) = 𝑋) | ||
| Theorem | latabs2 18400 | Lattice absorption law. From definition of lattice in [Kalmbach] p. 14. (chabs2 31479 analog.) (Contributed by NM, 8-Nov-2011.) |
| ⊢ 𝐵 = (Base‘𝐾) & ⊢ ∨ = (join‘𝐾) & ⊢ ∧ = (meet‘𝐾) ⇒ ⊢ ((𝐾 ∈ Lat ∧ 𝑋 ∈ 𝐵 ∧ 𝑌 ∈ 𝐵) → (𝑋 ∧ (𝑋 ∨ 𝑌)) = 𝑋) | ||
| < Previous Next > |
| Copyright terms: Public domain | < Previous Next > |