src/HOL/HOL.thy
changeset 9970 dfe4747c8318
parent 9950 879e88b1e552
child 10383 a092ae7bb2a6
equal deleted inserted replaced
9969:4753185f1dd2 9970:dfe4747c8318
   157   (*Extensionality is built into the meta-logic, and this rule expresses
   157   (*Extensionality is built into the meta-logic, and this rule expresses
   158     a related property.  It is an eta-expanded version of the traditional
   158     a related property.  It is an eta-expanded version of the traditional
   159     rule, and similar to the ABS rule of HOL.*)
   159     rule, and similar to the ABS rule of HOL.*)
   160   ext:          "(!!x::'a. (f x ::'b) = g x) ==> (%x. f x) = (%x. g x)"
   160   ext:          "(!!x::'a. (f x ::'b) = g x) ==> (%x. f x) = (%x. g x)"
   161 
   161 
   162   selectI:      "P (x::'a) ==> P (@x. P x)"
   162   someI:        "P (x::'a) ==> P (@x. P x)"
   163 
   163 
   164   impI:         "(P ==> Q) ==> P-->Q"
   164   impI:         "(P ==> Q) ==> P-->Q"
   165   mp:           "[| P-->Q;  P |] ==> Q"
   165   mp:           "[| P-->Q;  P |] ==> Q"
   166 
   166 
   167 defs
   167 defs