HomeHome Higher-Order Logic Explorer
Theorem List (p. 1 of 3)
< Previous  Next >
Browser slow? Try the
Unicode version.

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

Theorem List for Higher-Order Logic Explorer - 1-100   *Has distinct variable group(s)
TypeLabelDescription
Statement
 
0.1  Foundations
 
Syntaxtv 1 A var is a term.
term x:al
 
Syntaxht 2 The type of all functions from type al to type be.
type (al -> be)
 
Syntaxhb 3 The type of booleans (true and false).
type *
 
Syntaxhi 4 The type of individuals.
type iota
 
Syntaxkc 5 A combination (function application).
term (FT)
 
Syntaxkl 6 A lambda abstraction.
term \x:al T
 
Syntaxke 7 The equality term.
term =
 
Syntaxkt 8 Truth term.
term T.
 
Syntaxkbr 9 Infix operator.
term [AFB]
 
Syntaxkct 10 Context operator.
term (A, B)
 
SyntaxwffMMJ2 11 Internal axiom for mmj2 use.
wff A |= B
 
SyntaxwffMMJ2t 12 Internal axiom for mmj2 use.
wff A:al
 
Theoremidi 13 The identity inference.
|- R |= A   =>   |- R |= A
 
Theoremidt 14 The identity inference.
|- A:al   =>   |- A:al
 
Axiomax-syl 15 Syllogism inference.
|- R |= S   &   |- S |= T   =>   |- R |= T
 
Theoremsyl 16 Syllogism inference.
|- R |= S   &   |- S |= T   =>   |- R |= T
 
Axiomax-jca 17 Join common antecedents.
|- R |= S   &   |- R |= T   =>   |- R |= (S, T)
 
Theoremjca 18 Syllogism inference.
|- R |= S   &   |- R |= T   =>   |- R |= (S, T)
 
Theoremsyl2anc 19 Syllogism inference.
|- R |= S   &   |- R |= T   &   |- (S, T) |= A   =>   |- R |= A
 
Axiomax-simpl 20 Extract an assumption from the context.
|- R:*   &   |- S:*   =>   |- (R, S) |= R
 
Axiomax-simpr 21 Extract an assumption from the context.
|- R:*   &   |- S:*   =>   |- (R, S) |= S
 
Theoremsimpl 22 Extract an assumption from the context.
|- R:*   &   |- S:*   =>   |- (R, S) |= R
 
Theoremsimpr 23 Extract an assumption from the context.
|- R:*   &   |- S:*   =>   |- (R, S) |= S
 
Axiomax-id 24 The identity inference.
|- R:*   =>   |- R |= R
 
Theoremid 25 The identity inference.
|- R:*   =>   |- R |= R
 
Axiomax-trud 26 Deduction form of tru 41.
|- R:*   =>   |- R |= T.
 
Theoremtrud 27 Deduction form of tru 41.
|- R:*   =>   |- R |= T.
 
Theorema1i 28 Change an empty context into any context.
|- R:*   &   |- T. |= A   =>   |- R |= A
 
Axiomax-cb1 29 A context has type boolean.

This and the next few axioms are not strictly necessary, and are conservative on any theorem for which every variable has a specified type, but by adding this axiom we can save some typehood hypotheses in many theorems. The easy way to see that this axiom is conservative is to note that every axiom and inference rule that constructs a theorem of the form R |= A where R and A are type variables, also ensures that R:* and A:*. Thus it is impossible to prove any theorem |- R |= A unless both |- R:* and |- A:* had been previously derived, so it is conservative to deduce |- R:* from |- R |= A. The same remark applies to the construction of the theorem (A, B):*- there is only one rule that creates a formula of this type, namely wct 44, and it requires that A:* and B:* be previously established, so it is safe to reverse the process in wctl 31 and wctr 32.

|- R |= A   =>   |- R:*
 
Axiomax-cb2 30 A theorem has type boolean. (This axiom is unnecessary; see ax-cb1 29.)
|- R |= A   =>   |- A:*
 
