WOLFRAM NOTEBOOK

Where do human-found theorems live in metamathematical space?

Cf where in 3D x,y,z space did people build cities on earth?

Boolean Algebra

Entailment cone should give the true theorems, but not as efficiently

Can we tighten up what we find in the “entailment target/retention zone” [ “directed entailments” ]

Ordinary theorem proving: we know the target, we want to find a single path
Traditional entailment cone: the entailments go out in all directions ... as opposed to making a “phased array” or an antenna in a particular direction

What are the proofs of interesting statements like?

In[]:=
interesting=First/@{{a==aa,"idempotent law for and"},{a==aa,"idempotent law for or"},{ab==ba,"commutativity for and"},{ab==ba,"commutativity for or"},{a==a,"law of double negation"},{aa==bb,"definition of false (law of noncontradiction)"},{aa==bb,"definition of true (law of excluded middle)"},{(ab)==ab,"de Morgan law"},{(ab)==ab,"de Morgan law"},{a==a(ab),"absorption law"},{a==aab,"absorption law"},{(ab)c==a(bc),"associativity of and"},{(ab)c==a(bc),"associativity of or"}};
In[]:=
AxiomaticTheory["BooleanAxioms"]
Out[]=
{a.,b.}
a.b.b.a.,
{a.,b.,c.}
a.(b.c.)a.b.a.c.,
{a.,b.}
a.b.
b.
a.,
{a.,b.}
a.b.
b.
a.,
{a.,b.}
a.b.b.a.,
{a.,b.,c.}
a.b.c.(a.b.)(a.c.)
In[]:=
interesting/.{Square->OverBar,Vee->CirclePlus,Wedge->CircleTimes}
Out[]=
aaa,aaa,abba,abba,a
a
,
a
a
b
b,
a
a
b
b,
ab
a
b
,
ab
a
b
,aa(ab),aaab,(ab)ca(bc),(ab)ca(bc)
In[]:=
FindReplacePath[ForAll[a,aaa],AxiomaticTheory["BooleanAxioms"]]
Out[]=
Statementaaa,PathTestSuccess
Message: Path sides match the original statement
Tag: Path
,RewriteTestSuccess
Message: Running rewrite sequence reproduced the path.
Tag: Rewrite
,Justification{{{Axiom,1},Right,{}},{{Axiom,3},Right,{}},{{Axiom,2},Left,{}}},RewritesReplace[x1_x1x2$11_
x2$11_
]/*ReplaceAll[x2$11_a._],Replace[x1_x2_x1_x3_x1(x2x3)],Replace[x1_(x2_
x2_
)x1],Path{a._a._,a._a._a._
a._
,a._(a._
a._
),a._}
In[]:=
FindEquationalProof[ForAll[a,aaa],AxiomaticTheory["BooleanAxioms"]]
Out[]=
ProofObject
Logic: EquationalLogic
Steps: 7
Theorem:
a
aaa
In[]:=
FindReplacePath[ForAll[{a,b,c},#],AxiomaticTheory["BooleanAxioms"],"Path"]&/@aaa,aaa,abba,abba,a
a
,
a
a
b
b,
a
a
b
b,
ab
a
b
,
ab
a
b
,aa(ab),aaab,(ab)ca(bc),(ab)ca(bc)
justifyLemma
::wrongOrientation
:Reversing wrong orientation for {SubstitutionLemma,6}, because x1((x2
x2
)x3)x1x1x3 don't match x1_x1_x2_x1b
b
x2 with orientation 1.
justifyLemma
::wrongOrientation
:Reversing wrong orientation for {SubstitutionLemma,6}, because x1(x2
x2
)x3x1(x1x3) don't match x1_(x1_x2_)x1b
b
x2 with orientation 1.
justifyLemma
::badOrientation
:Bad orientation for lemma {CriticalPairLemma,25}
justifyLemma
::badOrientation
:Bad orientation for lemma {CriticalPairLemma,26}
justifyLemma
::badOrientation
:Bad orientation for lemma {CriticalPairLemma,25}
General
:Further output of justifyLemma::badOrientation will be suppressed during this calculation.
Out[]=
{a._a._,a._a._a._
a._
,a._(a._
a._
),a._},
11
,(a._b._)c._,(b._a._)c._,(b._a._)(c._a._
a._
),(b._a._)(c._a._)(c._
a._
),(b._a._)(c._a._)((c._
a._
)(c._
c._
)),(b._a._)(c._a._)((c._
c._
)(c._
a._
)),(b._a._)(c._a._)(c._
c._
a._
),(b._a._)(c._a._)c._
c._
a._
c._
c._
,
189
,(a._c._)(b._a._)b._
b._
a._
,(a._c._)(b._a._)b._
b._
(b._
a._
),(a._c._)(b._a._)(b._
a._
)b._
b._
,(a._c._)(b._a._)(b._
a._
),(a._c._)(b._a._
a._
),(a._a._)a._,a._(a._a._),a._(a._a._)
large output
show less
show more
show all
set size limit...
In[]:=
Length/@%
Out[]=
{4,4,2,2,16,6,6,704,704,34,36,205,205}
NOTE: LeafCount wrong because of _’s
In[]:=
MapThread[ListLinePlot[#,Frame->True,PlotLabel->#2]&,Map[LeafCount,%9,{2}],aaa,aaa,abba,abba,a
a
,
a
a
b
b,
a
a
b
b,
ab
a
b
,
ab
a
b
,aa(ab),aaab,(ab)ca(bc),(ab)ca(bc)]
Out[]=
,
,
,
,
,
,
,
,
,
,
,
,

Note that this is after cut elimination ....

Approximate the branching ratio for the entailment cone

With intermediate lemmas

Wannabe theorems:
I.e. there are no new variables generated.... [at least after canonicalization]

Other Axiom Systems

[ There are 3 proofs here; ATP found 1 ] [ There are many theorems; you pick the one you want ]

ATP is good if you already know the theorem you want

Discovering new theorems (e.g. my Boolean algebra axiom) is hard with ATP

General approach: use models to find plausible theorems

Start from the axioms and find all models consistent with the axioms ... then ask what relations satisfy those models

Directed Theorem Enumeration

Instead of making the whole entailment cone, we only want “interesting theorems”

In the Metamath database, we’re seeing a skeleton of the entailment cone

Metamath Database

Imagine the entailment cone from the axioms of set theory

The MM database has a very thin skeleton of that entailment cone

For the sake of argument, let’s assume MM’s proofs are minimal

Can we estimate whether the skeleton is uniform across the entailment cone

Guess is it’s not uniform in the EC, but instead it’s built out in towers....
Is there something special about the towers?

The big point is that higher-level math is possible; therefore having a sparse collection of towers may be “enough”

I.e. you can talk about math without going through all the detail of the whole entailment cone

What are the TEGs of the MM database?

The substitution entailment is more complicated in MM [ but it’s a simpler form of substitution, where it just replaces the variables ]

Each definition introduces a function symbol....

MM is embedding all math in an explicit entailment graph ...

But most mathematical conclusions (AKA mathematical motion) never has to look down to axioms/emes/....
E.g. in physics we have laws of motion that don’t talk about the atoms of space....
Analog in math is “human-level proofs”
[ E.g. Euclid picked “human-like axioms” ]
Extreme coarse graining:
In a math result, you’re not necessarily talking about something very specific at the level of axioms, and certainly not at the level of emes....
Wolfram Cloud

You are using a browser not supported by the Wolfram Cloud

Supported browsers include recent versions of Chrome, Edge, Firefox and Safari.


I understand and wish to continue anyway »

You are using a browser not supported by the Wolfram Cloud. Supported browsers include recent versions of Chrome, Edge, Firefox and Safari.