do not touch quick_and_dirty;
authorwenzelm
Tue, 28 Aug 2007 11:25:32 +0200
changeset 24447 fbd6d7cbf6dd
parent 24446 bb7a85ea57cf
child 24448 46a32e245617
do not touch quick_and_dirty;
src/HOL/ex/NBE.thy
src/HOL/ex/Refute_Examples.thy
--- a/src/HOL/ex/NBE.thy	Tue Aug 28 11:25:31 2007 +0200
+++ b/src/HOL/ex/NBE.thy	Tue Aug 28 11:25:32 2007 +0200
@@ -5,8 +5,6 @@
 
 theory NBE imports Main Executable_Set begin
 
-ML"set quick_and_dirty"
-
 declare Let_def[simp]
 
 consts_code undefined ("(raise Match)")
--- a/src/HOL/ex/Refute_Examples.thy	Tue Aug 28 11:25:31 2007 +0200
+++ b/src/HOL/ex/Refute_Examples.thy	Tue Aug 28 11:25:32 2007 +0200
@@ -518,8 +518,6 @@
   not generate certain axioms for recursion operators.  Without these
   axioms, refute may find spurious countermodels. *}
 
-ML {* reset quick_and_dirty *}
-
 text {* unit *}
 
 lemma "P (x::unit)"