Syntaxwctl 31 Reverse closure for the type of a context. (This axiom is unnecessary; see ax-cb1 29.)
|- (S, T):*   =>   |- S:*
 
Syntaxwctr 32 Reverse closure for the type of a context. (This axiom is unnecessary; see ax-cb1 29.)
|- (S, T):*   =>   |- T:*
 
Theoremmpdan 33 Modus ponens deduction.
|- R |= S   &   |- (R, S) |= T   =>   |- R |= T
 
Theoremsyldan 34 Syllogism inference.
|- (R, S) |= T   &   |- (R, T) |= A   =>   |- (R, S) |= A
 
Theoremsimpld 35 Extract an assumption from the context.
|- R |= (S, T)   =>   |- R |= S
 
Theoremsimprd 36 Extract an assumption from the context.
|- R |= (S, T)   =>   |- R |= T
 
Theoremtrul 37 Deduction form of tru 41.
|- (T., R) |= S   =>   |- R |= S
 
Syntaxweq 38 The equality function has type al -> al -> *, i.e. it is polymorphic over all types, but the left and right type must agree.
|- = :(al -> (al -> *))
 
Axiomax-refl 39 Reflexivity of equality.
|- A:al   =>   |- T. |= (( = A)A)
 
Theoremwtru 40 Truth type.
|- T.:*
 
Theoremtru 41 Tautology is provable.
|- T. |= T.
 
Axiomax-eqmp 42 Modus ponens for equality.
|- R |= A   &   |- R |= (( = A)B)   =>   |- R |= B
 
Axiomax-ded 43 Deduction theorem for equality.
|- (R, S) |= T   &   |- (R, T) |= S   =>   |- R |= (( = S)T)
 
Syntaxwct 44 The type of a context.
|- S:*   &   |- T:*   =>   |- (S, T):*
 
Syntaxwc 45 The type of a combination.
|- F:(al -> be)   &   |- T:al   =>   |- (FT):be
 
Axiomax-ceq 46 Equality theorem for combination.
|- F:(al -> be)   &   |- T:(al -> be)   &   |- A:al   &   |- B:al   =>   |- ((( = F)T), (( = A)B)) |= (( = (FA))(TB))
 
Theoremeqcomx 47 Commutativity of equality.
|- A:al   &   |- B:al   &   |- R |= (( = A)B)   =>   |- R |= (( = B)A)
 
Theoremmpbirx 48 Deduction from equality inference.
|- B:*   &   |- R |= A   &   |- R |= (( = B)A)   =>   |- R |= B
 
Theoremancoms 49 Swap the two elements of a context.
|- (R, S) |= T   =>   |- (S, R) |= T
 
Theoremadantr 50 Extract an assumption from the context.
|- R |= T   &   |- S:*   =>   |- (R, S) |= T
 
Theoremadantl 51 Extract an assumption from the context.
|- R |= T   &   |- S:*   =>   |- (S, R) |= T
 
Theoremct1 52 Introduce a right conjunct.
|- R |= S   &   |- T:*   =>   |- (R, T) |= (S, T)
 
Theoremct2 53 Introduce a left conjunct.
|- R |= S   &   |- T:*   =>   |- (T, R) |= (T, S)
 
Theoremsylan 54 Syllogism inference.
|- R |= S   &   |- (S, T) |= A   =>   |- (R, T) |= A
 
Theoreman32s 55 Commutation identity for context.
|- ((R, S), T) |= A   =>   |- ((R, T), S) |= A
 
Theoremanasss 56 Associativity for context.
|- ((R, S), T) |= A   =>   |- (R, (S, T)) |= A
 
Theoremanassrs 57 Associativity for context.
|- (R, (S, T)) |= A   =>   |- ((R, S), T) |= A
 
Syntaxwv 58 The type of a typed variable.
|- x:al:al
 
Syntaxwl 59 The type of a lambda abstraction.
|- T:be   =>   |- \x:al T:(al -> be)
 
Axiomax-beta 60 Axiom of beta-substitution.
|- A:be   =>   |- T. |= (( = (\x:al Ax:al))A)
 
