src/HOL/Examples/Ackermann.thy
changeset 72029 83456d9f0ed5
parent 71930 35a2ac83a262
child 73531 c89922715bf5
--- 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 \<open>A Tail-Recursive, Stack-Based Ackermann's Function\<close>
 
 theory Ackermann imports Main