HomeHome Intuitionistic Logic Explorer
Theorem List (p. 3 of 102)
< 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 - 201-300   *Has distinct variable group(s)
TypeLabelDescription
Statement
 
Theorem3bitr4i 201 A chained inference from transitive law for logical equivalence. This inference is frequently used to apply a definition to both sides of a logical equivalence. (Contributed by NM, 5-Aug-1993.)
(𝜑𝜓)    &   (𝜒𝜑)    &   (𝜃𝜓)       (𝜒𝜃)
 
Theorem3bitr4ri 202 A chained inference from transitive law for logical equivalence. (Contributed by NM, 2-Sep-1995.)
(𝜑𝜓)    &   (𝜒𝜑)    &   (𝜃𝜓)       (𝜃𝜒)
 
Theorem3bitrd 203 Deduction from transitivity of biconditional. (Contributed by NM, 13-Aug-1999.)
(𝜑 → (𝜓𝜒))    &   (𝜑 → (𝜒𝜃))    &   (𝜑 → (𝜃𝜏))       (𝜑 → (𝜓𝜏))
 
Theorem3bitrrd 204 Deduction from transitivity of biconditional. (Contributed by NM, 4-Aug-2006.)
(𝜑 → (𝜓𝜒))    &   (𝜑 → (𝜒𝜃))    &   (𝜑 → (𝜃𝜏))       (𝜑 → (𝜏𝜓))
 
Theorem3bitr2d 205 Deduction from transitivity of biconditional. (Contributed by NM, 4-Aug-2006.)
(𝜑 → (𝜓𝜒))    &   (𝜑 → (𝜃𝜒))    &   (𝜑 → (𝜃𝜏))       (𝜑 → (𝜓𝜏))
 
Theorem3bitr2rd 206 Deduction from transitivity of biconditional. (Contributed by NM, 4-Aug-2006.)
(𝜑 → (𝜓𝜒))    &   (𝜑 → (𝜃𝜒))    &   (𝜑 → (𝜃𝜏))       (𝜑 → (𝜏𝜓))
 
Theorem3bitr3d 207 Deduction from transitivity of biconditional. Useful for converting conditional definitions in a formula. (Contributed by NM, 24-Apr-1996.)
(𝜑 → (𝜓𝜒))    &   (𝜑 → (𝜓𝜃))    &   (𝜑 → (𝜒𝜏))       (𝜑 → (𝜃𝜏))
 
Theorem3bitr3rd 208 Deduction from transitivity of biconditional. (Contributed by NM, 4-Aug-2006.)
(𝜑 → (𝜓𝜒))    &   (𝜑 → (𝜓𝜃))    &   (𝜑 → (𝜒𝜏))       (𝜑 → (𝜏𝜃))
 
Theorem3bitr4d 209 Deduction from transitivity of biconditional. Useful for converting conditional definitions in a formula. (Contributed by NM, 18-Oct-1995.)
(𝜑 → (𝜓𝜒))    &   (𝜑 → (𝜃𝜓))    &   (𝜑 → (𝜏𝜒))       (𝜑 → (𝜃𝜏))
 
Theorem3bitr4rd 210 Deduction from transitivity of biconditional. (Contributed by NM, 4-Aug-2006.)
(𝜑 → (𝜓𝜒))    &   (𝜑 → (𝜃𝜓))    &   (𝜑 → (𝜏𝜒))       (𝜑 → (𝜏𝜃))
 
Theorem3bitr3g 211 More general version of 3bitr3i 199. Useful for converting definitions in a formula. (Contributed by NM, 4-Jun-1995.)
(𝜑 → (𝜓𝜒))    &   (𝜓𝜃)    &   (𝜒𝜏)       (𝜑 → (𝜃𝜏))
 
Theorem3bitr4g 212 More general version of 3bitr4i 201. Useful for converting definitions in a formula. (Contributed by NM, 5-Aug-1993.)
(𝜑 → (𝜓𝜒))    &   (𝜃𝜓)    &   (𝜏𝜒)       (𝜑 → (𝜃𝜏))
 
