# HG changeset patch # User paulson # Date 1685453049 -3600 # Node ID 3d2db8057b9f3bc4bb91f29aeb014c674febcc8e # Parent 24b70433c2e86811389219be4a8c8bc40552ebd4 Hiding the constructor names, particularly to avoid conflicts involving "ext" diff -r 24b70433c2e8 -r 3d2db8057b9f src/HOL/Analysis/Urysohn.thy --- a/src/HOL/Analysis/Urysohn.thy Tue May 30 12:33:06 2023 +0100 +++ b/src/HOL/Analysis/Urysohn.thy Tue May 30 14:24:09 2023 +0100 @@ -1542,9 +1542,11 @@ base: "openin X U \ Alexandroff_open X (Some ` U)" | ext: "\compactin X C; closedin X C\ \ Alexandroff_open X (insert None (Some ` (topspace X - C)))" +hide_fact (open) base ext + lemma Alexandroff_open_iff: "Alexandroff_open X S \ (\U. (S = Some ` U \ openin X U) \ (S = insert None (Some ` (topspace X - U)) \ compactin X U \ closedin X U))" - by (meson Alexandroff_open.cases Alexandroff_open.ext base) + by (meson Alexandroff_open.cases Alexandroff_open.ext Alexandroff_open.base) lemma Alexandroff_open_Un_aux: assumes U: "openin X U" and "Alexandroff_open X T" @@ -1681,7 +1683,7 @@ then have eq: "\\ = Some ` (\ K\\. U K)" using image_iff by fastforce show ?thesis - unfolding eq by (simp add: U base openin_clauses(3)) + unfolding eq by (simp add: U Alexandroff_open.base openin_clauses(3)) qed qed