src/HOLCF/IOA/meta_theory/Abstraction.thy
changeset 5976 44290b71a85f
parent 4816 64f075872f69
child 10835 f4745d77e620
equal deleted inserted replaced
5975:cd19eaa90f45 5976:44290b71a85f
    68 
    68 
    69 (* thm about ex2seq which is not provable by induction as ex2seq is not continous *)
    69 (* thm about ex2seq which is not provable by induction as ex2seq is not continous *)
    70 ex2seq_abs_cex
    70 ex2seq_abs_cex
    71   "ex2seq (cex_abs h ex) = cex_absSeq h (ex2seq ex)" 
    71   "ex2seq (cex_abs h ex) = cex_absSeq h (ex2seq ex)" 
    72 
    72 
    73 (* analog to the proved thm strength_Box  *)
    73 (* analog to the proved thm strength_Box - proof skipped as trivial *)
    74 weak_Box
    74 weak_Box
    75 "temp_weakening P Q h 
    75 "temp_weakening P Q h 
    76  ==> temp_weakening ([] P) ([] Q) h"
    76  ==> temp_weakening ([] P) ([] Q) h"
    77 
    77 
    78 (* analog to the proved thm strength_Next  *)
    78 (* analog to the proved thm strength_Next - proof skipped as trivial *)
    79 weak_Next
    79 weak_Next
    80 "temp_weakening P Q h 
    80 "temp_weakening P Q h 
    81  ==> temp_weakening (Next P) (Next Q) h"
    81  ==> temp_weakening (Next P) (Next Q) h"
    82 
    82 
    83 end
    83 end