Theorembi3ant 213 Construct a biconditional in antecedent position. (Contributed by Wolf Lammen, 14-May-2013.)
(𝜑 → (𝜓𝜒))       (((𝜃𝜏) → 𝜑) → (((𝜏𝜃) → 𝜓) → ((𝜃𝜏) → 𝜒)))
 
Theorembisym 214 Express symmetries of theorems in terms of biconditionals. (Contributed by Wolf Lammen, 14-May-2013.)
(((𝜑𝜓) → (𝜒𝜃)) → (((𝜓𝜑) → (𝜃𝜒)) → ((𝜑𝜓) → (𝜒𝜃))))
 
Theoremimbi2i 215 Introduce an antecedent to both sides of a logical equivalence. (Contributed by NM, 5-Aug-1993.) (Proof shortened by Wolf Lammen, 6-Feb-2013.)
(𝜑𝜓)       ((𝜒𝜑) ↔ (𝜒𝜓))
 
Theorembibi2i 216 Inference adding a biconditional to the left in an equivalence. (Contributed by NM, 5-Aug-1993.) (Proof shortened by Andrew Salmon, 7-May-2011.) (Proof shortened by Wolf Lammen, 16-May-2013.)
(𝜑𝜓)       ((𝜒𝜑) ↔ (𝜒𝜓))
 
Theorembibi1i 217 Inference adding a biconditional to the right in an equivalence. (Contributed by NM, 5-Aug-1993.)
(𝜑𝜓)       ((𝜑𝜒) ↔ (𝜓𝜒))
 
Theorembibi12i 218 The equivalence of two equivalences. (Contributed by NM, 5-Aug-1993.)
(𝜑𝜓)    &   (𝜒𝜃)       ((𝜑𝜒) ↔ (𝜓𝜃))
 
Theoremimbi2d 219 Deduction adding an antecedent to both sides of a logical equivalence. (Contributed by NM, 5-Aug-1993.)
(𝜑 → (𝜓𝜒))       (𝜑 → ((𝜃𝜓) ↔ (𝜃𝜒)))
 
Theoremimbi1d 220 Deduction adding a consequent to both sides of a logical equivalence. (Contributed by NM, 5-Aug-1993.) (Proof shortened by Wolf Lammen, 17-Sep-2013.)
(𝜑 → (𝜓𝜒))       (𝜑 → ((𝜓𝜃) ↔ (𝜒𝜃)))
 
Theorembibi2d 221 Deduction adding a biconditional to the left in an equivalence. (Contributed by NM, 5-Aug-1993.) (Proof shortened by Wolf Lammen, 19-May-2013.)
(𝜑 → (𝜓𝜒))       (𝜑 → ((𝜃𝜓) ↔ (𝜃𝜒)))
 
Theorembibi1d 222 Deduction adding a biconditional to the right in an equivalence. (Contributed by NM, 5-Aug-1993.)
(𝜑 → (𝜓𝜒))       (𝜑 → ((𝜓𝜃) ↔ (𝜒𝜃)))
 
Theoremimbi12d 223 Deduction joining two equivalences to form equivalence of implications. (Contributed by NM, 5-Aug-1993.)
(𝜑 → (𝜓𝜒))    &   (𝜑 → (𝜃𝜏))       (𝜑 → ((𝜓𝜃) ↔ (𝜒𝜏)))
 
Theorembibi12d 224 Deduction joining two equivalences to form equivalence of biconditionals. (Contributed by NM, 5-Aug-1993.)
(𝜑 → (𝜓𝜒))    &   (𝜑 → (𝜃𝜏))       (𝜑 → ((𝜓𝜃) ↔ (𝜒𝜏)))
 
Theoremimbi1 225 Theorem *4.84 of [WhiteheadRussell] p. 122. (Contributed by NM, 3-Jan-2005.)
((𝜑𝜓) → ((𝜑𝜒) ↔ (𝜓𝜒)))
 