Axiomax-distrc 61 Distribution of combination over substitution.
|- A:be   &   |- B:al   &   |- F:(be -> ga)   =>   |- T. |= (( = (\x:al (FA)B))((\x:al FB)(\x:al AB)))
 
Axiomax-leq 62* Equality theorem for abstraction.
|- A:be   &   |- B:be   &   |- R |= (( = A)B)   =>   |- R |= (( = \x:al A)\x:al B)
 
Axiomax-distrl 63* Distribution of lambda abstraction over substitution.
|- A:ga   &   |- B:al   =>   |- T. |= (( = (\x:al \y:be AB))\y:be (\x:al AB))
 
Syntaxwov 64 Type of an infix operator.
|- F:(al -> (be -> ga))   &   |- A:al   &   |- B:be   =>   |- [AFB]:ga
 
Definitiondf-ov 65 Infix operator. This is a simple metamath way of cleaning up the syntax of all these infix operators to make them a bit more readable than the curried representation.
|- F:(al -> (be -> ga))   &   |- A:al   &   |- B:be   =>   |- T. |= (( = [AFB])((FA)B))
 
Theoremdfov1 66 Forward direction of df-ov 65.
|- F:(al -> (be -> *))   &   |- A:al   &   |- B:be   &   |- R |= [AFB]   =>   |- R |= ((FA)B)
 
Theoremdfov2 67 Reverse direction of df-ov 65.
|- F:(al -> (be -> *))   &   |- A:al   &   |- B:be   &   |- R |= ((FA)B)   =>   |- R |= [AFB]
 
Theoremweqi 68 Type of an equality.
|- A:al   &   |- B:al   =>   |- [A = B]:*
 
Syntaxeqtypi 69 Deduce equality of types from equality of expressions. (This is unnecessary but eliminates a lot of hypotheses.)
|- A:al   &   |- R |= [A = B]   =>   |- B:al
 
Theoremeqcomi 70 Commutativity of equality.
|- A:al   &   |- R |= [A = B]   =>   |- R |= [B = A]
 
Syntaxeqtypri 71 Deduce equality of types from equality of expressions. (This is unnecessary but eliminates a lot of hypotheses.)
|- A:al   &   |- R |= [B = A]   =>   |- B:al
 
Theoremmpbi 72 Deduction from equality inference.
|- R |= A   &   |- R |= [A = B]   =>   |- R |= B
 
Theoremeqid 73 Reflexivity of equality.
|- R:*   &   |- A:al   =>   |- R |= [A = A]
 
Theoremded 74 Deduction theorem for equality.
|- (R, S) |= T   &   |- (R, T) |= S   =>   |- R |= [S = T]
 
Theoremdedi 75 Deduction theorem for equality.
|- S |= T   &   |- T |= S   =>   |- T. |= [S = T]
 
Theoremeqtru 76 If a statement is provable, then it is equivalent to truth.
|- R |= A   =>   |- R |= [T. = A]
 
Theoremmpbir 77 Deduction from equality inference.
|- R |= A   &   |- R |= [B = A]   =>   |- R |= B
 
Theoremceq12 78 Equality theorem for combination.
|- F:(al -> be)   &   |- A:al   &   |- R |= [F = T]   &   |- R |= [A = B]   =>   |- R |= [(FA) = (TB)]
 
Theoremceq1 79 Equality theorem for combination.
|- F:(al -> be)   &   |- A:al   &   |- R |= [F = T]   =>   |- R |= [(FA) = (TA)]
 
Theoremceq2 80 Equality theorem for combination.
|- F:(al -> be)   &   |- A:al   &   |- R |= [A = B]   =>   |- R |= [(FA) = (FB)]
 
Theoremleq 81* Equality theorem for lambda abstraction.
|- A:be   &   |- R |= [A = B]   =>   |- R |= [\x:al A = \x:al B]
 
Theorembeta 82 Axiom of beta-substitution.
|- A:be   =>   |- T. |= [(\x:al Ax:al) = A]
 
