src/FOL/IFOL.thy
changeset 18708 4b3dadb4fe33
parent 18523 9446cb8e1f65
child 18813 fc35dcc2558b
--- a/src/FOL/IFOL.thy	Thu Jan 19 15:45:10 2006 +0100
+++ b/src/FOL/IFOL.thy	Thu Jan 19 21:22:08 2006 +0100
@@ -194,9 +194,7 @@
   and [Pure.elim 2] = allE notE' impE'
   and [Pure.intro] = exI disjI2 disjI1
 
-setup {*
-  [ContextRules.addSWrapper (fn tac => hyp_subst_tac ORELSE' tac)]
-*}
+setup {* ContextRules.addSWrapper (fn tac => hyp_subst_tac ORELSE' tac) *}
 
 
 lemma iff_not_sym: "~ (Q <-> P) ==> ~ (P <-> Q)"