src/HOL/IMP/Sec_TypingT.thy
changeset 63539 70d4d9e5707b
parent 54864 a064732223ad
child 67406 23307fd33906
--- a/src/HOL/IMP/Sec_TypingT.thy	Thu Jul 21 10:52:27 2016 +0200
+++ b/src/HOL/IMP/Sec_TypingT.thy	Fri Jul 22 08:02:37 2016 +0200
@@ -107,9 +107,9 @@
     have "s = s' (\<le> l)" by auto
     moreover
     from termi_if_non0[OF 1 0, of t] obtain t' where
-      "(IF b THEN c1 ELSE c2,t) \<Rightarrow> t'" ..
+      t': "(IF b THEN c1 ELSE c2,t) \<Rightarrow> t'" ..
     moreover
-    from confinement[OF this 1] `\<not> sec b \<le> l`
+    from confinement[OF t' 1] `\<not> sec b \<le> l`
     have "t = t' (\<le> l)" by auto
     ultimately
     show ?case using `s = t (\<le> l)` by auto
@@ -134,9 +134,9 @@
     have "s = s' (\<le> l)" by auto
     moreover
     from termi_if_non0[OF 1 0, of t] obtain t' where
-      "(IF b THEN c1 ELSE c2,t) \<Rightarrow> t'" ..
+      t': "(IF b THEN c1 ELSE c2,t) \<Rightarrow> t'" ..
     moreover
-    from confinement[OF this 1] `\<not> sec b \<le> l`
+    from confinement[OF t' 1] `\<not> sec b \<le> l`
     have "t = t' (\<le> l)" by auto
     ultimately
     show ?case using `s = t (\<le> l)` by auto