diff -r 759532ef0885 -r 83456d9f0ed5 src/HOL/Examples/Ackermann.thy --- a/src/HOL/Examples/Ackermann.thy Sun Jul 12 18:10:06 2020 +0000 +++ b/src/HOL/Examples/Ackermann.thy Mon Jul 13 17:08:45 2020 +0200 @@ -1,3 +1,7 @@ +(* Title: HOL/Examples/Ackermann.thy + Author: Larry Paulson +*) + section \A Tail-Recursive, Stack-Based Ackermann's Function\ theory Ackermann imports Main