src/HOL/Library/Quantified_Premise_Simproc.thy
changeset 71989 bad75618fb82
parent 71988 ace45a11a45e
child 71990 66beb9d92e43
--- a/src/HOL/Library/Quantified_Premise_Simproc.thy	Thu Jul 02 08:49:04 2020 +0000
+++ /dev/null	Thu Jan 01 00:00:00 1970 +0000
@@ -1,9 +0,0 @@
-(* Author: Florian Haftmann, TU München *)
-
-theory Quantified_Premise_Simproc
-  imports Main
-begin
-
-declare [[simproc add: defined_all]]
-
-end