src/HOL/Hoare/Hoare_Syntax.thy
changeset 72990 db8f94656024
parent 72987 b1be35908165
child 74503 403ce50e6a2a
equal deleted inserted replaced
72989:5906162c8dd4 72990:db8f94656024
     1 (*  Title:      HOL/Hoare/Hoare_Syntax.thy
     1 (*  Title:      HOL/Hoare/Hoare_Syntax.thy
     2     Author:     Leonor Prensa Nieto & Tobias Nipkow
     2     Author:     Leonor Prensa Nieto & Tobias Nipkow
     3     Author:     Walter Guttmann (extension to total-correctness proofs)
     3     Author:     Walter Guttmann (extension to total-correctness proofs)
       
     4 *)
     4 
     5 
     5 Concrete syntax for Hoare logic, with translations for variables.
     6 section \<open>Concrete syntax for Hoare logic, with translations for variables\<close>
     6 *)
       
     7 
     7 
     8 theory Hoare_Syntax
     8 theory Hoare_Syntax
     9   imports Main
     9   imports Main
    10 begin
    10 begin
    11 
    11