changeset 57634 | efc00b9b8680 |
parent 56488 | 535cfc7fc301 |
child 58112 | 8081087096ad |
--- a/src/HOL/BNF_Examples/Compat.thy Thu Jul 24 00:24:00 2014 +0200 +++ b/src/HOL/BNF_Examples/Compat.thy Thu Jul 24 00:24:00 2014 +0200 @@ -1,3 +1,12 @@ +(* Title: HOL/BNF_Examples/Compat.thy + Author: Jasmin Blanchette, TU Muenchen + Copyright 2014 + +Tests for compatibility with the old datatype package. +*) + +header {* Tests for Compatibility with the Old Datatype Package *} + theory Compat imports Main begin