changeset 180 | 8f443f2ed1f6 |
parent 173 | b51cb9aef3ae |
child 181 | 4d54702229fd |
--- a/thys/Abacus.thy Mon Feb 18 00:18:56 2013 +0000 +++ b/thys/Abacus.thy Mon Feb 18 13:26:27 2013 +0000 @@ -38,7 +38,7 @@ fun mult :: "nat \<Rightarrow> nat \<Rightarrow> nat \<Rightarrow> nat \<Rightarrow> nat \<Rightarrow> abc_prog" where - "mult m1 m2 n p e = [Dec m1 e]@ plus m1 m2 p 1" + "mult m1 m2 n p e = [Dec m1 e]@ plus m2 n p 1" fun expo :: "nat \<Rightarrow> nat \<Rightarrow> nat \<Rightarrow> nat \<Rightarrow> nat \<Rightarrow> abc_prog" where