src/HOL/IMP/Abs_Int1_const.thy
changeset 51389 8a9f0503b1c0
parent 51372 d315e9a9ee72
child 51711 df3426139651
--- a/src/HOL/IMP/Abs_Int1_const.thy	Sun Mar 10 14:36:18 2013 +0100
+++ b/src/HOL/IMP/Abs_Int1_const.thy	Sun Mar 10 18:29:10 2013 +0100
@@ -30,7 +30,7 @@
 
 definition "a < (b::const) = (a \<le> b & ~ b \<le> a)"
 
-fun join_const where
+fun sup_const where
 "Const m \<squnion> Const n = (if n=m then Const m else Any)" |
 "_ \<squnion> _ = Any"
 
@@ -48,11 +48,11 @@
 next
   case goal6 thus ?case by(cases x, cases y, simp_all)
 next
-  case goal7 thus ?case by(cases y, cases x, simp_all)
+  case goal5 thus ?case by(cases y, cases x, simp_all)
 next
-  case goal8 thus ?case by(cases z, cases y, cases x, simp_all)
+  case goal7 thus ?case by(cases z, cases y, cases x, simp_all)
 next
-  case goal5 thus ?case by(simp add: top_const_def)
+  case goal8 thus ?case by(simp add: top_const_def)
 qed
 
 end