src/HOL/HOLCF/Universal.thy
changeset 61605 1bf7b186542e
parent 61169 4de9ff3ea29a
child 62175 8ffc4d0e652d
equal deleted inserted replaced
61604:bb20f11dd842 61605:1bf7b186542e
   834     by (rule exI, rule inj_place)
   834     by (rule exI, rule inj_place)
   835 qed
   835 qed
   836 
   836 
   837 end
   837 end
   838 
   838 
   839 interpretation compact_basis!:
   839 interpretation compact_basis:
   840   ideal_completion below Rep_compact_basis
   840   ideal_completion below Rep_compact_basis
   841     "approximants :: 'a::bifinite \<Rightarrow> 'a compact_basis set"
   841     "approximants :: 'a::bifinite \<Rightarrow> 'a compact_basis set"
   842 proof -
   842 proof -
   843   obtain a :: "nat \<Rightarrow> 'a \<rightarrow> 'a" where "approx_chain a"
   843   obtain a :: "nat \<Rightarrow> 'a \<rightarrow> 'a" where "approx_chain a"
   844     using bifinite ..
   844     using bifinite ..