Theoremimbi2 226 Theorem *4.85 of [WhiteheadRussell] p. 122. (Contributed by NM, 3-Jan-2005.) (Proof shortened by Wolf Lammen, 19-May-2013.)
((𝜑𝜓) → ((𝜒𝜑) ↔ (𝜒𝜓)))
 
Theoremimbi1i 227 Introduce a consequent to both sides of a logical equivalence. (Contributed by NM, 5-Aug-1993.) (Proof shortened by Wolf Lammen, 17-Sep-2013.)
(𝜑𝜓)       ((𝜑𝜒) ↔ (𝜓𝜒))
 
Theoremimbi12i 228 Join two logical equivalences to form equivalence of implications. (Contributed by NM, 5-Aug-1993.)
(𝜑𝜓)    &   (𝜒𝜃)       ((𝜑𝜒) ↔ (𝜓𝜃))
 
Theorembibi1 229 Theorem *4.86 of [WhiteheadRussell] p. 122. (Contributed by NM, 3-Jan-2005.)
((𝜑𝜓) → ((𝜑𝜒) ↔ (𝜓𝜒)))
 
Theorembiimt 230 A wff is equivalent to itself with true antecedent. (Contributed by NM, 28-Jan-1996.)
(𝜑 → (𝜓 ↔ (𝜑𝜓)))
 
Theorempm5.5 231 Theorem *5.5 of [WhiteheadRussell] p. 125. (Contributed by NM, 3-Jan-2005.)
(𝜑 → ((𝜑𝜓) ↔ 𝜓))
 
Theorema1bi 232 Inference rule introducing a theorem as an antecedent. (Contributed by NM, 5-Aug-1993.) (Proof shortened by Wolf Lammen, 11-Nov-2012.)
𝜑       (𝜓 ↔ (𝜑𝜓))
 
Theorempm5.501 233 Theorem *5.501 of [WhiteheadRussell] p. 125. (Contributed by NM, 3-Jan-2005.) (Revised by NM, 24-Jan-2013.)
(𝜑 → (𝜓 ↔ (𝜑𝜓)))
 
Theoremibib 234 Implication in terms of implication and biconditional. (Contributed by NM, 31-Mar-1994.) (Proof shortened by Wolf Lammen, 24-Jan-2013.)
((𝜑𝜓) ↔ (𝜑 → (𝜑𝜓)))
 
Theoremibibr 235 Implication in terms of implication and biconditional. (Contributed by NM, 29-Apr-2005.) (Proof shortened by Wolf Lammen, 21-Dec-2013.)
((𝜑𝜓) ↔ (𝜑 → (𝜓𝜑)))
 
Theoremtbt 236 A wff is equivalent to its equivalence with truth. (Contributed by NM, 18-Aug-1993.) (Proof shortened by Andrew Salmon, 13-May-2011.)
𝜑       (𝜓 ↔ (𝜓𝜑))
 
Theorembi2.04 237 Logical equivalence of commuted antecedents. Part of Theorem *4.87 of [WhiteheadRussell] p. 122. (Contributed by NM, 5-Aug-1993.)
((𝜑 → (𝜓𝜒)) ↔ (𝜓 → (𝜑𝜒)))
 
Theorempm5.4 238 Antecedent absorption implication. Theorem *5.4 of [WhiteheadRussell] p. 125. (Contributed by NM, 5-Aug-1993.)
((𝜑 → (𝜑𝜓)) ↔ (𝜑𝜓))
 
Theoremimdi 239 Distributive law for implication. Compare Theorem *5.41 of [WhiteheadRussell] p. 125. (Contributed by NM, 5-Aug-1993.)
((𝜑 → (𝜓𝜒)) ↔ ((𝜑𝜓) → (𝜑𝜒)))
 
Theorempm5.41 240 Theorem *5.41 of [WhiteheadRussell] p. 125. (Contributed by NM, 3-Jan-2005.) (Proof shortened by Wolf Lammen, 12-Oct-2012.)
(((𝜑𝜓) → (𝜑𝜒)) ↔ (𝜑 → (𝜓𝜒)))
 
