src/HOL/MetisExamples/BT.thy
changeset 26312 e9a65675e5e8
parent 25457 ba2bcae7aafd
child 27104 791607529f6d
--- a/src/HOL/MetisExamples/BT.thy	Mon Mar 17 22:34:25 2008 +0100
+++ b/src/HOL/MetisExamples/BT.thy	Mon Mar 17 22:34:26 2008 +0100
@@ -232,7 +232,7 @@
   done
 
 ML {*ResAtp.problem_name := "BT__bt_map_appnd"*}
-lemma bt_map_appnd:
+lemma (*bt_map_appnd:*)
      "bt_map f (appnd t1 t2) = appnd (bt_map f t1) (bt_map f t2)"
   apply (induct t1)
   apply (metis appnd.simps(1) bt_map_appnd)