src/HOL/ex/Execute_Choice.thy
changeset 58889 5b7a9633cfa8
parent 49929 70300f1b6835
child 61343 5b5656a63bd6
equal deleted inserted replaced
58888:9537bf1c4853 58889:5b7a9633cfa8
     1 (* Author: Florian Haftmann, TU Muenchen *)
     1 (* Author: Florian Haftmann, TU Muenchen *)
     2 
     2 
     3 header {* A simple cookbook example how to eliminate choice in programs. *}
     3 section {* A simple cookbook example how to eliminate choice in programs. *}
     4 
     4 
     5 theory Execute_Choice
     5 theory Execute_Choice
     6 imports Main "~~/src/HOL/Library/AList_Mapping"
     6 imports Main "~~/src/HOL/Library/AList_Mapping"
     7 begin
     7 begin
     8 
     8