src/HOL/Multivariate_Analysis/Brouwer_Fixpoint.thy
changeset 63129 e5cb3440af74
parent 63040 eb4ddd18d635
child 63301 d3c87eb0bad2
equal deleted inserted replaced
63128:24708cf4ba61 63129:e5cb3440af74
    17 (* ========================================================================= *)
    17 (* ========================================================================= *)
    18 
    18 
    19 section \<open>Results connected with topological dimension.\<close>
    19 section \<open>Results connected with topological dimension.\<close>
    20 
    20 
    21 theory Brouwer_Fixpoint
    21 theory Brouwer_Fixpoint
    22 imports Path_Connected
    22 imports Path_Connected Homeomorphism
    23 begin
    23 begin
    24 
    24 
    25 lemma bij_betw_singleton_eq:
    25 lemma bij_betw_singleton_eq:
    26   assumes f: "bij_betw f A B" and g: "bij_betw g A B" and a: "a \<in> A"
    26   assumes f: "bij_betw f A B" and g: "bij_betw g A B" and a: "a \<in> A"
    27   assumes eq: "(\<And>x. x \<in> A \<Longrightarrow> x \<noteq> a \<Longrightarrow> f x = g x)"
    27   assumes eq: "(\<And>x. x \<in> A \<Longrightarrow> x \<noteq> a \<Longrightarrow> f x = g x)"