src/HOL/Main.thy
changeset 18510 0a6c24f549c3
parent 18315 e52f867ab851
child 19607 07eeb832f28d
equal deleted inserted replaced
18509:d2d96f12a1fc 18510:0a6c24f549c3
    16 
    16 
    17 text {* \medskip Late clause setup: installs \emph{all} simprules and
    17 text {* \medskip Late clause setup: installs \emph{all} simprules and
    18   claset rules into the clause cache; cf.\ theory @{text
    18   claset rules into the clause cache; cf.\ theory @{text
    19   Reconstruction}. *}
    19   Reconstruction}. *}
    20 
    20 
    21 declare subset_refl [intro] 
    21 setup ResAxioms.setup
    22   text {*Ensures that this important theorem is not superseded by the
       
    23          simplifier's "== True" version.*}
       
    24 setup ResAxioms.clause_setup
       
    25 declare subset_refl [rule del]
       
    26   text {*Removed again because it harms blast's performance.*}
       
    27 
    22 
    28 end
    23 end