diff -r 4c54ef4dc84d -r 0fea8b7a14a1 ProgTutorial/Package/Ind_Code.thy --- a/ProgTutorial/Package/Ind_Code.thy Mon Oct 12 17:07:17 2009 +0200 +++ b/ProgTutorial/Package/Ind_Code.thy Tue Oct 13 22:57:25 2009 +0200 @@ -1,5 +1,5 @@ theory Ind_Code -imports "../Base" "../FirstSteps" Ind_General_Scheme +imports Ind_General_Scheme "../FirstSteps" begin section {* The Gory Details\label{sec:code} *}