src/HOL/Library/Infinite_Set.thy
changeset 55980 a8ad7f6dd217
parent 55952 9733ab5c1df6
child 55985 7e291ae244ea
equal deleted inserted replaced
55979:0cb8a2defb06 55980:a8ad7f6dd217
     3 *)
     3 *)
     4 
     4 
     5 header {* Infinite Sets and Related Concepts *}
     5 header {* Infinite Sets and Related Concepts *}
     6 
     6 
     7 theory Infinite_Set
     7 theory Infinite_Set
     8 imports Main
     8 imports Set_Interval
     9 begin
     9 begin
    10 
    10 
    11 subsection "Infinite Sets"
    11 subsection "Infinite Sets"
    12 
    12 
    13 text {*
    13 text {*
   552 
   552 
   553 lemma atmost_one_unique [elim]: "atmost_one S \<Longrightarrow> x \<in> S \<Longrightarrow> y \<in> S \<Longrightarrow> y = x"
   553 lemma atmost_one_unique [elim]: "atmost_one S \<Longrightarrow> x \<in> S \<Longrightarrow> y \<in> S \<Longrightarrow> y = x"
   554   by (simp add: atmost_one_def)
   554   by (simp add: atmost_one_def)
   555 
   555 
   556 end
   556 end
   557