Theoremimim21b 241 Simplify an implication between two implications when the antecedent of the first is a consequence of the antecedent of the second. The reverse form is useful in producing the successor step in induction proofs. (Contributed by Paul Chapman, 22-Jun-2011.) (Proof shortened by Wolf Lammen, 14-Sep-2013.)
((𝜓𝜑) → (((𝜑𝜒) → (𝜓𝜃)) ↔ (𝜓 → (𝜒𝜃))))
 
Theoremimpd 242 Importation deduction. (Contributed by NM, 31-Mar-1994.)
(𝜑 → (𝜓 → (𝜒𝜃)))       (𝜑 → ((𝜓𝜒) → 𝜃))
 
Theoremimp31 243 An importation inference. (Contributed by NM, 26-Apr-1994.)
(𝜑 → (𝜓 → (𝜒𝜃)))       (((𝜑𝜓) ∧ 𝜒) → 𝜃)
 
Theoremimp32 244 An importation inference. (Contributed by NM, 26-Apr-1994.)
(𝜑 → (𝜓 → (𝜒𝜃)))       ((𝜑 ∧ (𝜓𝜒)) → 𝜃)
 
Theoremexpd 245 Exportation deduction. (Contributed by NM, 20-Aug-1993.)
(𝜑 → ((𝜓𝜒) → 𝜃))       (𝜑 → (𝜓 → (𝜒𝜃)))
 
Theoremexpdimp 246 A deduction version of exportation, followed by importation. (Contributed by NM, 6-Sep-2008.)
(𝜑 → ((𝜓𝜒) → 𝜃))       ((𝜑𝜓) → (𝜒𝜃))
 
Theoremimpancom 247 Mixed importation/commutation inference. (Contributed by NM, 22-Jun-2013.)
((𝜑𝜓) → (𝜒𝜃))       ((𝜑𝜒) → (𝜓𝜃))
 
Theorempm3.3 248 Theorem *3.3 (Exp) of [WhiteheadRussell] p. 112. (Contributed by NM, 3-Jan-2005.) (Proof shortened by Wolf Lammen, 24-Mar-2013.)
(((𝜑𝜓) → 𝜒) → (𝜑 → (𝜓𝜒)))
 
Theorempm3.31 249 Theorem *3.31 (Imp) of [WhiteheadRussell] p. 112. (Contributed by NM, 3-Jan-2005.) (Proof shortened by Wolf Lammen, 24-Mar-2013.)
((𝜑 → (𝜓𝜒)) → ((𝜑𝜓) → 𝜒))
 
Theoremimpexp 250 Import-export theorem. Part of Theorem *4.87 of [WhiteheadRussell] p. 122. (Contributed by NM, 5-Aug-1993.) (Proof shortened by Wolf Lammen, 24-Mar-2013.)
(((𝜑𝜓) → 𝜒) ↔ (𝜑 → (𝜓𝜒)))
 
Theorempm3.21 251 Join antecedents with conjunction. Theorem *3.21 of [WhiteheadRussell] p. 111. (Contributed by NM, 5-Aug-1993.)
(𝜑 → (𝜓 → (𝜓𝜑)))
 
Theorempm3.22 252 Theorem *3.22 of [WhiteheadRussell] p. 111. (Contributed by NM, 3-Jan-2005.) (Proof shortened by Wolf Lammen, 13-Nov-2012.)
((𝜑𝜓) → (𝜓𝜑))
 
Theoremancom 253 Commutative law for conjunction. Theorem *4.3 of [WhiteheadRussell] p. 118. (Contributed by NM, 25-Jun-1998.) (Proof shortened by Wolf Lammen, 4-Nov-2012.)
((𝜑𝜓) ↔ (𝜓𝜑))
 
Theoremancomd 254 Commutation of conjuncts in consequent. (Contributed by Jeff Hankins, 14-Aug-2009.)
(𝜑 → (𝜓𝜒))       (𝜑 → (𝜒𝜓))
 
