src/HOL/Library/Linear_Temporal_Logic_on_Streams.thy
changeset 67399 eab6ce8368fa
parent 64911 f0e07600de47
child 67408 4a4c14b24800
--- a/src/HOL/Library/Linear_Temporal_Logic_on_Streams.thy	Wed Jan 10 15:21:49 2018 +0100
+++ b/src/HOL/Library/Linear_Temporal_Logic_on_Streams.thy	Wed Jan 10 15:25:09 2018 +0100
@@ -582,13 +582,13 @@
 lemma holds_Stream: "holds P (x ## s) \<longleftrightarrow> P x"
   by simp
 
-lemma holds_eq1[simp]: "holds (op = x) = HLD {x}"
+lemma holds_eq1[simp]: "holds ((=) x) = HLD {x}"
   by rule (auto simp: HLD_iff)
 
 lemma holds_eq2[simp]: "holds (\<lambda>y. y = x) = HLD {x}"
   by rule (auto simp: HLD_iff)
 
-lemma not_holds_eq[simp]: "holds (- op = x) = not (HLD {x})"
+lemma not_holds_eq[simp]: "holds (- (=) x) = not (HLD {x})"
   by rule (auto simp: HLD_iff)
 
 text \<open>Strong until\<close>