src/HOL/Real/HahnBanach/Aux.thy
changeset 9408 d3d56e1d2ec1
parent 9394 1ff8a6234c6a
child 9503 3324cbbecef8
equal deleted inserted replaced
9407:e8f6d918fde9 9408:d3d56e1d2ec1
     8 theory Aux = Real + Zorn:
     8 theory Aux = Real + Zorn:
     9 
     9 
    10 text {* Some existing theorems are declared as extra introduction
    10 text {* Some existing theorems are declared as extra introduction
    11 or elimination rules, respectively. *}
    11 or elimination rules, respectively. *}
    12 
    12 
    13 lemmas [intro??] = isLub_isUb
    13 lemmas [intro?] = isLub_isUb
    14 lemmas [intro??] = chainD 
    14 lemmas [intro?] = chainD 
    15 lemmas chainE2 = chainD2 [elimify]
    15 lemmas chainE2 = chainD2 [elimify]
    16 
    16 
    17 text_raw {* \medskip *}
    17 text_raw {* \medskip *}
    18 text{* Lemmas about sets. *}
    18 text{* Lemmas about sets. *}
    19 
    19