Theoremancoms 255 Inference commuting conjunction in antecedent. (Contributed by NM, 21-Apr-1994.)
((𝜑𝜓) → 𝜒)       ((𝜓𝜑) → 𝜒)
 
Theoremancomsd 256 Deduction commuting conjunction in antecedent. (Contributed by NM, 12-Dec-2004.)
(𝜑 → ((𝜓𝜒) → 𝜃))       (𝜑 → ((𝜒𝜓) → 𝜃))
 
Theorempm3.2i 257 Infer conjunction of premises. (Contributed by NM, 5-Aug-1993.)
𝜑    &   𝜓       (𝜑𝜓)
 
Theorempm3.43i 258 Nested conjunction of antecedents. (Contributed by NM, 5-Aug-1993.)
((𝜑𝜓) → ((𝜑𝜒) → (𝜑 → (𝜓𝜒))))
 
Theoremsimplbi 259 Deduction eliminating a conjunct. (Contributed by NM, 27-May-1998.)
(𝜑 ↔ (𝜓𝜒))       (𝜑𝜓)
 
Theoremsimprbi 260 Deduction eliminating a conjunct. (Contributed by NM, 27-May-1998.)
(𝜑 ↔ (𝜓𝜒))       (𝜑𝜒)
 
Theoremadantr 261 Inference adding a conjunct to the right of an antecedent. (Contributed by NM, 30-Aug-1993.)
(𝜑𝜓)       ((𝜑𝜒) → 𝜓)
 
Theoremadantl 262 Inference adding a conjunct to the left of an antecedent. (Contributed by NM, 30-Aug-1993.) (Proof shortened by Wolf Lammen, 23-Nov-2012.)
(𝜑𝜓)       ((𝜒𝜑) → 𝜓)
 
Theoremadantld 263 Deduction adding a conjunct to the left of an antecedent. (Contributed by NM, 4-May-1994.) (Proof shortened by Wolf Lammen, 20-Dec-2012.)
(𝜑 → (𝜓𝜒))       (𝜑 → ((𝜃𝜓) → 𝜒))
 
Theoremadantrd 264 Deduction adding a conjunct to the right of an antecedent. (Contributed by NM, 4-May-1994.)
(𝜑 → (𝜓𝜒))       (𝜑 → ((𝜓𝜃) → 𝜒))
 
Theoremmpan9 265 Modus ponens conjoining dissimilar antecedents. (Contributed by NM, 1-Feb-2008.) (Proof shortened by Andrew Salmon, 7-May-2011.)
(𝜑𝜓)    &   (𝜒 → (𝜓𝜃))       ((𝜑𝜒) → 𝜃)
 
Theoremsyldan 266 A syllogism deduction with conjoined antecents. (Contributed by NM, 24-Feb-2005.) (Proof shortened by Wolf Lammen, 6-Apr-2013.)
((𝜑𝜓) → 𝜒)    &   ((𝜑𝜒) → 𝜃)       ((𝜑𝜓) → 𝜃)
 
Theoremsylan 267 A syllogism inference. (Contributed by NM, 21-Apr-1994.) (Proof shortened by Wolf Lammen, 22-Nov-2012.)
(𝜑𝜓)    &   ((𝜓𝜒) → 𝜃)       ((𝜑𝜒) → 𝜃)
 
Theoremsylanb 268 A syllogism inference. (Contributed by NM, 18-May-1994.)
(𝜑𝜓)    &   ((𝜓𝜒) → 𝜃)       ((𝜑𝜒) → 𝜃)
 
Theoremsylanbr 269 A syllogism inference. (Contributed by NM, 18-May-1994.)
(𝜓𝜑)    &   ((𝜓𝜒) → 𝜃)       ((𝜑𝜒) → 𝜃)
 
Theoremsylan2 270 A syllogism inference. (Contributed by NM, 21-Apr-1994.) (Proof shortened by Wolf Lammen, 22-Nov-2012.)
(𝜑𝜒)    &   ((𝜓𝜒) → 𝜃)       ((𝜓𝜑) → 𝜃)
 
