src/HOL/ex/Computations.thy
changeset 66453 cc19f7ca2ed6
parent 64992 41e2c3617582
child 68660 4ce18f389f53
--- a/src/HOL/ex/Computations.thy	Fri Aug 18 13:55:05 2017 +0200
+++ b/src/HOL/ex/Computations.thy	Fri Aug 18 20:47:47 2017 +0200
@@ -5,7 +5,7 @@
 section \<open>Simple example for computations generated by the code generator\<close>
 
 theory Computations
-  imports "../Nat" "../Fun_Def" "../Num" "../Code_Numeral"
+  imports HOL.Nat HOL.Fun_Def HOL.Num HOL.Code_Numeral
 begin
 
 fun even :: "nat \<Rightarrow> bool"