file header
authorblanchet
Tue, 22 Mar 2016 12:39:37 +0100
changeset 62695 b287b56a6ce5
parent 62694 f50d7efc8fe3
child 62696 7325d8573fb8
file header
src/HOL/Datatype_Examples/Lift_BNF.thy
--- a/src/HOL/Datatype_Examples/Lift_BNF.thy	Tue Mar 22 12:39:37 2016 +0100
+++ b/src/HOL/Datatype_Examples/Lift_BNF.thy	Tue Mar 22 12:39:37 2016 +0100
@@ -1,3 +1,12 @@
+(*  Title:      HOL/Datatype_Examples/Lift_BNF.thy
+    Author:     Dmitriy Traytel, ETH Zürich
+    Copyright   2015
+
+Demonstration of the "lift_bnf" command.
+*)
+
+section {* Demonstration of the @{command lift_bnf} Command *}
+
 theory Lift_BNF
 imports Main
 begin