src/HOL/IMP/HoareT.thy
changeset 44177 b4b5cbca2519
parent 43158 686fa0a0696e
child 44890 22f665a2e91c
equal deleted inserted replaced
44176:eda112e9cdee 44177:b4b5cbca2519
     1 header{* Hoare Logic for Total Correctness *}
     1 header{* Hoare Logic for Total Correctness *}
     2 
     2 
     3 theory HoareT imports Hoare_Sound_Complete Util begin
     3 theory HoareT imports Hoare_Sound_Complete begin
     4 
     4 
     5 text{*
     5 text{*
     6 Now that we have termination, we can define
     6 Now that we have termination, we can define
     7 total validity, @{text"\<Turnstile>\<^sub>t"}, as partial validity and guaranteed termination:*}
     7 total validity, @{text"\<Turnstile>\<^sub>t"}, as partial validity and guaranteed termination:*}
     8 
     8