Home Linear Logic Proof Explorer
Theorem List (p. 4 of 4)
< Previous  Wrap >

Mirrors  >  Metamath Home Page  >  LLPE Home Page  >  Theorem List Contents       This page: Page List

Theorem List for Linear Logic Proof Explorer - 301-335   *Has distinct variable group(s)
TypeLabelDescription
Statement
 
Syntaxweqtru 301 Truth judgement.
wffP
 
Syntaxweqfal 302 Falsity judgement.
wffP
 
Definitiondf-eqtru 303 A shorthand way of saying that a church-encoded value is true. I would totally use this as a new typecode, so I could prove statements with instead of , but it turns out that adds needless complexity (and mmj2 doesn't like it).
(P = True ⧟ ⊨ P)
 
Definitiondf-eqfal 304 A shorthand way of saying that a church-encoded value is false. Note that this is not the opposite of df-eqtru 303 (although they do exclude each other), since there are many more things an expression could equal.
(P = False ⧟ ⊭ P)
 
Theoremdfeqtru1i 305 Introduce .
P = True       P
 
Theoremdfeqtru2i 306 Eliminate .
P        P = True
 
Theoremtru 307 True is true. Who'd've thunk it.
⊨ True
 
Syntaxnlimpl 308 Function representing logical implication.
nilad Impl
 
Syntaxnland 309 Function representing logical conjunction.
nilad And
 
Syntaxnlor 310 Function representing logical disjunction.
nilad Or
 
Syntaxnlnot 311 Function representing logical negation.
nilad Not
 
Syntaxnliff 312 Function representing logical biconditional.
nilad Iff
 
Definitiondf-limpl 313* Church-encoding of logical conjunction.
Impl = λaλb(baTrue)
 
Definitiondf-land 314* Church-encoding of logical conjunction.
And = λaλb(baFalse)
 
Definitiondf-lor 315* Church-encoding of logical disjunction.
Or = λaλb(Trueab)
 
Definitiondf-lnot 316* Church-encoding of logical negation.
Not = λaλxλy(yax)
 
Definitiondf-liff 317* Church-encoding of logical biconditional.
Iff = λaλb(ba(Not' b))
 
1.5  Quantifiers and equality

Oh boy. This is unexplored territory for me.

I'm just going to copy all the FOL axioms from set.mm and hope that works. I'm preeety sure that all those are valid theorems in linear logic; I'm just not sure whether they're sufficient. I think they are. Probably.

 
1.5.1  Axioms for predicate logic with equality
 
Syntaxwal 318 Universal quantifier. Characterized by ax-genOLD 323, ax-almd 324, ax-dis 325, ax-ex 326, ax-negf 330, ax-alcom 331.
wffx𝜑
 
Syntaxwex 319 Existential quantifier. Defined by df-ex 334.
wffx𝜑
 
Syntaxwnf 320 Not-free predicate. Defined by df-nf 335.
wffx𝜑
 
TheoremweqOLD 321 Equality. Charactrized by ax-ex 326, ax-sub 332, ax-aleq 333, ax-eqeu 327.
(𝜑𝜑)
 
Syntaxwel 322 Set element predicate. For the purposes of predicate logic, it's just an arbitrary operator.
wff xy
 
Axiomax-genOLD 323 Axiom of generalization. Universal quantifiers can be freely added to the start of an expression.
𝜑       x𝜑
 
Axiomax-almd 324 Quantified multiplicative disjunction. This "distributes" a quantifier over linear implication.
(∀x(𝜑𝜓) ⊸ (∀x𝜑 ⊸ ∀x𝜓))
 
Axiomax-dis 325* Distinctness principle. When the value of 𝜑 is independent of x, a quantifier can be added.
(𝜑 ⊸ ∀x𝜑)
 
Axiomax-ex 326 Axiom of existence. This axiom is secretly two useful axioms in one. It states that any y has an x that is equal to it. It also states that there exists something equal to itself, when y is substituted for x.
~ ∀x~ x = y
 
Axiomax-eqeu 327 Equality is Euclidean. Combined with ax-ex 326, this implies that equality is symmetric and transitive.
(x = y ⊸ (x = zy = z))
 
Axiomax-eleq1 328 Left equality for binary predicate. This consumes the equality.
(x = y ⊸ (xzyz))
 
Axiomax-eleq2 329 Right equality for binary predicate. This consumes the equality.
(x = y ⊸ (zxzy))
 
1.5.2  Auxiliary axioms for predicate logic with equality
 
Axiomax-negf 330 Axiom of quantified negation.
(~ ∀x𝜑 ⊸ ∀x~ ∀x𝜑)
 
Axiomax-alcom 331 Quantifier commutation.
(∀xy𝜑 ⊸ ∀yx𝜑)
 
Axiomax-sub 332 Axiom of variable substitution.
(x = y ⊸ (∀y𝜑 ⊸ ∀x(x = y𝜑)))
 
Axiomax-aleq 333 Quantified equality.
(~ x = y ⊸ (y = z ⊸ ∀x y = z))
 
Definitiondf-ex 334 Definition of existential quantifier. Dual of .
(∃x𝜑 ⧟ ~ ∀x~ 𝜑)
 
Definitiondf-nf 335 Definition of not-free predicate.
(Ⅎx𝜑 ⧟ (~ 𝜑 ⊸ ∀x𝜑))
    < Previous  Wrap >

Page List
Jump to page: Contents  1 1-100 2 101-200 3 201-300301-335
  Copyright terms: Public domain < Previous  Wrap >