Theoremsylan2b 271 A syllogism inference. (Contributed by NM, 21-Apr-1994.)
(𝜑𝜒)    &   ((𝜓𝜒) → 𝜃)       ((𝜓𝜑) → 𝜃)
 
Theoremsylan2br 272 A syllogism inference. (Contributed by NM, 21-Apr-1994.)
(𝜒𝜑)    &   ((𝜓𝜒) → 𝜃)       ((𝜓𝜑) → 𝜃)
 
Theoremsyl2an 273 A double syllogism inference. (Contributed by NM, 31-Jan-1997.)
(𝜑𝜓)    &   (𝜏𝜒)    &   ((𝜓𝜒) → 𝜃)       ((𝜑𝜏) → 𝜃)
 
Theoremsyl2anr 274 A double syllogism inference. (Contributed by NM, 17-Sep-2013.)
(𝜑𝜓)    &   (𝜏𝜒)    &   ((𝜓𝜒) → 𝜃)       ((𝜏𝜑) → 𝜃)
 
Theoremsyl2anb 275 A double syllogism inference. (Contributed by NM, 29-Jul-1999.)
(𝜑𝜓)    &   (𝜏𝜒)    &   ((𝜓𝜒) → 𝜃)       ((𝜑𝜏) → 𝜃)
 
Theoremsyl2anbr 276 A double syllogism inference. (Contributed by NM, 29-Jul-1999.)
(𝜓𝜑)    &   (𝜒𝜏)    &   ((𝜓𝜒) → 𝜃)       ((𝜑𝜏) → 𝜃)
 
Theoremsyland 277 A syllogism deduction. (Contributed by NM, 15-Dec-2004.)
(𝜑 → (𝜓𝜒))    &   (𝜑 → ((𝜒𝜃) → 𝜏))       (𝜑 → ((𝜓𝜃) → 𝜏))
 
Theoremsylan2d 278 A syllogism deduction. (Contributed by NM, 15-Dec-2004.)
(𝜑 → (𝜓𝜒))    &   (𝜑 → ((𝜃𝜒) → 𝜏))       (𝜑 → ((𝜃𝜓) → 𝜏))
 
Theoremsyl2and 279 A syllogism deduction. (Contributed by NM, 15-Dec-2004.)
(𝜑 → (𝜓𝜒))    &   (𝜑 → (𝜃𝜏))    &   (𝜑 → ((𝜒𝜏) → 𝜂))       (𝜑 → ((𝜓𝜃) → 𝜂))
 
Theorembiimpa 280 Inference from a logical equivalence. (Contributed by NM, 3-May-1994.)
(𝜑 → (𝜓𝜒))       ((𝜑𝜓) → 𝜒)
 
Theorembiimpar 281 Inference from a logical equivalence. (Contributed by NM, 3-May-1994.)
(𝜑 → (𝜓𝜒))       ((𝜑𝜒) → 𝜓)
 
Theorembiimpac 282 Inference from a logical equivalence. (Contributed by NM, 3-May-1994.)
(𝜑 → (𝜓𝜒))       ((𝜓𝜑) → 𝜒)
 
Theorembiimparc 283 Inference from a logical equivalence. (Contributed by NM, 3-May-1994.)
(𝜑 → (𝜓𝜒))       ((𝜒𝜑) → 𝜓)
 
Theoremiba 284 Introduction of antecedent as conjunct. Theorem *4.73 of [WhiteheadRussell] p. 121. (Contributed by NM, 30-Mar-1994.) (Revised by NM, 24-Mar-2013.)
(𝜑 → (𝜓 ↔ (𝜓𝜑)))
 
Theoremibar 285 Introduction of antecedent as conjunct. (Contributed by NM, 5-Dec-1995.) (Revised by NM, 24-Mar-2013.)
(𝜑 → (𝜓 ↔ (𝜑𝜓)))
 
Theorembiantru 286 A wff is equivalent to its conjunction with truth. (Contributed by NM, 5-Aug-1993.)
𝜑       (𝜓 ↔ (𝜓𝜑))
 
