--
You received this message because you are subscribed to the Google Groups "Metamath" group.
To unsubscribe from this group and stop receiving emails from it, send an email to metamath+u...@googlegroups.com.
To post to this group, send email to meta...@googlegroups.com.
Visit this group at https://groups.google.com/group/metamath.
For more options, visit https://groups.google.com/d/optout.
Was Binets Formula already
proved in meta math?
Just currious, a quick search didn't
show for example an Isabelle/HOL proof.
I remember Isabelle/HOL has strong induction. You could
invoke it somehow, this was part of some exercise in 2015.
Deriving strong induction in meta math should be possible,
so I guess it would be even bootstrappable. But still its
a challenging mixed problem...
On Sunday, April 21, 2019 at 4:11:15 PM UTC+2, Mario Carneiro wrote:
No, metamath doesn't even have the Fibonacci numbers AFAIK. In fact, the formula would probably be used as the definition of the fibonacci numbers, because a Fibonacci style recursion would be more complicated to define. Then the trick would be showing that Fn is an integer, and the defining equations hold.
On Sun, Apr 21, 2019 at 9:35 AM j4n bur53 <burs...@gmail.com> wrote:
Was Binets Formula already--
proved in meta math?
Just currious, a quick search didn't
show for example an Isabelle/HOL proof.
On Sunday, April 21, 2019 at 10:47:30 AM UTC+2, OlivierBinda wrote:I say.
The design of MetaMath is pretty strong and has withstood the test of time.
Let's just build the tooling that will really make it shine and prove
them wrong.
I have been experimenting with metamath tooling and it already looks to
me like there is a lot that can be done there.
In one month, I hope to go even further (just started working on stuff
with antecedents, right now).
Time will tell...
Olivier
You received this message because you are subscribed to the Google Groups "Metamath" group.
To unsubscribe from this group and stop receiving emails from it, send an email to meta...@googlegroups.com.
To post to this group, send email to meta...@googlegroups.com.
Visit this group at https://groups.google.com/group/metamath.
For more options, visit https://groups.google.com/d/optout.
prove forall n Q(n), instead forall n P(n). I guess forall n Q(n),
implies forall n P(n). So fibonacci is kind of a limited horizon
recursion, we only need to look back to a fixed number k of
elements where k=2, which makes it not a truely strong
recursion example, where k would be unbounded. Somehow I
am at loss, what a true example could be, although I have seen
some on the internet, but they were more complex, where the
objects what needs to look back were polynomials. So a
more number theoretic example, I did not yet find.
Am Sonntag, 28. April 2019 17:04:36 UTC+2 schrieb j4n bur53:Cool!
BTW: The discussion elsewhere about strong vs weak, took an interesting
turn. We are still looking for a convincing example for strong induction. Since
somebody suggested to solve Binets Formula problem, with a different
induction predicate
So instead prove via strong induction:
P(n) <=> fib(n) = binets_formula(n)
One can try the following weak induction:
Simply prove via weak induction:
Q(n) <=> P(n) /\ P(n+1)
Right?
But this wont say strong induction is useless. It says only that our
pedagogical search for a better illustration of strong induction cases
has not yet succeeded.
To unsubscribe from this group and stop receiving emails from it, send an email to meta...@googlegroups.com.
Thanks for the hint! Catalan numbers could indeed
be an interesting candidate. Now discussion started
meandering around axiom of choice, and I got
lost in metamath.
So to see
Theorem ac5 => Theorem ac7
I would need to look at:
http://us.metamath.org/mpegif/dfac4.html
What I want to see would be some byproduct?
Why is dfac4 called dfxxx like a definition?
Because it can be used like a definition?
Byproduct as in, simplified view:
A <=> B
--------------------------
(A => B) & (B => A)
----------------------------
A => B
So A=>B is a spinoff of having a proof A<=>B. But proofs work
more complex showing (CHOICE <=> A) <=> (CHOICE <=> B).
There are also "byproduct" helpers around, not of the "=>" kind,
more of the "<=>". But this helper explicitly mentions CHOICE,
like this here:
http://us.metamath.org/mpegif/axaci.html
Is this "architecture" genuinly metamath, or was it borrowed
from somewhere else?
Disclaimer: I call here A x B "sum" type and A -> B "product"
type. Not to be confused with disjoint sum A + B which is
not the same as cross product A x B.
Am Freitag, 17. Mai 2019 17:31:16 UTC+2 schrieb j4n bur53:Now there was an interesting thread somewhere else.
We observed that when we type predicates as:
Unary predicate: D
Binary predicate: D x D
We might obtain, i.e. shape shifting between arities, not
allowed in first order logic, FOL:
P(<x,y>) <=> P(x,y)
If P is a class symbol, does the same also happen in
metamath somehow? My own solution to the problem would
be to see unary respectively binary predicates as has
having this signature:
Unary predicate: D -> B
Binary predicate: D -> D -> B
where B={0,1}. But not sure how to resurect class
symbols then, and create a metamath zero, well I guess
it would be a metamath two, since metamath zero is
already used for an other project, a metamath with arity.
But there are a lot of options around. What should
the pairing function do? Should we have sum types at
all. The initial example assumes pairing function is, i.e.
without sum type, <_,_> : D -> D -> D.
but if we have sum type, we could say pair is <_,_> :
D -> D -> D x D. but in set theory there might be an inclusion
of the sum type, i.e. D x D subset D. So that sum types
dont seem to be viable to fix anything.
Am Sonntag, 12. Mai 2019 20:03:12 UTC+2 schrieb j4n bur53:Catalan numbers are natural numbers. A new question.
Was there ever already done something in metamath
about Cantor Pairing? Some theorems in metamath
about this little quadratic polynomial:
Cantor polynomial
P(x,y) = 1/2 ((x+y)*(x+y+1)) + x
https://en.wikipedia.org/wiki/Fueter%E2%80%93P%C3%B3lya_theorem
Googling "pairing" site:metamath.org
didn't give me something. Just currious.
Am Samstag, 11. Mai 2019 02:17:01 UTC+2 schrieb j4n bur53:
Thanks for the hint! Catalan numbers could indeed
be an interesting candidate. Now discussion started
meandering around axiom of choice, and I got
lost in metamath.
So to see
Theorem ac5 => Theorem ac7
I would need to look at:
http://us.metamath.org/mpegif/dfac4.html
What I want to see would be some byproduct?
Why is dfac4 called dfxxx like a definition?
Because it can be used like a definition?
To unsubscribe from this group and stop receiving emails from it, send an email to metamath+u...@googlegroups.com.
To post to this group, send email to meta...@googlegroups.com.
Visit this group at https://groups.google.com/group/metamath.
To view this discussion on the web visit https://groups.google.com/d/msgid/metamath/8b306044-0d76-4f24-9bc4-aec9423b3a90%40googlegroups.com.
Because I have every once a day an idea, I didn't wanted to
contributed to the explosion of threads by just posting every
new embrionic thought, in a new thread.
To view this discussion on the web visit https://groups.google.com/d/msgid/metamath/8b306044-0d76-4f24-9bc4-aec9423b3a90%40googlegroups.com.
For more options, visit https://groups.google.com/d/optout.
--
You received this message because you are subscribed to the Google Groups "Metamath" group.
To unsubscribe from this group and stop receiving emails from it, send an email to metamath+u...@googlegroups.com.
To post to this group, send email to meta...@googlegroups.com.
Visit this group at https://groups.google.com/group/metamath.
To view this discussion on the web visit https://groups.google.com/d/msgid/metamath/4fb5bb2e-1705-45d8-8d29-20b24bfad44f%40googlegroups.com.
You also answered in the past here:
Mario Carneiro
https://groups.google.com/d/msg/metamath/La4LEDM5ASI/OM8yhrU4CQAJ
Whats so different in my new question? Did I provoke something
because I mentioned metamath zero? I don't know how metamath
zero would handle the case. I only wanted to find a name
for what I am working on. So I called it metamath one. But
if you feel better, I can also call it metamath minus one. If
this makes you feel better, well then.
Ha Ha, some people are really fun, and they will never apologize.
Am Freitag, 17. Mai 2019 20:06:24 UTC+2 schrieb j4n bur53:Also Norman Megill didn't mind answering a question here.
I guess he has better manners than you have. Insulting people
with no grounds.
Am Freitag, 17. Mai 2019 20:05:08 UTC+2 schrieb j4n bur53:So far I have only use this thread for most of my thoughts. You can't
say I have polluted everyones elses thread, this a false allegation
and some harassement.
To view this discussion on the web visit https://groups.google.com/d/msgid/metamath/4fb5bb2e-1705-45d8-8d29-20b24bfad44f%40googlegroups.com.
For more options, visit https://groups.google.com/d/optout.
--
You received this message because you are subscribed to the Google Groups "Metamath" group.
To unsubscribe from this group and stop receiving emails from it, send an email to metamath+u...@googlegroups.com.
To post to this group, send email to meta...@googlegroups.com.
Visit this group at https://groups.google.com/group/metamath.
To view this discussion on the web visit https://groups.google.com/d/msgid/metamath/2ea5d8cf-1dd1-45fe-aaa7-1c7db17e2799%40googlegroups.com.
As a matter of facts, Mario is already experimenting with x86 semantics
in his MM0 repository, although at this point I do not really know what
is the status and the plan. He wrote something in this post:
--
You received this message because you are subscribed to the Google Groups "Metamath" group.
To unsubscribe from this group and stop receiving emails from it, send an email to metamath+u...@googlegroups.com.
To view this discussion on the web visit https://groups.google.com/d/msgid/metamath/8880c819-6bd9-4fb8-bae5-afe317e8157e%40googlegroups.com.