src/HOL/Types_To_Sets/Examples/Unoverload_Def.thy
author wenzelm
Mon, 23 Oct 2023 12:08:38 +0200
changeset 78817 30bcf149054d
parent 69689 ab5a8a2519b0
permissions -rw-r--r--
clarified modules;

(*  Title:      HOL/Types_To_Sets/Examples/Unoverload_Def.thy
    Author:     Fabian Immler, CMU
*)
theory Unoverload_Def
  imports
    "../Types_To_Sets"
    Complex_Main
begin

unoverload_definition closed_def
  and compact_eq_Heine_Borel
  and cauchy_filter_def
  and Cauchy_uniform
  and nhds_def
  and complete_uniform
  and module_def
  and vector_space_def
  and module_hom_axioms_def
  and module_hom_def
  and VS_linear: Vector_Spaces.linear_def
  and linear_def

end