src/HOL/Set.thy
changeset 14479 0eca4aabf371
parent 14398 c5c47703f763
child 14551 2cb6ff394bfb
equal deleted inserted replaced
14478:bdf6b7adc3ec 14479:0eca4aabf371
  1945   by blast
  1945   by blast
  1946 
  1946 
  1947 lemma vimage_mono: "A \<subseteq> B ==> f -` A \<subseteq> f -` B"
  1947 lemma vimage_mono: "A \<subseteq> B ==> f -` A \<subseteq> f -` B"
  1948   -- {* monotonicity *}
  1948   -- {* monotonicity *}
  1949   by blast
  1949   by blast
       
  1950 
       
  1951 
       
  1952 subsection {* Getting the Contents of a Singleton Set *}
       
  1953 
       
  1954 constdefs
       
  1955   contents :: "'a set => 'a"
       
  1956    "contents X == THE x. X = {x}"
       
  1957 
       
  1958 lemma contents_eq [simp]: "contents {x} = x"
       
  1959 by (simp add: contents_def)
  1950 
  1960 
  1951 
  1961 
  1952 subsection {* Transitivity rules for calculational reasoning *}
  1962 subsection {* Transitivity rules for calculational reasoning *}
  1953 
  1963 
  1954 lemma forw_subst: "a = b ==> P b ==> P a"
  1964 lemma forw_subst: "a = b ==> P b ==> P a"