author | wenzelm |
Wed, 13 Oct 2021 00:02:35 +0200 | |
changeset 74505 | ce8152fb021b |
parent 74504 | 7422950f3955 |
child 74506 | d97c48dc87fa |
--- a/src/HOL/Hoare/ExamplesTC.thy Tue Oct 12 20:58:00 2021 +0200 +++ b/src/HOL/Hoare/ExamplesTC.thy Wed Oct 13 00:02:35 2021 +0200 @@ -27,7 +27,7 @@ Here is the total-correctness proof for the same program. It needs the additional invariant \<open>m \<le> a\<close>. \<close> -ML \<open>\<^const_syntax>\<open>HOL.eq\<close>\<close> + lemma multiply_by_add_tc: "VARS m s a b [a=A \<and> b=B] m := 0; s := 0;