src/ZF/Order.thy
changeset 67399 eab6ce8368fa
parent 63901 4ce989e962e0
child 69587 53982d5ec0bb
--- a/src/ZF/Order.thy	Wed Jan 10 15:21:49 2018 +0100
+++ b/src/ZF/Order.thy	Wed Jan 10 15:25:09 2018 +0100
@@ -348,7 +348,7 @@
 apply (simp add: linear_def ord_iso_def, safe)
 apply (drule_tac x1 = "f`x" and x = "f`y" in bspec [THEN bspec])
 apply (safe elim!: bij_is_fun [THEN apply_type])
-apply (drule_tac t = "op ` (converse (f))" in subst_context)
+apply (drule_tac t = "(`) (converse (f))" in subst_context)
 apply (simp add: left_inverse_bij)
 done