Forgot a couple of checks for the quick_and_dirty flag the other day.
authorskalberg
Mon, 19 Apr 2004 10:57:26 +0200
changeset 14627 5d137da82f03
parent 14626 dfb8d2977263
child 14628 8086e5beef0e
Forgot a couple of checks for the quick_and_dirty flag the other day.
src/HOL/Import/import_syntax.ML
--- a/src/HOL/Import/import_syntax.ML	Mon Apr 19 09:31:00 2004 +0200
+++ b/src/HOL/Import/import_syntax.ML	Mon Apr 19 10:57:26 2004 +0200
@@ -156,14 +156,20 @@
     end
 
 fun create_int_thms thyname thy =
-    case ImportData.get thy of
-	None => ImportData.put (Some (fst (Replay.setup_int_thms thyname thy))) thy
-      | Some _ => error "Import data not closed - forgotten an end_setup, mayhap?"
+    if !SkipProof.quick_and_dirty
+    then thy
+    else
+	case ImportData.get thy of
+	    None => ImportData.put (Some (fst (Replay.setup_int_thms thyname thy))) thy
+	  | Some _ => error "Import data not closed - forgotten an end_setup, mayhap?"
 
 fun clear_int_thms thy =
-    case ImportData.get thy of
-	None => error "Import data already cleared - forgotten a setup_theory?"
-      | Some _ => ImportData.put None thy
+    if !SkipProof.quick_and_dirty
+    then thy
+    else
+	case ImportData.get thy of
+	    None => error "Import data already cleared - forgotten a setup_theory?"
+	  | Some _ => ImportData.put None thy
 
 val setup_theory = P.name
 		       >>