diff -r b93e6b458433 -r ca1ad6660b4a src/HOL/Import/Import_Setup.thy --- a/src/HOL/Import/Import_Setup.thy Thu Jan 16 12:12:32 2025 +0100 +++ b/src/HOL/Import/Import_Setup.thy Thu Jan 16 12:41:55 2025 +0100 @@ -3,7 +3,7 @@ Author: Alexander Krauss, QAware GmbH *) -section \Importer machinery and required theorems\ +section \Importer machinery\ theory Import_Setup imports Main @@ -11,19 +11,6 @@ begin ML_file \import_data.ML\ - -lemma light_ex_imp_nonempty: "P t \ \x. x \ Collect P" - by auto - -lemma typedef_hol2hollight: - "type_definition Rep Abs (Collect P) \ Abs (Rep a) = a \ P r = (Rep (Abs r) = r)" - by (metis type_definition.Rep_inverse type_definition.Abs_inverse - type_definition.Rep mem_Collect_eq) - -lemma ext2: "(\x. f x = g x) \ f = g" - by (rule ext) - ML_file \import_rule.ML\ end -