# HG changeset patch # User wenzelm # Date 1527970475 -7200 # Node ID 46d5a9f428e1b3d0d2fd1d7d6f7d573550dad60e # Parent 67a4db47e4f6fb3cf2524ff6a41763d0e057e008 more formal comments; diff -r 67a4db47e4f6 -r 46d5a9f428e1 src/HOL/Library/Extended_Real.thy --- a/src/HOL/Library/Extended_Real.thy Sat Jun 02 22:11:09 2018 +0200 +++ b/src/HOL/Library/Extended_Real.thy Sat Jun 02 22:14:35 2018 +0200 @@ -627,9 +627,10 @@ "real_of_ereal y < x \ (\y\ \ \ \ y < ereal x) \ (\y\ = \ \ 0 < x)" by (cases y) auto -(*To help with inferences like a < ereal x \ x < y \ a < ereal y, +text \ + To help with inferences like \<^prop>\a < ereal x \ x < y \ a < ereal y\, where x and y are real. -*) +\ lemma le_ereal_le: "a \ ereal x \ x \ y \ a \ ereal y" using ereal_less_eq(3) order.trans by blast diff -r 67a4db47e4f6 -r 46d5a9f428e1 src/HOL/Library/Lub_Glb.thy --- a/src/HOL/Library/Lub_Glb.thy Sat Jun 02 22:11:09 2018 +0200 +++ b/src/HOL/Library/Lub_Glb.thy Sat Jun 02 22:14:35 2018 +0200 @@ -221,7 +221,7 @@ lemma isLub_mono_imp_LIMSEQ: fixes X :: "nat \ real" - assumes u: "isLub UNIV {x. \n. X n = x} u" (* FIXME: use 'range X' *) + assumes u: "isLub UNIV {x. \n. X n = x} u" (* FIXME: use \range X\ *) assumes X: "\m n. m \ n \ X m \ X n" shows "X \ u" proof -