src/FOL/FOL.thy
changeset 34914 e391c3de0f6b
parent 32960 69916a850301
child 34989 b5c6e59e2cd7
--- a/src/FOL/FOL.thy	Sun Jan 10 18:39:50 2010 +0100
+++ b/src/FOL/FOL.thy	Sun Jan 10 18:41:07 2010 +0100
@@ -383,6 +383,8 @@
     val atomize = @{thms induct_atomize}
     val rulify = @{thms induct_rulify}
     val rulify_fallback = @{thms induct_rulify_fallback}
+    fun dest_def _ = NONE
+    fun trivial_tac _ = no_tac
   );
 *}