diff -r 066bb557570f -r 7619080e49f0 src/HOL/SetInterval.thy --- a/src/HOL/SetInterval.thy Wed Aug 15 09:02:11 2007 +0200 +++ b/src/HOL/SetInterval.thy Wed Aug 15 12:52:56 2007 +0200 @@ -153,19 +153,19 @@ subsection {*Two-sided intervals*} -lemma greaterThanLessThan_iff [simp]: +lemma greaterThanLessThan_iff [simp,noatp]: "(i : {l<.. {m.. i | m \ i & j \ (n::'a::linorder))" apply(auto simp:linorder_not_le) apply(rule ccontr)