Theoremdistrc 83 Distribution of combination over substitution.
|- F:(be -> ga)   &   |- A:be   &   |- B:al   =>   |- T. |= [(\x:al (FA)B) = ((\x:al FB)(\x:al AB))]
 
Theoremdistrl 84* Distribution of lambda abstraction over substitution.
|- A:ga   &   |- B:al   =>   |- T. |= [(\x:al \y:be AB) = \y:be (\x:al AB)]
 
Theoremeqtri 85 Transitivity of equality.
|- A:al   &   |- R |= [A = B]   &   |- R |= [B = C]   =>   |- R |= [A = C]
 
Theorem3eqtr4i 86 Transitivity of equality.
|- A:al   &   |- R |= [A = B]   &   |- R |= [S = A]   &   |- R |= [T = B]   =>   |- R |= [S = T]
 
Theorem3eqtr3i 87 Transitivity of equality.
|- A:al   &   |- R |= [A = B]   &   |- R |= [A = S]   &   |- R |= [B = T]   =>   |- R |= [S = T]
 
Theoremoveq123 88 Equality theorem for binary operation.
|- F:(al -> (be -> ga))   &   |- A:al   &   |- B:be   &   |- R |= [F = S]   &   |- R |= [A = C]   &   |- R |= [B = T]   =>   |- R |= [[AFB] = [CST]]
 
Theoremoveq1 89 Equality theorem for binary operation.
|- F:(al -> (be -> ga))   &   |- A:al   &   |- B:be   &   |- R |= [A = C]   =>   |- R |= [[AFB] = [CFB]]
 
Theoremoveq12 90 Equality theorem for binary operation.
|- F:(al -> (be -> ga))   &   |- A:al   &   |- B:be   &   |- R |= [A = C]   &   |- R |= [B = T]   =>   |- R |= [[AFB] = [CFT]]
 
Theoremoveq2 91 Equality theorem for binary operation.
|- F:(al -> (be -> ga))   &   |- A:al   &   |- B:be   &   |- R |= [B = T]   =>   |- R |= [[AFB] = [AFT]]
 
Theoremoveq 92 Equality theorem for binary operation.
|- F:(al -> (be -> ga))   &   |- A:al   &   |- B:be   &   |- R |= [F = S]   =>   |- R |= [[AFB] = [ASB]]
 
Axiomax-hbl1 93 x is bound in \xA.
|- A:ga   &   |- B:al   =>   |- T. |= [(\x:al \x:be AB) = \x:be A]
 
Theoremhbl1 94 Inference form of ax-hbl1 93.
|- A:ga   &   |- B:al   &   |- R:*   =>   |- R |= [(\x:al \x:be AB) = \x:be A]
 
Axiomax-17 95* If x does not appear in A, then any substitution to A yields A again, i.e. \xA is a constant function.
|- A:be   &   |- B:al   =>   |- T. |= [(\x:al AB) = A]
 
Theorema17i 96* Inference form of ax-17 95.
|- A:be   &   |- B:al   &   |- R:*   =>   |- R |= [(\x:al AB) = A]
 
Theoremhbxfrf 97* Transfer a hypothesis builder to an equivalent expression.
|- T:be   &   |- B:al   &   |- R |= [T = A]   &   |- (S, R) |= [(\x:al AB) = A]   =>   |- (S, R) |= [(\x:al TB) = T]
 
Theoremhbxfr 98* Transfer a hypothesis builder to an equivalent expression.
|- T:be   &   |- B:al   &   |- R |= [T = A]   &   |- R |= [(\x:al AB) = A]   =>   |- R |= [(\x:al TB) = T]
 
Theoremhbth 99* Hypothesis builder for a theorem.
|- B:al   &   |- R |= A   =>   |- R |= [(\x:al AB) = A]
 
Theoremhbc 100 Hypothesis builder for combination.
|- F:(be -> ga)   &   |- A:be   &   |- B:al   &   |- R |= [(\x:al FB) = F]   &   |- R |= [(\x:al AB) = A]   =>   |- R |= [(\x:al (FA)B) = (FA)]
    < Previous  Next >

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