tuned identifier
authornipkow
Tue, 12 Feb 2013 12:22:44 +0100
changeset 51037 0a6d84c41dbf
parent 51036 e7b54119c436
child 51038 73ddb9e6f6e8
tuned identifier
src/HOL/IMP/Abs_Int2.thy
--- a/src/HOL/IMP/Abs_Int2.thy	Tue Feb 12 11:54:29 2013 +0100
+++ b/src/HOL/IMP/Abs_Int2.thy	Tue Feb 12 12:22:44 2013 +0100
@@ -105,8 +105,8 @@
   (if res then bfilter b1 True (bfilter b2 True S)
    else bfilter b1 False S \<squnion> bfilter b2 False S)" |
 "bfilter (Less e1 e2) res S =
-  (let (res1,res2) = filter_less' res (aval'' e1 S) (aval'' e2 S)
-   in afilter e1 res1 (afilter e2 res2 S))"
+  (let (a1,a2) = filter_less' res (aval'' e1 S) (aval'' e2 S)
+   in afilter e1 a1 (afilter e2 a2 S))"
 
 lemma afilter_in_L: "S \<in> L X \<Longrightarrow> vars e \<subseteq> X \<Longrightarrow> afilter e a S \<in> L X"
 by(induction e arbitrary: a S)