src/HOL/ex/Set_Comprehension_Pointfree_Tests.thy
changeset 49070 9819d49d2f39
parent 49064 d862b0d56c49
child 49123 f93433b451b8
     1.1 --- a/src/HOL/ex/Set_Comprehension_Pointfree_Tests.thy	Fri Jun 01 08:32:26 2012 +0200
     1.2 +++ b/src/HOL/ex/Set_Comprehension_Pointfree_Tests.thy	Fri Jun 01 12:45:22 2012 +0200
     1.3 @@ -7,7 +7,7 @@
     1.4  
     1.5  theory Set_Comprehension_Pointfree_Tests
     1.6  imports Main
     1.7 -uses "~~/src/HOL/ex/set_comprehension_pointfree.ML"
     1.8 +uses "set_comprehension_pointfree.ML"
     1.9  begin
    1.10  
    1.11  simproc_setup finite_Collect ("finite (Collect P)") = {* Set_Comprehension_Pointfree.simproc *}