jagomart
digital resources
picture1_Outline


 114x       Filetype PDF       File size 0.06 MB       Source: www.isa-afp.org


File: Outline
fun with functions tobias nipkow december 12 2009 abstract this is a collection of cute puzzles of the form show that if a function satises the following constraints it must ...

icon picture PDF Filetype PDF | Posted on 29 Jan 2023 | 2 years ago
Partial capture of text on file.
                                               Fun With Functions
                                                      Tobias Nipkow
                                                    December 12, 2009
                                                         Abstract
                                 This is a collection of cute puzzles of the form “Show that if a
                              function satisfies the following constraints, it must be ...” Please add
                              further examples to this collection!
                            Apart from the one about factorial, they all come from the delightful
                         booklet by Terence Tao [1] but go back to Math Olympiads and similar
                         events.
                            Please add further examples of this kind, either directly or by sending
                         them to me. Let us make this a growing body of fun!
                         theory FunWithFunctions imports Complex-Main begin
                            See[1]. WasfirstbroughttoourattentionbyHerbertEhlerwhoprovided
                         a similar proof.
                         theorem identity1: fixes f :: nat ⇒ nat
                                     V
                         assumes fff:   n. f (f (n)) < f (Suc(n))
                         shows f(n) = n
                         hproofi
                            See [1]. Possible extension: Should also hold if the range of f is the reals!
                         lemma identity2: fixes f :: nat ⇒ nat
                         assumes f(k) = k and k ≥ 2
                         and f-times: Vm n. f(m∗n) = f(m)∗f(n)
                         and f-mono: Vm n. m
						
									
										
									
																
													
					
The words contained in this file might help you see if this file matches what you are looking for:

...Fun with functions tobias nipkow december abstract this is a collection of cute puzzles the form show that if function satises following constraints it must be please add further examples to apart from one about factorial they all come delightful booklet by terence tao but go back math olympiads and similar events kind either directly or sending them me let us make growing body theory funwithfunctions imports complex main begin see wasrstbroughttoourattentionbyherbertehlerwhoprovided proof theorem identity xes f nat v assumes n suc shows hproofi possible extension should also hold range reals lemma k times vm m mono...

no reviews yet
Please Login to review.