src/CTT/ex/Typechecking.thy
changeset 58974 cbc2ac19d783
parent 58972 5b026cfc5f04
child 58976 b38a54bbfbd6
--- a/src/CTT/ex/Typechecking.thy	Tue Nov 11 11:47:53 2014 +0100
+++ b/src/CTT/ex/Typechecking.thy	Tue Nov 11 13:40:13 2014 +0100
@@ -6,7 +6,7 @@
 section "Easy examples: type checking and type deduction"
 
 theory Typechecking
-imports CTT
+imports "../CTT"
 begin
 
 subsection {* Single-step proofs: verifying that a type is well-formed *}