src/HOL/BNF_Least_Fixpoint.thy
changeset 58274 4a84e94e58a2
parent 58211 c1f3fa32d322
child 58275 280ede57a6a9
--- a/src/HOL/BNF_Least_Fixpoint.thy	Tue Sep 09 20:51:36 2014 +0200
+++ b/src/HOL/BNF_Least_Fixpoint.thy	Tue Sep 09 20:51:36 2014 +0200
@@ -16,6 +16,9 @@
   "datatype_compat" :: thy_decl
 begin
 
+ML {* proofs := 2 *} (*###*)
+ML {* Proofterm.proofs_enabled () *}
+
 lemma subset_emptyI: "(\<And>x. x \<in> A \<Longrightarrow> False) \<Longrightarrow> A \<subseteq> {}"
   by blast