tuned header;
authorwenzelm
Fri, 01 Jun 2012 12:45:22 +0200
changeset 48055 9819d49d2f39
parent 48054 60bcc6cf17d6
child 48056 396749e9daaf
tuned header;
src/HOL/ex/Set_Comprehension_Pointfree_Tests.thy
src/HOL/ex/set_comprehension_pointfree.ML
--- a/src/HOL/ex/Set_Comprehension_Pointfree_Tests.thy	Fri Jun 01 08:32:26 2012 +0200
+++ b/src/HOL/ex/Set_Comprehension_Pointfree_Tests.thy	Fri Jun 01 12:45:22 2012 +0200
@@ -7,7 +7,7 @@
 
 theory Set_Comprehension_Pointfree_Tests
 imports Main
-uses "~~/src/HOL/ex/set_comprehension_pointfree.ML"
+uses "set_comprehension_pointfree.ML"
 begin
 
 simproc_setup finite_Collect ("finite (Collect P)") = {* Set_Comprehension_Pointfree.simproc *}
--- a/src/HOL/ex/set_comprehension_pointfree.ML	Fri Jun 01 08:32:26 2012 +0200
+++ b/src/HOL/ex/set_comprehension_pointfree.ML	Fri Jun 01 12:45:22 2012 +0200
@@ -1,4 +1,4 @@
-(*  Title:      HOL/Tools/set_comprehension_pointfree.ML
+(*  Title:      HOL/ex/set_comprehension_pointfree.ML
     Author:     Felix Kuperjans, Lukas Bulwahn, TU Muenchen
 
 Simproc for rewriting set comprehensions to pointfree expressions.