author | huffman |
Fri, 03 Jun 2005 23:30:31 +0200 | |
changeset 16213 | 88ddef269510 |
parent 16212 | 422f836f6b39 |
child 16214 | e3816a7db016 |
--- a/src/HOLCF/Discrete.thy Fri Jun 03 23:29:48 2005 +0200 +++ b/src/HOLCF/Discrete.thy Fri Jun 03 23:30:31 2005 +0200 @@ -68,7 +68,7 @@ by (fast dest: discr_chain0 elim: arg_cong) lemma cont_discr [iff]: "cont(%x::('a::type)discr. f x)" -apply (unfold cont is_lub_def is_ub_def) +apply (unfold cont_def is_lub_def is_ub_def) apply (simp add: discr_chain_f_range0) done