src/HOL/Library/Simps_Case_Conv.thy
changeset 69568 de09a7261120
parent 67724 63e305429f8a
child 69605 a96320074298
--- a/src/HOL/Library/Simps_Case_Conv.thy	Sun Dec 30 10:30:41 2018 +0100
+++ b/src/HOL/Library/Simps_Case_Conv.thy	Tue Jan 01 17:04:53 2019 +0100
@@ -3,7 +3,7 @@
 *)
 
 theory Simps_Case_Conv
-imports Main
+imports Case_Converter
   keywords "simps_of_case" "case_of_simps" :: thy_decl
   abbrevs "simps_of_case" "case_of_simps" = ""
 begin