src/HOL/Library/Quantified_Premise_Simproc.thy
author wenzelm
Mon, 13 Apr 2020 22:08:14 +0200
changeset 71751 abf3e80bd815
parent 71518 bae868febc53
child 71886 4f4695757980
permissions -rw-r--r--
tuned NEWS;

(* Author: Florian Haftmann, TU München *)

theory Quantified_Premise_Simproc
  imports Main
begin

simproc_setup defined_forall ("\<And>x. PROP P x") = \<open>K Quantifier1.rearrange_All\<close>

end