src/HOL/Record.thy
changeset 62117 86a31308a8e1
parent 61955 e96292f32c3c
child 67091 1393c2340eec
--- a/src/HOL/Record.thy	Mon Jan 11 00:04:23 2016 +0100
+++ b/src/HOL/Record.thy	Sun Jan 10 19:37:21 2016 -0800
@@ -10,7 +10,9 @@
 
 theory Record
 imports Quickcheck_Exhaustive
-keywords "record" :: thy_decl
+keywords
+  "record" :: thy_decl and
+  "print_record" :: diag
 begin
 
 subsection \<open>Introduction\<close>