Theorembiantrur 287 A wff is equivalent to its conjunction with truth. (Contributed by NM, 3-Aug-1994.)
𝜑       (𝜓 ↔ (𝜑𝜓))
 
Theorembiantrud 288 A wff is equivalent to its conjunction with truth. (Contributed by NM, 2-Aug-1994.) (Proof shortened by Wolf Lammen, 23-Oct-2013.)
(𝜑𝜓)       (𝜑 → (𝜒 ↔ (𝜒𝜓)))
 
Theorembiantrurd 289 A wff is equivalent to its conjunction with truth. (Contributed by NM, 1-May-1995.) (Proof shortened by Andrew Salmon, 7-May-2011.)
(𝜑𝜓)       (𝜑 → (𝜒 ↔ (𝜓𝜒)))
 
Theoremjca 290 Deduce conjunction of the consequents of two implications ("join consequents with 'and'"). (Contributed by NM, 5-Aug-1993.) (Proof shortened by Wolf Lammen, 25-Oct-2012.)
(𝜑𝜓)    &   (𝜑𝜒)       (𝜑 → (𝜓𝜒))
 
Theoremjcad 291 Deduction conjoining the consequents of two implications. (Contributed by NM, 5-Aug-1993.) (Proof shortened by Wolf Lammen, 23-Jul-2013.)
(𝜑 → (𝜓𝜒))    &   (𝜑 → (𝜓𝜃))       (𝜑 → (𝜓 → (𝜒𝜃)))
 
Theoremjca31 292 Join three consequents. (Contributed by Jeff Hankins, 1-Aug-2009.)
(𝜑𝜓)    &   (𝜑𝜒)    &   (𝜑𝜃)       (𝜑 → ((𝜓𝜒) ∧ 𝜃))
 
Theoremjca32 293 Join three consequents. (Contributed by FL, 1-Aug-2009.)
(𝜑𝜓)    &   (𝜑𝜒)    &   (𝜑𝜃)       (𝜑 → (𝜓 ∧ (𝜒𝜃)))
 
Theoremjcai 294 Deduction replacing implication with conjunction. (Contributed by NM, 5-Aug-1993.)
(𝜑𝜓)    &   (𝜑 → (𝜓𝜒))       (𝜑 → (𝜓𝜒))
 
Theoremjctil 295 Inference conjoining a theorem to left of consequent in an implication. (Contributed by NM, 31-Dec-1993.)
(𝜑𝜓)    &   𝜒       (𝜑 → (𝜒𝜓))
 
Theoremjctir 296 Inference conjoining a theorem to right of consequent in an implication. (Contributed by NM, 31-Dec-1993.)
(𝜑𝜓)    &   𝜒       (𝜑 → (𝜓𝜒))
 
Theoremjctl 297 Inference conjoining a theorem to the left of a consequent. (Contributed by NM, 31-Dec-1993.) (Proof shortened by Wolf Lammen, 24-Oct-2012.)
𝜓       (𝜑 → (𝜓𝜑))
 
Theoremjctr 298 Inference conjoining a theorem to the right of a consequent. (Contributed by NM, 18-Aug-1993.) (Proof shortened by Wolf Lammen, 24-Oct-2012.)
𝜓       (𝜑 → (𝜑𝜓))
 
Theoremjctild 299 Deduction conjoining a theorem to left of consequent in an implication. (Contributed by NM, 21-Apr-2005.)
(𝜑 → (𝜓𝜒))    &   (𝜑𝜃)       (𝜑 → (𝜓 → (𝜃𝜒)))
 
Theoremjctird 300 Deduction conjoining a theorem to right of consequent in an implication. (Contributed by NM, 21-Apr-2005.)
(𝜑 → (𝜓𝜒))    &   (𝜑𝜃)       (𝜑 → (𝜓 → (𝜒𝜃)))
    < Previous  Next >

Page List
Jump to page: Contents  1 1-100 2 101-200201-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-10124
  Copyright terms: Public domain < Previous  Next >