src/HOL/Library/Old_Recdef.thy
changeset 46947 b8c7eb0c2f89
parent 46942 f5c2d66faa04
child 46950 d0181abdbdac
--- a/src/HOL/Library/Old_Recdef.thy	Thu Mar 15 17:45:54 2012 +0100
+++ b/src/HOL/Library/Old_Recdef.thy	Thu Mar 15 19:02:34 2012 +0100
@@ -6,7 +6,7 @@
 
 theory Old_Recdef
 imports Wfrec
-keywords "recdef" :: thy_decl
+keywords "recdef" :: thy_decl and "permissive" "congs" "hints"
 uses
   ("~~/src/HOL/Tools/TFL/casesplit.ML")
   ("~~/src/HOL/Tools/TFL/utils.ML")
@@ -42,7 +42,7 @@
 lemma tfl_eq_True: "(x = True) --> x"
   by blast
 
-lemma tfl_rev_eq_mp: "(x = y) --> y --> x";
+lemma tfl_rev_eq_mp: "(x = y) --> y --> x"
   by blast
 
 lemma tfl_simp_thm: "(x --> y) --> (x = x') --> (x' --> y)"