src/HOL/IMP/Denotational.thy
changeset 58889 5b7a9633cfa8
parent 52402 c2f30ba4bb98
child 62217 527488dc8b90
equal deleted inserted replaced
58888:9537bf1c4853 58889:5b7a9633cfa8
     1 (* Authors: Heiko Loetzbeyer, Robert Sandner, Tobias Nipkow *)
     1 (* Authors: Heiko Loetzbeyer, Robert Sandner, Tobias Nipkow *)
     2 
     2 
     3 header "Denotational Semantics of Commands"
     3 section "Denotational Semantics of Commands"
     4 
     4 
     5 theory Denotational imports Big_Step begin
     5 theory Denotational imports Big_Step begin
     6 
     6 
     7 type_synonym com_den = "(state \<times> state) set"
     7 type_synonym com_den = "(state \<times> state) set"
     8 
     8