changeset 41956 | c15ef1b85035 |
parent 41457 | 3bb2f035203f |
child 55447 | aa41ecbdc205 |
--- a/src/HOL/Predicate_Compile_Examples/Code_Prolog_Examples.thy Sun Mar 13 20:56:00 2011 +0100 +++ b/src/HOL/Predicate_Compile_Examples/Code_Prolog_Examples.thy Sun Mar 13 21:21:48 2011 +0100 @@ -1,5 +1,5 @@ theory Code_Prolog_Examples -imports Code_Prolog +imports "~~/src/HOL/Library/Code_Prolog" begin section {* Example append *}